src/HOL/Transcendental.thy
changeset 56541 0e3abadbef39
parent 56536 aefb4a8da31f
child 56544 b60d5d119489
--- a/src/HOL/Transcendental.thy	Fri Apr 11 17:53:16 2014 +0200
+++ b/src/HOL/Transcendental.thy	Fri Apr 11 22:53:33 2014 +0200
@@ -687,9 +687,7 @@
   let ?diff = "\<lambda>i x. (f (x0 + x) i - f x0 i) / x"
 
   let ?r = "r / (3 * real ?N)"
-  have "0 < 3 * real ?N" by auto
-  from divide_pos_pos[OF `0 < r` this]
-  have "0 < ?r" .
+  from `0 < r` have "0 < ?r" by simp
 
   let ?s = "\<lambda>n. SOME s. 0 < s \<and> (\<forall> x. x \<noteq> 0 \<and> \<bar> x \<bar> < s \<longrightarrow> \<bar> ?diff n x - f' x0 n \<bar> < ?r)"
   def S' \<equiv> "Min (?s ` {..< ?N })"