summaryrefslogtreecommitdiff
path: root/src/Helium/Algebra/Ordered/StrictTotal/Properties/Field.agda
diff options
context:
space:
mode:
authorGreg Brown <greg.brown@cl.cam.ac.uk>2022-04-04 15:51:22 +0100
committerGreg Brown <greg.brown@cl.cam.ac.uk>2022-04-04 15:51:22 +0100
commit6acd0e87fa8ab2a3230626b37f1cd02181810a1a (patch)
tree21f96be343fc8ad7a8afa595c13d19b408de9e0e /src/Helium/Algebra/Ordered/StrictTotal/Properties/Field.agda
parent4cd820506e0fd2a5595a11555fc2a6206757b3cd (diff)
Add some more ordered division ring properties.
Diffstat (limited to 'src/Helium/Algebra/Ordered/StrictTotal/Properties/Field.agda')
-rw-r--r--src/Helium/Algebra/Ordered/StrictTotal/Properties/Field.agda21
1 files changed, 21 insertions, 0 deletions
diff --git a/src/Helium/Algebra/Ordered/StrictTotal/Properties/Field.agda b/src/Helium/Algebra/Ordered/StrictTotal/Properties/Field.agda
index 51a054e..33578e0 100644
--- a/src/Helium/Algebra/Ordered/StrictTotal/Properties/Field.agda
+++ b/src/Helium/Algebra/Ordered/StrictTotal/Properties/Field.agda
@@ -23,6 +23,16 @@ open Field field′
open import Algebra.Properties.Ring Unordered.ring public
renaming (-0#≈0# to -0≈0)
+open import Helium.Algebra.Properties.AlmostGroup *-almostGroup public
+ renaming
+ ( x≉0⇒∙-cancelˡ to x≉0⇒*-cancelˡ
+ ; x≉0⇒∙-cancelʳ to x≉0⇒*-cancelʳ
+ ; ⁻¹-anti-homo-∙ to ⁻¹-anti-homo-*
+ ; identityˡ-unique to *-identityˡ-unique
+ ; identityʳ-unique to *-identityʳ-unique
+ ; inverseˡ-unique to *-inverseˡ-unique
+ ; inverseʳ-unique to *-inverseʳ-unique
+ )
open import Algebra.Properties.Semiring.Mult.TCOptimised Unordered.semiring public
open import Algebra.Properties.CommutativeSemiring.Exp.TCOptimised Unordered.commutativeSemiring public
open import Helium.Relation.Binary.Properties.StrictTotalOrder strictTotalOrder public
@@ -97,4 +107,15 @@ open import Helium.Algebra.Ordered.StrictTotal.Properties.DivisionRing divisionR
; x>1∧n≢0⇒x^n>1; 0≤x<1∧n≢0⇒x^n<1
; x≥1⇒x^n≥1; 0≤x≤1⇒x^n≤1
+
+ ; x>0⇒x⁻¹>0 ; x<0⇒x⁻¹<0
+
+ ; x⁻¹>0⇒x>0 ; x⁻¹<0⇒x<0
+
+ ; x>1⇒x⁻¹<1; 0<x<1⇒x⁻¹>1
+
+ ; x⁻¹>1⇒x<1; 0<x⁻¹<1⇒x>1
+
+ ; -‿⁻¹-comm
+ ; x≉0⇒x⁻¹≉0
)