File tree 2 files changed +14
-0
lines changed
src/Algebra/Construct/Flip
2 files changed +14
-0
lines changed Original file line number Diff line number Diff line change @@ -1602,7 +1602,9 @@ 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#
1605
1606
ring : Ring a ℓ → Ring a ℓ
1607
+ commutativeRing : CommutativeRing a ℓ → CommutativeRing a ℓ
1606
1608
```
1607
1609
1608
1610
* Added new definition to ` Algebra.Definitions ` :
Original file line number Diff line number Diff line change @@ -200,6 +200,14 @@ 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
+
203
211
204
212
------------------------------------------------------------------------
205
213
-- Bundles
@@ -282,3 +290,7 @@ ring : Ring a ℓ → Ring a ℓ
282
290
ring r = record { isRing = isRing r.isRing }
283
291
where module r = Ring r
284
292
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