Localization of monoidal categories #
Let C
be a monoidal category equipped with a class of morphisms W
which
is compatible with the monoidal category structure: this means W
is multiplicative and stable by left and right whiskerings (this is
the type class W.IsMonoidal
). Let L : C ⥤ D
be a localization functor
for W
. In the file, we construct a monoidal category structure
on D
such that the localization functor is monoidal. The structure
is actually defined on a type synonym LocalizedMonoidal L W ε
.
Here, the data ε : L.obj (𝟙_ C) ≅ unit
is an isomorphism to some
object unit : D
which allows the user to provide a preferred choice
of a unit object.
A class of morphisms W
in a monoidal category is monoidal if it is multiplicative
and stable under left and right whiskering. Under this condition, the localized
category can be equipped with a monoidal category structure, see LocalizedMonoidal
.
- whiskerLeft (X : C) {Y₁ Y₂ : C} (g : Y₁ ⟶ Y₂) (hg : W g) : W (MonoidalCategoryStruct.whiskerLeft X g)
- whiskerRight {X₁ X₂ : C} (f : X₁ ⟶ X₂) (hf : W f) (Y : C) : W (MonoidalCategoryStruct.whiskerRight f Y)
Instances
Given a monoidal category C
, a localization functor L : C ⥤ D
with respect
to W : MorphismProperty C
which satisfies W.IsMonoidal
, and a choice
of object unit : D
with an isomorphism L.obj (𝟙_ C) ≅ unit
, this is a
type synonym for D
on which we define the localized monoidal category structure.
Equations
- CategoryTheory.LocalizedMonoidal L W x✝ = D
Instances For
The monoidal functor from a monoidal category C
to
its localization LocalizedMonoidal L W ε
.
Equations
Instances For
The isomorphism ε : L.obj (𝟙_ C) ≅ unit
,
as (toMonoidalCategory L W ε).obj (𝟙_ C) ≅ unit
.
Equations
Instances For
The localized tensor product, as a bifunctor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
The bifunctor tensorBifunctor
on LocalizedMonoidal L W ε
is induced by
curriedTensor C
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
The left unitor in the localized monoidal category LocalizedMonoidal L W ε
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The right unitor in the localized monoidal category LocalizedMonoidal L W ε
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The associator in the localized monoidal category LocalizedMonoidal L W ε
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
The compatibility isomorphism of the monoidal functor toMonoidalCategory L W ε
with respect to the tensor product.
Equations
- CategoryTheory.Localization.Monoidal.μ L W ε X Y = ((CategoryTheory.Localization.Monoidal.tensorBifunctorIso L W ε).app X).app Y
Instances For
Equations
- CategoryTheory.Localization.Monoidal.instMonoidalCategoryLocalizedMonoidal L W ε = CategoryTheory.MonoidalCategory.mk ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯ ⋯
Equations
- One or more equations did not get rendered due to their size.