Documentation

Mathlib.RepresentationTheory.Homological.GroupHomology.FiniteCyclic

Group homology of a finite cyclic group #

Let k be a commutative ring, G a group and A a k-linear G-representation. Given endomorphisms φ, ψ : A ⟶ A such that φ ∘ ψ = ψ ∘ φ = 0, denote by Chains(A, φ, ψ) the periodic chain complex ... ⟶ A --φ--> A --ψ--> A --φ--> A --ψ--> A ⟶ 0.

When G is finite and generated by g : G, then P := Chains(k[G], N, ρ(g) - Id) (with ρ the left regular representation) is a projective resolution of k as a trivial representation. In this file we show that for A : Rep k G, (A ⊗ P)_G is isomorphic to Chains(A, N, ρ_A(g) - Id) as a complex of k-modules, and hence the homology of this complex computes group homology.

Main definitions #

Given a finite cyclic group G generated by g : G and a k-linear G-representation A, the period chain complex ... ⟶ (A ⊗ₖ k[G])_G --⟦Id ⊗ N⟧--> (A ⊗ₖ k[G])_G --⟦Id ⊗ (ρ(g⁻¹) - 𝟙)⟧--> (A ⊗ₖ k[G])_G ⟶ 0 is isomorphic as a complex in ModuleCat k to ... ⟶ A --N--> A --(ρ(g) - 𝟙)--> A --N--> A --(ρ(g) - 𝟙)--> A ⟶ 0.

Equations
Instances For
    @[reducible, inline]

    Given a finite cyclic group G generated by g and A : Rep k G, H₀(G, A) is isomorphic to the cokernel of ρ(g) - Id(A).

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      noncomputable def Rep.FiniteCyclicGroup.groupHomologyIsoEven {k G : Type u} [CommRing k] [CommGroup G] [Fintype G] (A : Rep k G) (g : G) [DecidableEq G] (hg : ∀ (x : G), x Subgroup.zpowers g) (i : ) [h₀ : NeZero i] (hi : Even i) :

      Given a finite cyclic group G generated by g and A : Rep k G, Hᵢ(G, A) is isomorphic to the homology of the short complex of k-modules A --(ρ(g) - 𝟙)--> A --N--> A when i is nonzero and even.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[reducible, inline]
        noncomputable abbrev Rep.FiniteCyclicGroup.groupHomologyπEven {k G : Type u} [CommRing k] [CommGroup G] [Fintype G] (A : Rep k G) (g : G) [DecidableEq G] (hg : ∀ (x : G), x Subgroup.zpowers g) (i : ) [NeZero i] (hi : Even i) :

        Given a finite cyclic group G generated by g and A : Rep k G, this is the quotient map Ker(N) ⟶ Ker(N)/Im(ρ(g) - Id(A)) ≅ Hᵢ(G, A) for any nonzero even i.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          noncomputable def Rep.FiniteCyclicGroup.groupHomologyIsoOdd {k G : Type u} [CommRing k] [CommGroup G] [Fintype G] (A : Rep k G) (g : G) [DecidableEq G] (hg : ∀ (x : G), x Subgroup.zpowers g) (i : ) (hi : Odd i) :

          Given a finite cyclic group G generated by g and A : Rep k G, Hⁱ(G, A) is isomorphic to the homology of the short complex of k-modules A --N--> A --(ρ(g) - 𝟙)--> A when i is odd.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[reducible, inline]
            noncomputable abbrev Rep.FiniteCyclicGroup.groupHomologyπOdd {k G : Type u} [CommRing k] [CommGroup G] [Fintype G] (A : Rep k G) (g : G) [DecidableEq G] (hg : ∀ (x : G), x Subgroup.zpowers g) (i : ) (hi : Odd i) :

            Given a finite cyclic group G generated by g and A : Rep k G, this is the quotient map Ker(ρ(g) - Id(A)) ⟶ Ker(ρ(g) - Id(A))/Im(N) ≅ Hᵢ(G, A) for any odd i.

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