src/HOL/Analysis/Further_Topology.thy
changeset 66827 c94531b5007d
parent 65064 a4abec71279a
child 66884 c2128ab11f61
--- a/src/HOL/Analysis/Further_Topology.thy	Tue Oct 10 14:03:51 2017 +0100
+++ b/src/HOL/Analysis/Further_Topology.thy	Tue Oct 10 17:15:37 2017 +0100
@@ -1183,7 +1183,7 @@
                  and hin: "\<And>x. x \<in> C \<inter> K \<Longrightarrow> h x \<in> ball a d \<inter> U"
     proof (rule homeomorphism_grouping_points_exists_gen [of C "ball a d \<inter> U" "C \<inter> K" "S \<union> C"])
       show "openin (subtopology euclidean C) (ball a d \<inter> U)"
-        by (metis Topology_Euclidean_Space.open_ball \<open>C \<subseteq> U\<close> \<open>ball a d \<inter> U \<subseteq> C\<close> inf.absorb_iff2 inf.orderE inf_assoc open_openin openin_subtopology)
+        by (metis open_ball \<open>C \<subseteq> U\<close> \<open>ball a d \<inter> U \<subseteq> C\<close> inf.absorb_iff2 inf.orderE inf_assoc open_openin openin_subtopology)
       show "openin (subtopology euclidean (affine hull C)) C"
         by (metis \<open>a \<in> C\<close> \<open>openin (subtopology euclidean U) C\<close> affine_hull_eq affine_hull_openin all_not_in_conv \<open>affine U\<close>)
       show "ball a d \<inter> U \<noteq> {}"