src/HOL/Topological_Spaces.thy
changeset 60040 1fa1023b13b9
parent 60036 218fcc645d22
child 60150 bd773c47ad0b
--- a/src/HOL/Topological_Spaces.thy	Sun Apr 12 11:33:50 2015 +0200
+++ b/src/HOL/Topological_Spaces.thy	Sun Apr 12 11:34:09 2015 +0200
@@ -1636,7 +1636,7 @@
     by (rule compactE)
   from `D \<subseteq> ?C` have "\<forall>x\<in>D. eventually (\<lambda>y. y \<notin> x) (nhds y)" by auto
   with `finite D` have "eventually (\<lambda>y. y \<notin> \<Union>D) (nhds y)"
-    by (simp add: eventually_Ball_finite)
+    by (simp add: eventually_ball_finite)
   with `s \<subseteq> \<Union>D` have "eventually (\<lambda>y. y \<notin> s) (nhds y)"
     by (auto elim!: eventually_mono [rotated])
   thus "\<exists>t. open t \<and> y \<in> t \<and> t \<subseteq> - s"