Documentation

Mathlib.CategoryTheory.Comma.Over.Pullback

Adjunctions related to the over category #

In a category with pullbacks, for any morphism f : X ⟶ Y, the functor Over.map f : Over X ⥤ Over Y has a right adjoint Over.pullback f.

In a category with binary products, for any object X the functor Over.forget X : Over X ⥤ C has a right adjoint Over.star X.

Main declarations #

TODO #

Show star X itself has a right adjoint provided C is cartesian closed and has pullbacks.

def CategoryTheory.Over.pullback {C : Type u} [Category.{v, u} C] [Limits.HasPullbacks C] {X Y : C} (f : X Y) :
Functor (Over Y) (Over X)

In a category with pullbacks, a morphism f : X ⟶ Y induces a functor Over Y ⥤ Over X, by pulling back a morphism along f.

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

    Over.map f is left adjoint to Over.pullback f.

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

      pullback (𝟙 X) : Over X ⥤ Over X is the identity functor.

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

        pullback commutes with composition (up to natural isomorphism).

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

          The functor from C to Over X which sends Y : C to π₁ : X ⨯ Y ⟶ X, sometimes denoted X*.

          Equations
          Instances For
            @[simp]
            theorem CategoryTheory.Over.star_obj_left {C : Type u} [Category.{v, u} C] (X : C) [Limits.HasBinaryProducts C] (X✝ : C) :
            ((star X).obj X✝).left = (X X✝)
            @[simp]
            theorem CategoryTheory.Over.star_map_left {C : Type u} [Category.{v, u} C] (X : C) [Limits.HasBinaryProducts C] {X✝ Y✝ : C} (f : X✝ Y✝) :

            The functor Over.forget X : Over X ⥤ C has a right adjoint given by star X.

            Note that the binary products assumption is necessary: the existence of a right adjoint to Over.forget X is equivalent to the existence of each binary product X ⨯ -.

            Equations
            Instances For

              Note that the binary products assumption is necessary: the existence of a right adjoint to Over.forget X is equivalent to the existence of each binary product X ⨯ -.

              When C has pushouts, a morphism f : X ⟶ Y induces a functor Under X ⥤ Under Y, by pushing a morphism forward along f.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                @[simp]
                theorem CategoryTheory.Under.pushout_map {C : Type u} [Category.{v, u} C] [Limits.HasPushouts C] {X Y : C} (f : X Y) (x : Under X) {x' : Under X} {u : x x'} :
                @[simp]
                theorem CategoryTheory.Under.pushout_obj {C : Type u} [Category.{v, u} C] [Limits.HasPushouts C] {X Y : C} (f : X Y) (x : Under X) :

                Under.pushout f is left adjoint to Under.map f.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  @[simp]
                  theorem CategoryTheory.Under.mapPushoutAdj_unit_app {C : Type u} [Category.{v, u} C] [Limits.HasPushouts C] {X Y : C} (f : X Y) (X✝ : Under X) :

                  pushout (𝟙 X) : Under X ⥤ Under X is the identity functor.

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

                    pushout commutes with composition (up to natural isomorphism).

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

                      If X : C is initial, then the under category of X is equivalent to C.

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