src/HOL/Analysis/Topology_Euclidean_Space.thy
changeset 64394 141e1ed8d5a0
parent 64320 ba194424b895
child 64539 a868c83aa66e
--- a/src/HOL/Analysis/Topology_Euclidean_Space.thy	Tue Oct 25 11:55:38 2016 +0200
+++ b/src/HOL/Analysis/Topology_Euclidean_Space.thy	Tue Oct 25 15:46:07 2016 +0100
@@ -8985,6 +8985,18 @@
     done
 qed
 
+lemma homeomorphic_spheres:
+  fixes a b ::"'a::real_normed_vector"
+  assumes "0 < d"  "0 < e"
+  shows "(sphere a d) homeomorphic (sphere b e)"
+unfolding homeomorphic_minimal
+    apply(rule_tac x="\<lambda>x. b + (e/d) *\<^sub>R (x - a)" in exI)
+    apply(rule_tac x="\<lambda>x. a + (d/e) *\<^sub>R (x - b)" in exI)
+    using assms
+    apply (auto intro!: continuous_intros
+      simp: dist_commute dist_norm pos_divide_less_eq mult_strict_left_mono)
+    done
+
 subsection\<open>Inverse function property for open/closed maps\<close>
 
 lemma continuous_on_inverse_open_map: