diff -r 5352449209b1 -r 160eaf566bcb src/HOL/Analysis/Homeomorphism.thy --- a/src/HOL/Analysis/Homeomorphism.thy Mon Oct 07 21:51:31 2019 +0200 +++ b/src/HOL/Analysis/Homeomorphism.thy Tue Oct 08 10:26:40 2019 +0000 @@ -533,9 +533,8 @@ unfolding f_def using \norm b = 1\ norm_eq_1 by (force simp: field_simps inner_add_right inner_diff_right) moreover have "f ` T \ T" - unfolding f_def using assms - apply (auto simp: field_simps inner_add_right inner_diff_right) - by (metis add_0 diff_zero mem_affine_3_minus) + unfolding f_def using assms \subspace T\ + by (auto simp add: inner_add_right inner_diff_right mem_affine_3_minus subspace_mul) moreover have "{x. b\x = 0} \ T \ f ` ({x. norm x = 1 \ b\x \ 1} \ T)" apply clarify apply (rule_tac x = "g x" in image_eqI, auto)