Documentation

Mathlib.CategoryTheory.Limits.Elements

Limits in the category of elements #

We show that if C has limits of shape I and A : C ⥤ Type w preserves limits of shape I, then the category of elements of A has limits of shape I and the forgetful functor π : A.Elements ⥤ C creates them.

noncomputable def CategoryTheory.CategoryOfElements.CreatesLimitsAux.liftedConeElement' {C : Type u} [Category.{v, u} C] {A : Functor C (Type w)} {I : Type u₁} [Category.{v₁, u₁} I] [Small.{w, u₁} I] (F : Functor I A.Elements) :
Limits.limit ((F.comp (π A)).comp A)

(implementation) A system (Fi, fi)_i of elements induces an element in lim_i A(Fi).

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem CategoryTheory.CategoryOfElements.CreatesLimitsAux.π_liftedConeElement' {C : Type u} [Category.{v, u} C] {A : Functor C (Type w)} {I : Type u₁} [Category.{v₁, u₁} I] [Small.{w, u₁} I] (F : Functor I A.Elements) (i : I) :
    Limits.limit.π ((F.comp (π A)).comp A) i (liftedConeElement' F) = (F.obj i).snd

    (implementation) A system (Fi, fi)_i of elements induces an element in A(lim_i Fi).

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

      (implementation) The constructured limit cone.

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

        (implementation) The constructed limit cone is a lift of the limit cone in C.

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

          (implementation) The constuctured limit cone is a limit cone.

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