Presheaves of functions #
We construct some simple examples of presheaves of functions on a topological space.
presheafToTypes X T
, whereT : X → Type
, is the presheaf of dependently-typed (not-necessarily continuous) functionspresheafToType X T
, whereT : Type
, is the presheaf of (not-necessarily-continuous) functions to a fixed target typeT
presheafToTop X T
, whereT : TopCat
, is the presheaf of continuous functions into a topological spaceT
presheafToTopCommRing X R
, whereR : TopCommRingCat
is the presheaf valued inCommRing
of functions functions into a topological ringR
- as an example of the previous construction,
presheafToTopCommRing X (TopCommRingCat.of ℂ)
is the presheaf of rings of continuous complex-valued functions onX
.
The presheaf of dependently typed functions on X
, with fibres given by a type family T
.
There is no requirement that the functions are continuous, here.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
theorem
TopCat.presheafToTypes_obj
(X : TopCat)
{T : ↑X → Type v}
{U : (TopologicalSpace.Opens ↑X)ᵒᵖ}
:
(X.presheafToTypes T).obj U = ((x : ↥(Opposite.unop U)) → T ↑x)
@[simp]
theorem
TopCat.presheafToTypes_map
(X : TopCat)
{T : ↑X → Type v}
{U V : (TopologicalSpace.Opens ↑X)ᵒᵖ}
{i : U ⟶ V}
{f : (X.presheafToTypes T).obj U}
:
(X.presheafToTypes T).map i f = fun (x : ↥(Opposite.unop V)) => f ((fun (x : ↥(Opposite.unop V)) => ⟨↑x, ⋯⟩) x)
The presheaf of functions on X
with values in a type T
.
There is no requirement that the functions are continuous, here.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
theorem
TopCat.presheafToType_obj
(X : TopCat)
{T : Type v}
{U : (TopologicalSpace.Opens ↑X)ᵒᵖ}
:
(X.presheafToType T).obj U = (↥(Opposite.unop U) → T)
@[simp]
theorem
TopCat.presheafToType_map
(X : TopCat)
{T : Type v}
{U V : (TopologicalSpace.Opens ↑X)ᵒᵖ}
{i : U ⟶ V}
{f : (X.presheafToType T).obj U}
:
(X.presheafToType T).map i f = f ∘ fun (x : ↥(Opposite.unop V)) => ⟨↑x, ⋯⟩
The presheaf of continuous functions on X
with values in fixed target topological space
T
.
Equations
- X.presheafToTop T = (TopologicalSpace.Opens.toTopCat X).op.comp (CategoryTheory.yoneda.obj T)
Instances For
@[simp]
theorem
TopCat.presheafToTop_obj
(X T : TopCat)
(U : (TopologicalSpace.Opens ↑X)ᵒᵖ)
:
(X.presheafToTop T).obj U = ((TopologicalSpace.Opens.toTopCat X).obj (Opposite.unop U) ⟶ T)