Local properties of smooth functions which depend on both the source and target #
In this file, we consider local properties of functions between manifolds, which depend on both the
source and the target: more precisely, properties P of functions f : M → N such that
f has property P if and only if there is a suitable pair of charts on M and N, respectively,
such that f read in these charts has a particular form.
The motivating example of this general description are immersions and submersions:
f : M → N is an immersion at x iff there are charts φ and ψ of M and N around x and
f x, respectively, such that in these charts, f looks like u ↦ (u, 0). Similarly, f is a
submersion at x iff it looks like a projection (u, v) ↦ u in suitable charts near x and f x.
Studying such local properties allows proving several lemmas about immersions and submersions
only once. In IsImmersionEmbedding.lean, we prove that being an immersion at x is indeed a
local property of this form.
Main definitions and results #
Manifold.LocalSourceTargetPropertyAtcaptures a local property of the above form: for eachf : M → N, and pair of chartsφofMandψofN, the local property is either safisfied or not. We ask that the property be stable under congruence and under restriction ofφ.Manifold.LiftSourceTargetPropertyAt f x P, wherePis aLocalSourceTargetPropertyAt, defines a local property of functions of the above shape:fhas this property atxif there exist chartsφandψsuch thatP f φ ψholds.Manifold.LiftSourceTargetPropertyAt.congr_of_eventuallyEq: iffhas propertyPatxandgequalsfnearx, thengalso has propertyPatx.
Structure recording good behaviour of a property of functions M → N w.r.t. to compatible
choices of both a chart on M and N. Currently, we ask for the property being stable under
restriction of the domain chart, and local in the target.
Motivating examples are immersions and submersions of smooth manifolds.
- mono_source {f : M → N} {φ : OpenPartialHomeomorph M H} {ψ : OpenPartialHomeomorph N G} {s : Set M} : IsOpen s → P f φ ψ → P f (φ.restr s) ψ
- congr {f g : M → N} {φ : OpenPartialHomeomorph M H} {ψ : OpenPartialHomeomorph N G} : Set.EqOn f g φ.source → P f φ ψ → P g φ ψ
Instances For
Data witnessing the fact that f has local property P at x
- domChart : OpenPartialHomeomorph M H
A choice of chart on the domain
Mof the local propertyPoffatx: w.r.t. this chart andcodChart,fhas the local propertyPatx. - codChart : OpenPartialHomeomorph N G
A choice of chart on the target
Nof the local propertyPoffatx: w.r.t. this chart anddomChart,fhas the local propertyPatx.
Instances For
The induced property by a local property P: it is satisfied for f at x iff there exist
charts φ and ψ of M and N around x and f x, respectively, such that f satisfies P
w.r.t. φ and ψ.
The motivating example are smooth immersions and submersions: the corresponding condition is that
f look like the inclusion u ↦ (u, 0) (resp. a projection (u, v) ↦ u)
in the charts φ and ψ.
Equations
- Manifold.LiftSourceTargetPropertyAt I I' n f x P = Nonempty (Manifold.LocalPresentationAt I I' n f x P)
Instances For
A choice of charts witnessing the local property P of f at x.
Equations
Instances For
A choice of chart on the domain M of a local property of f at x:
w.r.t. this chart and h.codChart, f has the local property P at x.
The particular chart is arbitrary, but this choice matches the witness given by h.codChart.
Equations
Instances For
A choice of chart on the co-domain N of a local property of f at x:
w.r.t. this chart and h.domChart, f has the local property P at x
The particular chart is arbitrary, but this choice matches the witness given by h.domChart.
Equations
Instances For
If P is a local property, by monotonicity w.r.t. restricting domChart,
if f is continuous at x, to prove LiftSourceTargetPropertyAt I I' n f x P
we need not check the condition f '' domChart.source ⊆ codChart.source.
If P is monotone w.r.t. restricting domChart and closed under congruence,
if f has property P at x and f and g are eventually equal near x,
then g has property P at x.
If P is monotone w.r.t. restricting domChart and closed under congruence,
and f and g are eventually equal near x,
then f has property P at x if and only if g has property P at x.