|
8 | 8 |
|
9 | 9 | module Relation.Binary.Consequences where
|
10 | 10 |
|
11 |
| -open import Data.Empty using (⊥-elim) |
12 | 11 | open import Data.Product.Base using (_,_)
|
13 | 12 | open import Data.Sum.Base as Sum using (inj₁; inj₂; [_,_]′)
|
14 | 13 | open import Function.Base using (_∘_; _∘₂_; _$_; flip)
|
15 | 14 | open import Level using (Level)
|
16 | 15 | open import Relation.Binary.Core
|
17 | 16 | open import Relation.Binary.Definitions
|
18 |
| -open import Relation.Nullary.Negation.Core using (¬_) |
| 17 | +open import Relation.Nullary.Negation.Core using (¬_; contradiction) |
19 | 18 | open import Relation.Nullary.Decidable.Core
|
20 | 19 | using (yes; no; recompute; map′; dec⇒maybe)
|
21 | 20 | open import Relation.Unary using (∁; Pred)
|
@@ -121,7 +120,7 @@ module _ {_≈_ : Rel A ℓ₁} {_<_ : Rel A ℓ₂} where
|
121 | 120 | irrefl (antisym x<y y<x) x<y
|
122 | 121 |
|
123 | 122 | asym⇒antisym : Asymmetric _<_ → Antisymmetric _≈_ _<_
|
124 |
| - asym⇒antisym asym x<y y<x = ⊥-elim (asym x<y y<x) |
| 123 | + asym⇒antisym asym x<y y<x = contradiction y<x (asym x<y) |
125 | 124 |
|
126 | 125 | asym⇒irr : _<_ Respects₂ _≈_ → Symmetric _≈_ →
|
127 | 126 | Asymmetric _<_ → Irreflexive _≈_ _<_
|
@@ -157,16 +156,16 @@ module _ {_≈_ : Rel A ℓ₁} {_<_ : Rel A ℓ₂} where
|
157 | 156 | _<_ Respectsʳ _≈_
|
158 | 157 | trans∧tri⇒respʳ sym ≈-tr <-tr tri {x} {y} {z} y≈z x<y with tri x z
|
159 | 158 | ... | tri< x<z _ _ = x<z
|
160 |
| - ... | tri≈ _ x≈z _ = ⊥-elim (tri⇒irr tri (≈-tr x≈z (sym y≈z)) x<y) |
161 |
| - ... | tri> _ _ z<x = ⊥-elim (tri⇒irr tri (sym y≈z) (<-tr z<x x<y)) |
| 159 | + ... | tri≈ _ x≈z _ = contradiction x<y (tri⇒irr tri (≈-tr x≈z (sym y≈z))) |
| 160 | + ... | tri> _ _ z<x = contradiction (<-tr z<x x<y) (tri⇒irr tri (sym y≈z)) |
162 | 161 |
|
163 | 162 | trans∧tri⇒respˡ : Transitive _≈_ →
|
164 | 163 | Transitive _<_ → Trichotomous _≈_ _<_ →
|
165 | 164 | _<_ Respectsˡ _≈_
|
166 | 165 | trans∧tri⇒respˡ ≈-tr <-tr tri {z} {_} {y} x≈y x<z with tri y z
|
167 | 166 | ... | tri< y<z _ _ = y<z
|
168 |
| - ... | tri≈ _ y≈z _ = ⊥-elim (tri⇒irr tri (≈-tr x≈y y≈z) x<z) |
169 |
| - ... | tri> _ _ z<y = ⊥-elim (tri⇒irr tri x≈y (<-tr x<z z<y)) |
| 167 | + ... | tri≈ _ y≈z _ = contradiction x<z (tri⇒irr tri (≈-tr x≈y y≈z)) |
| 168 | + ... | tri> _ _ z<y = contradiction (<-tr x<z z<y) (tri⇒irr tri x≈y) |
170 | 169 |
|
171 | 170 | trans∧tri⇒resp : Symmetric _≈_ → Transitive _≈_ →
|
172 | 171 | Transitive _<_ → Trichotomous _≈_ _<_ →
|
|
0 commit comments