File tree 2 files changed +10
-0
lines changed
2 files changed +10
-0
lines changed Original file line number Diff line number Diff line change @@ -249,6 +249,12 @@ Additions to existing modules
249
249
x \\ y = (x ⁻¹) ∙ y
250
250
```
251
251
252
+ * In ` Algebra.Structures.IsCancellativeCommutativeSemiring ` add the
253
+ extra property as an exposed definition:
254
+ ``` agda
255
+ *-cancelʳ-nonZero : AlmostRightCancellative 0# *
256
+ ```
257
+
252
258
* In ` Data.Container.Indexed.Core ` :
253
259
``` agda
254
260
Subtrees o c = (r : Response c) → X (next c r)
Original file line number Diff line number Diff line change @@ -573,6 +573,10 @@ record IsCancellativeCommutativeSemiring (+ * : Op₂ A) (0# 1# : A) : Set (a
573
573
574
574
open IsCommutativeSemiring isCommutativeSemiring public
575
575
576
+ *-cancelʳ-nonZero : AlmostRightCancellative 0# *
577
+ *-cancelʳ-nonZero = Consequences.comm∧almostCancelˡ⇒almostCancelʳ setoid
578
+ *-comm *-cancelˡ-nonZero
579
+
576
580
record IsIdempotentSemiring (+ * : Op₂ A) (0# 1# : A) : Set (a ⊔ ℓ) where
577
581
field
578
582
isSemiring : IsSemiring + * 0# 1#
You can’t perform that action at this time.
0 commit comments