Documentation

Mathlib.CategoryTheory.Adjunction.Evaluation

Adjunctions involving evaluation #

We show that evaluation of functors have adjoints, given the existence of (co)products.

The left adjoint of evaluation.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem CategoryTheory.evaluationLeftAdjoint_map_app {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] (D : Type u₂) [CategoryTheory.Category.{v₂, u₂} D] [∀ (a b : C), CategoryTheory.Limits.HasCoproductsOfShape (a b) D] (c : C) {x✝ d₂ : D} (f : x✝ d₂) (x✝¹ : C) :

    The adjunction showing that evaluation is a right adjoint.

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

      See also the file CategoryTheory.Limits.FunctorCategory.EpiMono for a similar result under a HasPullbacks assumption.

      The right adjoint of evaluation.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem CategoryTheory.evaluationRightAdjoint_map_app {C : Type u₁} [CategoryTheory.Category.{v₁, u₁} C] (D : Type u₂) [CategoryTheory.Category.{v₂, u₂} D] [∀ (a b : C), CategoryTheory.Limits.HasProductsOfShape (a b) D] (c : C) {X✝ Y✝ : D} (f : X✝ Y✝) (x✝ : C) :

        The adjunction showing that evaluation is a left adjoint.

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

          See also the file CategoryTheory.Limits.FunctorCategory.EpiMono for a similar result under a HasPushouts assumption.