File tree 1 file changed +2
-2
lines changed
1 file changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -17,7 +17,7 @@ open import Algebra.Bundles using (Magma; Semigroup; CommutativeSemigroup;
17
17
open import Algebra.Definitions.RawMagma using (_,_)
18
18
open import Algebra.Morphism
19
19
open import Algebra.Consequences.Propositional
20
- using (comm+ cancelˡ⇒cancelʳ; comm∧distrʳ⇒distrˡ; comm∧distrˡ⇒distrʳ)
20
+ using (comm∧ cancelˡ⇒cancelʳ; comm∧distrʳ⇒distrˡ; comm∧distrˡ⇒distrʳ)
21
21
open import Algebra.Construct.NaturalChoice.Base
22
22
using (MinOperator; MaxOperator)
23
23
import Algebra.Construct.NaturalChoice.MinMaxOp as MinMaxOp
@@ -561,7 +561,7 @@ open ≤-Reasoning
561
561
+-cancelˡ-≡ (suc m) _ _ eq = +-cancelˡ-≡ m _ _ (cong pred eq)
562
562
563
563
+-cancelʳ-≡ : RightCancellative _≡_ _+_
564
- +-cancelʳ-≡ = comm+ cancelˡ⇒cancelʳ +-comm +-cancelˡ-≡
564
+ +-cancelʳ-≡ = comm∧ cancelˡ⇒cancelʳ +-comm +-cancelˡ-≡
565
565
566
566
+-cancel-≡ : Cancellative _≡_ _+_
567
567
+-cancel-≡ = +-cancelˡ-≡ , +-cancelʳ-≡
You can’t perform that action at this time.
0 commit comments