Skip to content

Commit 66b5974

Browse files
Fix #2396 by removing redundant zero in IsNonAssociativeRing
The zero field in the IsNonAssociativeRing was redundant, and could be replaced with a proof based on the other properties.
1 parent 18ab15e commit 66b5974

File tree

1 file changed

+9
-7
lines changed

1 file changed

+9
-7
lines changed

src/Algebra/Structures.agda

+9-7
Original file line numberDiff line numberDiff line change
@@ -799,7 +799,6 @@ record IsNonAssociativeRing (+ * : Op₂ A) (-_ : Op₁ A) (0# 1# : A) : Set (a
799799
*-cong : Congruent₂ *
800800
*-identity : Identity 1# *
801801
distrib : * DistributesOver +
802-
zero : Zero 0# *
803802

804803
open IsAbelianGroup +-isAbelianGroup public
805804
renaming
@@ -827,18 +826,21 @@ record IsNonAssociativeRing (+ * : Op₂ A) (-_ : Op₁ A) (0# 1# : A) : Set (a
827826
; isGroup to +-isGroup
828827
)
829828

830-
zeroˡ : LeftZero 0# *
831-
zeroˡ = proj₁ zero
832-
833-
zeroʳ : RightZero 0# *
834-
zeroʳ = proj₂ zero
835-
836829
distribˡ : * DistributesOverˡ +
837830
distribˡ = proj₁ distrib
838831

839832
distribʳ : * DistributesOverʳ +
840833
distribʳ = proj₂ distrib
841834

835+
zeroˡ : LeftZero 0# *
836+
zeroˡ = Consequences.assoc∧distribʳ∧idʳ∧invʳ⇒zeˡ setoid +-cong *-cong +-assoc distribʳ +-identityʳ -‿inverseʳ
837+
838+
zeroʳ : RightZero 0# *
839+
zeroʳ = Consequences.assoc∧distribˡ∧idʳ∧invʳ⇒zeʳ setoid +-cong *-cong +-assoc distribˡ +-identityʳ -‿inverseʳ
840+
841+
zero : Zero 0# *
842+
zero = zeroˡ , zeroʳ
843+
842844
*-isMagma : IsMagma *
843845
*-isMagma = record
844846
{ isEquivalence = isEquivalence

0 commit comments

Comments
 (0)