Documentation

Mathlib.RepresentationTheory.Homological.GroupHomology.Basic

The group homology of a k-linear G-representation #

Let k be a commutative ring and G a group. This file defines the group homology of A : Rep k G to be the homology of the complex $$\dots \to \bigoplus_{G^2} A \to \bigoplus_{G^1} A \to \bigoplus_{G^0} A$$ with differential $d_n$ sending $a\cdot (g_0, \dots, g_n)$ to $$\rho(g_0^{-1})(a)\cdot (g_1, \dots, g_n)$$ $$+ \sum_{i = 0}^{n - 1}(-1)^{i + 1}a\cdot (g_0, \dots, g_ig_{i + 1}, \dots, g_n)$$ $$+ (-1)^{n + 1}a\cdot (g_0, \dots, g_{n - 1})$$ (where ρ is the representation attached to A).

We have a k-linear isomorphism $\bigoplus_{G^n} A \cong (A \otimes_k \left(\bigoplus_{G^n} k[G]\right))_G$ given by Rep.coinvariantsTensorFreeLEquiv. If we conjugate the $n$th differential in $(A \otimes_k P)_G$ by this isomorphism, where P is the bar resolution of k as a trivial k-linear G-representation, then the resulting map agrees with the differential $d_n$ defined above, a fact we prove.

Hence our $d_n$ squares to zero, and we get $\mathrm{H}_n(G, A) \cong \mathrm{Tor}_n(A, k),$ where $\mathrm{Tor}$ is defined by deriving the second argument of the functor $(A, B) \mapsto (A \otimes_k B)_G.$

Main definitions #

Implementation notes #

Group homology is typically stated for G-modules, or equivalently modules over the group ring ℤ[G]. However, can be generalized to any commutative ring k, which is what we use. Moreover, we express k[G]-module structures on a module k-module A using the Rep definition. We avoid using instances Module (MonoidAlgebra k G) A so that we do not run into possible scalar action diamonds.

Note that the existing definition of Tor in Mathlib.CategoryTheory.Monoidal.Tor is for monoidal categories, and the bifunctor we need to derive here maps to ModuleCat k. Hence we define Rep.Tor k G n by instead left-deriving the second argument of Rep.coinvariantsTensor k G: $(A, B) \mapsto (A \otimes_k B)_G$. The functor Rep.coinvariantsTensor k G is naturally isomorphic to the functor sending A, B to A ⊗[k[G]] B, where we give A the k[G]ᵐᵒᵖ-module structure defined by g • a := A.ρ g⁻¹ a, but currently mathlib's TensorProduct is only defined for commutative rings.

TODO #

