Smooth immersions #
In this file, we define C^n immersions between C^n manifolds.
The correct definition in the infinite-dimensional setting differs from the standard
finite-dimensional definition (concerning the mfderiv being injective): future pull requests will
prove that our definition implies the latter, and that both are equivalent for finite-dimensional
manifolds.
This definition can be conveniently formulated in terms of local properties: f is an immersion at
x iff there exist suitable charts near x and f x such that f has a nice form w.r.t. these
charts. Most results below can be deduced from more abstract results about such local properties.
This shortens the overall argument, as the definition of submersions has the same general form.
Main definitions #
IsImmersionAtOfComplement F I J n f xmeans a mapf : M → NbetweenC^nmanifoldsMandNis an immersion atx : M: there are chartsφandψofMandNaroundxandf x, respectively, such that in these charts,flooks likeu ↦ (u, 0), w.r.t. some equivalenceE' ≃L[𝕜] E × F. We do not demand thatfbe differentiable (this follows from this definition).IsImmersionAt I J n f xmeans thatfis aC^nimmersion atx : Mfor some choice of a complementFof the model normed spaceEofMin the model normed spaceE'ofN. In most cases, prefer this definition overIsImmersionAtOfComplement.IsImmersionOfComplement F I J n fmeansf : M → Nis an immersion at every pointx : M, w.r.t. the chosen complementF.IsImmersion I J n fmeansf : M → Nis an immersion at every pointx : M, w.r.t. some global choice of complement.
Main results #
IsImmersionAt.congr_of_eventuallyEq: being an immersion is a local property. Iffandgagree nearxandfis an immersion atx, so isgIsImmersionAtOfComplement.congr_F,IsImmersionOfComplement.congr_F: being an immersion (atx) w.r.t.Fis stable under replacing the complementFby an isomorphic copy
Implementation notes #
- In most applications, there is no need to control the chosen complement in the definition of
immersions, so
IsImmersion(At)is perfectly fine to use. Such control will be helpful, however, when considering the local characterisation of submanifolds: locally, a submanifold is described either as the image of an immersion, or the preimage of a submersion --- w.r.t. the same complement. Having access to a definition version with complements allows stating this equivalence cleanly. - To avoid a free universe variable in
IsImmersion(At), we ask for a complement in the same universe as the model normed space forN. We provide convenience constructors which do not have this restriction (recovering usability). The underlying observation is that the equivalence in the definition of immersions allows shrinking the universe of the complement: this is implemented inIsImmersion(At)OfComplement.smallandIsImmersion(At)OfComplement.smallEquiv.
TODO #
- The converse to
IsImmersionAtOfComplement.congr_Falso holds: any two complements are isomorphic, as they are isomorphic to the cokernel of the differentialmfderiv I J f x. - The set where
IsImmersionAt(OfComplement)holds is open. IsImmersionAt.contMDiffAt: if f is an immersion atx, it isC^natx.IsImmersion.contMDiff: if f is an immersion, it isC^n.IsImmersionAt.prodMap: the product of two immersions is an immersion.- If
fis an immersion atx, its differential splits, hence is injective. - If
f : M → Nis a map between Banach manifolds,mfderiv I J f xsplitting impliesfis an immersion atx. (This requires the inverse function theorem.) IsImmersionAt.comp: iff : M → Nandg: N → N'are maps between Banach manifolds such thatfis an immersion atx : Mandgis an immersion atf x, theng ∘ fis an immersion atx.IsImmersion.comp: the composition of immersions (between Banach manifolds) is an immersion- If
f : M → Nis a map between finite-dimensional manifolds,mfderiv I J f xbeing injective impliesfis an immersion atx.
References #
The local property of being an immersion at a point: f : M → N is an immersion at x if
there exist charts φ and ψ of M and N around x and f x, respectively, such that in these
charts, f looks like the inclusion u ↦ (u, 0).
This definition has a fixed parameter F, which is a choice of complement of E in the model
normed space E' of N: being an immersion at x includes a choice of linear isomorphism
between E × F and E'.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Being an immersion at x is a local property.
f : M → N is a C^n immersion at x if 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).
Additionally, we demand that f map φ.source into ψ.source.
NB. We don't know the particular atlasses used for M and N, so asking for φ and ψ to be
in the atlas would be too optimistic: lying in the maximalAtlas is sufficient.
This definition has a fixed parameter F, which is a choice of complement of E in E':
being an immersion at x includes a choice of linear isomorphism between E × F and E'.
While the particular choice of complement is often not important, chosing a complement is useful
in some settings, such as proving that embedded submanifolds are locally given either by an
immersion or a submersion.
Unless you have a particular reason, prefer to use IsImmersionAt instead.
Equations
- Manifold.IsImmersionAtOfComplement F I J n f x = Manifold.LiftSourceTargetPropertyAt I J n f x (Manifold.ImmersionAtProp F I J M N)
Instances For
f : M → N is a C^n immersion at x if 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).
Additionally, we demand that f map φ.source into ψ.source.
NB. We don't know the particular atlasses used for M and N, so asking for φ and ψ to be
in the atlas would be too optimistic: lying in the maximalAtlas is sufficient.
Implicit in this definition is an abstract choice F of a complement of E in E': being an
immersion at x includes a choice of linear isomorphism between E × F and E', which is
where the choice of F enters.
If you need stronger control over the complement F, use IsImmersionAtOfComplement instead.
Equations
- Manifold.IsImmersionAt I J n f x = ∃ (F : Type ?u.29) (x_1 : NormedAddCommGroup F) (x_2 : NormedSpace 𝕜 F), Manifold.IsImmersionAtOfComplement F I J n f x
Instances For
f : M → N is a C^n immersion at x if 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).
This version does not assume that f maps φ.source to ψ.source,
but that f is continuous at x.
A choice of chart on the domain M of an immersion f at x:
w.r.t. this chart and the data h.codChart and h.equiv,
f will look like an inclusion u ↦ (u, 0) in these extended charts.
The particular chart is arbitrary, but this choice matches the witnesses given by
h.codChart and h.codChart.
Instances For
A choice of chart on the co-domain N of an immersion f at x:
w.r.t. this chart and the data h.domChart and h.equiv,
f will look like an inclusion u ↦ (u, 0) in these extended charts.
The particular chart is arbitrary, but this choice matches the witnesses given by
h.equiv and h.domChart.
Instances For
A linear equivalence E × F ≃L[𝕜] E'' which belongs to the data of an immersion f at x:
the particular equivalence is arbitrary, but this choice matches the witnesses given by
h.domChart and h.codChart.
Equations
- h.equiv = Classical.choose ⋯
Instances For
If f is an immersion at x, it maps its domain chart's target (h.domChart.extend I).target
to its codomain chart's target (h.domChart.extend J).target.
Roig and Domingues' [roigdomingues1992] definition of immersions only asks for this inclusion
between the targets of the local charts: using mathlib's formalisation conventions, that condition
is slightly weaker than source_subset_preimage_source: the latter implies that
h.codChart.extend J ∘ f maps h.domChart.source to
(h.codChart.extend J).target = (h.codChart.extend I) '' h.codChart.source,
but that does not imply f maps h.domChart.source to h.codChartSource;
a priori f could map some point f ∘ h.domChart.extend I x ∉ h.codChart.source into the target.
Note that this difference only occurs because of our design using junk values;
this is not a mathematically meaningful difference.`
At the same time, this condition is fairly weak: it is implied, for instance, by f being
continuous at x (see mk_of_continuousAt), which is easy to ascertain in practice.
See target_subset_preimage_target for a version stated using preimages instead of images.
If f is an immersion at x, its domain chart's target (h.domChart.extend I).target
is mapped to it codomain chart's target (h.domChart.extend J).target:
see map_target_subset_target for a version stated using images.
If f is an immersion at x and g = f on some neighbourhood of x,
then g is an immersion at x.
If f = g on some neighbourhood of x,
then f is an immersion at x if and only if g is an immersion at x.
Given an immersion f at x, this is a choice of complement which lives in the same universe
as the model space for the co-domain of f: this is useful to avoid universe restrictions.
Equations
Instances For
Equations
Equations
Given an immersion f at x w.r.t. a complement F, this construction provides
a continuous linear equivalence from F to the small complement of F:
mathematically, this is just the identity map; however, this is technically useful as it enables
us to always work with hf.smallComplement.
Equations
- hf.smallEquiv = (Equiv.continuousLinearEquiv 𝕜 (equivShrink F).symm).symm
Instances For
Being an immersion at x w.r.t. F is stable under replacing F by an isomorphic copy.
If f is an immersion at x w.r.t. some complement F, it is an immersion at x.
Note that the proof contains a small formalisation-related subtlety: F can live in any universe,
while being an immersion at x requires the existence of a complement in the same universe as
the model normed space of N. This is solved by smallComplement and smallEquiv.
f : M → N is a C^n immersion at x if 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).
This version does not assume that f maps φ.source to ψ.source,
but that f is continuous at x.
A choice of complement of the model normed space E of M in the model normed space
E' of N
Equations
Instances For
Equations
Equations
A choice of chart on the domain M of an immersion f at x:
w.r.t. this chart and the data h.codChart and h.equiv,
f will look like an inclusion u ↦ (u, 0) in these extended charts.
The particular chart is arbitrary, but this choice matches the witnesses given by
h.codChart and h.codChart.
Instances For
A choice of chart on the co-domain N of an immersion f at x:
w.r.t. this chart and the data h.domChart and h.equiv,
f will look like an inclusion u ↦ (u, 0) in these extended charts.
The particular chart is arbitrary, but this choice matches the witnesses given by
h.equiv and h.domChart.
Instances For
A linear equivalence E × F ≃L[𝕜] E'' which belongs to the data of an immersion f at x:
the particular equivalence is arbitrary, but this choice matches the witnesses given by
h.domChart and h.codChart.
Instances For
If f is an immersion at x, it maps its domain chart's target to its codomain chart's target:
(h.domChart.extend I).target to (h.domChart.extend J).target.
Roig and Domingues' [roigdomingues1992] definition of immersions only asks for this inclusion
between the targets of the local charts: using mathlib's formalisation conventions, that condition
is slightly weaker than source_subset_preimage_source: the latter implies that
h.codChart.extend J ∘ f maps h.domChart.source to
(h.codChart.extend J).target = (h.codChart.extend I) '' h.codChart.source,
but that does not imply f maps h.domChart.source to h.codChartSource;
a priori f could map some point f ∘ h.domChart.extend I x ∉ h.codChart.source into the target.
Note that this difference only occurs because of our design using junk values;
this is not a mathematically meaningful difference.`
At the same time, this condition is fairly weak: it is implied, for instance, by f being
continuous at x (see mk_of_continuousAt), which is easy to ascertain in practice.
See target_subset_preimage_target for a version stated using preimages instead of images.
If f is an immersion at x, its domain chart's target (h.domChart.extend I).target
is mapped to it codomain chart's target (h.domChart.extend J).target:
see map_target_subset_target for a version stated using images.
If f is an immersion at x and g = f on some neighbourhood of x,
then g is an immersion at x.
If f = g on some neighbourhood of x,
then f is an immersion at x if and only if g is an immersion at x.
f : M → N is a C^n immersion if around each point x ∈ M,
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).
In other words, f is an immersion at each x ∈ M.
This definition has a fixed parameter F, which is a choice of complement of E in E':
being an immersion at x includes a choice of linear isomorphism between E × F and E'.
Equations
- Manifold.IsImmersionOfComplement F I J n f = ∀ (x : M), Manifold.IsImmersionAtOfComplement F I J n f x
Instances For
f : M → N is a C^n immersion if around each point x ∈ M,
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).
Implicit in this definition is an abstract choice F of a complement of E in E':
being an immersion includes a choice of linear isomorphism between E × F and E', which is where
the choice of F enters. If you need stronger control over the complement F,
use IsImmersionOfComplement instead.
Note that our global choice of complement is a bit stronger than asking f to be an immersion at
each x ∈ M w.r.t. to potentially varying complements: see isImmersionAt for details.
Equations
- Manifold.IsImmersion I J n f = ∃ (F : Type ?u.30) (x : NormedAddCommGroup F) (x_1 : NormedSpace 𝕜 F), Manifold.IsImmersionOfComplement F I J n f
Instances For
If f is an immersion, it is an immersion at each point.
If f = g and f is an immersion, so is g.
Being an immersion w.r.t. F is stable under replacing F by an isomorphic copy.
If f is an immersion w.r.t. some complement F, it is an immersion.
Note that the proof contains a small formalisation-related subtlety: F can live in any universe,
while being an immersion requires the existence of a complement in the same universe as
the model normed space of N. This is solved by smallComplement and smallEquiv.
A choice of complement of the model normed space E of M in the model normed space
E' of N
Equations
Instances For
Equations
Equations
If f is an immersion, it is an immersion at each point.
Note that the converse statement is false in general:
if f is an immersion at each x, but with the choice of complement possibly depending on x,
there need not be a global choice of complement for which f is an immersion at each point.
The complement of f at x is isomorphic to the cokernel of mfderiv I J f x, but the mfderiv
of f at (even nearby) points x and x' are not directly related. They have the same rank
(the dimension of E, as will follow from injectivity), but if E'' is infinite-dimensional this
is not conclusive. If E'' is infinite-dimensional, this dimension can indeed change between
different connected of M.
If f = g and f is an immersion, so is g.