Documentation

Mathlib.CategoryTheory.GuitartExact.KanExtension

Guitart exact squares and Kan extensions #

Given a Guitart exact square w : T ⋙ R ⟶ L ⋙ B,

     T
  C₁ ⥤ C₂
L |     | R
  v     v
  C₃ ⥤ C₄
     B

we show that an extension F' : C₄ ⥤ D of F : C₂ ⥤ D along R is a pointwise left Kan extension at B.obj X₃ iff the composition T ⋙ F' is a pointwise left Kan extension at X₃ of B ⋙ F'.

@[reducible, inline]
abbrev CategoryTheory.Functor.LeftExtension.compTwoSquare {C₁ : Type u₁} {C₂ : Type u₂} {C₃ : Type u₃} {C₄ : Type u₄} {D : Type u₅} [Category.{v₁, u₁} C₁] [Category.{v₂, u₂} C₂] [Category.{v₃, u₃} C₃] [Category.{v₄, u₄} C₄] [Category.{v₅, u₅} D] {T : Functor C₁ C₂} {L : Functor C₁ C₃} {R : Functor C₂ C₄} {B : Functor C₃ C₄} {F : Functor C₂ D} (E : R.LeftExtension F) (w : TwoSquare T L R B) :

Given a square w : TwoSquare T L R B (consisting of a natural transformation T ⋙ R ⟶ L ⋙ B), this is the obvious map R.LeftExtension F → L.LeftExtension (T ⋙ F) obtained by the precomposition with B and the postcomposition with w.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    noncomputable def CategoryTheory.Functor.LeftExtension.isPointwiseLeftKanExtensionAtCompTwoSquareEquiv {C₁ : Type u₁} {C₂ : Type u₂} {C₃ : Type u₃} {C₄ : Type u₄} {D : Type u₅} [Category.{v₁, u₁} C₁] [Category.{v₂, u₂} C₂] [Category.{v₃, u₃} C₃] [Category.{v₄, u₄} C₄] [Category.{v₅, u₅} D] {T : Functor C₁ C₂} {L : Functor C₁ C₃} {R : Functor C₂ C₄} {B : Functor C₃ C₄} {F : Functor C₂ D} (E : R.LeftExtension F) (w : TwoSquare T L R B) (X₃ : C₃) [(w.costructuredArrowRightwards X₃).Final] :

    If w : TwoSquare T L R B is a Guitart exact square, and E is a left extension of F along R, then E is a pointwise left Kan extension of F along R at B.obj X₃ iff E.compTwoSquare w is a pointwise left Kan extension of T ⋙ F along L at X₃.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem CategoryTheory.Functor.LeftExtension.nonempty_isPointwiseLeftKanExtensionAt_compTwoSquare_iff {C₁ : Type u₁} {C₂ : Type u₂} {C₃ : Type u₃} {C₄ : Type u₄} {D : Type u₅} [Category.{v₁, u₁} C₁] [Category.{v₂, u₂} C₂] [Category.{v₃, u₃} C₃] [Category.{v₄, u₄} C₄] [Category.{v₅, u₅} D] {T : Functor C₁ C₂} {L : Functor C₁ C₃} {R : Functor C₂ C₄} {B : Functor C₃ C₄} {F : Functor C₂ D} (E : R.LeftExtension F) (w : TwoSquare T L R B) (X₃ : C₃) [(w.costructuredArrowRightwards X₃).Final] :
      noncomputable def CategoryTheory.Functor.LeftExtension.IsPointwiseLeftKanExtension.compTwoSquare {C₁ : Type u₁} {C₂ : Type u₂} {C₃ : Type u₃} {C₄ : Type u₄} {D : Type u₅} [Category.{v₁, u₁} C₁] [Category.{v₂, u₂} C₂] [Category.{v₃, u₃} C₃] [Category.{v₄, u₄} C₄] [Category.{v₅, u₅} D] {T : Functor C₁ C₂} {L : Functor C₁ C₃} {R : Functor C₂ C₄} {B : Functor C₃ C₄} {F : Functor C₂ D} {E : R.LeftExtension F} (h : E.IsPointwiseLeftKanExtension) (w : TwoSquare T L R B) [w.GuitartExact] :

      If w : TwoSquare T L R B is a Guitart exact square, and E is a pointwise left Kan extension of F along R, then E.compTwoSquare w is a pointwise left Kan extension of T ⋙ F along L.

      Equations
      Instances For
        noncomputable def CategoryTheory.Functor.LeftExtension.isPointwiseLeftKanExtensionOfCompTwoSquare {C₁ : Type u₁} {C₂ : Type u₂} {C₃ : Type u₃} {C₄ : Type u₄} {D : Type u₅} [Category.{v₁, u₁} C₁] [Category.{v₂, u₂} C₂] [Category.{v₃, u₃} C₃] [Category.{v₄, u₄} C₄] [Category.{v₅, u₅} D] {T : Functor C₁ C₂} {L : Functor C₁ C₃} {R : Functor C₂ C₄} {B : Functor C₃ C₄} {F : Functor C₂ D} (E : R.LeftExtension F) (w : TwoSquare T L R B) [w.GuitartExact] [B.EssSurj] (h : (E.compTwoSquare w).IsPointwiseLeftKanExtension) :

        If w : TwoSquare T L R B is a Guitart exact square, with B essentially surjective, and E is a left extension of F along R, then E is a pointwise left Kan extension of F along R provided E.compTwoSquare w is a pointwise left Kan extension of T ⋙ F along L.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          noncomputable def CategoryTheory.Functor.LeftExtension.isPointwiseLeftKanExtensionEquivOfGuitartExact {C₁ : Type u₁} {C₂ : Type u₂} {C₃ : Type u₃} {C₄ : Type u₄} {D : Type u₅} [Category.{v₁, u₁} C₁] [Category.{v₂, u₂} C₂] [Category.{v₃, u₃} C₃] [Category.{v₄, u₄} C₄] [Category.{v₅, u₅} D] {T : Functor C₁ C₂} {L : Functor C₁ C₃} {R : Functor C₂ C₄} {B : Functor C₃ C₄} {F : Functor C₂ D} (E : R.LeftExtension F) (w : TwoSquare T L R B) [w.GuitartExact] [B.EssSurj] :

          If w : TwoSquare T L R B is a Guitart exact square, with B essentially surjective, and E is a left extension of F along R, then E is a pointwise left Kan extension of F along R iff E.compTwoSquare w is a pointwise left Kan extension of T ⋙ F along L.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            theorem CategoryTheory.TwoSquare.hasPointwiseLeftKanExtensionAt_iff {C₁ : Type u₁} {C₂ : Type u₂} {C₃ : Type u₃} {C₄ : Type u₄} {D : Type u₅} [Category.{v₁, u₁} C₁] [Category.{v₂, u₂} C₂] [Category.{v₃, u₃} C₃] [Category.{v₄, u₄} C₄] [Category.{v₅, u₅} D] {T : Functor C₁ C₂} {L : Functor C₁ C₃} {R : Functor C₂ C₄} {B : Functor C₃ C₄} (w : TwoSquare T L R B) (F : Functor C₂ D) (X₃ : C₃) [(w.costructuredArrowRightwards X₃).Final] :
            theorem CategoryTheory.TwoSquare.hasPointwiseLeftKanExtension_iff {C₁ : Type u₁} {C₂ : Type u₂} {C₃ : Type u₃} {C₄ : Type u₄} {D : Type u₅} [Category.{v₁, u₁} C₁] [Category.{v₂, u₂} C₂] [Category.{v₃, u₃} C₃] [Category.{v₄, u₄} C₄] [Category.{v₅, u₅} D] {T : Functor C₁ C₂} {L : Functor C₁ C₃} {R : Functor C₂ C₄} {B : Functor C₃ C₄} (w : TwoSquare T L R B) [w.GuitartExact] [B.EssSurj] (F : Functor C₂ D) :
            theorem CategoryTheory.TwoSquare.hasPointwiseLeftKanExtension {C₁ : Type u₁} {C₂ : Type u₂} {C₃ : Type u₃} {C₄ : Type u₄} {D : Type u₅} [Category.{v₁, u₁} C₁] [Category.{v₂, u₂} C₂] [Category.{v₃, u₃} C₃] [Category.{v₄, u₄} C₄] [Category.{v₅, u₅} D] {T : Functor C₁ C₂} {L : Functor C₁ C₃} {R : Functor C₂ C₄} {B : Functor C₃ C₄} (w : TwoSquare T L R B) [w.GuitartExact] (F : Functor C₂ D) [R.HasPointwiseLeftKanExtension F] :
            theorem CategoryTheory.TwoSquare.hasLeftKanExtension {C₁ : Type u₁} {C₂ : Type u₂} {C₃ : Type u₃} {C₄ : Type u₄} {D : Type u₅} [Category.{v₁, u₁} C₁] [Category.{v₂, u₂} C₂] [Category.{v₃, u₃} C₃] [Category.{v₄, u₄} C₄] [Category.{v₅, u₅} D] {T : Functor C₁ C₂} {L : Functor C₁ C₃} {R : Functor C₂ C₄} {B : Functor C₃ C₄} (w : TwoSquare T L R B) [w.GuitartExact] (F : Functor C₂ D) [R.HasPointwiseLeftKanExtension F] :