Documentation

Mathlib.CategoryTheory.Triangulated.Functor

Triangulated functors #

In this file, when C and D are categories equipped with a shift by and F : C ⥤ D is a functor which commutes with the shift, we define the induced functor F.mapTriangle : Triangle C ⥤ Triangle D on the categories of triangles. When C and D are pretriangulated, a triangulated functor is such a functor F which also sends distinguished triangles to distinguished triangles: this defines the typeclass Functor.IsTriangulated.

@[simp]

The functor Triangle C ⥤ Triangle D that is induced by a functor F : C ⥤ D which commutes with shift by .

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

    The functor F.mapTriangle commutes with the shift.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      Equations
      • F.instCommShiftTriangleMapTriangleInt = { iso := F.mapTriangleCommShiftIso, zero := , add := }

      F.mapTriangle commutes with the rotation of triangles.

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

        A functor which commutes with the shift by is triangulated if it sends distinguished triangles to distinguished triangles.

        • map_distinguished : TCategoryTheory.Pretriangulated.distinguishedTriangles, F.mapTriangle.obj T CategoryTheory.Pretriangulated.distinguishedTriangles
        Instances
          theorem CategoryTheory.Functor.IsTriangulated.map_distinguished {C : Type u_1} {D : Type u_2} [CategoryTheory.Category.{u_3, u_1} C] [CategoryTheory.Category.{u_4, u_2} D] [CategoryTheory.HasShift C ] [CategoryTheory.HasShift D ] {F : CategoryTheory.Functor C D} [F.CommShift ] [CategoryTheory.Limits.HasZeroObject C] [CategoryTheory.Limits.HasZeroObject D] [CategoryTheory.Preadditive C] [CategoryTheory.Preadditive D] [∀ (n : ), (CategoryTheory.shiftFunctor C n).Additive] [∀ (n : ), (CategoryTheory.shiftFunctor D n).Additive] [CategoryTheory.Pretriangulated C] [CategoryTheory.Pretriangulated D] [self : F.IsTriangulated] (T : CategoryTheory.Pretriangulated.Triangle C) :
          T CategoryTheory.Pretriangulated.distinguishedTrianglesF.mapTriangle.obj T CategoryTheory.Pretriangulated.distinguishedTriangles
          theorem CategoryTheory.Functor.map_distinguished {C : Type u_1} {D : Type u_2} [CategoryTheory.Category.{u_3, u_1} C] [CategoryTheory.Category.{u_4, u_2} D] [CategoryTheory.HasShift C ] [CategoryTheory.HasShift D ] (F : CategoryTheory.Functor C D) [F.CommShift ] [CategoryTheory.Limits.HasZeroObject C] [CategoryTheory.Limits.HasZeroObject D] [CategoryTheory.Preadditive C] [CategoryTheory.Preadditive D] [∀ (n : ), (CategoryTheory.shiftFunctor C n).Additive] [∀ (n : ), (CategoryTheory.shiftFunctor D n).Additive] [CategoryTheory.Pretriangulated C] [CategoryTheory.Pretriangulated D] [F.IsTriangulated] (T : CategoryTheory.Pretriangulated.Triangle C) (hT : T CategoryTheory.Pretriangulated.distinguishedTriangles) :
          F.mapTriangle.obj T CategoryTheory.Pretriangulated.distinguishedTriangles