diff -r d2daeef3ce47 -r 36209dfb981e src/HOL/Analysis/Homeomorphism.thy --- a/src/HOL/Analysis/Homeomorphism.thy Wed May 02 12:48:08 2018 +0100 +++ b/src/HOL/Analysis/Homeomorphism.thy Wed May 02 23:32:47 2018 +0100 @@ -963,7 +963,7 @@ then obtain f g where fg: "homeomorphism (sphere 0 1 - {i}) {x. i \ x = 0} f g" by (force simp: homeomorphic_def) have "h ` (+) (- a) ` S \ T" - using heq span_clauses(1) span_linear_image by blast + using heq span_superset span_linear_image by blast then have "g ` h ` (+) (- a) ` S \ g ` {x. i \ x = 0}" using Tsub by (simp add: image_mono) also have "... \ sphere 0 1 - {i}" @@ -987,8 +987,8 @@ apply (simp add: homeomorphic_def homeomorphism_def) apply (rule_tac x="g \ h" in exI) apply (rule_tac x="k \ f" in exI) - apply (auto simp: ghcont kfcont span_clauses(1) homeomorphism_apply2 [OF fg] image_comp) - apply (force simp: o_def homeomorphism_apply2 [OF fg] span_clauses(1)) + apply (auto simp: ghcont kfcont span_superset homeomorphism_apply2 [OF fg] image_comp) + apply (force simp: o_def homeomorphism_apply2 [OF fg] span_superset) done finally have Shom: "S homeomorphic (g \ h) ` (+) (- a) ` S" . show ?thesis