Presheaves on a topological space #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
We define presheaf C X simply as (opens X)ᵒᵖ ⥤ C,
and inherit the category structure with natural transformations as morphisms.
We define
pushforward_obj {X Y : Top.{w}} (f : X ⟶ Y) (ℱ : X.presheaf C) : Y.presheaf Cwith notationf _* ℱand forℱ : X.presheaf Cprovide the natural isomorphismspushforward.id : (𝟙 X) _* ℱ ≅ ℱpushforward.comp : (f ≫ g) _* ℱ ≅ g _* (f _* ℱ)along with their@[simp]lemmas.
We also define the functors pushforward and pullback between the categories
X.presheaf C and Y.presheaf C, and provide their adjunction at
pushforward_pullback_adjunction.
The category of C-valued presheaves on a (bundled) topological space X.
Equations
- Top.presheaf C X = ((topological_space.opens ↥X)ᵒᵖ ⥤ C)
 
The restriction of a section along an inclusion of open sets.
For x : F.obj (op V), we provide the notation x |_ₕ i (h stands for hom) for i : U ⟶ V,
and the notation x |_ₗ U ⟪i⟫ (l stands for le) for i : U ≤ V.
Equations
- Top.presheaf.restrict x h = ⇑(F.map h.op) x
 
The restriction of a section along an inclusion of open sets.
For x : F.obj (op V), we provide the notation x |_ U, where the proof U ≤ V is inferred by
the tactic Top.presheaf.restrict_tac'
Pushforward a presheaf on X along a continuous map f : X ⟶ Y, obtaining a presheaf
on Y.
Equations
- f _* ℱ = (topological_space.opens.map f).op ⋙ ℱ
 
An equality of continuous maps induces a natural isomorphism between the pushforwards of a presheaf along those maps.
Equations
The natural isomorphism between the pushforward of a presheaf along the identity continuous map and the original presheaf.
The natural isomorphism between the pushforward of a presheaf along the composition of two continuous maps and the corresponding pushforward of a pushforward.
A morphism of presheaves gives rise to a morphisms of the pushforwards of those presheaves.
Equations
- Top.presheaf.pushforward_map f α = {app := λ (U : (topological_space.opens ↥Y)ᵒᵖ), α.app ((topological_space.opens.map f).op.obj U), naturality' := _}
 
Pullback a presheaf on Y along a continuous map f : X ⟶ Y, obtaining a presheaf on X.
This is defined in terms of left Kan extensions, which is just a fancy way of saying "take the colimits over the open sets whose preimage contains U".
Equations
Pulling back along continuous maps is functorial.
Equations
If f '' U is open, then f⁻¹ℱ U ≅ ℱ (f '' U).
Equations
- Top.presheaf.pullback_obj_obj_of_image_open f ℱ U H = let x : category_theory.costructured_arrow (topological_space.opens.map f).op (opposite.op U) := category_theory.costructured_arrow.mk (category_theory.hom_of_le _).op in (category_theory.limits.colimit.is_colimit (category_theory.Lan.diagram (topological_space.opens.map f).op ℱ (opposite.op U))).cocone_point_unique_up_to_iso (category_theory.limits.colimit_of_diagram_terminal {lift := λ (s : category_theory.limits.cone (category_theory.functor.empty (category_theory.costructured_arrow (topological_space.opens.map f).op (opposite.op U)))), category_theory.costructured_arrow.hom_mk (id (category_theory.hom_of_le _).op) _, fac' := _, uniq' := _} (category_theory.Lan.diagram (topological_space.opens.map f).op ℱ (opposite.op U)))
 
The pullback along the identity is isomorphic to the original presheaf.
Equations
The pushforward functor.
Equations
- Top.presheaf.pushforward C f = {obj := Top.presheaf.pushforward_obj f, map := Top.presheaf.pushforward_map f, map_id' := _, map_comp' := _}
 
A homeomorphism of spaces gives an equivalence of categories of presheaves.
Equations
If H : X ≅ Y is a homeomorphism,
then given an H _* ℱ ⟶ 𝒢, we may obtain an ℱ ⟶ H ⁻¹ _* 𝒢.
Equations
If H : X ≅ Y is a homeomorphism,
then given an H _* ℱ ⟶ 𝒢, we may obtain an ℱ ⟶ H ⁻¹ _* 𝒢.
Equations
- Top.presheaf.pushforward_to_of_iso H₁ H₂ = ⇑(((Top.presheaf.presheaf_equiv_of_iso C H₁.symm).to_adjunction.hom_equiv ℱ 𝒢).symm) H₂
 
Pullback a presheaf on Y along a continuous map f : X ⟶ Y, obtaining a presheaf
on X.
Equations
The pullback and pushforward along a continuous map are adjoint to each other.
Pulling back along a homeomorphism is the same as pushing forward along its inverse.
Pulling back along the inverse of a homeomorphism is the same as pushing forward along it.