Skip to content

Commit 6630bd9

Browse files
Kleene algebra (#1730)
1 parent 01e94a5 commit 6630bd9

File tree

4 files changed

+81
-31
lines changed

4 files changed

+81
-31
lines changed

CHANGELOG.md

+4
Original file line numberDiff line numberDiff line change
@@ -892,6 +892,7 @@ Other minor changes
892892
record RawLoop c ℓ : Set (suc (c ⊔ ℓ))
893893
record Loop c ℓ : Set (suc (c ⊔ ℓ))
894894
record RingWithoutOne c ℓ : Set (suc (c ⊔ ℓ))
895+
record KleeneAlgebra c ℓ : Set (suc (c ⊔ ℓ))
895896
```
896897
and the existing record `Lattice` now provides
897898
```agda
@@ -937,6 +938,8 @@ Other minor changes
937938
InvertibleUnitalMagma (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
938939
quasigroup : Quasigroup a ℓ₁ → Quasigroup b ℓ₂ → Quasigroup (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
939940
loop : Loop a ℓ₁ → Loop b ℓ₂ → Loop (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
941+
kleeneAlgebra : KleeneAlgebra a ℓ₁ → KleeneAlgebra b ℓ₂ →
942+
KleeneAlgebra (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
940943
```
941944

942945
* Added new definition to `Algebra.Definitions`:
@@ -972,6 +975,7 @@ Other minor changes
972975
record IsQuasigroup (∙ \\ // : Op₂ A) : Set (a ⊔ ℓ)
973976
record IsLoop (∙ \\ // : Op₂ A) (ε : A) : Set (a ⊔ ℓ)
974977
record IsRingWithoutOne (+ * : Op₂ A) (-_ : Op₁ A) (0# : A) : Set (a ⊔ ℓ)
978+
record IsKleeneAlgebra (+ * : Op₂ A) (0# 1# : A) : Set (a ⊔ ℓ)
975979
```
976980
and the existing record `IsLattice` now provides
977981
```

src/Algebra/Bundles.agda

+30
Original file line numberDiff line numberDiff line change
@@ -750,6 +750,36 @@ record CancellativeCommutativeSemiring c ℓ : Set (suc (c ⊔ ℓ)) where
750750
; _≉_
751751
)
752752

753+
record KleeneAlgebra c ℓ : Set (suc (c ⊔ ℓ)) where
754+
infixl 7 _*_
755+
infixl 6 _+_
756+
infix 4 _≈_
757+
field
758+
Carrier : Set c
759+
_≈_ : Rel Carrier ℓ
760+
_+_ : Op₂ Carrier
761+
_*_ : Op₂ Carrier
762+
0# : Carrier
763+
1# : Carrier
764+
isKleeneAlgebra : IsKleeneAlgebra _≈_ _+_ _*_ 0# 1#
765+
766+
open IsKleeneAlgebra isKleeneAlgebra public
767+
768+
semiring : Semiring _ _
769+
semiring = record { isSemiring = isSemiring }
770+
771+
open Semiring semiring public
772+
using
773+
( _≉_; +-rawMagma; +-magma; +-unitalMagma; +-commutativeMagma
774+
; +-semigroup; +-commutativeSemigroup
775+
; *-rawMagma; *-magma; *-semigroup
776+
; +-rawMonoid; +-monoid; +-commutativeMonoid
777+
; *-rawMonoid; *-monoid
778+
; nearSemiring; semiringWithoutOne
779+
; semiringWithoutAnnihilatingZero
780+
; rawSemiring
781+
)
782+
753783
------------------------------------------------------------------------
754784
-- Bundles with 2 binary operations, 1 unary operation & 1 element
755785
------------------------------------------------------------------------

src/Algebra/Construct/DirectProduct.agda

+39-31
Original file line numberDiff line numberDiff line change
@@ -130,6 +130,16 @@ commutativeSemigroup G H = record
130130
}
131131
} where module G = CommutativeSemigroup G; module H = CommutativeSemigroup H
132132

133+
unitalMagma : UnitalMagma a ℓ₁ UnitalMagma b ℓ₂ UnitalMagma (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
134+
unitalMagma M N = record
135+
{ ε = M.ε , N.ε
136+
; isUnitalMagma = record
137+
{ isMagma = Magma.isMagma (magma M.magma N.magma)
138+
; identity = (M.identityˡ , N.identityˡ <*>_)
139+
, (M.identityʳ , N.identityʳ <*>_)
140+
}
141+
} where module M = UnitalMagma M; module N = UnitalMagma N
142+
133143
monoid : Monoid a ℓ₁ Monoid b ℓ₂ Monoid (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
134144
monoid M N = record
135145
{ ε = M.ε , N.ε
@@ -163,6 +173,27 @@ idempotentCommutativeMonoid M N = record
163173
module M = IdempotentCommutativeMonoid M
164174
module N = IdempotentCommutativeMonoid N
165175

176+
invertibleMagma : InvertibleMagma a ℓ₁ InvertibleMagma b ℓ₂ InvertibleMagma (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
177+
invertibleMagma M N = record
178+
{ _⁻¹ = map M._⁻¹ N._⁻¹
179+
; isInvertibleMagma = record
180+
{ isMagma = Magma.isMagma (magma M.magma N.magma)
181+
; inverse = (λ x (M.inverseˡ , N.inverseˡ) <*> x)
182+
, (λ x (M.inverseʳ , N.inverseʳ) <*> x)
183+
; ⁻¹-cong = map M.⁻¹-cong N.⁻¹-cong
184+
}
185+
} where module M = InvertibleMagma M; module N = InvertibleMagma N
186+
187+
invertibleUnitalMagma : InvertibleUnitalMagma a ℓ₁ InvertibleUnitalMagma b ℓ₂ InvertibleUnitalMagma (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
188+
invertibleUnitalMagma M N = record
189+
{ ε = M.ε , N.ε
190+
; isInvertibleUnitalMagma = record
191+
{ isInvertibleMagma = InvertibleMagma.isInvertibleMagma (invertibleMagma M.invertibleMagma N.invertibleMagma)
192+
; identity = (M.identityˡ , N.identityˡ <*>_)
193+
, (M.identityʳ , N.identityʳ <*>_)
194+
}
195+
} where module M = InvertibleUnitalMagma M; module N = InvertibleUnitalMagma N
196+
166197
group : Group a ℓ₁ Group b ℓ₂ Group (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
167198
group G H = record
168199
{ _⁻¹ = map G._⁻¹ H._⁻¹
@@ -225,6 +256,14 @@ commutativeSemiring R S = record
225256
}
226257
} where module R = CommutativeSemiring R; module S = CommutativeSemiring S
227258

259+
kleeneAlgebra : KleeneAlgebra a ℓ₁ KleeneAlgebra b ℓ₂ KleeneAlgebra (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
260+
kleeneAlgebra K L = record
261+
{ isKleeneAlgebra = record
262+
{ isSemiring = Semiring.isSemiring (semiring K.semiring L.semiring)
263+
; +-idem = λ x (K.+-idem , L.+-idem) <*> x
264+
}
265+
} where module K = KleeneAlgebra K; module L = KleeneAlgebra L
266+
228267
ring : Ring a ℓ₁ Ring b ℓ₂ Ring (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
229268
ring R S = record
230269
{ -_ = uncurry (λ x y R.-_ x , S.-_ y)
@@ -252,37 +291,6 @@ commutativeRing R S = record
252291
}
253292
} where module R = CommutativeRing R; module S = CommutativeRing S
254293

255-
unitalMagma : UnitalMagma a ℓ₁ UnitalMagma b ℓ₂ UnitalMagma (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
256-
unitalMagma M N = record
257-
{ ε = M.ε , N.ε
258-
; isUnitalMagma = record
259-
{ isMagma = Magma.isMagma (magma M.magma N.magma)
260-
; identity = (M.identityˡ , N.identityˡ <*>_)
261-
, (M.identityʳ , N.identityʳ <*>_)
262-
}
263-
} where module M = UnitalMagma M; module N = UnitalMagma N
264-
265-
invertibleMagma : InvertibleMagma a ℓ₁ InvertibleMagma b ℓ₂ InvertibleMagma (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
266-
invertibleMagma M N = record
267-
{ _⁻¹ = map M._⁻¹ N._⁻¹
268-
; isInvertibleMagma = record
269-
{ isMagma = Magma.isMagma (magma M.magma N.magma)
270-
; inverse = (λ x (M.inverseˡ , N.inverseˡ) <*> x)
271-
, (λ x (M.inverseʳ , N.inverseʳ) <*> x)
272-
; ⁻¹-cong = map M.⁻¹-cong N.⁻¹-cong
273-
}
274-
} where module M = InvertibleMagma M; module N = InvertibleMagma N
275-
276-
invertibleUnitalMagma : InvertibleUnitalMagma a ℓ₁ InvertibleUnitalMagma b ℓ₂ InvertibleUnitalMagma (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
277-
invertibleUnitalMagma M N = record
278-
{ ε = M.ε , N.ε
279-
; isInvertibleUnitalMagma = record
280-
{ isInvertibleMagma = InvertibleMagma.isInvertibleMagma (invertibleMagma M.invertibleMagma N.invertibleMagma)
281-
; identity = (M.identityˡ , N.identityˡ <*>_)
282-
, (M.identityʳ , N.identityʳ <*>_)
283-
}
284-
} where module M = InvertibleUnitalMagma M; module N = InvertibleUnitalMagma N
285-
286294
quasigroup : Quasigroup a ℓ₁ Quasigroup b ℓ₂ Quasigroup (a ⊔ b) (ℓ₁ ⊔ ℓ₂)
287295
quasigroup M N = record
288296
{ _\\_ = zip M._\\_ N._\\_

src/Algebra/Structures.agda

+8
Original file line numberDiff line numberDiff line change
@@ -496,6 +496,14 @@ record IsCancellativeCommutativeSemiring (+ * : Op₂ A) (0# 1# : A) : Set (a
496496

497497
open IsCommutativeSemiring isCommutativeSemiring public
498498

499+
500+
record IsKleeneAlgebra (+ * : Op₂ A) (0# 1# : A) : Set (a ⊔ ℓ) where
501+
field
502+
isSemiring : IsSemiring + * 0# 1#
503+
+-idem : Idempotent +
504+
505+
open IsSemiring isSemiring public
506+
499507
------------------------------------------------------------------------
500508
-- Structures with 2 binary operations, 1 unary operation & 1 element
501509
------------------------------------------------------------------------

0 commit comments

Comments
 (0)