The action of trifunctors on graded objects #
Given a trifunctor F. C₁ ⥤ C₂ ⥤ C₃ ⥤ C₄
and types I₁
, I₂
and I₃
, we define a functor
GradedObject I₁ C₁ ⥤ GradedObject I₂ C₂ ⥤ GradedObject I₃ C₃ ⥤ GradedObject (I₁ × I₂ × I₃) C₄
(see mapTrifunctor
). When we have a map p : I₁ × I₂ × I₃ → J
and suitable coproducts
exists, we define a functor
GradedObject I₁ C₁ ⥤ GradedObject I₂ C₂ ⥤ GradedObject I₃ C₃ ⥤ GradedObject J C₄
(see mapTrifunctorMap
) which sends graded objects X₁
, X₂
, X₃
to the graded object
which sets j
to the coproduct of the objects ((F.obj (X₁ i₁)).obj (X₂ i₂)).obj (X₃ i₃)
for p ⟨i₁, i₂, i₃⟩ = j
.
This shall be used in order to construct the associator isomorphism for the monoidal
category structure on GradedObject I C
induced by a monoidal structure on C
and
an additive monoid structure on I
(TODO @joelriou).
Auxiliary definition for mapTrifunctor
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given a trifunctor F : C₁ ⥤ C₂ ⥤ C₃ ⥤ C₄
and types I₁
, I₂
, I₃
,
this is the obvious functor
GradedObject I₁ C₁ ⥤ GradedObject I₂ C₂ ⥤ GradedObject I₃ C₃ ⥤ GradedObject (I₁ × I₂ × I₃) C₄
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The natural transformation mapTrifunctor F I₁ I₂ I₃ ⟶ mapTrifunctor F' I₁ I₂ I₃
induced by a natural transformation F ⟶ F
of trifunctors.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The natural isomorphism mapTrifunctor F I₁ I₂ I₃ ≅ mapTrifunctor F' I₁ I₂ I₃
induced by a natural isomorphism F ≅ F
of trifunctors.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given a trifunctor F : C₁ ⥤ C₂ ⥤ C₃ ⥤ C₃
, graded objects X₁ : GradedObject I₁ C₁
,
X₂ : GradedObject I₂ C₂
, X₃ : GradedObject I₃ C₃
, and a map p : I₁ × I₂ × I₃ → J
,
this is the J
-graded object sending j
to the coproduct of
((F.obj (X₁ i₁)).obj (X₂ i₂)).obj (X₃ i₃)
for p ⟨i₁, i₂, i₃⟩ = k
.
Equations
- CategoryTheory.GradedObject.mapTrifunctorMapObj F p X₁ X₂ X₃ = ((((CategoryTheory.GradedObject.mapTrifunctor F I₁ I₂ I₃).obj X₁).obj X₂).obj X₃).mapObj p
Instances For
The obvious inclusion
((F.obj (X₁ i₁)).obj (X₂ i₂)).obj (X₃ i₃) ⟶ mapTrifunctorMapObj F p X₁ X₂ X₃ j
when
p ⟨i₁, i₂, i₃⟩ = j
.
Equations
- CategoryTheory.GradedObject.ιMapTrifunctorMapObj F p X₁ X₂ X₃ i₁ i₂ i₃ j h = ((((CategoryTheory.GradedObject.mapTrifunctor F I₁ I₂ I₃).obj X₁).obj X₂).obj X₃).ιMapObj p (i₁, i₂, i₃) j h
Instances For
The maps mapTrifunctorMapObj F p X₁ X₂ X₃ ⟶ mapTrifunctorMapObj F p Y₁ Y₂ Y₃
which
express the functoriality of mapTrifunctorMapObj
, see mapTrifunctorMap
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- ⋯ = h
Given a trifunctor F : C₁ ⥤ C₂ ⥤ C₃ ⥤ C₄
, a map p : I₁ × I₂ × I₃ → J
, and
graded objects X₁ : GradedObject I₁ C₁
, X₂ : GradedObject I₂ C₂
and X₃ : GradedObject I₃ C₃
,
this is the J
-graded object sending j
to the coproduct of
((F.obj (X₁ i₁)).obj (X₂ i₂)).obj (X₃ i₃)
for p ⟨i₁, i₂, i₃⟩ = j
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given a trifunctor F : C₁ ⥤ C₂ ⥤ C₃ ⥤ C₄
and a map p : I₁ × I₂ × I₃ → J
,
this is the functor
GradedObject I₁ C₁ ⥤ GradedObject I₂ C₂ ⥤ GradedObject I₃ C₃ ⥤ GradedObject J C₄
sending X₁ : GradedObject I₁ C₁
, X₂ : GradedObject I₂ C₂
and X₃ : GradedObject I₃ C₃
to the J
-graded object sending j
to the coproduct of
((F.obj (X₁ i₁)).obj (X₂ i₂)).obj (X₃ i₃)
for p ⟨i₁, i₂, i₃⟩ = j
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given a map r : I₁ × I₂ × I₃ → J
, a BifunctorComp₁₂IndexData r
consists of the data
of a type I₁₂
, maps p : I₁ × I₂ → I₁₂
and q : I₁₂ × I₃ → J
, such that r
is obtained
by composition of p
and q
.
- I₁₂ : Type u_11
an auxiliary type
- p : I₁ × I₂ → self.I₁₂
a map
I₁ × I₂ → I₁₂
- q : self.I₁₂ × I₃ → J
a map
I₁₂ × I₃ → J
Instances For
Given bifunctors F₁₂ : C₁ ⥤ C₂ ⥤ C₁₂
, G : C₁₂ ⥤ C₃ ⥤ C₄
, graded objects
X₁ : GradedObject I₁ C₁
, X₂ : GradedObject I₂ C₂
, X₃ : GradedObject I₃ C₃
and
ρ₁₂ : BifunctorComp₁₂IndexData r
, this asserts that for all i₁₂ : ρ₁₂.I₁₂
and i₃ : I₃
,
the functor G(-, X₃ i₃)
commutes with the coproducts of the F₁₂(X₁ i₁, X₂ i₂)
such that ρ₁₂.p ⟨i₁, i₂⟩ = i₁₂
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The inclusion of (G.obj ((F₁₂.obj (X₁ i₁)).obj (X₂ i₂))).obj (X₃ i₃)
in
mapBifunctorMapObj G ρ₁₂.q (mapBifunctorMapObj F₁₂ ρ₁₂.p X₁ X₂) X₃ j
when r (i₁, i₂, i₃) = j
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The cofan consisting of the inclusions given by ιMapBifunctor₁₂BifunctorMapObj
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The cofan cofan₃MapBifunctor₁₂BifunctorMapObj
is a colimit, see the induced isomorphism
mapBifunctorComp₁₂MapObjIso
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The action on graded objects of a trifunctor obtained by composition of two bifunctors can be computed as a composition of the actions of these two bifunctors.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Constructor for morphisms from
mapBifunctorMapObj G ρ₁₂.q (mapBifunctorMapObj F₁₂ ρ₁₂.p X₁ X₂) X₃ j
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Given a map r : I₁ × I₂ × I₃ → J
, a BifunctorComp₂₃IndexData r
consists of the data
of a type I₂₃
, maps p : I₂ × I₃ → I₂₃
and q : I₁ × I₂₃ → J
, such that r
is obtained
by composition of p
and q
.
- I₂₃ : Type u_11
an auxiliary type
- p : I₂ × I₃ → self.I₂₃
a map
I₂ × I₃ → I₂₃
- q : I₁ × self.I₂₃ → J
a map
I₁ × I₂₃ → J
Instances For
Given bifunctors F : C₁ ⥤ C₂₃ ⥤ C₄
, G₂₃ : C₂ ⥤ C₃ ⥤ C₂₃
, graded objects
X₁ : GradedObject I₁ C₁
, X₂ : GradedObject I₂ C₂
, X₃ : GradedObject I₃ C₃
and
ρ₂₃ : BifunctorComp₂₃IndexData r
, this asserts that for all i₁ : I₁
and i₂₃ : ρ₂₃.I₂₃
,
the functor F(X₁ i₁, _)
commutes with the coproducts of the G₂₃(X₂ i₂, X₃ i₃)
such that ρ₂₃.p ⟨i₂, i₃⟩ = i₂₃
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The inclusion of (F.obj (X₁ i₁)).obj ((G₂₃.obj (X₂ i₂)).obj (X₃ i₃))
in
mapBifunctorMapObj F ρ₂₃.q X₁ (mapBifunctorMapObj G₂₃ ρ₂₃.p X₂ X₃) j
when r (i₁, i₂, i₃) = j
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The cofan consisting of the inclusions given by ιMapBifunctorBifunctor₂₃MapObj
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The cofan cofan₃MapBifunctorBifunctor₂₃MapObj
is a colimit, see the induced isomorphism
mapBifunctorComp₁₂MapObjIso
.
Instances For
The action on graded objects of a trifunctor obtained by composition of two bifunctors can be computed as a composition of the actions of these two bifunctors.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Constructor for morphisms from
mapBifunctorMapObj F ρ₂₃.q X₁ (mapBifunctorMapObj G₂₃ ρ₂₃.p X₂ X₃) j
.
Equations
- One or more equations did not get rendered due to their size.