mathlib3 documentation

representation_theory.group_cohomology.resolution

The structure of the k[G]-module k[Gⁿ] #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file contains facts about an important k[G]-module structure on k[Gⁿ], where k is a commutative ring and G is a group. The module structure arises from the representation G →* End(k[Gⁿ]) induced by the diagonal action of G on Gⁿ.

In particular, we define an isomorphism of k-linear G-representations between k[Gⁿ⁺¹] and k[G] ⊗ₖ k[Gⁿ] (on which G acts by ρ(g₁)(g₂ ⊗ x) = (g₁ * g₂) ⊗ x).

This allows us to define a k[G]-basis on k[Gⁿ⁺¹], by mapping the natural k[G]-basis of k[G] ⊗ₖ k[Gⁿ] along the isomorphism.

We then define the standard resolution of k as a trivial representation, by taking the alternating face map complex associated to an appropriate simplicial k-linear G-representation. This simplicial object is the linearization of the simplicial G-set given by the universal cover of the classifying space of G, EG. We prove this simplicial G-set EG is isomorphic to the Čech nerve of the natural arrow of G-sets G ⟶ {pt}.

We then use this isomorphism to deduce that as a complex of k-modules, the standard resolution of k as a trivial G-representation is homotopy equivalent to the complex with k at 0 and 0 elsewhere.

Putting this material together allows us to define group_cohomology.ProjectiveResolution, the standard projective resolution of k as a trivial k-linear G-representation.

Main definitions #

Implementation notes #

We express k[G]-module structures on a module k-module V using the representation definition. We avoid using instances module (G →₀ k) V so that we do not run into possible scalar action diamonds.

We also use the category theory library to bundle the type k[Gⁿ] - or more generally k[H] when H has G-action - and the representation together, as a term of type Rep k G, and call it Rep.of_mul_action k G H. This enables us to express the fact that certain maps are G-equivariant by constructing morphisms in the category Rep k G, i.e., representations of G over k.

An isomorphism of G-sets Gⁿ⁺¹ ≅ G × Gⁿ, where G acts by left multiplication on Gⁿ⁺¹ and G but trivially on Gⁿ. The map sends (g₀, ..., gₙ) ↦ (g₀, (g₀⁻¹g₁, g₁⁻¹g₂, ..., gₙ₋₁⁻¹gₙ)), and the inverse is (g₀, (g₁, ..., gₙ)) ↦ (g₀, g₀g₁, g₀g₁g₂, ..., g₀g₁...gₙ).

Equations
noncomputable def group_cohomology.resolution.diagonal_succ (k G : Type u) [comm_ring k] [group G] (n : ) :

An isomorphism of k-linear representations of G from k[Gⁿ⁺¹] to k[G] ⊗ₖ k[Gⁿ] (on which G acts by ρ(g₁)(g₂ ⊗ x) = (g₁ * g₂) ⊗ x) sending (g₀, ..., gₙ) to g₀ ⊗ (g₀⁻¹g₁, g₁⁻¹g₂, ..., gₙ₋₁⁻¹gₙ). The inverse sends g₀ ⊗ (g₁, ..., gₙ) to (g₀, g₀g₁, ..., g₀g₁...gₙ).

Equations
theorem group_cohomology.resolution.diagonal_succ_inv_single_left {k G : Type u} [comm_ring k] {n : } [group G] (g : G) (f : (fin n G) →₀ k) (r : k) :

The k[G]-linear isomorphism k[G] ⊗ₖ k[Gⁿ] ≃ k[Gⁿ⁺¹], where the k[G]-module structure on the lefthand side is tensor_product.left_module, whilst that of the righthand side comes from representation.as_module. Allows us to use basis.algebra_tensor_product to get a k[G]-basis of the righthand side.

Equations

A k[G]-basis of k[Gⁿ⁺¹], coming from the k[G]-linear isomorphism k[G] ⊗ₖ k[Gⁿ] ≃ k[Gⁿ⁺¹].

Equations
noncomputable def Rep.diagonal_hom_equiv {k G : Type u} [comm_ring k] (n : ) [group G] (A : Rep k G) :
(Rep.of_mul_action k G (fin (n + 1) G) A) ≃ₗ[k] (fin n G) A

Given a k-linear G-representation A, the set of representation morphisms Hom(k[Gⁿ⁺¹], A) is k-linearly isomorphic to the set of functions Gⁿ → A.

Equations
theorem Rep.diagonal_hom_equiv_apply {k G : Type u} [comm_ring k] {n : } [group G] {A : Rep k G} (f : Rep.of_mul_action k G (fin (n + 1) G) A) (x : fin n G) :

Given a k-linear G-representation A, diagonal_hom_equiv is a k-linear isomorphism of the set of representation morphisms Hom(k[Gⁿ⁺¹], A) with Fun(Gⁿ, A). This lemma says that this sends a morphism of representations f : k[Gⁿ⁺¹] ⟶ A to the function (g₁, ..., gₙ) ↦ f(1, g₁, g₁g₂, ..., g₁g₂...gₙ).

