Documentation

Mathlib.Geometry.Manifold.WhitneyEmbedding

Whitney embedding theorem #

In this file we prove a version of the Whitney embedding theorem: for any compact real manifold M, for sufficiently large n there exists a smooth embedding M → ℝ^n.

TODO #

Tags #

partition of unity, smooth bump function, whitney theorem

Whitney embedding theorem #

In this section we prove a version of the Whitney embedding theorem: for any compact real manifold M, for sufficiently large n there exists a smooth embedding M → ℝ^n.

Smooth embedding of M into (E × ℝ) ^ ι.

Equations
Instances For
    theorem SmoothBumpCovering.embeddingPiTangent_coe {ι : Type uι} {E : Type uE} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] {H : Type uH} [TopologicalSpace H] {I : ModelWithCorners E H} {M : Type uM} [TopologicalSpace M] [ChartedSpace H M] [SmoothManifoldWithCorners I M] [T2Space M] [hi : Fintype ι] {s : Set M} (f : SmoothBumpCovering ι I M s) :
    (SmoothBumpCovering.embeddingPiTangent f) = fun (x : M) (i : ι) => ((f.toFun i) x (extChartAt I (f.c i)) x, (f.toFun i) x)

    Baby version of the Whitney weak embedding theorem: if M admits a finite covering by supports of bump functions, then for some n it can be immersed into the n-dimensional Euclidean space.

    Baby version of the Whitney weak embedding theorem: if M admits a finite covering by supports of bump functions, then for some n it can be embedded into the n-dimensional Euclidean space.