Centers of subgroups #
The center of a group G
is the set of elements that commute with everything in G
Equations
- Subgroup.center G = { carrier := Set.center G, mul_mem' := ⋯, one_mem' := ⋯, inv_mem' := ⋯ }
Instances For
The center of an additive group G
is the set of elements that commute with
everything in G
Equations
- AddSubgroup.center G = { carrier := Set.addCenter G, add_mem' := ⋯, zero_mem' := ⋯, neg_mem' := ⋯ }
Instances For
@[simp]
@[simp]
@[simp]
theorem
Subgroup.centerCongr_symm_apply_coe
{G : Type u_1}
[Group G]
{H : Type u_2}
[Group H]
(e : G ≃* H)
(s : ↥(Subsemigroup.center H))
:
@[simp]
theorem
AddSubgroup.centerCongr_symm_apply_coe
{G : Type u_1}
[AddGroup G]
{H : Type u_2}
[AddGroup H]
(e : G ≃+ H)
(s : ↥(AddSubsemigroup.center H))
:
@[simp]
theorem
AddSubgroup.centerCongr_apply_coe
{G : Type u_1}
[AddGroup G]
{H : Type u_2}
[AddGroup H]
(e : G ≃+ H)
(r : ↥(AddSubsemigroup.center G))
:
@[simp]
theorem
Subgroup.centerCongr_apply_coe
{G : Type u_1}
[Group G]
{H : Type u_2}
[Group H]
(e : G ≃* H)
(r : ↥(Subsemigroup.center G))
:
The center of a group is isomorphic to the center of its opposite.
Instances For
The center of an additive group is isomorphic to the center of its opposite.
Instances For
@[simp]
theorem
Subgroup.centerToMulOpposite_symm_apply_coe
(G : Type u_1)
[Group G]
(r : ↥(Subsemigroup.center Gᵐᵒᵖ))
:
@[simp]
theorem
AddSubgroup.centerToAddOpposite_apply_coe
(G : Type u_1)
[AddGroup G]
(r : ↥(AddSubsemigroup.center G))
:
@[simp]
theorem
AddSubgroup.centerToAddOpposite_symm_apply_coe
(G : Type u_1)
[AddGroup G]
(r : ↥(AddSubsemigroup.center Gᵃᵒᵖ))
:
@[simp]
theorem
Subgroup.centerToMulOpposite_apply_coe
(G : Type u_1)
[Group G]
(r : ↥(Subsemigroup.center G))
:
For a group with zero, the center of the units is the same as the units of the center.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
theorem
Subgroup.val_centerUnitsEquivUnitsCenter_apply_coe
(G₀ : Type u_2)
[GroupWithZero G₀]
(a : ↥(center G₀ˣ))
:
@[simp]
theorem
Subgroup.val_centerUnitsEquivUnitsCenter_symm_apply_coe
(G₀ : Type u_2)
[GroupWithZero G₀]
(u : (↥(Submonoid.center G₀))ˣ)
:
A group is commutative if the center is the whole group
Equations
Instances For
theorem
IsConj.eq_of_left_mem_center
{M : Type u_2}
[Monoid M]
{g h : M}
(H : IsConj g h)
(Hg : g ∈ Set.center M)
:
theorem
IsConj.eq_of_right_mem_center
{M : Type u_2}
[Monoid M]
{g h : M}
(H : IsConj g h)
(Hh : h ∈ Set.center M)
:
theorem
ConjClasses.mk_bijOn
(G : Type u_2)
[Group G]
:
Set.BijOn ConjClasses.mk (↑(Subgroup.center G)) (noncenter G)ᶜ