Binary (co)products of type-valued functors #
Defines an explicit construction of binary products and coproducts of type-valued functors.
Also defines isomorphisms to the categorical product and coproduct, respectively.
prod F G
is the explicit binary product of type-valued functors F
and G
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The first projection of prod F G
, onto F
.
Equations
- CategoryTheory.FunctorToTypes.prod.fst = { app := fun (x : C) (a : (CategoryTheory.FunctorToTypes.prod F G).obj x) => a.1, naturality := ⋯ }
Instances For
The second projection of prod F G
, onto G
.
Equations
- CategoryTheory.FunctorToTypes.prod.snd = { app := fun (x : C) (a : (CategoryTheory.FunctorToTypes.prod F G).obj x) => a.2, naturality := ⋯ }
Instances For
Given natural transformations F ⟶ F₁
and F ⟶ F₂
, construct
a natural transformation F ⟶ prod F₁ F₂
.
Equations
- CategoryTheory.FunctorToTypes.prod.lift τ₁ τ₂ = { app := fun (x : C) (y : F.obj x) => (τ₁.app x y, τ₂.app x y), naturality := ⋯ }
Instances For
The binary fan whose point is prod F G
.
Equations
- CategoryTheory.FunctorToTypes.binaryProductCone F G = CategoryTheory.Limits.BinaryFan.mk CategoryTheory.FunctorToTypes.prod.fst CategoryTheory.FunctorToTypes.prod.snd
Instances For
prod F G
is a limit cone.
Equations
- CategoryTheory.FunctorToTypes.binaryProductLimit F G = { lift := fun (s : CategoryTheory.Limits.BinaryFan F G) => CategoryTheory.FunctorToTypes.prod.lift s.fst s.snd, fac := ⋯, uniq := ⋯ }
Instances For
prod F G
is a binary product for F
and G
.
Equations
- CategoryTheory.FunctorToTypes.binaryProductLimitCone F G = { cone := CategoryTheory.FunctorToTypes.binaryProductCone F G, isLimit := CategoryTheory.FunctorToTypes.binaryProductLimit F G }
Instances For
The categorical binary product of type-valued functors is prod F G
.
Equations
Instances For
Construct an element of (F ⨯ G).obj a
from an element of F.obj a
and
an element of G.obj a
.
Equations
- CategoryTheory.FunctorToTypes.prodMk x y = (CategoryTheory.FunctorToTypes.binaryProductIso F G).inv.app a (x, y)
Instances For
(F ⨯ G).obj a
is in bijection with the product of F.obj a
and G.obj a
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
coprod F G
is the explicit binary coproduct of type-valued functors F
and G
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The left inclusion of F
into coprod F G
.
Equations
Instances For
The right inclusion of G
into coprod F G
.
Equations
Instances For
Given natural transformations F₁ ⟶ F
and F₂ ⟶ F
, construct
a natural transformation coprod F₁ F₂ ⟶ F
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The binary cofan whose point is coprod F G
.
Equations
- CategoryTheory.FunctorToTypes.binaryCoproductCocone F G = CategoryTheory.Limits.BinaryCofan.mk CategoryTheory.FunctorToTypes.coprod.inl CategoryTheory.FunctorToTypes.coprod.inr
Instances For
coprod F G
is a colimit cocone.
Equations
- One or more equations did not get rendered due to their size.
Instances For
coprod F G
is a binary coproduct for F
and G
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The categorical binary coproduct of type-valued functors is coprod F G
.
Equations
Instances For
Construct an element of (F ⨿ G).obj a
from an element of F.obj a
Equations
- CategoryTheory.FunctorToTypes.coprodInl x = (CategoryTheory.FunctorToTypes.binaryCoproductIso F G).inv.app a (Sum.inl x)
Instances For
Construct an element of (F ⨿ G).obj a
from an element of G.obj a
Equations
- CategoryTheory.FunctorToTypes.coprodInr x = (CategoryTheory.FunctorToTypes.binaryCoproductIso F G).inv.app a (Sum.inr x)
Instances For
(F ⨿ G).obj a
is in bijection with disjoint union of F.obj a
and G.obj a
.
Equations
- One or more equations did not get rendered due to their size.