Skip to content

Commit 5baffde

Browse files
committed
added CommutativeRing to the tally
1 parent d23bc6f commit 5baffde

File tree

2 files changed

+14
-0
lines changed

2 files changed

+14
-0
lines changed

CHANGELOG.md

+2
Original file line numberDiff line numberDiff line change
@@ -1602,7 +1602,9 @@ Other minor changes
16021602
zero : Zero ≈ ε ∙ → Zero ≈ ε (flip ∙)
16031603
distributes : (≈ DistributesOver ∙) + → (≈ DistributesOver (flip ∙)) +
16041604
isRing : IsRing ≈ + * - 0# 1# → IsRing ≈ + (flip *) - 0# 1#
1605+
isCommutativeRing : IsCommutativeRing ≈ + * - 0# 1# → IsCommutativeRing ≈ + (flip *) - 0# 1#
16051606
ring : Ring a ℓ → Ring a ℓ
1607+
commutativeRing : CommutativeRing a ℓ → CommutativeRing a ℓ
16061608
```
16071609

16081610
* Added new definition to `Algebra.Definitions`:

src/Algebra/Construct/Flip/Op.agda

+12
Original file line numberDiff line numberDiff line change
@@ -200,6 +200,14 @@ module _ {≈ : Rel A ℓ} {+ * : Op₂ A} { - : Op₁ A} {0# 1# : A} where
200200
where
201201
module r = IsRing r
202202

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+
203211

204212
------------------------------------------------------------------------
205213
-- Bundles
@@ -282,3 +290,7 @@ ring : Ring a ℓ → Ring a ℓ
282290
ring r = record { isRing = isRing r.isRing }
283291
where module r = Ring r
284292

293+
commutativeRing : CommutativeRing a ℓ CommutativeRing a ℓ
294+
commutativeRing r = record { isCommutativeRing = isCommutativeRing r.isCommutativeRing }
295+
where module r = CommutativeRing r
296+

0 commit comments

Comments
 (0)