theorem Rep.diagonal_hom_equiv_symm_apply {k G : Type u} [comm_ring k] {n : } [group G] {A : Rep k G} (f : (fin n G) A) (x : fin (n + 1) G) :
((((Rep.diagonal_hom_equiv n A).symm) f).hom) (finsupp.single x 1) = ((A.ρ) (x 0)) (f (λ (i : fin n), (x (fin.cast_succ i))⁻¹ * x i.succ))

Given a k-linear G-representation A, diagonal_hom_equiv is a k-linear isomorphism of the set of representation morphisms Hom(k[Gⁿ⁺¹], A) with Fun(Gⁿ, A). This lemma says that the inverse map sends a function f : Gⁿ → A to the representation morphism sending (g₀, ... gₙ) ↦ ρ(g₀)(f(g₀⁻¹g₁, g₁⁻¹g₂, ..., gₙ₋₁⁻¹gₙ)), where ρ is the representation attached to A.

theorem Rep.diagonal_hom_equiv_symm_partial_prod_succ {k G : Type u} [comm_ring k] {n : } [group G] {A : Rep k G} (f : (fin n G) A) (g : fin (n + 1) G) (a : fin (n + 1)) :

Auxiliary lemma for defining group cohomology, used to show that the isomorphism diagonal_hom_equiv commutes with the differentials in two complexes which compute group cohomology.

The simplicial G-set sending [n] to Gⁿ⁺¹ equipped with the diagonal action of G.

Equations

When the category is G-Set, cech_nerve_terminal_from of G with the left regular action is isomorphic to EG, the universal cover of the classifying space of G as a simplicial G-set.

Equations

The free functor Type u ⥤ Module.{u} k applied to the universal cover of the classifying space of G as a simplicial set, augmented by the map from fin 1 → G to the terminal object in Type u.

Equations

If we augment the universal cover of the classifying space of G as a simplicial set by the map from fin 1 → G to the terminal object in Type u, then apply the free functor Type u ⥤ Module.{u} k, the resulting augmented simplicial k-module has an extra degeneracy.

Equations
noncomputable def group_cohomology.resolution (k G : Type u) [comm_ring k] [monoid G] :

The standard resolution of k as a trivial representation, defined as the alternating face map complex of a simplicial k-linear G-representation.

Equations
noncomputable def group_cohomology.resolution.d (k : Type u) [comm_ring k] (G : Type u) (n : ) :
((fin (n + 1) G) →₀ k) →ₗ[k] (fin n G) →₀ k

The k-linear map underlying the differential in the standard resolution of k as a trivial k-linear G-representation. It sends (g₀, ..., gₙ) ↦ ∑ (-1)ⁱ • (g₀, ..., ĝᵢ, ..., gₙ).

Equations
@[simp]
theorem group_cohomology.resolution.d_of {k : Type u} [comm_ring k] {G : Type u} {n : } (c : fin (n + 1) G) :
noncomputable def group_cohomology.resolution.X_iso (k G : Type u) [comm_ring k] [monoid G] (n : ) :

The nth object of the standard resolution of k is definitionally isomorphic to k[Gⁿ⁺¹] equipped with the representation induced by the diagonal action of G.

Equations

Simpler expression for the differential in the standard resolution of k as a G-representation. It sends (g₀, ..., gₙ₊₁) ↦ ∑ (-1)ⁱ • (g₀, ..., ĝᵢ, ..., gₙ₊₁).

The standard resolution of k as a trivial representation as a complex of k-modules.

Equations

If we apply the free functor Type u ⥤ Module.{u} k to the universal cover of the classifying space of G as a simplicial set, then take the alternating face map complex, the result is isomorphic to the standard resolution of the trivial G-representation k as a complex of k-modules.

Equations
noncomputable def group_cohomology.resolution.ε (k G : Type u) [comm_ring k] [monoid G] :

The hom of k-linear G-representations k[G¹] → k sending ∑ nᵢgᵢ ↦ ∑ nᵢ.

Equations

The homotopy equivalence of complexes of k-modules between the standard resolution of k as a trivial G-representation, and the complex which is k at 0 and 0 everywhere else, acts as ∑ nᵢgᵢ ↦ ∑ nᵢ : k[G¹] → k at 0.

The chain map from the standard resolution of k to k[0] given by ∑ nᵢgᵢ ↦ ∑ nᵢ in degree zero.

Equations
Instances for group_cohomology.resolution.ε_to_single₀

Given a k-linear G-representation V, Extⁿ(k, V) (where k is a trivial k-linear G-representation) is isomorphic to the nth cohomology group of Hom(P, V), where P is the standard resolution of k called group_cohomology.resolution k G.

Equations