src/HOL/Analysis/Function_Topology.thy
changeset 65036 ab7e11730ad8
parent 64911 f0e07600de47
child 66827 c94531b5007d
--- a/src/HOL/Analysis/Function_Topology.thy	Sun Feb 19 11:58:51 2017 +0100
+++ b/src/HOL/Analysis/Function_Topology.thy	Tue Feb 21 15:04:01 2017 +0000
@@ -967,7 +967,7 @@
     by blast
   define m where "m = Min {(1/2)^(to_nat i) * e i|i. i \<in> I}"
   have "m > 0" if "I\<noteq>{}"
-    unfolding m_def apply (rule Min_grI) using \<open>finite I\<close> \<open>I \<noteq> {}\<close> \<open>\<And>i. e i > 0\<close> by auto
+    unfolding m_def Min_gr_iff using \<open>finite I\<close> \<open>I \<noteq> {}\<close> \<open>\<And>i. e i > 0\<close> by auto
   moreover have "{y. dist x y < m} \<subseteq> U"
   proof (auto)
     fix y assume "dist x y < m"