@@ -16,7 +16,6 @@ import Algebra.Lattice.Properties.BooleanAlgebra as BooleanAlgebraProperties
16
16
open import Data.Bool.Base
17
17
using (Bool; true; false; not; _∧_; _∨_; _xor_ ; if_then_else_; T; _≤_; _<_
18
18
; b≤b; f≤t; f<t)
19
- open import Data.Empty using (⊥; ⊥-elim)
20
19
open import Data.Product.Base using (_×_; _,_; proj₁; proj₂)
21
20
open import Data.Sum.Base using (_⊎_; inj₁; inj₂; [_,_])
22
21
open import Function.Base using (_⟨_⟩_; const; id)
@@ -42,6 +41,7 @@ open import Relation.Binary.PropositionalEquality.Properties
42
41
using (module ≡-Reasoning ; setoid; decSetoid; isEquivalence)
43
42
open import Relation.Nullary.Decidable.Core
44
43
using (True; yes; no; fromWitness ; toWitness)
44
+ open import Relation.Nullary.Negation.Core using (contradiction)
45
45
import Relation.Unary as U
46
46
47
47
open import Algebra.Definitions {A = Bool} _≡_
@@ -657,10 +657,10 @@ not-¬ {true} refl ()
657
657
not-¬ {false} refl ()
658
658
659
659
¬-not : ∀ {x y} → x ≢ y → x ≡ not y
660
- ¬-not {true} {true} x≢y = ⊥-elim ( x≢y refl)
660
+ ¬-not {true} {true} x≢y = contradiction refl x≢y
661
661
¬-not {true} {false} _ = refl
662
662
¬-not {false} {true} _ = refl
663
- ¬-not {false} {false} x≢y = ⊥-elim ( x≢y refl)
663
+ ¬-not {false} {false} x≢y = contradiction refl x≢y
664
664
665
665
------------------------------------------------------------------------
666
666
-- Properties of _xor_
0 commit comments