Generic construction of a sheaf from a local_invariant_prop on a manifold #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file constructs the sheaf-of-types of functions f : M → M' (for charted spaces M, M')
which satisfy the lifted property lift_prop P associated to some locally invariant (in the sense
of structure_groupoid.local_invariant_prop) property P on the model spaces of M and M'. For
example, differentiability and smoothness are locally invariant properties in this sense, so this
construction can be used to construct the sheaf of differentiable functions on a manifold and the
sheaf of smooth functions on a manifold.
The mathematical work is in associating a Top.local_predicate to a
structure_groupoid.local_invariant_prop: that is, showing that a differential-geometric "locally
invariant" property is preserved under restriction and gluing.
Main definitions #
structure_groupoid.local_invariant_prop.local_predicate: theTop.local_predicate(in the sheaf-theoretic sense) on functions from open subsets ofMintoM', which states whether such functions satisfylift_prop P.structure_groupoid.local_invariant_prop.sheaf: the sheaf-of-types of functionsf : M → M'which satisfy the lifted propertylift_prop P.
Equations
Let P be a local_invariant_prop for functions between spaces with the groupoids G, G'
and let M, M' be charted spaces modelled on the model spaces of those groupoids. Then there is
an induced local_predicate on the functions from M to M', given by lift_prop P.
Equations
- structure_groupoid.local_invariant_prop.local_predicate M M' hG = {to_prelocal_predicate := {pred := λ {U : topological_space.opens ↥(Top.of M)} (f : ↥U → M'), charted_space.lift_prop P f, res := _}, locality := _}
Let P be a local_invariant_prop for functions between spaces with the groupoids G, G'
and let M, M' be charted spaces modelled on the model spaces of those groupoids. Then there is
a sheaf of types on M which, to each open set U in M, associates the type of bundled
functions from U to M' satisfying the lift of P.
Equations
Equations
- structure_groupoid.local_invariant_prop.sheaf_has_coe_to_fun M M' hG U = {coe := λ (a : (structure_groupoid.local_invariant_prop.sheaf M M' hG).val.obj U), a.val}