File tree Expand file tree Collapse file tree 2 files changed +6
-2
lines changed
src/Relation/Nullary/Negation Expand file tree Collapse file tree 2 files changed +6
-2
lines changed Original file line number Diff line number Diff line change @@ -17,6 +17,10 @@ Non-backwards compatible changes
17
17
Minor improvements
18
18
------------------
19
19
20
+ * The type of ` Relation.Nullary.Negation.Core.contradiction-irr ` has been further
21
+ weakened so that the negated hypothesis ` ¬ A ` is marked as irrelevant. This is
22
+ safe to do, in view of ` Relation.Nullary.Recomputable.Properties.¬-recompute ` .
23
+
20
24
* Refactored usages of ` +-∸-assoc 1 ` to ` ∸-suc ` in:
21
25
``` agda
22
26
README.Data.Fin.Relation.Unary.Top
Original file line number Diff line number Diff line change @@ -47,11 +47,11 @@ _¬-⊎_ = [_,_]
47
47
------------------------------------------------------------------------
48
48
-- Uses of negation
49
49
50
- contradiction-irr : .A → ¬ A → Whatever
50
+ contradiction-irr : .A → .( ¬ A) → Whatever
51
51
contradiction-irr a ¬a = ⊥-elim-irr (¬a a)
52
52
53
53
contradiction : A → ¬ A → Whatever
54
- contradiction a = contradiction-irr a
54
+ contradiction a ¬a = contradiction-irr a ¬ a
55
55
56
56
contradiction₂ : A ⊎ B → ¬ A → ¬ B → Whatever
57
57
contradiction₂ (inj₁ a) ¬a ¬b = contradiction a ¬a
You can’t perform that action at this time.
0 commit comments