The left-derived functors given by deriving the second argument of A, B ↦ (A ⊗[k] B)_G.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem Rep.Tor_map (k G : Type u) [CommRing k] [Group G] (n : ) {X✝ Y✝ : Rep k G} (f : X✝ Y✝) :
    @[simp]
    theorem Rep.Tor_obj (k G : Type u) [CommRing k] [Group G] (n : ) (X : Rep k G) :
    (Tor k G n).obj X = ((coinvariantsTensor k G).obj X).leftDerived n
    theorem Rep.isZero_Tor_succ_of_projective {k G : Type u} [CommRing k] [Group G] (X Y : Rep k G) [CategoryTheory.Projective Y] (n : ) :

    The higher Tor groups for X and Y are zero if Y is projective.

    @[reducible, inline]

    Given a k-linear G-representation A, this is the chain complex (A ⊗[k] P)_G, where P is the bar resolution of k as a trivial representation.

    Equations
    Instances For
      def groupHomology.inhomogeneousChains.d {k G : Type u} [CommRing k] [Group G] (A : Rep k G) (n : ) :
      ModuleCat.of k ((Fin (n + 1)G) →₀ A.V) ModuleCat.of k ((Fin nG) →₀ A.V)

      The differential in the complex of inhomogeneous chains used to calculate group homology.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem groupHomology.inhomogeneousChains.d_single {k G : Type u} [CommRing k] [Group G] {A : Rep k G} (n : ) (g : Fin (n + 1)G) (a : A.V) :
        (CategoryTheory.ConcreteCategory.hom (d A n)) (Finsupp.single g a) = Finsupp.single (fun (i : Fin n) => g i.succ) ((A.ρ (g 0)⁻¹) a) + j : Fin (n + 1), (-1) ^ (j + 1) Finsupp.single (j.contractNth (fun (x1 x2 : G) => x1 * x2) g) a
        @[reducible, inline]
        noncomputable abbrev groupHomology.inhomogeneousChains {k G : Type u} [CommRing k] [Group G] (A : Rep k G) [DecidableEq G] :

        Given a k-linear G-representation A, this is the complex of inhomogeneous chains $$\dots \to \bigoplus_{G^1} A \to \bigoplus_{G^0} A \to 0$$ which calculates the group homology of A.

        Equations
        Instances For
          theorem groupHomology.inhomogeneousChains.d_def {k G : Type u} [CommRing k] [Group G] (A : Rep k G) [DecidableEq G] (n : ) :
          (inhomogeneousChains A).d (n + 1) n = d A n

          Given a k-linear G-representation A, the complex of inhomogeneous chains is isomorphic to (A ⊗[k] P)_G, where P is the bar resolution of k as a trivial G-representation.

          Equations
          Instances For
            @[reducible, inline]
            abbrev groupHomology.cycles {k G : Type u} [CommRing k] [Group G] (A : Rep k G) [DecidableEq G] (n : ) :

            The n-cycles Zₙ(G, A) of a k-linear G-representation A, i.e. the kernel of the differential Cₙ(G, A) ⟶ Cₙ₋₁(G, A) in the complex of inhomogeneous chains.

            Equations
            Instances For
              @[reducible, inline]
              abbrev groupHomology.iCycles {k G : Type u} [CommRing k] [Group G] (A : Rep k G) [DecidableEq G] (n : ) :

              The natural inclusion of the n-cycles Zₙ(G, A) into the n-chains Cₙ(G, A).

              Equations
              Instances For
                @[reducible, inline]
                abbrev groupHomology.toCycles {k G : Type u} [CommRing k] [Group G] (A : Rep k G) [DecidableEq G] (i j : ) :

                This is the map from i-chains to j-cycles induced by the differential in the complex of inhomogeneous chains.

                Equations
                Instances For
                  def groupHomology {k G : Type u} [CommRing k] [Group G] [DecidableEq G] (A : Rep k G) (n : ) :

                  The group homology of a k-linear G-representation A, as the homology of its complex of inhomogeneous chains.

                  Equations
                  Instances For
                    @[reducible, inline]
                    abbrev groupHomology.π {k G : Type u} [CommRing k] [Group G] [DecidableEq G] (A : Rep k G) (n : ) :

                    The natural map from n-cycles to nth group homology for a k-linear G-representation A.

                    Equations
                    Instances For
                      theorem groupHomology_induction_on {k G : Type u} [CommRing k] [Group G] [DecidableEq G] {A : Rep k G} {n : } {C : (groupHomology A n)Prop} (x : (groupHomology A n)) (h : ∀ (x : (groupHomology.cycles A n)), C ((CategoryTheory.ConcreteCategory.hom (groupHomology.π A n)) x)) :
                      C x
                      def groupHomologyIsoTor {k G : Type u} [CommRing k] [Group G] [DecidableEq G] (A : Rep k G) (n : ) :
                      groupHomology A n ((Rep.Tor k G n).obj A).obj (Rep.trivial k G k)

                      The nth group homology of a k-linear G-representation A is isomorphic to Torₙ(A, k) (taken in Rep k G), where k is a trivial k-linear G-representation.

                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For