Documentation

Mathlib.CategoryTheory.Adjunction.Over

Adjunctions related to the over category #

Construct the left adjoint star X to Over.forget X : Over X ⥤ C.

TODO #

Show star X itself has a left adjoint provided C is locally cartesian closed.

@[simp]
theorem CategoryTheory.star_obj_hom {C : Type u} [CategoryTheory.Category.{v, u} C] (X : C) [CategoryTheory.Limits.HasBinaryProducts C] (X : C) :
((CategoryTheory.star X).obj X).hom = CategoryTheory.Limits.prod.fst

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

Instances For

    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 ⨯ -.

    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 ⨯ -.