Documentation

Mathlib.GroupTheory.Subsemigroup.Centralizer

Centralizers in semigroups, as subsemigroups. #

Main definitions #

We provide Monoid.centralizer, AddMonoid.centralizer, Subgroup.centralizer, and AddSubgroup.centralizer in other files.

The centralizer of a subset of a semigroup M.

Equations
Instances For

    The centralizer of a subset of an additive semigroup.

    Equations
    Instances For
      @[simp]
      theorem Subsemigroup.coe_centralizer {M : Type u_1} (S : Set M) [Semigroup M] :
      (Subsemigroup.centralizer S) = S.centralizer
      @[simp]
      theorem AddSubsemigroup.coe_centralizer {M : Type u_1} (S : Set M) [AddSemigroup M] :
      (AddSubsemigroup.centralizer S) = S.addCentralizer
      theorem Subsemigroup.mem_centralizer_iff {M : Type u_1} {S : Set M} [Semigroup M] {z : M} :
      z Subsemigroup.centralizer S gS, g * z = z * g
      theorem AddSubsemigroup.mem_centralizer_iff {M : Type u_1} {S : Set M} [AddSemigroup M] {z : M} :
      z AddSubsemigroup.centralizer S gS, g + z = z + g
      instance Subsemigroup.decidableMemCentralizer {M : Type u_1} {S : Set M} [Semigroup M] (a : M) [Decidable (∀ bS, b * a = a * b)] :
      Equations
      instance AddSubsemigroup.decidableMemCentralizer {M : Type u_1} {S : Set M} [AddSemigroup M] (a : M) [Decidable (∀ bS, b + a = a + b)] :
      Equations
      @[reducible, inline]
      abbrev Subsemigroup.closureCommSemigroupOfComm (M : Type u_1) [Semigroup M] {s : Set M} (hcomm : as, bs, a * b = b * a) :

      If all the elements of a set s commute, then closure s is a commutative semigroup.

      Equations
      Instances For
        @[reducible, inline]
        abbrev AddSubsemigroup.closureAddCommSemigroupOfComm (M : Type u_1) [AddSemigroup M] {s : Set M} (hcomm : as, bs, a + b = b + a) :

        If all the elements of a set s commute, then closure s forms an additive commutative semigroup.

        Equations
        Instances For