Skip to content

Commit cbfc19e

Browse files
committed
add: Algebra.Definitions.Central
1 parent 38f22ec commit cbfc19e

File tree

2 files changed

+8
-0
lines changed

2 files changed

+8
-0
lines changed

CHANGELOG.md

Lines changed: 5 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -126,6 +126,11 @@ Additions to existing modules
126126
∀ w x y z → ((w ∙ x) ◦ (y ∙ z)) ≈ ((((w ◦ y) ∙ (w ◦ z)) ∙ (x ◦ y)) ∙ (x ◦ z))
127127
```
128128

129+
* In `Algebra.Definitions`:
130+
```agda
131+
Central : Op₂ A → A → Set _
132+
```
133+
129134
* In `Algebra.Lattice.Properties.BooleanAlgebra.XorRing`:
130135
```agda
131136
⊕-∧-isBooleanRing : IsBooleanRing _⊕_ _∧_ id ⊥ ⊤

src/Algebra/Definitions.agda

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -50,6 +50,9 @@ Associative _∙_ = ∀ x y z → ((x ∙ y) ∙ z) ≈ (x ∙ (y ∙ z))
5050
Commutative : Op₂ A Set _
5151
Commutative _∙_ = x y (x ∙ y) ≈ (y ∙ x)
5252

53+
Central : Op₂ A A Set _
54+
Central _∙_ x = y (x ∙ y) ≈ (y ∙ x)
55+
5356
LeftIdentity : A Op₂ A Set _
5457
LeftIdentity e _∙_ = x (e ∙ x) ≈ x
5558

0 commit comments

Comments
 (0)