@@ -944,8 +944,8 @@ distribʳ-⊖-+-neg m n o = begin
944
944
; ⁻¹-cong = cong (-_)
945
945
}
946
946
947
- +-isAbelianGroup : IsAbelianGroup _+_ +0 (-_)
948
- +-isAbelianGroup = record
947
+ +-0- isAbelianGroup : IsAbelianGroup _+_ +0 (-_)
948
+ +-0- isAbelianGroup = record
949
949
{ isGroup = +-0-isGroup
950
950
; comm = +-comm
951
951
}
@@ -980,7 +980,7 @@ distribʳ-⊖-+-neg m n o = begin
980
980
981
981
+-0-abelianGroup : AbelianGroup 0ℓ 0ℓ
982
982
+-0-abelianGroup = record
983
- { isAbelianGroup = +-isAbelianGroup
983
+ { isAbelianGroup = +-0- isAbelianGroup
984
984
}
985
985
986
986
------------------------------------------------------------------------
@@ -1522,7 +1522,7 @@ private
1522
1522
1523
1523
+-*-isRing : IsRing _+_ _*_ -_ 0ℤ 1ℤ
1524
1524
+-*-isRing = record
1525
- { +-isAbelianGroup = +-isAbelianGroup
1525
+ { +-isAbelianGroup = +-0- isAbelianGroup
1526
1526
; *-cong = cong₂ _*_
1527
1527
; *-assoc = *-assoc
1528
1528
; *-identity = *-identity
@@ -1539,12 +1539,6 @@ private
1539
1539
------------------------------------------------------------------------
1540
1540
-- Bundles
1541
1541
1542
- *-rawMagma : RawMagma 0ℓ 0ℓ
1543
- *-rawMagma = record { _≈_ = _≡_ ; _∙_ = _*_ }
1544
-
1545
- *-1-rawMonoid : RawMonoid 0ℓ 0ℓ
1546
- *-1-rawMonoid = record { _≈_ = _≡_ ; _∙_ = _*_ ; ε = 1ℤ }
1547
-
1548
1542
*-magma : Magma 0ℓ 0ℓ
1549
1543
*-magma = record
1550
1544
{ isMagma = *-isMagma
@@ -2387,3 +2381,11 @@ pos-distrib-* m n = sym (pos-* m n)
2387
2381
"Warning: pos-distrib-* was deprecated in v2.0
2388
2382
Please use pos-* instead."
2389
2383
#-}
2384
+ +-isAbelianGroup = +-0-isAbelianGroup
2385
+ {-# WARNING_ON_USAGE +-isAbelianGroup
2386
+ "Warning: +-isAbelianGroup was deprecated in v2.0
2387
+ Please use +-0-isAbelianGroup instead."
2388
+ #-}
2389
+ {- issue1844/issue1755: raw bundles have moved to `Data.X.Base` -}
2390
+ open Data.Integer.Base public
2391
+ using (*-rawMagma; *-1-rawMonoid)
0 commit comments