Documentation

Mathlib.GroupTheory.Subgroup.Zpowers

Subgroups generated by an element #

Tags #

subgroup, subgroups

def Subgroup.zpowers {G : Type u_1} [inst : Group G] (g : G) :

The subgroup generated by an element.

Equations
  • One or more equations did not get rendered due to their size.
@[simp]
theorem Subgroup.mem_zpowers {G : Type u_1} [inst : Group G] (g : G) :
@[simp]
theorem Subgroup.range_zpowersHom {G : Type u_1} [inst : Group G] (g : G) :
theorem Subgroup.zpowers_subset {G : Type u_1} [inst : Group G] {a : G} {K : Subgroup G} (h : a K) :
theorem Subgroup.mem_zpowers_iff {G : Type u_1} [inst : Group G] {g : G} {h : G} :
h Subgroup.zpowers g k, g ^ k = h
@[simp]
theorem Subgroup.zpow_mem_zpowers {G : Type u_1} [inst : Group G] (g : G) (k : ) :
@[simp]
theorem Subgroup.npow_mem_zpowers {G : Type u_1} [inst : Group G] (g : G) (k : ) :
@[simp]
theorem Subgroup.forall_zpowers {G : Type u_1} [inst : Group G] {x : G} {p : { x // x Subgroup.zpowers x }Prop} :
((g : { x // x Subgroup.zpowers x }) → p g) (m : ) → p { val := x ^ m, property := (_ : y, (fun x x_1 => x ^ x_1) x y = x ^ m) }
@[simp]
theorem Subgroup.exists_zpowers {G : Type u_1} [inst : Group G] {x : G} {p : { x // x Subgroup.zpowers x }Prop} :
(g, p g) m, p { val := x ^ m, property := (_ : y, (fun x x_1 => x ^ x_1) x y = x ^ m) }
theorem Subgroup.forall_mem_zpowers {G : Type u_1} [inst : Group G] {x : G} {p : GProp} :
((g : G) → g Subgroup.zpowers xp g) (m : ) → p (x ^ m)
theorem Subgroup.exists_mem_zpowers {G : Type u_1} [inst : Group G] {x : G} {p : GProp} :
(g, g Subgroup.zpowers x p g) m, p (x ^ m)
def AddSubgroup.zmultiples {A : Type u_1} [inst : AddGroup A] (a : A) :

The subgroup generated by an element.

Equations
@[simp]
theorem AddSubgroup.mem_zmultiples {G : Type u_1} [inst : AddGroup G] (g : G) :
abbrev AddSubgroup.zmultiples_subset.match_1 {G : Type u_1} [inst : AddGroup G] {a : G} (motive : (x : G) → x AddSubgroup.zmultiples aProp) :
(x : G) → (hx : x AddSubgroup.zmultiples a) → ((i : ) → motive ((fun x x_1 => x_1 x) a i) (_ : y, (fun x x_1 => x_1 x) a y = (fun x x_1 => x_1 x) a i)) → motive x hx
Equations
  • One or more equations did not get rendered due to their size.
theorem AddSubgroup.zmultiples_subset {G : Type u_1} [inst : AddGroup G] {a : G} {K : AddSubgroup G} (h : a K) :
theorem AddSubgroup.mem_zmultiples_iff {G : Type u_1} [inst : AddGroup G] {g : G} {h : G} :
@[simp]
theorem AddSubgroup.zsmul_mem_zmultiples {G : Type u_1} [inst : AddGroup G] (g : G) (k : ) :
@[simp]
theorem AddSubgroup.nsmul_mem_zmultiples {G : Type u_1} [inst : AddGroup G] (g : G) (k : ) :
@[simp]
theorem AddSubgroup.forall_zmultiples {G : Type u_1} [inst : AddGroup G] {x : G} {p : { x // x AddSubgroup.zmultiples x }Prop} :
((g : { x // x AddSubgroup.zmultiples x }) → p g) (m : ) → p { val := m x, property := (_ : y, (fun x x_1 => x_1 x) x y = m x) }
theorem AddSubgroup.forall_mem_zmultiples {G : Type u_1} [inst : AddGroup G] {x : G} {p : GProp} :
((g : G) → g AddSubgroup.zmultiples xp g) (m : ) → p (m x)
@[simp]
theorem AddSubgroup.exists_zmultiples {G : Type u_1} [inst : AddGroup G] {x : G} {p : { x // x AddSubgroup.zmultiples x }Prop} :
(g, p g) m, p { val := m x, property := (_ : y, (fun x x_1 => x_1 x) x y = m x) }
theorem AddSubgroup.exists_mem_zmultiples {G : Type u_1} [inst : AddGroup G] {x : G} {p : GProp} :
(g, g AddSubgroup.zmultiples x p g) m, p (m x)
@[simp]
theorem AddSubgroup.int_cast_mul_mem_zmultiples {R : Type u_1} [inst : Ring R] (r : R) (k : ) :
@[simp]
@[simp]
theorem AddMonoidHom.map_zmultiples {G : Type u_1} [inst : AddGroup G] {N : Type u_2} [inst : AddGroup N] (f : G →+ N) (x : G) :
@[simp]
theorem MonoidHom.map_zpowers {G : Type u_1} [inst : Group G] {N : Type u_2} [inst : Group N] (f : G →* N) (x : G) :
theorem ofMul_image_zpowers_eq_zmultiples_ofMul {G : Type u_1} [inst : Group G] {x : G} :
Additive.ofMul '' ↑(Subgroup.zpowers x) = ↑(AddSubgroup.zmultiples (Additive.ofMul x))
theorem ofAdd_image_zmultiples_eq_zpowers_ofAdd {A : Type u_1} [inst : AddGroup A] {x : A} :
Multiplicative.ofAdd '' ↑(AddSubgroup.zmultiples x) = ↑(Subgroup.zpowers (Multiplicative.ofAdd x))
abbrev AddSubgroup.zmultiples_isCommutative.match_1 {G : Type u_1} [inst : AddGroup G] (g : G) (motive : { x // x AddSubgroup.zmultiples g }Prop) :
(x : { x // x AddSubgroup.zmultiples g }) → ((val : G) → (w : ) → (h₂ : (fun x x_1 => x_1 x) g w = val) → motive { val := val, property := (_ : y, (fun x x_1 => x_1 x) g y = val) }) → motive x
Equations
@[simp]
theorem AddSubgroup.zmultiples_le {G : Type u_1} [inst : AddGroup G] {g : G} {H : AddSubgroup G} :
@[simp]
theorem Subgroup.zpowers_le {G : Type u_1} [inst : Group G] {g : G} {H : Subgroup G} :
@[simp]
theorem AddSubgroup.zmultiples_eq_bot {G : Type u_1} [inst : AddGroup G] {g : G} :
@[simp]
theorem Subgroup.zpowers_eq_bot {G : Type u_1} [inst : Group G] {g : G} :
@[simp]