@@ -35,7 +35,7 @@ open import Relation.Binary.Core using (_⇒_; _Preserves_⟶_; _Preserves₂_
35
35
open import Relation.Binary.Bundles
36
36
using (Setoid; DecSetoid; Preorder; TotalPreorder; Poset; TotalOrder; DecTotalOrder; StrictPartialOrder; StrictTotalOrder; DenseLinearOrder)
37
37
open import Relation.Binary.Structures
38
- using (IsEquivalence; IsDecEquivalence; IsApartnessRelation; IsTotalPreorder; IsPreorder; IsPartialOrder; IsTotalOrder; IsDecTotalOrder; IsStrictPartialOrder; IsStrictTotalOrder; IsDenseLinearOrder)
38
+ using (IsEquivalence; IsDecEquivalence; IsApartnessRelation; IsTightApartnessRelation; IsTotalPreorder; IsPreorder; IsPartialOrder; IsTotalOrder; IsDecTotalOrder; IsStrictPartialOrder; IsStrictTotalOrder; IsDenseLinearOrder)
39
39
open import Relation.Binary.Definitions
40
40
using (Reflexive; Symmetric; Transitive; Cotransitive; Tight; Decidable; Antisymmetric; Asymmetric; Dense; Total; Trans; Trichotomous; Irreflexive; Irrelevant; _Respectsˡ_; _Respectsʳ_; _Respects₂_; tri≈; tri<; tri>)
41
41
import Relation.Binary.Consequences as BC
@@ -139,8 +139,13 @@ p ≃? q = Dec.map′ *≡* drop-*≡* (↥ p ℤ.* ↧ q ℤ.≟ ↥ q ℤ.*
139
139
}
140
140
141
141
≄-tight : Tight _≃_ _≄_
142
- proj₁ (≄-tight p q) ¬p≄q = Dec.decidable-stable (p ≃? q) ¬p≄q
143
- proj₂ (≄-tight p q) p≃q p≄q = p≄q p≃q
142
+ ≄-tight p q = Dec.decidable-stable (p ≃? q)
143
+
144
+ ≄-isTightApartnessRelation : IsTightApartnessRelation _≃_ _≄_
145
+ ≄-isTightApartnessRelation = record
146
+ { isApartnessRelation = ≄-isApartnessRelation
147
+ ; tight = ≄-tight
148
+ }
144
149
145
150
≃-setoid : Setoid 0ℓ 0ℓ
146
151
≃-setoid = record
@@ -1399,15 +1404,14 @@ nonNeg*nonNeg⇒nonNeg p q = nonNegative
1399
1404
+-*-isHeytingCommutativeRing : IsHeytingCommutativeRing _≃_ _≄_ _+_ _*_ -_ 0ℚᵘ 1ℚᵘ
1400
1405
+-*-isHeytingCommutativeRing = record
1401
1406
{ isCommutativeRing = +-*-isCommutativeRing
1402
- ; isApartnessRelation = ≄-isApartnessRelation
1403
- ; #⇒invertible = ≄⇒invertible
1404
- ; invertible⇒# = invertible⇒≄
1407
+ ; isTightApartnessRelation = ≄-isTightApartnessRelation
1405
1408
}
1406
1409
1407
1410
+-*-isHeytingField : IsHeytingField _≃_ _≄_ _+_ _*_ -_ 0ℚᵘ 1ℚᵘ
1408
1411
+-*-isHeytingField = record
1409
1412
{ isHeytingCommutativeRing = +-*-isHeytingCommutativeRing
1410
- ; tight = ≄-tight
1413
+ ; #⇒invertible = ≄⇒invertible
1414
+ ; invertible⇒# = invertible⇒≄
1411
1415
}
1412
1416
1413
1417
------------------------------------------------------------------------
0 commit comments