Skip to content

Commit ce8e4af

Browse files
authored
fix: naming convention (#2838)
1 parent bb57f49 commit ce8e4af

File tree

2 files changed

+58
-10
lines changed

2 files changed

+58
-10
lines changed

CHANGELOG.md

Lines changed: 9 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -48,6 +48,15 @@ Deprecated names
4848
interchange ↦ medial
4949
```
5050

51+
* In `Relation.Nullary.Negation`:
52+
```agda
53+
∃⟶¬∀¬ ↦ ∃⇒¬∀¬
54+
∀⟶¬∃¬ ↦ ∀⇒¬∃¬
55+
¬∃⟶∀¬ ↦ ¬∃⇒∀¬
56+
∀¬⟶¬∃ ↦ ∀¬⇒¬∃
57+
∃¬⟶¬∀ ↦ ∃¬⇒¬∀
58+
```
59+
5160
New modules
5261
-----------
5362

src/Relation/Nullary/Negation.agda

Lines changed: 49 additions & 10 deletions
Original file line numberDiff line numberDiff line change
@@ -32,20 +32,20 @@ open import Relation.Nullary.Negation.Core public
3232
------------------------------------------------------------------------
3333
-- Quantifier juggling
3434

35-
¬∀¬ : ∃ P ¬ ( x ¬ P x)
36-
¬∀¬ = flip uncurry
35+
¬∀¬ : ∃ P ¬ ( x ¬ P x)
36+
¬∀¬ = flip uncurry
3737

38-
¬∃¬ : ( x P x) ¬ ∃ λ x ¬ P x
39-
¬∃¬ ∀xPx (x , ¬Px) = ¬Px (∀xPx x)
38+
¬∃¬ : ( x P x) ¬ ∃ λ x ¬ P x
39+
¬∃¬ ∀xPx (x , ¬Px) = ¬Px (∀xPx x)
4040

41-
¬∃∀¬ : ¬ ∃ (λ x P x) x ¬ P x
42-
¬∃∀¬ = curry
41+
¬∃∀¬ : ¬ ∃ (λ x P x) x ¬ P x
42+
¬∃∀¬ = curry
4343

44-
∀¬¬∃ : ( x ¬ P x) ¬ ∃ (λ x P x)
45-
∀¬¬∃ = uncurry
44+
∀¬¬∃ : ( x ¬ P x) ¬ ∃ (λ x P x)
45+
∀¬¬∃ = uncurry
4646

47-
∃¬¬∀ : ∃ (λ x ¬ P x) ¬ ( x P x)
48-
∃¬¬∀ = flip ∀¬∃¬
47+
∃¬¬∀ : ∃ (λ x ¬ P x) ¬ ( x P x)
48+
∃¬¬∀ = flip ∀¬∃¬
4949

5050
------------------------------------------------------------------------
5151
-- Double Negation
@@ -106,3 +106,42 @@ private
106106
helper : ∃ (λ b A if b then B else C) (A B) ⊎ (A C)
107107
helper (true , f) = inj₁ f
108108
helper (false , f) = inj₂ f
109+
110+
111+
------------------------------------------------------------------------
112+
-- DEPRECATED NAMES
113+
------------------------------------------------------------------------
114+
-- Please use the new names as continuing support for the old names is
115+
-- not guaranteed.
116+
117+
-- Version 2.4
118+
119+
∃⟶¬∀¬ = ∃⇒¬∀¬
120+
{-# WARNING_ON_USAGE ∃⟶¬∀¬
121+
"Warning: ∃⟶¬∀¬ was deprecated in v2.4.
122+
Please use ∃⇒¬∀¬ instead."
123+
#-}
124+
125+
∀⟶¬∃¬ = ∀⇒¬∃¬
126+
{-# WARNING_ON_USAGE ∀⟶¬∃¬
127+
"Warning: ∀⟶¬∃¬ was deprecated in v2.4.
128+
Please use ∀⇒¬∃¬ instead."
129+
#-}
130+
131+
¬∃⟶∀¬ = ¬∃⇒∀¬
132+
{-# WARNING_ON_USAGE ¬∃⟶∀¬
133+
"Warning: ¬∃⟶∀¬ was deprecated in v2.4.
134+
Please use ¬∃⇒∀¬ instead."
135+
#-}
136+
137+
∀¬⟶¬∃ = ∀¬⇒¬∃
138+
{-# WARNING_ON_USAGE ∀¬⟶¬∃
139+
"Warning: ∀¬⟶¬∃ was deprecated in v2.4.
140+
Please use ∀¬⇒¬∃ instead."
141+
#-}
142+
143+
∃¬⟶¬∀ = ∃¬⇒¬∀
144+
{-# WARNING_ON_USAGE ∃¬⟶¬∀
145+
"Warning: ∃¬⟶¬∀ was deprecated in v2.4.
146+
Please use ∃¬⇒¬∀ instead."
147+
#-}

0 commit comments

Comments
 (0)