summaryrefslogtreecommitdiff
path: root/src/Helium/Algebra/Ordered/StrictTotal/Properties/CommutativeRing.agda
diff options
context:
space:
mode:
authorGreg Brown <greg.brown@cl.cam.ac.uk>2022-04-04 12:34:14 +0100
committerGreg Brown <greg.brown@cl.cam.ac.uk>2022-04-04 12:34:14 +0100
commite3f5e2a708452c8cde9af7f08ab6f00afe0f859a (patch)
tree53f48f4d174b50b5b5f473b6f1d7b77b2033f807 /src/Helium/Algebra/Ordered/StrictTotal/Properties/CommutativeRing.agda
parentba95dc7d15cab1af40da896114b7dd9aad5afda0 (diff)
Remove redundant cancel property.
It is in the standard library as `⁻¹-injective`.
Diffstat (limited to 'src/Helium/Algebra/Ordered/StrictTotal/Properties/CommutativeRing.agda')
-rw-r--r--src/Helium/Algebra/Ordered/StrictTotal/Properties/CommutativeRing.agda2
1 files changed, 1 insertions, 1 deletions
diff --git a/src/Helium/Algebra/Ordered/StrictTotal/Properties/CommutativeRing.agda b/src/Helium/Algebra/Ordered/StrictTotal/Properties/CommutativeRing.agda
index d303c99..aa265c8 100644
--- a/src/Helium/Algebra/Ordered/StrictTotal/Properties/CommutativeRing.agda
+++ b/src/Helium/Algebra/Ordered/StrictTotal/Properties/CommutativeRing.agda
@@ -59,7 +59,7 @@ open import Helium.Algebra.Ordered.StrictTotal.Properties.Ring ring public
; n≢0∧n×x≥0⇒x≥0; n≢0∧n×x≤0⇒x≤0
; -‿anti-mono-<; -‿anti-mono-≤
- ; -‿cancel; -‿anti-cancel-<; -‿anti-cancel-≤
+ ; -‿anti-cancel-<; -‿anti-cancel-≤
; x<0⇒-x>0; x>0⇒-x<0; x≤0⇒-x≥0; x≥0⇒-x≤0
; -x<0⇒x>0; -x>0⇒x<0; -x≤0⇒x≥0; -x≥0⇒x≤0