Functors out of sums of categories. #
This file records the universal property of sums of categories as an equivalence of
categories Sum.functorEquiv : A ⊕ A' ⥤ B ≌ (A ⥤ B) × (A' ⥤ B)
, and characterizes its
precompositions with the left and right inclusion as corresponding to the projections on
the product side.
The equivalence between functors from a sum and the product of the functor categories.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Composing the forward direction of functorEquiv
with the first projection is the same as
precomposition with inl_ A A'
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Composing the forward direction of functorEquiv
with the second projection is the same as
precomposition with inr_ A A'
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Composing the backward direction of functorEquiv
with precomposition with inl_ A A'
.
is naturally isomorphic to the first projection.
Equations
- CategoryTheory.Sum.functorEquivInverseCompWhiskeringLeftInlIso = CategoryTheory.NatIso.ofComponents (fun (x : CategoryTheory.Functor A B × CategoryTheory.Functor A' B) => x.1.inlCompSum' x.2) ⋯
Instances For
Composing the backward direction of functorEquiv
with the second projection is the same as
precomposition with inr_ A A'
.
Equations
- CategoryTheory.Sum.functorEquivInverseCompWhiskeringLeftInrIso = CategoryTheory.NatIso.ofComponents (fun (x : CategoryTheory.Functor A B × CategoryTheory.Functor A' B) => x.1.inrCompSum' x.2) ⋯
Instances For
A consequence of functorEquiv
: we can construct a natural transformation of functors
A ⊕ A' ⥤ B
from the data of natural transformations of their whiskering with inl_
and inr_
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A consequence of functorEquiv
: we can construct a natural isomorphism of functors
A ⊕ A' ⥤ B
from the data of natural isomorphisms of their whiskering with inl_
and inr_
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
functorEquiv A A' B
transforms Swap.equivalence
into Prod.braiding
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The equivalence Sum.functorEquiv
sends associativity of sums to associativity of products
Equations
- One or more equations did not get rendered due to their size.