Documentation

Mathlib.CategoryTheory.ChosenFiniteProducts.FunctorCategory

Functor categories have chosen finite products #

If C is a category with chosen finite products, then so is J ⥤ C.

The chosen terminal object in J ⥤ C is terminal.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem CategoryTheory.Functor.chosenProd_map {J : Type u_1} {C : Type u_2} [CategoryTheory.Category.{u_3, u_1} J] [CategoryTheory.Category.{u_4, u_2} C] [CategoryTheory.ChosenFiniteProducts C] (F₁ : CategoryTheory.Functor J C) (F₂ : CategoryTheory.Functor J C) :
    ∀ {X Y : J} (φ : X Y), (F₁.chosenProd F₂).map φ = CategoryTheory.MonoidalCategory.tensorHom (F₁.map φ) (F₂.map φ)

    The chosen binary product on J ⥤ C.

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

      The first projection chosenProd F₁ F₂ ⟶ F₁.

      Equations
      Instances For

        The second projection chosenProd F₁ F₂ ⟶ F₂.

        Equations
        Instances For

          Functor.chosenProd F₁ F₂ is a binary product of F₁ and F₂.

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