(Co)induced representations of a finite index subgroup #
Given a commutative ring k
, a finite index subgroup S ≤ G
, and a k
-linear S
-representation
A
, this file defines an isomorphism $Ind_S^G(A) ≅ Coind_S^G(A)$. Given g : G
and a : A
, the
forward map sends ⟦g ⊗ₜ[k] a⟧
to the function G → A
supported at sg
by ρ(s)(a)
for s : S
and which is 0 elsewhere. Meanwhile, the inverse sends f : G → A
to ∑ᵢ ⟦gᵢ ⊗ₜ[k] f(gᵢ)⟧
for
1 ≤ i ≤ n
, where g₁, ..., gₙ
is a set of right coset representatives of S
.
Main definitions #
Rep.indCoindIso A
: An isomorphismInd_S^G(A) ≅ Coind_S^G(A)
for a finite index subgroupS ≤ G
and ak
-linearS
-representationA
.Rep.indCoindNatIso k S
: A natural isomorphism between the functorsInd_S^G
andCoind_S^G
.
TODO #
- Add Shapiro's lemma, using this isomorphism.
Let S ≤ G
be a subgroup and (A, ρ)
a k
-linear S
-representation. Then given g : G
and
a : A
, this is the function G → A
sending sg
to ρ(s)(a)
for all s : S
and everything else
to 0.
Equations
- A.indToCoindAux g = LinearMap.pi fun (g₁ : G) => if h : (QuotientGroup.rightRel S) g₁ g then A.ρ ⟨g₁ * g⁻¹, ⋯⟩ else 0
Instances For
Let S ≤ G
be a subgroup and A
a k
-linear S
-representation. This is the k
-linear map
Ind_S^G(A) →ₗ[k] Coind_S^G(A)
sending (⟦g ⊗ₜ[k] a⟧, sg) ↦ ρ(s)(a)
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Let S ≤ G
be a finite index subgroup, g₁, ..., gₙ
a set of right coset representatives of
S
, and A
a k
-linear S
-representation. This is the k
-linear map
Coind_S^G(A) →ₗ[k] Ind_S^G(A)
sending f : G → A
to ∑ᵢ ⟦gᵢ ⊗ₜ[k] f(gᵢ)⟧
for 1 ≤ i ≤ n
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Let S ≤ G
be a finite index subgroup, g₁, ..., gₙ
a set of right coset representatives of
S
, and A
a k
-linear S
-representation. This is an isomorphism Ind_S^G(A) ≅ Coind_S^G(A)
.
The forward map sends (⟦g ⊗ₜ[k] a⟧, sg) ↦ ρ(s)(a)
, and the inverse sends f : G → A
to
∑ᵢ ⟦gᵢ ⊗ₜ[k] f(gᵢ)⟧
for 1 ≤ i ≤ n
.
Equations
- A.indCoindIso = Action.mkIso { hom := ModuleCat.ofHom A.indToCoind, inv := ModuleCat.ofHom A.coindToInd, hom_inv_id := ⋯, inv_hom_id := ⋯ } ⋯
Instances For
Given a finite index subgroup S ≤ G
, this is a natural isomorphism between the Ind_S^G
and
Coind_G^S
functors Rep k S ⥤ Rep k G
.
Equations
- Rep.indCoindNatIso k S = CategoryTheory.NatIso.ofComponents (fun (x : Rep k ↥S) => x.indCoindIso) ⋯
Instances For
Given a finite index subgroup S ≤ G
, Ind_S^G
is right adjoint to the restriction functor
Res k G ⥤ Res k S
, since it is naturally isomorphic to Coind_S^G
.
Equations
- Rep.resIndAdjunction k S = (Rep.resCoindAdjunction k S.subtype).ofNatIsoRight (Rep.indCoindNatIso k S).symm
Instances For
Given a finite index subgroup S ≤ G
, Coind_S^G
is left adjoint to the restriction functor
Res k G ⥤ Res k S
, since it is naturally isomorphic to Ind_S^G
.
Equations
- Rep.coindResAdjunction k S = (Rep.indResAdjunction k S.subtype).ofNatIsoLeft (Rep.indCoindNatIso k S)