mathlib3 documentation

category_theory.localization.construction

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 #

@[nolint]
  • 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

The relations by which we take the quotient in order to get the localized category.

@[nolint]

The localized category obtained by formally inverting the morphisms in W : morphism_property C

Equations
Instances for category_theory.morphism_property.localization
@[reducible]
def category_theory.localization.construction.Winv {C : Type u_1} [category_theory.category C] {W : category_theory.morphism_property C} {X Y : C} (w : X Y) (hw : W w) :
(category_theory.morphism_property.Q (λ {X Y : C} (w : X Y), W w)).obj Y (category_theory.morphism_property.Q (λ {X Y : C} (w : X Y), W w)).obj X

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
theorem category_theory.localization.construction.uniq {C : Type u_1} [category_theory.category C] {W : category_theory.morphism_property C} {D : Type u_3} [category_theory.category D] (G₁ G₂ : W.localization D) (h : W.Q G₁ = W.Q G₂) :
G₁ = G₂

The canonical bijection between objects in a category and its localization with respect to a morphism_property W

Equations

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

theorem category_theory.localization.construction.morphism_property_is_top' {C : Type u_1} [category_theory.category C] {W : category_theory.morphism_property C} (P : category_theory.morphism_property W.localization) (hP₁ : ⦃X Y : C⦄ (f : X Y), P (W.Q.map f)) (hP₂ : ⦃X Y : W.localization⦄ (e : X Y), P e.hom P e.inv) (hP₃ : P.stable_under_composition) :
P =

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.

Equations

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₂.

Equations
theorem category_theory.localization.construction.nat_trans_hcomp_injective {C : Type u_1} [category_theory.category C] {W : category_theory.morphism_property C} {D : Type u_3} [category_theory.category D] {F G : W.localization D} {τ₁ τ₂ : F G} (h : 𝟙 W.Q τ₁ = 𝟙 W.Q τ₂) :
τ₁ = τ₂