Documentation

Mathlib.CategoryTheory.Center.Localization

Localization of the center of a category #

Given a localization functor L : C ⥤ D with respect to W : MorphismProperty C, we define a localization map CatCenter C → CatCenter D for the centers of these categories. In case L is an additive functor between preadditive categories, we promote this to a ring morphism CatCenter C →+* CatCenter D.

Given r : CatCenter C and L : C ⥤ D a localization functor with respect to W : MorphismProperty D, this is the induced element in CatCenter D obtained by localization.

Equations
Instances For
    @[simp]
    theorem CategoryTheory.CatCenter.localization_app {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] (r : CatCenter C) (L : Functor C D) (W : MorphismProperty C) [L.IsLocalization W] (X : C) :
    (r.localization L W).app (L.obj X) = L.map (r.app X)
    theorem CategoryTheory.CatCenter.ext_of_localization {C : Type u₁} [Category.{v₁, u₁} C] {D : Type u₂} [Category.{v₂, u₂} D] (L : Functor C D) (W : MorphismProperty C) [L.IsLocalization W] (r s : CatCenter D) (h : ∀ (X : C), r.app (L.obj X) = s.app (L.obj X)) :
    r = s

    The morphism of rings CatCenter C →+* CatCenter D when L : C ⥤ D is an additive localization functor between preadditive categories.

    Equations
    Instances For