Skip to content

Commit 429e617

Browse files
authored
\[ refactor \] add rawSetoid fields to Algebra.Bundles.Raw (#2536)
1 parent b429588 commit 429e617

File tree

2 files changed

+16
-3
lines changed

2 files changed

+16
-3
lines changed

CHANGELOG.md

+5
Original file line numberDiff line numberDiff line change
@@ -183,6 +183,11 @@ Additions to existing modules
183183
rawKleeneAlgebra : RawKleeneAlgebra _ _
184184
```
185185

186+
* In `Algebra.Bundles.Raw.*`
187+
```agda
188+
rawSetoid : RawSetoid c ℓ
189+
```
190+
186191
* In `Algebra.Bundles.Raw.RawRingWithoutOne`
187192
```agda
188193
rawNearSemiring : RawNearSemiring c ℓ

src/Algebra/Bundles/Raw.agda

+11-3
Original file line numberDiff line numberDiff line change
@@ -10,6 +10,7 @@ module Algebra.Bundles.Raw where
1010

1111
open import Algebra.Core
1212
open import Relation.Binary.Core using (Rel)
13+
open import Relation.Binary.Bundles.Raw using (RawSetoid)
1314
open import Level using (suc; _⊔_)
1415
open import Relation.Nullary.Negation.Core using (¬_)
1516

@@ -27,6 +28,11 @@ record RawSuccessorSet c ℓ : Set (suc (c ⊔ ℓ)) where
2728
suc# : Op₁ Carrier
2829
zero# : Carrier
2930

31+
rawSetoid : RawSetoid c ℓ
32+
rawSetoid = record { _≈_ = _≈_ }
33+
34+
open RawSetoid rawSetoid public using (_≉_)
35+
3036
------------------------------------------------------------------------
3137
-- Raw bundles with 1 binary operation
3238
------------------------------------------------------------------------
@@ -39,9 +45,11 @@ record RawMagma c ℓ : Set (suc (c ⊔ ℓ)) where
3945
_≈_ : Rel Carrier ℓ
4046
_∙_ : Op₂ Carrier
4147

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

4654
------------------------------------------------------------------------
4755
-- Raw bundles with 1 binary operation & 1 element

0 commit comments

Comments
 (0)