Documentation

Mathlib.CategoryTheory.Limits.Constructions.Over.Connected

Connected limits in the over category #

Shows that the forgetful functor Over B ⥤ C creates and preserves connected limits, the latter without assuming that C has any limits. In particular, Over B has any connected limit which C has.

(Impl) Given a diagram in the over category, produce a natural transformation from the diagram legs to the specific object.

Equations
Instances For

    (Impl) Given a cone in the base category, raise it to a cone in the over category. Note this is where the connected assumption is used.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CategoryTheory.Over.CreatesConnected.raiseCone_π_app {J : Type u'} [Category.{v', u'} J] {C : Type u} [Category.{v, u} C] [IsConnected J] {B : C} {F : Functor J (Over B)} (c : Limits.Cone (F.comp (forget B))) (j : J) :
      (raiseCone c).π.app j = homMk (c.π.app j)

      (Impl) Show that the raised cone is a limit.

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

        The forgetful functor from the over category creates any connected limit.

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

        The forgetful functor from the over category preserves any connected limit.

        The over category has any connected limit which the original category has.