Documentation

Mathlib.CategoryTheory.Abelian.Injective.Dimension

Injective dimension #

In an abelian category C, we shall say that X : C has Injective dimension < n if all Ext Y X i vanish when n ≤ i. This defines a type class HasInjectiveDimensionLT X n. We also define a type class HasInjectiveDimensionLE X n as an abbreviation for HasInjectiveDimensionLT X (n + 1). (Note that the fact that X is a zero object is equivalent to the condition HasInjectiveDimensionLT X 0, but this cannot be expressed in terms of HasInjectiveDimensionLE.)

We also define the Injective dimension in WithBot ℕ∞ as injectiveDimension, injectiveDimension X = ⊥ iff X is zero and acts in common sense in the non-negative values.

An object X in an abelian category has Injective dimension < n if all Ext X Y i vanish when n ≤ i. See also HasInjectiveDimensionLE. (Do not use the subsingleton' field directly. Use the constructor HasInjectiveDimensionLT.mk, and the lemmas hasInjectiveDimensionLT_iff and Ext.eq_zero_of_hasInjectiveDimensionLT.)

Instances
    @[reducible, inline]

    An object X in an abelian category has Injective dimension ≤ n if all Ext X Y i vanish when n + 1 ≤ i

    Equations
    Instances For
      theorem CategoryTheory.HasInjectiveDimensionLT.subsingleton {C : Type u} [Category.{v, u} C] [Abelian C] [HasExt C] (X : C) (n : ) [hX : HasInjectiveDimensionLT X n] (i : ) (hi : n i) (Y : C) :
      theorem CategoryTheory.HasInjectiveDimensionLT.mk {C : Type u} [Category.{v, u} C] [Abelian C] [HasExt C] {X : C} {n : } (hX : ∀ (i : ), n i∀ ⦃Y : C⦄ (e : Abelian.Ext Y X i), e = 0) :
      theorem CategoryTheory.Abelian.Ext.eq_zero_of_hasInjectiveDimensionLT {C : Type u} [Category.{v, u} C] [Abelian C] [HasExt C] {X Y : C} {i : } (e : Ext Y X i) (n : ) [HasInjectiveDimensionLT X n] (hi : n i) :
      e = 0
      theorem CategoryTheory.hasInjectiveDimensionLT_iff {C : Type u} [Category.{v, u} C] [Abelian C] (X : C) (n : ) [HasExt C] :
      HasInjectiveDimensionLT X n ∀ (i : ), n i∀ ⦃Y : C⦄ (e : Abelian.Ext Y X i), e = 0
      noncomputable def CategoryTheory.injectiveDimension {C : Type u} [Category.{v, u} C] [Abelian C] (X : C) :

      The injective dimension of an object in an abelian category.

      Equations
      Instances For