Skip to content

Commit 5c155c3

Browse files
committed
fixup! use qualified import instead of renaming
1 parent 7a5394f commit 5c155c3

File tree

1 file changed

+3
-2
lines changed

1 file changed

+3
-2
lines changed

src/Relation/Unary/Properties.agda

Lines changed: 3 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -17,7 +17,8 @@ open import Relation.Binary.Definitions
1717
hiding (Decidable; Universal; Irrelevant; Empty)
1818
open import Relation.Binary.PropositionalEquality.Core using (refl; _≗_)
1919
open import Relation.Unary
20-
open import Relation.Nullary.Decidable using (yes; no; _⊎-dec_; _×-dec_; ¬?; map′; does) renaming (does-≡ to does-≡′)
20+
import Relation.Nullary.Decidable as Dec
21+
open import Relation.Nullary.Decidable using (yes; no; _⊎-dec_; _×-dec_; ¬?; map′; does)
2122
open import Function.Base using (id; _$_; _∘_)
2223

2324
private
@@ -239,7 +240,7 @@ _~? P? = P? ∘ swap
239240

240241
does-≡ : {P : Pred A ℓ} (P? P?′ : Decidable P)
241242
does ∘ P? ≗ does ∘ P?′
242-
does-≡ P? P?′ x = does-≡ (P? x) (P?′ x)
243+
does-≡ P? P?′ x = Dec.does-≡ (P? x) (P?′ x)
243244

244245
does-≐ : {P : Pred A ℓ₁} {Q : Pred A ℓ₂} P ≐ Q
245246
(P? : Decidable P) (Q? : Decidable Q)

0 commit comments

Comments
 (0)