External product of diagrams in a monoidal category #
In a monoidal category C
, given a pair of diagrams K₁ : J₁ ⥤ C
and K₂ : J₂ ⥤ C
, we
introduce the external product K₁ ⊠ K₂ : J₁ × J₂ ⥤ C
as the bifunctor (j₁, j₂) ↦ K₁ j₁ ⊗ K₂ j₂
.
The notation - ⊠ -
is scoped to MonoidalCategory.ExternalProduct
.
The (curried version of the) external product bifunctor: given diagrams
K₁ : J₁ ⥤ C
and K₂ : J₂ ⥤ C
, this is the bifunctor j₁ ↦ j₂ ↦ K₁ j₁ ⊗ K₂ j₂
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The external product bifunctor: given diagrams
K₁ : J₁ ⥤ C
and K₂ : J₂ ⥤ C
, this is the bifunctor (j₁, j₂) ↦ K₁ j₁ ⊗ K₂ j₂
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
An abbreviation for the action of externalProductBifunctor J₁ J₂ C
on objects.
Equations
Instances For
Notation for externalProduct
.
Do open scoped CategoryTheory.MonoidalCategory.ExternalProduct
to bring this notation in scope.
Equations
- One or more equations did not get rendered due to their size.
Instances For
When both diagrams have the same source category, composing the external product with
the diagonal gives the pointwise functor tensor product.
Note that (externalProductCompDiagIso _ _).app (F₁, F₂) : Functor.diag J₁ ⋙ F₁ ⊠ F₂ ≅ F₁ ⊗ F₂
type checks.
Equations
- One or more equations did not get rendered due to their size.
Instances For
When C
is braided, there is an isomorphism Prod.swap _ _ ⋙ F₁ ⊠ F₂ ≅ F₂ ⊠ F₁
, natural
in both F₁
and F₂
.
Note that (externalProductSwap _ _ _).app (F₁, F₂) : Prod.swap _ _ ⋙ F₁ ⊠ F₂ ≅ F₂ ⊠ F₁
type checks.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A version of externalProductSwap
phrased in terms of the curried functors.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Composing F₁ × F₂
with G₁ ⊠ G₂
is isomorphic to (F₁ ⋙ G₁) ⊠ (F₂ ⋙ G₂)
.
Equations
- One or more equations did not get rendered due to their size.