Subsheaf of types #
We define the sub(pre)sheaf of a type valued presheaf.
Main results #
CategoryTheory.Subpresheaf
: A subpresheaf of a presheaf of types.CategoryTheory.Subpresheaf.sheafify
: The sheafification of a subpresheaf as a subpresheaf. Note that this is a sheaf only when the whole sheaf is.CategoryTheory.Subpresheaf.sheafify_isSheaf
: The sheafification is a sheafCategoryTheory.Subpresheaf.sheafifyLift
: The descent of a map into a sheaf to the sheafification.CategoryTheory.GrothendieckTopology.imageSheaf
: The image sheaf of a morphism.CategoryTheory.GrothendieckTopology.imageFactorization
: The image sheaf as aLimits.imageFactorization
.
The sheafification of a subpresheaf as a subpresheaf. Note that this is a sheaf only when the whole presheaf is a sheaf.
Equations
- CategoryTheory.Subpresheaf.sheafify J G = { obj := fun (U : Cᵒᵖ) => {s : F.obj U | G.sieveOfSection s ∈ J (Opposite.unop U)}, map := ⋯ }
Instances For
The lift of a presheaf morphism onto the sheafification subpresheaf.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A morphism factors through the sheafification of the image presheaf.
Equations
Instances For
The image sheaf of a morphism between sheaves, defined to be the sheafification of
image_presheaf
.
Equations
- CategoryTheory.Sheaf.image f = { val := (CategoryTheory.Subpresheaf.sheafify J (CategoryTheory.Subpresheaf.range f.val)).toPresheaf, cond := ⋯ }
Instances For
A morphism factors through the image sheaf.
Equations
- CategoryTheory.Sheaf.toImage f = { val := CategoryTheory.Subpresheaf.toRangeSheafify J f.val }
Instances For
The inclusion of the image sheaf to the target.
Equations
- CategoryTheory.Sheaf.imageι f = { val := (CategoryTheory.Subpresheaf.sheafify J (CategoryTheory.Subpresheaf.range f.val)).ι }
Instances For
The mono factorization given by image_sheaf
for a morphism.
Equations
Instances For
The mono factorization given by image_sheaf
for a morphism is an image.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Alias of CategoryTheory.Subpresheaf.toRangeSheafify
.
A morphism factors through the sheafification of the image presheaf.
Instances For
Alias of CategoryTheory.Sheaf.image
.
The image sheaf of a morphism between sheaves, defined to be the sheafification of
image_presheaf
.
Equations
Instances For
Alias of CategoryTheory.Sheaf.toImage
.
A morphism factors through the image sheaf.
Instances For
Alias of CategoryTheory.Sheaf.imageι
.
The inclusion of the image sheaf to the target.
Instances For
Alias of CategoryTheory.Sheaf.toImage_ι
.