Regular wreath product #
This file defines the regular wreath product of groups, and the canonical maps in and out of the
product. The regular wreath product of D
and Q
is the product (Q → D) × Q
with the group
operation ⟨a₁, a₂⟩ * ⟨b₁, b₂⟩ = ⟨a₁ * (fun x ↦ b₁ (a₂⁻¹ * x)), a₂ * b₂⟩
.
Main definitions #
RegularWreathProduct D Q
: The regular wreath product of groupsD
andQ
.rightHom
: The canonical projectionD ≀ᵣ Q →* Q
.inl
: The canonical mapQ →* D ≀ᵣ Q
.toPerm
: The homomorphism fromD ≀ᵣ Q
toEquiv.Perm (Λ × Q)
, whereΛ
is aD
-set.IteratedWreathProduct G n
: The iterated wreath product of a groupG
n
times.Sylow.mulEquivIteratedWreathProduct
: The isomorphism between the Sylowp
-subgroup ofPerm p^n
and the iterated wreath product of the cyclic group of orderp
n
times.
Notation #
This file introduces the global notation D ≀ᵣ Q
for RegularWreathProduct D Q
.
Tags #
group, regular wreath product, sylow p-subgroup
The regular wreath product of groups Q
and D
. It is the product (Q → D) × Q
with the group
operation ⟨a₁, a₂⟩ * ⟨b₁, b₂⟩ = ⟨a₁ * (fun x ↦ b₁ (a₂⁻¹ * x)), a₂ * b₂⟩
.
- left : Q → D
The function of Q → D
- right : Q
The element of Q
Instances For
The regular wreath product of groups Q
and D
. It is the product (Q → D) × Q
with the group
operation ⟨a₁, a₂⟩ * ⟨b₁, b₂⟩ = ⟨a₁ * (fun x ↦ b₁ (a₂⁻¹ * x)), a₂ * b₂⟩
.
Equations
- «term_≀ᵣ_» = Lean.ParserDescr.trailingNode `«term_≀ᵣ_» 65 66 (Lean.ParserDescr.binary `andthen (Lean.ParserDescr.symbol " ≀ᵣ ") (Lean.ParserDescr.cat `term 66))
Instances For
The canonical projection map D ≀ᵣ Q →* Q
, as a group hom.
Equations
- RegularWreathProduct.rightHom = { toFun := RegularWreathProduct.right, map_one' := ⋯, map_mul' := ⋯ }
Instances For
Define an isomorphism from D₁ ≀ᵣ Q₁
to D₂ ≀ᵣ Q₂
given isomorphisms D₁ ≀ᵣ Q₁
and Q₁ ≃* Q₂
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- RegularWreathProduct.instMulActionProd D Q Λ = { toSMul := RegularWreathProduct.instSMulProd D Q Λ, one_smul := ⋯, mul_smul := ⋯ }
The map sending the wreath product D ≀ᵣ Q
to its representation as a permutation of Λ × Q
given D
-set Λ
.
Equations
- RegularWreathProduct.toPerm D Q Λ = MulAction.toPermHom (D ≀ᵣ Q) (Λ × Q)
Instances For
The wreath product of group G
iterated n
times.
Equations
Instances For
Equations
- instGroupIteratedWreathProduct G n = Nat.recAux (⋯.mpr inferInstance) (fun (n : ℕ) (ih : Group (IteratedWreathProduct G n)) => ⋯.mpr inferInstance) n
The homomorphism from IteratedWreathProduct G n
to Perm (Fin n → G)
.
Equations
- iteratedWreathToPermHom G 0 = 1
- iteratedWreathToPermHom G n.succ = (Equiv.Perm.permCongrHom (Fin.succFunEquiv G n).symm).toMonoidHom.comp (RegularWreathProduct.toPerm (IteratedWreathProduct G n) G (Fin n → G))
Instances For
The encoding of the Sylow p
-subgroups of Perm α
as an iterated wreath product.
Equations
- One or more equations did not get rendered due to their size.