This is file proves the existence of a sphere eversion from the local verson of the h-principle.
We define the relation of immersions R = immersion_sphere_rel ⊆ J¹(E, F)
which consist of all
(x, y, ϕ)
such that if x
is outside a ball around the origin with chosen radius R < 1
then
ϕ
must be injective on (ℝ ∙ x)ᗮ
(the orthogonal complement of the span of x
).
We show that R
is open and ample.
Furthermore, we define a formal solution of sphere eversion that is holonomic near 0
and 1
.
We have to be careful since we're not actually working on the sphere,
but in the ambient space E ≃ ℝ³
.
See loc_formal_eversion
for the choice and constaints of the solution.
Finally, we obtain the existence of sphere eversion from the parametric local h-principle,
proven in Local/ParametricHPrinciple
.
A map between vector spaces is a immersion viewed as a map on the sphere, when its
derivative at x ∈ 𝕊²
is injective on the orthogonal complement of x
(the tangent space to the sphere). Note that this implies f
is differentiable at every point
x ∈ 𝕊²
since otherwise D f x = 0
.
Equations
- SphereImmersion f = ∀ x ∈ Metric.sphere 0 1, Set.InjOn ⇑(D f x) ↑(Submodule.span ℝ {x})ᗮ
Instances For
The relation of immersionsof a two-sphere into its ambient Euclidean space.
Equations
- immersionSphereRel E F = {w : OneJet E F | w.1 ∉ Metric.ball 0 0.9 → Set.InjOn ⇑w.2.2 ↑(Submodule.span ℝ {w.1})ᗮ}
Instances For
The main ingredient of the linear map in the formal eversion of the sphere.
Equations
- locFormalEversionAuxφ ω t x = ω.rot (t, x) - (2 * t) • (Submodule.span ℝ {x}).subtypeL.comp (orthogonalProjection (Submodule.span ℝ {x}))
Instances For
A formal eversion of 𝕊²
, viewed as a homotopy.
Equations
- One or more equations did not get rendered due to their size.
Instances For
A formal eversion of 𝕊²
into its ambient Euclidean space.
The corresponding map E → E
is roughly a linear homotopy from id
at t = 0
to - id
at
t = 1
. The continuous linear maps are roughly rotations with angle t * π
. However, we have to
keep track of a few complications:
- We need the formal solution to be holonomic near
0
and1
. Therefore, we compose the above maps with a smooth step function that is constant0
neart = 0
and constant1
neart = 1
. - We need to modify the derivative of
ω.rot
to also have the right behavior on(ℝ ∙ x)
att = 1
(it is the identity, but it should be-id
). Therefore, we subtract(2 * t) • (submodule.subtypeL (ℝ ∙ x) ∘L orthogonal_projection (ℝ ∙ x))
, which is2t
times the identity on(ℝ ∙ x)
. - We have to make sure the family of continuous linear map is smooth at
x = 0
. Therefore, we multiply the family with a factor ofsmooth_step (‖x‖ ^ 2)
.
Equations
- locFormalEversion ω = { toFamilyJetSec := locFormalEversionAux ω, is_sol := ⋯ }