File tree Expand file tree Collapse file tree 1 file changed +3
-2
lines changed Expand file tree Collapse file tree 1 file changed +3
-2
lines changed Original file line number Diff line number Diff line change @@ -17,7 +17,8 @@ open import Relation.Binary.Definitions
17
17
hiding (Decidable; Universal; Irrelevant; Empty)
18
18
open import Relation.Binary.PropositionalEquality.Core using (refl; _≗_)
19
19
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)
21
22
open import Function.Base using (id; _$_; _∘_)
22
23
23
24
private
@@ -239,7 +240,7 @@ _~? P? = P? ∘ swap
239
240
240
241
does-≡ : {P : Pred A ℓ} → (P? P?′ : Decidable P) →
241
242
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)
243
244
244
245
does-≐ : {P : Pred A ℓ₁} {Q : Pred A ℓ₂} → P ≐ Q →
245
246
(P? : Decidable P) → (Q? : Decidable Q) →
You can’t perform that action at this time.
0 commit comments