src/HOL/Deriv.thy
changeset 56541 0e3abadbef39
parent 56480 093ea91498e6
child 57418 6ab1c7cb0b8d
--- a/src/HOL/Deriv.thy	Fri Apr 11 17:53:16 2014 +0200
+++ b/src/HOL/Deriv.thy	Fri Apr 11 22:53:33 2014 +0200
@@ -468,10 +468,8 @@
     fix h show "F h = 0"
     proof (rule ccontr)
       assume **: "F h \<noteq> 0"
-      then have h: "h \<noteq> 0"
-        by (clarsimp simp add: F.zero)
-      with ** have "0 < ?r h"
-        by (simp add: divide_pos_pos)
+      hence h: "h \<noteq> 0" by (clarsimp simp add: F.zero)
+      with ** have "0 < ?r h" by simp
       from LIM_D [OF * this] obtain s where s: "0 < s"
         and r: "\<And>x. x \<noteq> 0 \<Longrightarrow> norm x < s \<Longrightarrow> ?r x < ?r h" by auto
       from dense [OF s] obtain t where t: "0 < t \<and> t < s" ..