File tree 2 files changed +10
-0
lines changed
src/Relation/Nullary/Negation
2 files changed +10
-0
lines changed Original file line number Diff line number Diff line change @@ -287,3 +287,8 @@ Additions to existing modules
287
287
⊤-dec : Dec {a} ⊤
288
288
⊥-dec : Dec {a} ⊥
289
289
```
290
+
291
+ * In ` Relation.Nullary.Negation.Core ` :
292
+ ``` agda
293
+ contra-diagonal : (A → ¬ A) → ¬ A
294
+ ```
Original file line number Diff line number Diff line change @@ -60,6 +60,11 @@ contradiction₂ (inj₂ b) ¬a ¬b = contradiction b ¬b
60
60
contraposition : (A → B) → ¬ B → ¬ A
61
61
contraposition f ¬b a = contradiction (f a) ¬b
62
62
63
+ -- Self-contradictory propositions are false by 'diagonalisation'
64
+
65
+ contra-diagonal : (A → ¬ A) → ¬ A
66
+ contra-diagonal self a = self a a
67
+
63
68
-- Everything is stable in the double-negation monad.
64
69
stable : ¬ ¬ Stable A
65
70
stable ¬[¬¬a→a] = ¬[¬¬a→a] (contradiction (¬[¬¬a→a] ∘ const))
You can’t perform that action at this time.
0 commit comments