File tree Expand file tree Collapse file tree 3 files changed +28
-1
lines changed Expand file tree Collapse file tree 3 files changed +28
-1
lines changed Original file line number Diff line number Diff line change @@ -278,7 +278,13 @@ Other minor additions
278
278
recompute : .(Coprime n d) → Coprime n d
279
279
```
280
280
281
- * Added new types and constructors to ` Data.Rational.Unnormalised ` :
281
+ * Add proof to ` Algebra.Morphism.RingMonomorphism ` :
282
+ ``` agda
283
+ isCommutativeRing : IsCommutativeRing _≈₂_ _⊕_ _⊛_ ⊝_ 0#₂ 1#₂ →
284
+ IsCommutativeRing _≈₁_ _+_ _*_ -_ 0# 1#
285
+ ```
286
+
287
+ * Added new types and constructors to ` Data.Rational ` :
282
288
``` agda
283
289
NonZero : Pred ℚ 0ℓ
284
290
Positive : Pred ℚ 0ℓ
@@ -295,6 +301,12 @@ Other minor additions
295
301
nonNegative : p ≥ 0ℚ → NonNegative p
296
302
```
297
303
304
+ * Added proofs to ` Data.Rational.Properties ` :
305
+ ``` agda
306
+ +-*-isCommutativeRing : IsCommutativeRing _+_ _*_ -_ 0ℚ 1ℚ
307
+ +-*-commutativeRing : CommutativeRing 0ℓ 0ℓ
308
+ ```
309
+
298
310
* Added new types and constructors to ` Data.Rational.Unnormalised `
299
311
``` agda
300
312
_≠_ : Rel ℚᵘ 0ℓ
Original file line number Diff line number Diff line change @@ -127,3 +127,10 @@ isRing isRing = record
127
127
; distrib = distrib R.+-isGroup R.*-isMagma R.distrib
128
128
; zero = zero R.+-isGroup R.*-isMagma R.zero
129
129
} where module R = IsRing isRing
130
+
131
+ isCommutativeRing : IsCommutativeRing _≈₂_ _⊕_ _⊛_ ⊝_ 0#₂ 1#₂ →
132
+ IsCommutativeRing _≈₁_ _+_ _*_ -_ 0# 1#
133
+ isCommutativeRing isCommRing = record
134
+ { isRing = isRing C.isRing
135
+ ; *-comm = *-comm C.*-isMagma C.*-comm
136
+ } where module C = IsCommutativeRing isCommRing
Original file line number Diff line number Diff line change @@ -818,6 +818,9 @@ private
818
818
+-*-isRing : IsRing _+_ _*_ -_ 0ℚ 1ℚ
819
819
+-*-isRing = *-Monomorphism.isRing ℚᵘ.+-*-isRing
820
820
821
+ +-*-isCommutativeRing : IsCommutativeRing _+_ _*_ -_ 0ℚ 1ℚ
822
+ +-*-isCommutativeRing = *-Monomorphism.isCommutativeRing ℚᵘ.+-*-isCommutativeRing
823
+
821
824
------------------------------------------------------------------------
822
825
-- Packages
823
826
@@ -846,6 +849,11 @@ private
846
849
{ isRing = +-*-isRing
847
850
}
848
851
852
+ +-*-commutativeRing : CommutativeRing 0ℓ 0ℓ
853
+ +-*-commutativeRing = record
854
+ { isCommutativeRing = +-*-isCommutativeRing
855
+ }
856
+
849
857
------------------------------------------------------------------------
850
858
-- DEPRECATED NAMES
851
859
------------------------------------------------------------------------
You can’t perform that action at this time.
0 commit comments