Bousfield localization #
Given a predicate P : C → Prop
on the objects of a category C
,
we define Localization.LeftBousfield.W P : MorphismProperty C
as the class of morphisms f : X ⟶ Y
such that for any Z : C
such that P Z
, the precomposition with f
induces a bijection
(Y ⟶ Z) ≃ (X ⟶ Z)
.
(This construction is part of left Bousfield localization in the context of model categories.)
When G ⊣ F
is an adjunction with F : C ⥤ D
fully faithful, then
G : D ⥤ C
is a localization functor for the class W (· ∈ Set.range F.obj)
,
which then identifies to the inverse image by G
of the class of
isomorphisms in C
.
References #
- https://ncatlab.org/nlab/show/left+Bousfield+localization+of+model+categories
Given a predicate P : C → Prop
, this is the class of morphisms f : X ⟶ Y
such that for all Z : C
such that P Z
, the precomposition with f
induces
a bijection (Y ⟶ Z) ≃ (X ⟶ Z)
.
Equations
- CategoryTheory.Localization.LeftBousfield.W P f = ∀ (Z : C), P Z → Function.Bijective fun (g : x ⟶ Z) => CategoryTheory.CategoryStruct.comp f g
Instances For
The bijection (Y ⟶ Z) ≃ (X ⟶ Z)
induced by f : X ⟶ Y
when LeftBousfield.W P f
and P Z
.
Equations
- hf.homEquiv Z hZ = Equiv.ofBijective (fun (g : Y ⟶ Z) => CategoryTheory.CategoryStruct.comp f g) ⋯
Instances For
Equations
- ⋯ = ⋯
Equations
- ⋯ = ⋯