File tree Expand file tree Collapse file tree 2 files changed +10
-0
lines changed
src/Relation/Nullary/Negation Expand file tree Collapse file tree 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
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+ ```
Original file line number Diff line number Diff line change @@ -60,6 +60,11 @@ contradiction₂ (inj₂ b) ¬a ¬b = contradiction b ¬b
6060contraposition : (A → B) → ¬ B → ¬ A
6161contraposition 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.
6469stable : ¬ ¬ Stable A
6570stable ¬[¬¬a→a] = ¬[¬¬a→a] (contradiction (¬[¬¬a→a] ∘ const))
You can’t perform that action at this time.
0 commit comments