Documentation

Mathlib.CategoryTheory.Limits.MorphismProperty

(Co)limits in subcategories of comma categories defined by morphism properties #

noncomputable def CategoryTheory.MorphismProperty.Comma.forgetCreatesLimitOfClosed {T : Type u_1} [Category.{u_5, u_1} T] (P : MorphismProperty T) {A : Type u_2} {B : Type u_3} {J : Type u_4} [Category.{u_6, u_2} A] [Category.{u_7, u_3} B] [Category.{u_8, u_4} J] {L : Functor A T} {R : Functor B T} (D : Functor J (MorphismProperty.Comma L R P )) (h : Limits.ClosedUnderLimitsOfShape J fun (f : Comma L R) => P f.hom) [Limits.HasLimit (D.comp (forget L R P ))] :

If P is closed under limits of shape J in Comma L R, then when D has a limit in Comma L R, the forgetful functor creates this limit.

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

    If Comma L R has limits of shape J and Comma L R is closed under limits of shape J, then forget L R P ⊤ ⊤ creates limits of shape J.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem CategoryTheory.CostructuredArrow.closedUnderLimitsOfShape_discrete_empty {T : Type u_1} [Category.{u_4, u_1} T] (P : MorphismProperty T) {A : Type u_2} [Category.{u_3, u_2} A] {L : Functor A T} [L.Faithful] [L.Full] {Y : A} [P.ContainsIdentities] [P.RespectsIso] :
      theorem CategoryTheory.Over.closedUnderLimitsOfShape_discrete_empty {T : Type u_1} [Category.{u_2, u_1} T] (P : MorphismProperty T) {X : T} [P.ContainsIdentities] [P.RespectsIso] :
      theorem CategoryTheory.Over.closedUnderLimitsOfShape_pullback {T : Type u_1} [Category.{u_2, u_1} T] (P : MorphismProperty T) {X : T} [Limits.HasPullbacks T] [P.IsStableUnderComposition] [P.IsStableUnderBaseChange] [P.HasOfPostcompProperty P] :

      Let P be stable under composition and base change. If P satisfies cancellation on the right, the subcategory of Over X defined by P is closed under pullbacks.

      Without the cancellation property, this does not in general. Consider for example P = Function.Surjective on Type.

      Equations
      • One or more equations did not get rendered due to their size.
      noncomputable instance CategoryTheory.MorphismProperty.Over.createsLimitsOfShape_walkingCospan {T : Type u_1} [Category.{u_2, u_1} T] (P : MorphismProperty T) (X : T) [Limits.HasPullbacks T] [P.IsStableUnderComposition] [P.IsStableUnderBaseChange] [P.HasOfPostcompProperty P] :

      If P is stable under composition, base change and satisfies post-cancellation, Over.forget P ⊤ X creates pullbacks.

      Equations
      @[instance 900]
      instance CategoryTheory.MorphismProperty.Over.hasPullbacks {T : Type u_1} [Category.{u_2, u_1} T] (P : MorphismProperty T) (X : T) [Limits.HasPullbacks T] [P.IsStableUnderComposition] [P.IsStableUnderBaseChange] [P.HasOfPostcompProperty P] :

      If P is stable under composition, base change and satisfies post-cancellation, P.Over ⊤ X has pullbacks