Skip to content

Commit

Permalink
New chart stability lemma statement
Browse files Browse the repository at this point in the history
  • Loading branch information
PatrickMassot committed Dec 6, 2023
1 parent ab5ccbd commit d731a32
Showing 1 changed file with 9 additions and 0 deletions.
9 changes: 9 additions & 0 deletions SphereEversion/Global/LocalisationData.lean
Original file line number Diff line number Diff line change
Expand Up @@ -155,6 +155,15 @@ theorem ε_spec (ld : LocalisationData I I' f) :
range (g ∘ ld.φ i) ⊆ range (ld.ψj i) :=
(localisation_stability ld).choose_spec.choose_spec.choose_spec

theorem exists_stability_dist {f : M → M'} (hf : Continuous f) :
∃ ε > (0 : M → ℝ), Continuous ε ∧
∀ x : M,
∃ φ : OpenSmoothEmbedding 𝓘(ℝ, E) E I M,
∃ ψ : OpenSmoothEmbedding 𝓘(ℝ, E') E' I' M',
x ∈ range φ ∧
∀ (g : M → M'), (∀ m, dist (g m) (f m) < ε m) → range (g ∘ φ) ⊆ range ψ := by
sorry

end LocalisationData

end

0 comments on commit d731a32

Please sign in to comment.