Documentation

Mathlib.Algebra.Homology.DifferentialObject

Homological complexes are differential graded objects. #

We verify that a HomologicalComplex indexed by an AddCommGroup is essentially the same thing as a differential graded object.

This equivalence is probably not particularly useful in practice; it's here to check that definitions match up as expected.

We first prove some results about differential graded objects.

Porting note: after the port, move these to their own file.

@[reducible, inline]

Since eqToHom only preserves the fact that X.X i = X.X j but not i = j, this definition is used to aid the simplifier.

Equations
Instances For

    The functor from differential graded objects to homological complexes.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem HomologicalComplex.homologicalComplexToDGO_obj_d {β : Type u_1} [AddCommGroup β] (b : β) (V : Type u_2) [CategoryTheory.Category.{u_3, u_2} V] [CategoryTheory.Limits.HasZeroMorphisms V] (X : HomologicalComplex V (ComplexShape.up' b)) (i : β) :
      ((HomologicalComplex.homologicalComplexToDGO b V).obj X).d i = X.d i ((fun (b_1 : β) => b_1 + { as := 1 }.as b) i)

      The functor from homological complexes to differential graded objects.

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

        The category of differential graded objects in V is equivalent to the category of homological complexes in V.

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