Complements #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define the complement of a subgroup.
Main definitions #
is_complement S T
whereS
andT
are subsets ofG
states that everyg : G
can be written uniquely as a products * t
fors ∈ S
,t ∈ T
.left_transversals T
whereT
is a subset ofG
is the set of all left-complements ofT
, i.e. the set of allS : set G
that contain exactly one element of each left coset ofT
.right_transversals S
whereS
is a subset ofG
is the set of all right-complements ofS
, i.e. the set of allT : set G
that contain exactly one element of each right coset ofS
.transfer_transversal H g
is a specificleft_transversal
ofH
that is used in the computation of the transfer homomorphism evaluated at an elementg : G
.
Main results #
is_complement_of_coprime
: Subgroups of coprime order are complements.
S
and T
are complements if (*) : S × T → G
is a bijection.
This notion generalizes left transversals, right transversals, and complementary subgroups.
H
and K
are complements if (*) : H × K → G
is a bijection
H
and K
are complements if (*) : H × K → G
is a bijection
The set of left-complements of T : set G
Equations
- add_subgroup.left_transversals T = {S : set G | add_subgroup.is_complement S T}
Instances for ↥add_subgroup.left_transversals
The set of left-complements of T : set G
Equations
- subgroup.left_transversals T = {S : set G | subgroup.is_complement S T}
Instances for ↥subgroup.left_transversals
The set of right-complements of S : set G
Equations
- subgroup.right_transversals S = {T : set G | subgroup.is_complement S T}
Instances for ↥subgroup.right_transversals
The set of right-complements of S : set G
Equations
- add_subgroup.right_transversals S = {T : set G | add_subgroup.is_complement S T}
Instances for ↥add_subgroup.right_transversals
A left transversal is in bijection with left cosets.
Equations
A left transversal is in bijection with left cosets.
Equations
A left transversal can be viewed as a function mapping each element of the group to the chosen representative from that left coset.
A left transversal can be viewed as a function mapping each element of the group to the chosen representative from that left coset.
A right transversal is in bijection with right cosets.
Equations
A right transversal is in bijection with right cosets.
Equations
A right transversal can be viewed as a function mapping each element of the group to the chosen representative from that right coset.
A right transversal can be viewed as a function mapping each element of the group to the chosen representative from that right coset.
Equations
- add_subgroup.left_transversals.add_action = {to_has_vadd := {vadd := λ (f : F) (T : ↥(add_subgroup.left_transversals ↑H)), ⟨f +ᵥ ↑T, _⟩}, zero_vadd := _, add_vadd := _}
Equations
- subgroup.left_transversals.mul_action = {to_has_smul := {smul := λ (f : F) (T : ↥(subgroup.left_transversals ↑H)), ⟨f • ↑T, _⟩}, one_smul := _, mul_smul := _}
Equations
Equations
Equations
Equations
Partition G ⧸ H
into orbits of the action of g : G
.
Equations
- H.quotient_equiv_sigma_zmod g = (mul_action.self_equiv_sigma_orbits ↥(subgroup.zpowers g) (G ⧸ H)).trans (equiv.sigma_congr_right (λ (q : mul_action.orbit_rel.quotient ↥(subgroup.zpowers g) (G ⧸ H)), mul_action.orbit_zpowers_equiv g (quotient.out' q)))
The transfer transversal as a function. Given a ⟨g⟩
-orbit q₀, g • q₀, ..., g ^ (m - 1) • q₀
in G ⧸ H
, an element g ^ k • q₀
is mapped to g ^ k • g₀
for a fixed choice of
representative g₀
of q₀
.
Equations
- H.transfer_function g = λ (q : G ⧸ H), g ^ ↑((⇑(H.quotient_equiv_sigma_zmod g) q).snd) * quotient.out' (quotient.out' (⇑(H.quotient_equiv_sigma_zmod g) q).fst)
The transfer transversal as a set. Contains elements of the form g ^ k • g₀
for fixed choices
of representatives g₀
of fixed choices of representatives q₀
of ⟨g⟩
-orbits in G ⧸ H
.
Equations
- H.transfer_set g = set.range (H.transfer_function g)
The transfer transversal. Contains elements of the form g ^ k • g₀
for fixed choices
of representatives g₀
of fixed choices of representatives q₀
of ⟨g⟩
-orbits in G ⧸ H
.
Equations
- H.transfer_transversal g = ⟨H.transfer_set g, _⟩