Documentation

Mathlib.CategoryTheory.WithTerminal.Cone

Relations between Cone, WithTerminal and Over #

Given categories C and J, an object X : C and a functor K : J ⥤ Over X, it has an obvious lift liftFromOver K : WithTerminal J ⥤ C, namely, send the terminal object to X. These two functors have equivalent categories of cones (coneEquiv). As a corollary, the limit of K is the limit of liftFromOver K, and viceversa.

The category of functors J ⥤ Over X can be seen as part of a comma category, namely the comma category constructed from the identity of the category of functors J ⥤ C and the functor that maps X : C to the constant functor J ⥤ C.

Given a functor K : J ⥤ Over X, it is mapped to a natural transformation from the obvious functor J ⥤ C to the constant functor X.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem CategoryTheory.WithTerminal.commaFromOver_map_left {C : Type u₁} [Category.{v₁, u₁} C] {J : Type w} [Category.{w', w} J] {X : C} {X✝ Y✝ : Functor J (Over X)} (f : X✝ Y✝) :
    @[simp]
    @[simp]

    For any functor K : J ⥤ Over X, there is a canonical extension WithTerminal J ⥤ C, that sends star to X.

    Equations
    Instances For
      @[simp]
      theorem CategoryTheory.WithTerminal.liftFromOver_obj_obj {C : Type u₁} [Category.{v₁, u₁} C] {J : Type w} [Category.{w', w} J] {X : C} (X✝ : Functor J (Over X)) (X✝ : WithTerminal J) :
      (liftFromOver.obj X✝).obj X✝ = match X✝ with | of x => (X✝.obj x).left | star => X
      @[simp]
      theorem CategoryTheory.WithTerminal.liftFromOver_map_app {C : Type u₁} [Category.{v₁, u₁} C] {J : Type w} [Category.{w', w} J] {X : C} {X✝ Y✝ : Functor J (Over X)} (f : X✝ Y✝) (x : WithTerminal J) :
      (liftFromOver.map f).app x = match x with | of x => (f.app x).left | star => CategoryStruct.id X
      @[simp]
      theorem CategoryTheory.WithTerminal.liftFromOver_obj_map {C : Type u₁} [Category.{v₁, u₁} C] {J : Type w} [Category.{w', w} J] {X : C} (X✝ : Functor J (Over X)) {X✝ Y : WithTerminal J} (f : X✝ Y) :
      (liftFromOver.obj X✝).map f = match X✝, Y, f with | of a, of a_1, f => (X✝.map (down f)).left | of x, star, x_1 => (X✝.obj x).hom | star, star, x => CategoryStruct.id X

      The extension of a functor to over categories behaves well with compositions.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem CategoryTheory.WithTerminal.liftFromOverComp_inv_app {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] {J : Type w} [Category.{w', w} J] {X : C} {K : Functor J (Over X)} {F : Functor C D} (x✝ : WithTerminal J) :

        Given a functor K : J ⥤ Over X and its extension liftFromOver K : WithTerminal J ⥤ C, there is an obvious equivalence between cones of these two functors. A cone of K is an object of Over X, so it has the form t ⟶ X. Equivalently, a cone of WithTerminal K is an object t : C, and we can recover the structure morphism as π.app X : t ⟶ X.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          @[simp]
          theorem CategoryTheory.WithTerminal.coneEquiv_functor_map_hom {C : Type u₁} [Category.{v₁, u₁} C] {J : Type w} [Category.{w', w} J] {X : C} {K : Functor J (Over X)} {t₁ t₂ : Limits.Cone K} (f : t₁ t₂) :

          A cone t of K : J ⥤ Over X is a limit if and only if the corresponding cone coneLift t of liftFromOver.obj K : WithTerminal K ⥤ C is a limit.

          Equations
          Instances For

            The category of functors J ⥤ Under X can be seen as part of a comma category, namely the comma category constructed from the identity of the category of functors J ⥤ C and the functor that maps X : C to the constant functor J ⥤ C.

            Given a functor K : J ⥤ Under X, it is mapped to a natural transformation to the obvious functor J ⥤ C from the constant functor X.

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

              For any functor K : J ⥤ Under X, there is a canonical extension WithInitial J ⥤ C, that sends star to X.

              Equations
              Instances For
                @[simp]
                theorem CategoryTheory.WithInitial.liftFromUnder_obj_obj {C : Type u₁} [Category.{v₁, u₁} C] {J : Type w} [Category.{w', w} J] {X : C} (X✝ : Functor J (Under X)) (X✝ : WithInitial J) :
                (liftFromUnder.obj X✝).obj X✝ = match X✝ with | of x => (X✝.obj x).right | star => X
                @[simp]
                theorem CategoryTheory.WithInitial.liftFromUnder_map_app {C : Type u₁} [Category.{v₁, u₁} C] {J : Type w} [Category.{w', w} J] {X : C} {X✝ Y✝ : Functor J (Under X)} (f : X✝ Y✝) (x : WithInitial J) :
                (liftFromUnder.map f).app x = match x with | of x => (f.app x).right | star => CategoryStruct.id X
                @[simp]
                theorem CategoryTheory.WithInitial.liftFromUnder_obj_map {C : Type u₁} [Category.{v₁, u₁} C] {J : Type w} [Category.{w', w} J] {X : C} (X✝ : Functor J (Under X)) {X✝ Y : WithInitial J} (f : X✝ Y) :
                (liftFromUnder.obj X✝).map f = match X✝, Y, f with | of a, of a_1, f => (X✝.map (down f)).right | star, of a, x => (X✝.obj a).hom | star, star, x => CategoryStruct.id X

                The extension of a functor to under categories behaves well with compositions.

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

                  Given a functor K : J ⥤ Under X and its extension liftFromUnder K : WithInitial J ⥤ C, there is an obvious equivalence between cocones of these two functors. A cocone of K is an object of Under X, so it has the form X ⟶ t. Equivalently, a cocone of WithInitial K is an object t : C, and we can recover the structure morphism as ι.app X : X ⟶ t.

                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    @[simp]
                    theorem CategoryTheory.WithInitial.coconeEquiv_functor_map_hom {C : Type u₁} [Category.{v₁, u₁} C] {J : Type w} [Category.{w', w} J] {X : C} {K : Functor J (Under X)} {t₁ t₂ : Limits.Cocone K} (f : t₁ t₂) :

                    A cocone t of K : J ⥤ Under X is a colimit if and only if the corresponding cocone coconeLift t of liftFromUnder.obj K : WithInitial K ⥤ C is a colimit.

                    Equations
                    Instances For