Cartesian products of categories #
We define the category instance on C × D
when C
and D
are categories.
We define:
sectL C Z
: the functorC ⥤ C × D
given byX ↦ ⟨X, Z⟩
sectR Z D
: the functorD ⥤ C × D
given byY ↦ ⟨Z, Y⟩
fst
: the functor⟨X, Y⟩ ↦ X
snd
: the functor⟨X, Y⟩ ↦ Y
swap
: the functorC × D ⥤ D × C
given by⟨X, Y⟩ ↦ ⟨Y, X⟩
(and the fact this is an equivalence)
We further define evaluation : C ⥤ (C ⥤ D) ⥤ D
and evaluationUncurried : C × (C ⥤ D) ⥤ D
,
and products of functors and natural transformations, written F.prod G
and α.prod β
.
prod C D
gives the cartesian product of two categories.
Equations
Two rfl lemmas that cannot be generated by @[simps]
.
Construct a morphism in a product category by giving its constituent components.
This constructor should be preferred over Prod.mk
, because lean infers better the
source and target of the resulting morphism.
Equations
Instances For
Construct a morphism in a product category by giving its constituent components.
This constructor should be preferred over Prod.mk
, because lean infers better the
source and target of the resulting morphism.
Equations
Instances For
The isomorphism between (X.1, X.2)
and X
.
Equations
Instances For
Construct an isomorphism in C × D
out of two isomorphisms in C
and D
.
Equations
Instances For
Category.uniformProd C D
is an additional instance specialised so both factors have the same
universe levels. This helps typeclass resolution.
Equations
sectL C Z
is the functor C ⥤ C × D
given by X ↦ (X, Z)
.
Equations
Instances For
sectR Z D
is the functor D ⥤ C × D
given by Y ↦ (Z, Y)
.
Equations
Instances For
fst
is the functor (X, Y) ↦ X
.
Equations
Instances For
snd
is the functor (X, Y) ↦ Y
.
Equations
Instances For
The functor swapping the factors of a cartesian product of categories, C × D ⥤ D × C
.
Equations
Instances For
Swapping the factors of a cartesian product of categories twice is naturally isomorphic to the identity functor.
Equations
Instances For
The equivalence, given by swapping factors, between C × D
and D × C
.
Equations
Instances For
Any morphism in a product factors as a morphsim whose left component is an identity followed by a morphism whose right component is an identity.
Any morphism in a product factors as a morphsim whose right component is an identity followed by a morphism whose left component is an identity.
The "evaluation at X
" functor, such that
(evaluation.obj X).obj F = F.obj X
,
which is functorial in both X
and F
.
Equations
Instances For
The "evaluation of F
at X
" functor,
as a functor C × (C ⥤ D) ⥤ D
.
Equations
Instances For
The constant functor followed by the evaluation functor is just the identity.
Equations
Instances For
The cartesian product of two functors.
Equations
Instances For
Similar to prod
, but both functors start from the same category A
Equations
Instances For
The product F.prod' G
followed by projection on the first component is isomorphic to F
Equations
Instances For
The product F.prod' G
followed by projection on the second component is isomorphic to G
Equations
Instances For
The diagonal functor.
Equations
Instances For
The cartesian product of two natural transformations.
Equations
Instances For
The cartesian product of two natural transformations where both functors have the same source.
Equations
Instances For
The cartesian product functor between functor categories
Equations
Instances For
The cartesian product of two natural isomorphisms.
Equations
Instances For
The cartesian product of two equivalences of categories.
Equations
Instances For
F.flip
composed with evaluation is the same as evaluating F
.
Equations
Instances For
F
composed with evaluation is the same as evaluating F.flip
.
Equations
Instances For
Whiskering by F
and then evaluating at a
is the same as evaluating at F.obj a
.
Equations
Instances For
Whiskering by F
and then evaluating at a
is the same as evaluating at F.obj a
.
Whiskering by F
and then evaluating at a
is the same as evaluating at F
and then
applying F
.
Equations
Instances For
Whiskering by F
and then evaluating at a
is the same as evaluating at F
and then
applying F
.
The forward direction for functorProdFunctorEquiv
Equations
Instances For
The backward direction for functorProdFunctorEquiv
Equations
Instances For
The unit isomorphism for functorProdFunctorEquiv
Equations
Instances For
The counit isomorphism for functorProdFunctorEquiv
Equations
Instances For
The equivalence of categories between (A ⥤ B) × (A ⥤ C)
and A ⥤ (B × C)
Equations
Instances For
The equivalence between the opposite of a product and the product of the opposites.