File tree Expand file tree Collapse file tree 2 files changed +8
-0
lines changed
Expand file tree Collapse file tree 2 files changed +8
-0
lines changed Original file line number Diff line number Diff 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 ⊥ ⊤
Original file line number Diff line number Diff line change @@ -50,6 +50,9 @@ Associative _∙_ = ∀ x y z → ((x ∙ y) ∙ z) ≈ (x ∙ (y ∙ z))
5050Commutative : Op₂ A → Set _
5151Commutative _∙_ = ∀ x y → (x ∙ y) ≈ (y ∙ x)
5252
53+ Central : Op₂ A → A → Set _
54+ Central _∙_ x = ∀ y → (x ∙ y) ≈ (y ∙ x)
55+
5356LeftIdentity : A → Op₂ A → Set _
5457LeftIdentity e _∙_ = ∀ x → (e ∙ x) ≈ x
5558
You can’t perform that action at this time.
0 commit comments