Rep k G
is the category of k
-linear representations of G
. #
If V : Rep k G
, there is a coercion that allows you to treat V
as a type,
and this type comes equipped with a Module k V
instance.
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 construct the categorical equivalence Rep k G ≌ ModuleCat (MonoidAlgebra k G)
.
We verify that Rep k G
is a k
-linear abelian symmetric monoidal category with all (co)limits.
Specialize the existing Action.ρ
, changing the type to Representation k G V
.
Instances For
Allows us to apply lemmas about the underlying ρ
, which would take an element g : G
rather
than g : MonCat.of G
as an argument.
The trivial k
-linear G
-representation on a k
-module V.
Instances For
The linearization of a type X
on which G
acts trivially is the trivial G
-representation
on k[X]
.
Instances For
The linearization of a type H
with a G
-action is definitionally isomorphic to the
k
-linear G
-representation on k[H]
induced by the G
-action on H
.
Instances For
Given an element x : A
, there is a natural morphism of representations k[G] ⟶ A
sending
g ↦ A.ρ(g)(x).
Instances For
Given a k
-linear G
-representation A
, there is a k
-linear isomorphism between
representation morphisms Hom(k[G], A)
and A
.
Instances For
Given a k
-linear G
-representation (A, ρ₁)
, this is the 'internal Hom' functor sending
(B, ρ₂)
to the representation Homₖ(A, B)
that maps g : G
and f : A →ₗ[k] B
to
(ρ₂ g) ∘ₗ f ∘ₗ (ρ₁ g⁻¹)
.
Instances For
Given a k
-linear G
-representation A
, this is the Hom-set bijection in the adjunction
A ⊗ - ⊣ ihom(A, -)
. It sends f : A ⊗ B ⟶ C
to a Rep k G
morphism defined by currying the
k
-linear map underlying f
, giving a map A →ₗ[k] B →ₗ[k] C
, then flipping the arguments.
Instances For
Porting note: if we generate this with @[simps]
the linter complains some types in the LHS
simplify.
Porting note: if we generate this with @[simps]
the linter complains some types in the LHS
simplify.
There is a k
-linear isomorphism between the sets of representation morphismsHom(A ⊗ B, C)
and Hom(B, Homₖ(A, C))
.
Instances For
There is a k
-linear isomorphism between the sets of representation morphismsHom(A ⊗ B, C)
and Hom(A, Homₖ(B, C))
.
Instances For
Tautological isomorphism to help Lean in typechecking.
Instances For
Auxiliary lemma for toModuleMonoidAlgebra
.
Auxiliary definition for toModuleMonoidAlgebra
.
Instances For
Functorially convert a representation of G
into a module over MonoidAlgebra k G
.
Instances For
Functorially convert a module over MonoidAlgebra k G
into a representation of G
.
Instances For
Auxiliary definition for equivalenceModuleMonoidAlgebra
.
Instances For
Auxiliary definition for equivalenceModuleMonoidAlgebra
.
Instances For
Auxiliary definition for equivalenceModuleMonoidAlgebra
.
Instances For
Auxiliary definition for equivalenceModuleMonoidAlgebra
.