fdRep k G
is the category of finite dimensional k
-linear representations of G
. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
If V : fdRep k G
, there is a coercion that allows you to treat V
as a type,
and this type comes equipped with module k V
and finite_dimensional k V
instances.
Also V.ρ
gives the homomorphism G →* (V →ₗ[k] V)
.
Conversely, given a homomorphism ρ : G →* (V →ₗ[k] V)
,
you can construct the bundled representation as Rep.of ρ
.
We verify that fdRep k G
is a k
-linear monoidal category, and rigid when G
is a group.
fdRep k G
has all finite limits.
TODO #
fdRep k G ≌ full_subcategory (finite_dimensional k)
- Upgrade the right rigid structure to a rigid structure
(this just needs to be done for
fgModule
). fdRep k G
has all finite colimits.fdRep k G
is abelian.fdRep k G ≌ fgModule (monoid_algebra k G)
.
Equations
Equations
- V.add_comm_group = id ((category_theory.forget₂ (fdRep k G) (fgModule k)).obj V).obj.is_add_comm_group
All hom spaces are finite dimensional.
The underlying linear_equiv
of an isomorphism of representations.
Equations
- fdRep.iso_to_linear_equiv i = fgModule.iso_to_linear_equiv ((Action.forget (fgModule k) (Mon.of G)).map_iso i)
Lift an unbundled representation to fdRep
.
Equations
- fdRep.Rep.category_theory.has_forget₂ = {forget₂ := (category_theory.forget₂ (fgModule k) (Module k)).map_Action (Mon.of G), forget_comp := _}
The forgetful functor to Rep k G
preserves hom-sets and their vector space structure
Equations
- X.forget₂_hom_linear_equiv Y = {to_fun := λ (f : (category_theory.forget₂ (fdRep k G) (Rep k G)).obj X ⟶ (category_theory.forget₂ (fdRep k G) (Rep k G)).obj Y), {hom := f.hom, comm' := _}, map_add' := _, map_smul' := _, inv_fun := λ (f : X ⟶ Y), {hom := (category_theory.forget₂ (fgModule k) (Module k)).map f.hom, comm' := _}, left_inv := _, right_inv := _}
Auxiliary definition for fdRep.dual_tensor_iso_lin_hom
.
Equations
When V
and W
are finite dimensional representations of a group G
, the isomorphism
dual_tensor_hom_equiv k V W
of vector spaces induces an isomorphism of representations.