Documentation

Mathlib.CategoryTheory.Triangulated.Opposite.Triangle

Triangles in the opposite category of a (pre)triangulated category #

Let C be a (pre)triangulated category. In CategoryTheory.Triangulated.Opposite.Basic, we have constructed a shift on Cᵒᵖ that will be part of a structure of (pre)triangulated category. In this file, we construct an equivalence of categories between (Triangle C)ᵒᵖ and Triangle Cᵒᵖ, called CategoryTheory.Pretriangulated.triangleOpEquivalence. It sends a triangle X ⟶ Y ⟶ Z ⟶ X⟦1⟧ in C to the triangle op Z ⟶ op Y ⟶ op X ⟶ (op Z)⟦1⟧ in Cᵒᵖ (without introducing signs).

References #

The functor which sends a triangle X ⟶ Y ⟶ Z ⟶ X⟦1⟧ in C to the triangle op Z ⟶ op Y ⟶ op X ⟶ (op Z)⟦1⟧ in Cᵒᵖ (without introducing signs).

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

    The functor which sends a triangle X ⟶ Y ⟶ Z ⟶ X⟦1⟧ in Cᵒᵖ to the triangle Z.unop ⟶ Y.unop ⟶ X.unop ⟶ Z.unop⟦1⟧ in C (without introducing signs).

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CategoryTheory.Pretriangulated.TriangleOpEquivalence.inverse_map (C : Type u_1) [CategoryTheory.Category.{u_2, u_1} C] [CategoryTheory.HasShift C ] {T₁ T₂ : CategoryTheory.Pretriangulated.Triangle Cᵒᵖ} (φ : T₁ T₂) :
      (CategoryTheory.Pretriangulated.TriangleOpEquivalence.inverse C).map φ = Quiver.Hom.op { hom₁ := φ.hom₃.unop, hom₂ := φ.hom₂.unop, hom₃ := φ.hom₁.unop, comm₁ := , comm₂ := , comm₃ := }

      The unit isomorphism of the equivalence triangleOpEquivalence C : (Triangle C)ᵒᵖ ≌ Triangle Cᵒᵖ .

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

        The counit isomorphism of the equivalence triangleOpEquivalence C : (Triangle C)ᵒᵖ ≌ Triangle Cᵒᵖ .

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

          An anti-equivalence between the categories of triangles in C and in Cᵒᵖ. A triangle in Cᵒᵖ shall be distinguished iff it correspond to a distinguished triangle in C via this equivalence.

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