File tree 2 files changed +16
-3
lines changed
2 files changed +16
-3
lines changed Original file line number Diff line number Diff line change @@ -183,6 +183,11 @@ Additions to existing modules
183
183
rawKleeneAlgebra : RawKleeneAlgebra _ _
184
184
```
185
185
186
+ * In ` Algebra.Bundles.Raw.* `
187
+ ``` agda
188
+ rawSetoid : RawSetoid c ℓ
189
+ ```
190
+
186
191
* In ` Algebra.Bundles.Raw.RawRingWithoutOne `
187
192
``` agda
188
193
rawNearSemiring : RawNearSemiring c ℓ
Original file line number Diff line number Diff line change @@ -10,6 +10,7 @@ module Algebra.Bundles.Raw where
10
10
11
11
open import Algebra.Core
12
12
open import Relation.Binary.Core using (Rel)
13
+ open import Relation.Binary.Bundles.Raw using (RawSetoid)
13
14
open import Level using (suc; _⊔_)
14
15
open import Relation.Nullary.Negation.Core using (¬_)
15
16
@@ -27,6 +28,11 @@ record RawSuccessorSet c ℓ : Set (suc (c ⊔ ℓ)) where
27
28
suc# : Op₁ Carrier
28
29
zero# : Carrier
29
30
31
+ rawSetoid : RawSetoid c ℓ
32
+ rawSetoid = record { _≈_ = _≈_ }
33
+
34
+ open RawSetoid rawSetoid public using (_≉_)
35
+
30
36
------------------------------------------------------------------------
31
37
-- Raw bundles with 1 binary operation
32
38
------------------------------------------------------------------------
@@ -39,9 +45,11 @@ record RawMagma c ℓ : Set (suc (c ⊔ ℓ)) where
39
45
_≈_ : Rel Carrier ℓ
40
46
_∙_ : Op₂ Carrier
41
47
42
- infix 4 _≉_
43
- _≉_ : Rel Carrier _
44
- x ≉ y = ¬ (x ≈ y)
48
+ rawSetoid : RawSetoid c ℓ
49
+ rawSetoid = record { _≈_ = _≈_ }
50
+
51
+ open RawSetoid rawSetoid public using (_≉_)
52
+
45
53
46
54
------------------------------------------------------------------------
47
55
-- Raw bundles with 1 binary operation & 1 element
You can’t perform that action at this time.
0 commit comments