Construction of the localized category #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file constructs the localized category, obtained by formally inverting
a class of maps W : morphism_property C
in a category C
.
We first construct a quiver loc_quiver W
whose objects are the same as those
of C
and whose maps are the maps in C
and placeholders for the formal
inverses of the maps in W
.
The localized category W.localization
is obtained by taking the quotient
of the path category of loc_quiver W
by the congruence generated by four
types of relations.
The obvious functor Q W : C ⥤ W.localization
satisfies the universal property
of the localization. Indeed, if G : C ⥤ D
sends morphisms in W
to isomorphisms
in D
(i.e. we have hG : W.is_inverted_by G
), then there exists a unique functor
G' : W.localization ⥤ D
such that Q W ≫ G' = G
. This G'
is lift G hG
.
The expected property of lift G hG
if expressed by the lemma fac
and the
uniqueness is expressed by uniq
.
References #
- obj : C
If W : morphism_property C
, loc_quiver W
is a quiver with the same objects
as C
, and whose morphisms are those in C
and placeholders for formal
inverses of the morphisms in W
.
Instances for category_theory.localization.construction.loc_quiver
- category_theory.localization.construction.loc_quiver.has_sizeof_inst
- category_theory.localization.construction.loc_quiver.quiver
Equations
- category_theory.localization.construction.loc_quiver.quiver W = {hom := λ (A B : category_theory.localization.construction.loc_quiver W), (A.obj ⟶ B.obj) ⊕ {f // W f}}
The object in the path category of loc_quiver W
attached to an object in
the category C
Equations
The morphism in the path category associated to a morphism in the original category.
Equations
The morphism in the path category corresponding to a formal inverse.
Equations
- category_theory.localization.construction.ψ₂ W w hw = category_theory.paths.of.map (sum.inr ⟨w, hw⟩)
- id : ∀ {C : Type u_1} [_inst_1 : category_theory.category C] {W : category_theory.morphism_property C} (X : C), category_theory.localization.construction.relations W (category_theory.localization.construction.ψ₁ W (𝟙 X)) (𝟙 (category_theory.localization.construction.ι_paths W X))
- comp : ∀ {C : Type u_1} [_inst_1 : category_theory.category C] {W : category_theory.morphism_property C} {X Y Z : C} (f : X ⟶ Y) (g : Y ⟶ Z), category_theory.localization.construction.relations W (category_theory.localization.construction.ψ₁ W (f ≫ g)) (category_theory.localization.construction.ψ₁ W f ≫ category_theory.localization.construction.ψ₁ W g)
- Winv₁ : ∀ {C : Type u_1} [_inst_1 : category_theory.category C] {W : category_theory.morphism_property C} {X Y : C} (w : X ⟶ Y) (hw : W w), category_theory.localization.construction.relations W (category_theory.localization.construction.ψ₁ W w ≫ category_theory.localization.construction.ψ₂ W w hw) (𝟙 (category_theory.localization.construction.ι_paths W X))
- Winv₂ : ∀ {C : Type u_1} [_inst_1 : category_theory.category C] {W : category_theory.morphism_property C} {X Y : C} (w : X ⟶ Y) (hw : W w), category_theory.localization.construction.relations W (category_theory.localization.construction.ψ₂ W w hw ≫ category_theory.localization.construction.ψ₁ W w) (𝟙 (category_theory.localization.construction.ι_paths W Y))
The relations by which we take the quotient in order to get the localized category.
The localized category obtained by formally inverting the morphisms
in W : morphism_property C
Equations
Instances for category_theory.morphism_property.localization
The obvious functor C ⥤ W.localization
Equations
- W.Q = {obj := λ (X : C), (category_theory.quotient.functor (category_theory.localization.construction.relations W)).obj (category_theory.paths.of.obj {obj := X}), map := λ (X Y : C) (f : X ⟶ Y), (category_theory.quotient.functor (category_theory.localization.construction.relations W)).map (category_theory.localization.construction.ψ₁ W f), map_id' := _, map_comp' := _}
Instances for category_theory.morphism_property.Q
The isomorphism in W.localization
associated to a morphism w
in W
Equations
- category_theory.localization.construction.Wiso w hw = {hom := W.Q.map w, inv := (category_theory.quotient.functor (category_theory.localization.construction.relations W)).map (category_theory.paths.of.map (sum.inr ⟨w, hw⟩)), hom_inv_id' := _, inv_hom_id' := _}
The formal inverse in W.localization
of a morphism w
in W
.
The lifting of a functor to the path category of loc_quiver W
Equations
- category_theory.localization.construction.lift_to_path_category G hG = category_theory.Quiv.lift {obj := λ (X : category_theory.localization.construction.loc_quiver W), G.obj X.obj, map := λ (X Y : category_theory.localization.construction.loc_quiver W) (ᾰ : X ⟶ Y), sum.cases_on ᾰ (λ (f : X.obj ⟶ Y.obj), G.map f) (λ (ᾰ : {f // W f}), ᾰ.cases_on (λ (g : Y.obj ⟶ X.obj) (hg : W g), category_theory.inv (G.map g)))}
The lifting of a functor C ⥤ D
inverting W
as a functor W.localization ⥤ D
Equations
Instances for category_theory.localization.construction.lift
The canonical bijection between objects in a category and its
localization with respect to a morphism_property W
A morphism_property
in W.localization
is satisfied by all
morphisms in the localized category if it contains the image of the
morphisms in the original category, the inverses of the morphisms
in W
and if it is stable under composition
A morphism_property
in W.localization
is satisfied by all
morphisms in the localized category if it contains the image of the
morphisms in the original category, if is stable under composition
and if the property is stable by passing to inverses.
If F₁
and F₂
are functors W.localization ⥤ D
and if we have
τ : W.Q ⋙ F₁ ⟶ W.Q ⋙ F₂
, we shall define a natural transformation F₁ ⟶ F₂
.
This is the app
field of this natural transformation.
If F₁
and F₂
are functors W.localization ⥤ D
, a natural transformation F₁ ⟶ F₂
can be obtained from a natural transformation W.Q ⋙ F₁ ⟶ W.Q ⋙ F₂
.
The functor (W.localization ⥤ D) ⥤ (W.functors_inverting D)
induced by the
composition with W.Q : C ⥤ W.localization
.
Equations
- category_theory.localization.construction.whiskering_left_equivalence.functor W D = category_theory.full_subcategory.lift (λ (F : C ⥤ D), W.is_inverted_by F) ((category_theory.whiskering_left C W.localization D).obj W.Q) _
The function (W.functors_inverting D) ⥤ (W.localization ⥤ D)
induced by
construction.lift
.
Equations
- category_theory.localization.construction.whiskering_left_equivalence.inverse W D = {obj := λ (G : W.functors_inverting D), category_theory.localization.construction.lift G.obj _, map := λ (G₁ G₂ : W.functors_inverting D) (τ : G₁ ⟶ G₂), category_theory.localization.construction.nat_trans_extension (category_theory.eq_to_hom _ ≫ τ ≫ category_theory.eq_to_hom _), map_id' := _, map_comp' := _}
The unit isomorphism of the equivalence of categories whiskering_left_equivalence W D
.
The counit isomorphism of the equivalence of categories whiskering_left_equivalence W D
.
The equivalence of categories (W.localization ⥤ D) ≌ (W.functors_inverting D)
induced by the composition with W.Q : C ⥤ W.localization
.
Equations
- category_theory.localization.construction.whiskering_left_equivalence W D = {functor := category_theory.localization.construction.whiskering_left_equivalence.functor W D _inst_2, inverse := category_theory.localization.construction.whiskering_left_equivalence.inverse W D _inst_2, unit_iso := category_theory.localization.construction.whiskering_left_equivalence.unit_iso W D _inst_2, counit_iso := category_theory.localization.construction.whiskering_left_equivalence.counit_iso W D _inst_2, functor_unit_iso_comp' := _}