mathlib3 documentation

group_theory.subsemigroup.center

Centers of magmas and semigroups #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

Main definitions #

We provide submonoid.center, add_submonoid.center, subgroup.center, add_subgroup.center, subsemiring.center, and subring.center in other files.

def set.center (M : Type u_1) [has_mul M] :
set M

The center of a magma.

Equations
def set.add_center (M : Type u_1) [has_add M] :
set M

The center of an additive magma.

Equations
theorem set.mem_add_center (M : Type u_1) [has_add M] {z : M} :
z set.add_center M (g : M), g + z = z + g
theorem set.mem_center_iff (M : Type u_1) [has_mul M] {z : M} :
z set.center M (g : M), g * z = z * g
@[protected, instance]
def set.decidable_mem_center (M : Type u_1) [has_mul M] [Π (a : M), decidable ( (b : M), b * a = a * b)] :
decidable_pred (λ (_x : M), _x set.center M)
Equations
@[simp]
@[simp]
theorem set.one_mem_center (M : Type u_1) [mul_one_class M] :
@[simp]
theorem set.zero_mem_center (M : Type u_1) [mul_zero_class M] :
@[simp]
theorem set.mul_mem_center {M : Type u_1} [semigroup M] {a b : M} (ha : a set.center M) (hb : b set.center M) :
@[simp]
theorem set.add_mem_add_center {M : Type u_1} [add_semigroup M] {a b : M} (ha : a set.add_center M) (hb : b set.add_center M) :
@[simp]
theorem set.inv_mem_center {M : Type u_1} [group M] {a : M} (ha : a set.center M) :
@[simp]
theorem set.neg_mem_add_center {M : Type u_1} [add_group M] {a : M} (ha : a set.add_center M) :
@[simp]
theorem set.add_mem_center {M : Type u_1} [distrib M] {a b : M} (ha : a set.center M) (hb : b set.center M) :
@[simp]
theorem set.neg_mem_center {M : Type u_1} [ring M] {a : M} (ha : a set.center M) :

In a group with zero, the center of the units is the preimage of the center.

@[simp]
theorem set.inv_mem_center₀ {M : Type u_1} [group_with_zero M] {a : M} (ha : a set.center M) :
@[simp]
theorem set.div_mem_center {M : Type u_1} [group M] {a b : M} (ha : a set.center M) (hb : b set.center M) :
@[simp]
theorem set.sub_mem_add_center {M : Type u_1} [add_group M] {a b : M} (ha : a set.add_center M) (hb : b set.add_center M) :
@[simp]
theorem set.div_mem_center₀ {M : Type u_1} [group_with_zero M] {a b : M} (ha : a set.center M) (hb : b set.center M) :
@[simp]

The center of a semigroup M is the set of elements that commute with everything in M

Equations
Instances for subsemigroup.center

The center of a semigroup M is the set of elements that commute with everything in M

Equations
Instances for add_subsemigroup.center
theorem subsemigroup.mem_center_iff {M : Type u_1} [semigroup M] {z : M} :
z subsemigroup.center M (g : M), g * z = z * g
theorem add_subsemigroup.mem_center_iff {M : Type u_1} [add_semigroup M] {z : M} :
z add_subsemigroup.center M (g : M), g + z = z + g
@[protected, instance]
def subsemigroup.decidable_mem_center {M : Type u_1} [semigroup M] (a : M) [decidable ( (b : M), b * a = a * b)] :
Equations
@[protected, instance]

The center of a semigroup is commutative.

Equations