Skip to content

Commit

Permalink
Prove new stability lemma using localization data.
Browse files Browse the repository at this point in the history
  • Loading branch information
PatrickMassot committed Dec 7, 2023
1 parent 8ef1e3f commit 9797490
Showing 1 changed file with 7 additions and 1 deletion.
8 changes: 7 additions & 1 deletion SphereEversion/Global/LocalisationData.lean
Original file line number Diff line number Diff line change
Expand Up @@ -164,7 +164,13 @@ theorem _root_.exists_stability_dist {f : M → M'} (hf : Continuous f) :
∃ ψ : OpenSmoothEmbedding 𝓘(ℝ, E') E' I' M',
x ∈ range φ ∧
∀ (g : M → M'), (∀ m, dist (g m) (f m) < ε m) → range (g ∘ φ) ⊆ range ψ := by
sorry
let L := stdLocalisationData E I E' I' hf
use L.ε, L.ε_pos, L.ε_cont
intro x
rcases mem_iUnion.mp <| eq_univ_iff_forall.mp L.h₁ x with ⟨i, hi⟩
use L.φ i, L.ψj i, mem_range_of_mem_image (φ L i) _ hi, ?_
have := L.ε_spec
tauto

end LocalisationData

Expand Down

0 comments on commit 9797490

Please sign in to comment.