Documentation

Mathlib.Algebra.Homology.HomotopyCategory.HomComplexCohomology

Cohomology of the hom complex #

Given -indexed cochain complexes K and L, and n : ℤ, we introduce a type HomComplex.CohomologyClass K L n which is the quotient of HomComplex.Cocycle K L n which identifies cohomologous cocycles. We construct this type of cohomology classes instead of using the homology API because Cochain K L can be considered both as a complex of abelian groups or as a complex of R-modules when the category is R-linear. This also complements the API around HomComplex which is centered on terms in types Cochain or Cocycle which are suitable for computations.

We also show that HomComplex.CohomologyClass K L n identifies to the type of morphisms between K and L⟦n⟧ in the homotopy category.

The subgroup of Cocycle K L n consisting of coboundaries.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem CochainComplex.HomComplex.mem_coboundaries_iff {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] {K L : CochainComplex C } {n : } (α : Cocycle K L n) (m : ) (hm : m + 1 = n) :
    α coboundaries K L n ∃ (β : Cochain K L m), δ m n β = α

    The type of cohomology classes of degree n in the complex of morphisms from K to L.

    Equations
    Instances For

      The additive map which sends a cohomology class to the corresponding morphism in the homotopy category.

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

        CohomologyClass K L m identifies to the cohomology of the complex HomComplex K L in degree m.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem CochainComplex.HomComplex.leftHomologyData'_H_coe {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (K L : CochainComplex C ) (n m p : ) (hm : n + 1 = m) (hp : m + 1 = p) :
          (leftHomologyData' K L n m p hm hp).H = CohomologyClass K L m
          @[simp]
          theorem CochainComplex.HomComplex.leftHomologyData'_K_coe {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (K L : CochainComplex C ) (n m p : ) (hm : n + 1 = m) (hp : m + 1 = p) :
          (leftHomologyData' K L n m p hm hp).K = Cocycle K L m