Skip to content

Commit 6d018a3

Browse files
authored
[ add ] obvious lemma about self-contradiction to Relation.Nullary.Negation.Core (#2693)
* add: obvious lemma about self-contradiction * add: obvious lemma about self-contradiction * fix: change name
1 parent 3880dec commit 6d018a3

File tree

2 files changed

+10
-0
lines changed

2 files changed

+10
-0
lines changed

CHANGELOG.md

+5
Original file line numberDiff line numberDiff line change
@@ -287,3 +287,8 @@ Additions to existing modules
287287
⊤-dec : Dec {a} ⊤
288288
⊥-dec : Dec {a} ⊥
289289
```
290+
291+
* In `Relation.Nullary.Negation.Core`:
292+
```agda
293+
contra-diagonal : (A → ¬ A) → ¬ A
294+
```

src/Relation/Nullary/Negation/Core.agda

+5
Original file line numberDiff line numberDiff line change
@@ -60,6 +60,11 @@ contradiction₂ (inj₂ b) ¬a ¬b = contradiction b ¬b
6060
contraposition : (A B) ¬ B ¬ A
6161
contraposition f ¬b a = contradiction (f a) ¬b
6262

63+
-- Self-contradictory propositions are false by 'diagonalisation'
64+
65+
contra-diagonal : (A ¬ A) ¬ A
66+
contra-diagonal self a = self a a
67+
6368
-- Everything is stable in the double-negation monad.
6469
stable : ¬ ¬ Stable A
6570
stable ¬[¬¬a→a] = ¬[¬¬a→a] (contradiction (¬[¬¬a→a] ∘ const))

0 commit comments

Comments
 (0)