Lifting of trifunctors #
In this file, in the context of the localization of categories, we extend the notion
of lifting of functors to the case of trifunctors
(see also the file Localization.Bifunctor
for the case of bifunctors).
The main result in this file is that we can localize "associator" isomorphisms
(see the definition Localization.associator
).
Classes of morphisms W₁ : MorphismProperty C₁
, W₂ : MorphismProperty C₂
and
W₃ : MorphismProperty C₃
are said to be inverted by F : C₁ ⥤ C₂ ⥤ C₃ ⥤ E
if
W₁.prod (W₂.prod W₃)
is inverted by the
functor currying₃.functor.obj F : C₁ × C₂ × C₃ ⥤ E
.
Equations
- W₁.IsInvertedBy₃ W₂ W₃ F = (W₁.prod (W₂.prod W₃)).IsInvertedBy (CategoryTheory.currying₃.functor.obj F)
Instances For
Given functors L₁ : C₁ ⥤ D₁
, L₂ : C₂ ⥤ D₂
, L₃ : C₃ ⥤ D₃
,
morphisms properties W₁
on C₁
, W₂
on C₂
, W₃
on C₃
, and
functors F : C₁ ⥤ C₂ ⥤ C₃ ⥤ E
and F' : D₁ ⥤ D₂ ⥤ D₃ ⥤ E
, we say
Lifting₃ L₁ L₂ L₃ W₁ W₂ W₃ F F'
holds if F
is induced by F'
, up to an isomorphism.
- iso' : ((((whiskeringLeft₃ E).obj L₁).obj L₂).obj L₃).obj F' ≅ F
the isomorphism
((((whiskeringLeft₃ E).obj L₁).obj L₂).obj L₃).obj F' ≅ F
expressing thatF
is induced byF'
up to an isomorphism
Instances
The isomorphism ((((whiskeringLeft₃ E).obj L₁).obj L₂).obj L₃).obj F' ≅ F
when Lifting₃ L₁ L₂ L₃ W₁ W₂ W₃ F F'
holds.
Equations
- CategoryTheory.Localization.Lifting₃.iso L₁ L₂ L₃ W₁ W₂ W₃ F F' = CategoryTheory.Localization.Lifting₃.iso' W₁ W₂ W₃
Instances For
Equations
- CategoryTheory.Localization.Lifting₃.uncurry L₁ L₂ L₃ W₁ W₂ W₃ F F' = { iso' := CategoryTheory.uncurry₃.mapIso (CategoryTheory.Localization.Lifting₃.iso L₁ L₂ L₃ W₁ W₂ W₃ F F') }
Given localization functor L₁ : C₁ ⥤ D₁
, L₂ : C₂ ⥤ D₂
and L₃ : C₃ ⥤ D₃
with respect to W₁ : MorphismProperty C₁
, W₂ : MorphismProperty C₂
and
W₃ : MorphismProperty C₃
respectively, and a trifunctor F : C₁ ⥤ C₂ ⥤ C₃ ⥤ E
which inverts W₁
, W₂
and W₃
, this is the induced localized
trifunctor D₁ ⥤ D₂ ⥤ D₃ ⥤ E
.
Equations
- CategoryTheory.Localization.lift₃ F hF L₁ L₂ L₃ = CategoryTheory.curry₃.obj (CategoryTheory.Localization.lift (CategoryTheory.uncurry₃.obj F) hF (L₁.prod (L₂.prod L₃)))
Instances For
Equations
- One or more equations did not get rendered due to their size.
The natural transformation F₁' ⟶ F₂'
of trifunctors induced by a
natural transformation τ : F₁ ⟶ F₂
when Lifting₃ L₁ L₂ L₃ W₁ W₂ W₃ F₁ F₁'
and Lifting₃ L₁ L₂ L₃ W₁ W₂ W₃ F₂ F₂'
hold.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The natural isomorphism F₁' ≅ F₂'
of trifunctors induced by a
natural isomorphism e : F₁ ≅ F₂
when Lifting₃ L₁ L₂ L₃ W₁ W₂ W₃ F₁ F₁'
and Lifting₃ L₁ L₂ L₃ W₁ W₂ W₃ F₂ F₂'
hold.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The construction bifunctorComp₁₂
of a trifunctor by composition of bifunctors
is compatible with localization.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The construction bifunctorComp₂₃
of a trifunctor by composition of bifunctors
is compatible with localization.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The associator isomorphism obtained by localization.
Equations
- One or more equations did not get rendered due to their size.