Documentation

Mathlib.GroupTheory.Subsemigroup.Center

Centers of semigroups, as subsemigroups. #

Main definitions #

We provide Submonoid.center, AddSubmonoid.center, Subgroup.center, AddSubgroup.center, Subsemiring.center, and Subring.center in other files.

References #

Set.center as a Subsemigroup. #

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

Equations
Instances For

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

    Equations
    Instances For

      The center of a magma is commutative and associative.

      Equations
      Instances For

        The center of an additive magma is commutative and associative.

        Equations
        Instances For
          theorem Subsemigroup.mem_center_iff {M : Type u_1} [Semigroup M] {z : M} :
          Iff (Membership.mem (center M) z) (∀ (g : M), Eq (HMul.hMul g z) (HMul.hMul z g))
          theorem AddSubsemigroup.mem_center_iff {M : Type u_1} [AddSemigroup M] {z : M} :
          Iff (Membership.mem (center M) z) (∀ (g : M), Eq (HAdd.hAdd g z) (HAdd.hAdd z g))
          def Subsemigroup.decidableMemCenter {M : Type u_1} [Semigroup M] (a : M) [Decidable (∀ (b : M), Eq (HMul.hMul b a) (HMul.hMul a b))] :
          Equations
          Instances For
            def AddSubsemigroup.decidableMemCenter {M : Type u_1} [AddSemigroup M] (a : M) [Decidable (∀ (b : M), Eq (HAdd.hAdd b a) (HAdd.hAdd a b))] :
            Equations
            Instances For