Skip to content

Commit 1785813

Browse files
committed
rename ≐? to map
1 parent c99296e commit 1785813

File tree

2 files changed

+5
-5
lines changed

2 files changed

+5
-5
lines changed

CHANGELOG.md

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -834,7 +834,7 @@ Additions to existing modules
834834

835835
* Added new proofs in `Relation.Nullary.Properties`:
836836
```agda
837-
≐? : P ≐ Q → Decidable P → Decidable Q
837+
map : P ≐ Q → Decidable P → Decidable Q
838838
does-≐ : P ≐ Q → (P? : Decidable P) → (Q? : Decidable Q) → does ∘ P? ≗ does ∘ Q?
839839
does-≡ : (P? P?′ : Decidable P) → does ∘ P? ≗ does ∘ P?′
840840
```

src/Relation/Unary/Properties.agda

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -200,9 +200,9 @@ U-Universal = λ _ → _
200200
------------------------------------------------------------------------
201201
-- Decidability properties
202202

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)
206206

207207
∁? : {P : Pred A ℓ} Decidable P Decidable (∁ P)
208208
∁? P? x = ¬? (P? x)
@@ -244,7 +244,7 @@ does-≡ P? P?′ x = Dec.does-≡ (P? x) (P?′ x)
244244
does-≐ : {P : Pred A ℓ₁} {Q : Pred A ℓ₂} P ≐ Q
245245
(P? : Decidable P) (Q? : Decidable Q)
246246
does ∘ P? ≗ does ∘ Q?
247-
does-≐ P≐Q P? = does-≡ (≐? P≐Q P?)
247+
does-≐ P≐Q P? = does-≡ (map P≐Q P?)
248248

249249
------------------------------------------------------------------------
250250
-- Irrelevant properties

0 commit comments

Comments
 (0)