summaryrefslogtreecommitdiff
path: root/src/Helium/Algebra/Ordered/StrictTotal/Properties/Group.agda
diff options
context:
space:
mode:
authorGreg Brown <greg.brown@cl.cam.ac.uk>2022-04-05 12:08:00 +0100
committerGreg Brown <greg.brown@cl.cam.ac.uk>2022-04-05 12:08:00 +0100
commit038d2109e78d9c688acfc3338140cc908151db76 (patch)
tree3687ed702cf13d728cffe23642a3fe6affb73310 /src/Helium/Algebra/Ordered/StrictTotal/Properties/Group.agda
parentb212c150ec0a9bf45cf6c28fba997693669e78d2 (diff)
Generalise 0 comparison to ≤.
Diffstat (limited to 'src/Helium/Algebra/Ordered/StrictTotal/Properties/Group.agda')
-rw-r--r--src/Helium/Algebra/Ordered/StrictTotal/Properties/Group.agda15
1 files changed, 15 insertions, 0 deletions
diff --git a/src/Helium/Algebra/Ordered/StrictTotal/Properties/Group.agda b/src/Helium/Algebra/Ordered/StrictTotal/Properties/Group.agda
index 5cf2d5b..81c57ad 100644
--- a/src/Helium/Algebra/Ordered/StrictTotal/Properties/Group.agda
+++ b/src/Helium/Algebra/Ordered/StrictTotal/Properties/Group.agda
@@ -213,3 +213,18 @@ x<y⇒ε<y∙x⁻¹ {x} {y} x<y = begin-strict
y ∙ (x ⁻¹ ∙ x) ≈⟨ ∙-congˡ (inverseˡ x) ⟩
y ∙ ε ≈⟨ identityʳ y ⟩
y ∎
+
+x≤y⇒ε≤y∙x⁻¹ : ∀ {x y} → x ≤ y → ε ≤ y ∙ x ⁻¹
+x≤y⇒ε≤y∙x⁻¹ {x} {y} x≤y = begin
+ ε ≈˘⟨ inverseʳ x ⟩
+ x ∙ x ⁻¹ ≤⟨ ∙-monoʳ-≤ x≤y ⟩
+ y ∙ x ⁻¹ ∎
+
+ε≤y∙x⁻¹⇒x≤y : ∀ {x y} → ε ≤ y ∙ x ⁻¹ → x ≤ y
+ε≤y∙x⁻¹⇒x≤y {x} {y} ε≤y∙x⁻¹ = begin
+ x ≈˘⟨ identityˡ x ⟩
+ ε ∙ x ≤⟨ ∙-monoʳ-≤ ε≤y∙x⁻¹ ⟩
+ y ∙ x ⁻¹ ∙ x ≈⟨ assoc y (x ⁻¹) x ⟩
+ y ∙ (x ⁻¹ ∙ x) ≈⟨ ∙-congˡ (inverseˡ x) ⟩
+ y ∙ ε ≈⟨ identityʳ y ⟩
+ y ∎