Subspace of invariants a group representation #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file introduces the subspace of invariants of a group representation
and proves basic results about it.
The main tool used is the average of all elements of the group, seen as an element of
monoid_algebra k G
. The action of this special element gives a projection onto the
subspace of invariants.
In order for the definition of the average element to make sense, we need to assume for most of the
results that the order of G
is invertible in k
(e. g. k
has characteristic 0
).
The average of all elements of the group G
, considered as an element of monoid_algebra k G
.
Equations
- group_algebra.average k G = ⅟ ↑(fintype.card G) • finset.univ.sum (λ (g : G), ⇑(monoid_algebra.of k G) g)
average k G
is invariant under left multiplication by elements of G
.
average k G
is invariant under right multiplication by elements of G
.
The subspace of invariants, consisting of the vectors fixed by all elements of G
.
The action of average k G
gives a projection map onto the subspace of invariants.
Equations
- ρ.average_map = ⇑(ρ.as_algebra_hom) (group_algebra.average k G)
The average_map
sends elements of V
to the subspace of invariants.
The average_map
acts as the identity on the subspace of invariants.
The invariants of the representation lin_hom X.ρ Y.ρ
correspond to the the representation
homomorphisms from X
to Y
Equations
- representation.lin_hom.invariants_equiv_fdRep_hom X Y = _.mpr (_.mpr ((representation.lin_hom.invariants_equiv_Rep_hom ((category_theory.forget₂ (fdRep k ↥G) (Rep k ↥G)).obj X) ((category_theory.forget₂ (fdRep k ↥G) (Rep k ↥G)).obj Y)).trans (X.forget₂_hom_linear_equiv Y)))