File tree 1 file changed +4
-4
lines changed
1 file changed +4
-4
lines changed Original file line number Diff line number Diff line change @@ -200,9 +200,9 @@ U-Universal = λ _ → _
200
200
------------------------------------------------------------------------
201
201
-- Decidability properties
202
202
203
- ≐? : {P : Pred A ℓ₁} {Q : Pred A ℓ₂} →
204
- P ≐ Q → Decidable P → Decidable Q
205
- ≐? (P⊆Q , Q⊆P) P? x = map′ P⊆Q Q⊆P (P? x)
203
+ map : {P : Pred A ℓ₁} {Q : Pred A ℓ₂} →
204
+ P ≐ Q → Decidable P → Decidable Q
205
+ map (P⊆Q , Q⊆P) P? x = map′ P⊆Q Q⊆P (P? x)
206
206
207
207
∁? : {P : Pred A ℓ} → Decidable P → Decidable (∁ P)
208
208
∁? P? x = ¬? (P? x)
@@ -244,7 +244,7 @@ does-≡ P? P?′ x = Dec.does-≡ (P? x) (P?′ x)
244
244
does-≐ : {P : Pred A ℓ₁} {Q : Pred A ℓ₂} → P ≐ Q →
245
245
(P? : Decidable P) → (Q? : Decidable Q) →
246
246
does ∘ P? ≗ does ∘ Q?
247
- does-≐ P≐Q P? = does-≡ (≐? P≐Q P?)
247
+ does-≐ P≐Q P? = does-≡ (map P≐Q P?)
248
248
249
249
------------------------------------------------------------------------
250
250
-- Irrelevant properties
You can’t perform that action at this time.
0 commit comments