Documentation

Mathlib.CategoryTheory.Monoidal.Tor

Tor, the left-derived functor of tensor product #

We define Tor C n : C ⥤ C ⥤ C, by left-deriving in the second factor of (X, Y) ↦ X ⊗ Y.

For now we have almost nothing to say about it!

It would be good to show that this is naturally isomorphic to the functor obtained by left-deriving in the first factor, instead. For now we define Tor' by left-deriving in the first factor, but showing Tor C n ≅ Tor' C n will require a bit more theory! Possibly it's best to axiomatize delta functors, and obtain a unique characterisation?

We define Tor C n : C ⥤ C ⥤ C by left-deriving in the second factor of (X, Y) ↦ X ⊗ Y.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem CategoryTheory.Tor_map (C : Type u_1) [Category.{u_2, u_1} C] [MonoidalCategory C] [Abelian C] [MonoidalPreadditive C] [HasProjectiveResolutions C] (n : ) {X✝ Y✝ : C} (f : X✝ Y✝) :
    @[simp]
    theorem CategoryTheory.Tor_obj (C : Type u_1) [Category.{u_2, u_1} C] [MonoidalCategory C] [Abelian C] [MonoidalPreadditive C] [HasProjectiveResolutions C] (n : ) (X : C) :
    (Tor C n).obj X = ((MonoidalCategory.tensoringLeft C).obj X).leftDerived n

    An alternative definition of Tor, where we left-derive in the first factor instead.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CategoryTheory.Tor'_obj_obj (C : Type u_1) [Category.{u_2, u_1} C] [MonoidalCategory C] [Abelian C] [MonoidalPreadditive C] [HasProjectiveResolutions C] (n : ) (k j : C) :
      ((Tor' C n).obj k).obj j = (((MonoidalCategory.tensoringRight C).obj j).leftDerived n).obj k
      @[simp]
      theorem CategoryTheory.Tor'_map_app' (C : Type u_1) [Category.{u_2, u_1} C] [MonoidalCategory C] [Abelian C] [MonoidalPreadditive C] [HasProjectiveResolutions C] (n : ) {X Y : C} (f : X Y) (Z : C) :
      ((Tor' C n).map f).app Z = (((MonoidalCategory.tensoringRight C).obj Z).leftDerived n).map f
      @[simp]
      theorem CategoryTheory.Tor'_obj_map (C : Type u_1) [Category.{u_2, u_1} C] [MonoidalCategory C] [Abelian C] [MonoidalPreadditive C] [HasProjectiveResolutions C] (n : ) {X Y : C} (Z : C) (f : X Y) :
      ((Tor' C n).obj Z).map f = (NatTrans.leftDerived ((MonoidalCategory.tensoringRight C).map f) n).app Z

      The higher Tor groups for X and Y are zero if Y is projective.

      The higher Tor' groups for X and Y are zero if X is projective.