Documentation

Mathlib.Algebra.Homology.HomotopyCategory.Shift

The shift on cochain complexes and on the homotopy category #

In this file, we show that for any preadditive category C, the categories CochainComplex C ℤ and HomotopyCategory C (ComplexShape.up ℤ) are equipped with a shift by .

@[simp]
theorem CochainComplex.shiftFunctor_map_f (C : Type u) [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (n : ) :
∀ {X Y : CochainComplex C } (φ : X Y) (i : ), ((CochainComplex.shiftFunctor C n).map φ).f i = φ.f (i + n)
@[simp]
theorem CochainComplex.shiftFunctor_obj_d (C : Type u) [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (n : ) (K : CochainComplex C ) (i : ) (j : ) :
((CochainComplex.shiftFunctor C n).obj K).d i j = n.negOnePow K.d (i + n) (j + n)

The shift functor by n : ℤ on CochainComplex C ℤ which sends a cochain complex K to the complex which is K.X (i + n) in degree i, and which multiplies the differentials by (-1)^n.

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

    The canonical isomorphism ((shiftFunctor C n).obj K).X i ≅ K.X m when m = i + n.

    Equations
    Instances For

      The shift functor by n on CochainComplex C ℤ identifies to the identity functor when n = 0.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem CochainComplex.shiftFunctorAdd'_inv_app_f (C : Type u) [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (n₁ : ) (n₂ : ) (n₁₂ : ) (h : n₁ + n₂ = n₁₂) (X : CochainComplex C ) (i : ) :
        ((CochainComplex.shiftFunctorAdd' C n₁ n₂ n₁₂ h).inv.app X).f i = (HomologicalComplex.XIsoOfEq X ).inv
        @[simp]
        theorem CochainComplex.shiftFunctorAdd'_hom_app_f (C : Type u) [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (n₁ : ) (n₂ : ) (n₁₂ : ) (h : n₁ + n₂ = n₁₂) (X : CochainComplex C ) (i : ) :
        ((CochainComplex.shiftFunctorAdd' C n₁ n₂ n₁₂ h).hom.app X).f i = (HomologicalComplex.XIsoOfEq X ).hom

        The compatibility of the shift functors on CochainComplex C ℤ with respect to the addition of integers.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem CochainComplex.shiftFunctor_obj_d' {C : Type u} [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (K : CochainComplex C ) (n : ) (i : ) (j : ) :
          ((CategoryTheory.shiftFunctor (CochainComplex C ) n).obj K).d i j = n.negOnePow K.d (i + { as := n }.as) (j + { as := n }.as)
          @[simp]
          theorem CochainComplex.shiftEval_hom_app (C : Type u) [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (n : ) (i : ) (i' : ) (hi : n + i = i') (X : CochainComplex C ) :
          (CochainComplex.shiftEval C n i i' hi).hom.app X = (HomologicalComplex.XIsoOfEq X ).hom
          @[simp]
          theorem CochainComplex.shiftEval_inv_app (C : Type u) [CategoryTheory.Category.{v, u} C] [CategoryTheory.Preadditive C] (n : ) (i : ) (i' : ) (hi : n + i = i') (X : CochainComplex C ) :
          (CochainComplex.shiftEval C n i i' hi).inv.app X = (HomologicalComplex.XIsoOfEq X ).inv

          Shifting cochain complexes by n and evaluating in a degree i identifies to the evaluation in degree i' when n + i = i'.

          Equations
          Instances For

            If h : Homotopy φ₁ φ₂ and n : ℤ, this is the induced homotopy between φ₁⟦n⟧' and φ₂⟦n⟧'.

            Equations
            • Homotopy.shift h n = { hom := fun (i j : ) => n.negOnePow h.hom (i + { as := n }.as) (j + { as := n }.as), zero := , comm := }
            Instances For