File tree 2 files changed +0
-14
lines changed
src/Algebra/Construct/Flip
2 files changed +0
-14
lines changed Original file line number Diff line number Diff line change @@ -1602,9 +1602,7 @@ Other minor changes
1602
1602
zero : Zero ≈ ε ∙ → Zero ≈ ε (flip ∙)
1603
1603
distributes : (≈ DistributesOver ∙) + → (≈ DistributesOver (flip ∙)) +
1604
1604
isRing : IsRing ≈ + * - 0# 1# → IsRing ≈ + (flip *) - 0# 1#
1605
- isCommutativeRing : IsCommutativeRing ≈ + * - 0# 1# → IsCommutativeRing ≈ + (flip *) - 0# 1#
1606
1605
ring : Ring a ℓ → Ring a ℓ
1607
- commutativeRing : CommutativeRing a ℓ → CommutativeRing a ℓ
1608
1606
```
1609
1607
1610
1608
* Added new definition to ` Algebra.Definitions ` :
Original file line number Diff line number Diff line change @@ -200,14 +200,6 @@ module _ {≈ : Rel A ℓ} {+ * : Op₂ A} { - : Op₁ A} {0# 1# : A} where
200
200
where
201
201
module r = IsRing r
202
202
203
- isCommutativeRing : IsCommutativeRing + * - 0# 1# → IsCommutativeRing + (flip *) - 0# 1#
204
- isCommutativeRing r = record
205
- { isRing = isRing r.isRing
206
- ; *-comm = commutative r.*-comm
207
- }
208
- where
209
- module r = IsCommutativeRing r
210
-
211
203
212
204
------------------------------------------------------------------------
213
205
-- Bundles
@@ -290,7 +282,3 @@ ring : Ring a ℓ → Ring a ℓ
290
282
ring r = record { isRing = isRing r.isRing }
291
283
where module r = Ring r
292
284
293
- commutativeRing : CommutativeRing a ℓ → CommutativeRing a ℓ
294
- commutativeRing r = record { isCommutativeRing = isCommutativeRing r.isCommutativeRing }
295
- where module r = CommutativeRing r
296
-
You can’t perform that action at this time.
0 commit comments