Documentation

Mathlib.CategoryTheory.Limits.Preserves.Ulift

ULift creates small (co)limits #

This file shows that uliftFunctor.{v, u} preserves all limits and colimits, including those potentially too big to exist in Type u.

As this functor is fully faithful, we also deduce that it creates u-small limits and colimits.

def CategoryTheory.Limits.Types.sectionsEquiv {J : Type u_1} [Category.{u_2, u_1} J] (K : Functor J (Type u)) :
K.sections (K.comp uliftFunctor.{v, u}).sections

The equivalence between K.sections and (K ⋙ uliftFunctor.{v, u}).sections. This is used to show that uliftFunctor preserves limits that are potentially too large to exist in the source category.

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

    The functor uliftFunctor : Type u ⥤ Type (max u v) creates u-small limits.

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

    The functor uliftFunctor : Type u ⥤ Type (max u v) creates u-small colimits.

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