Documentation

Mathlib.Algebra.Homology.DerivedCategory.Ext.Map

Map Between Ext Induced by Exact Functor #

In this file, we develope the map Ext^k (M, N) → Ext^k (F(M), F(N)), where F is an exact functor between abelian categories.

noncomputable def CategoryTheory.Abelian.Ext.mapExactFunctor {C : Type u} [Category.{v, u} C] [Abelian C] {D : Type u'} [Category.{v', u'} D] [Abelian D] (F : Functor C D) [F.Additive] [Limits.PreservesFiniteLimits F] [Limits.PreservesFiniteColimits F] [HasExt C] [HasExt D] {X Y : C} {n : } (f : Ext X Y n) :
Ext (F.obj X) (F.obj Y) n

The map between Ext induced by F.mapShiftedHomAddHom.

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

    The additive homomorphism between Ext induced by F.mapShiftedHomAddHom.

    Equations
    Instances For

      Upgrade of F.mapExtAddHom assuming F is linear.

      Equations
      Instances For