diff -r 515b6020cf5d -r c1b87ef4a1c3 src/HOL/Hyperreal/Integration.thy --- a/src/HOL/Hyperreal/Integration.thy Tue Jul 12 12:49:46 2005 +0200 +++ b/src/HOL/Hyperreal/Integration.thy Tue Jul 12 17:56:03 2005 +0200 @@ -429,7 +429,7 @@ prefer 2 apply simp apply (erule_tac [!] V= "\x'. x' ~= x & \x' + - x\ < s --> ?P x'" in thin_rl) apply (drule_tac x = v in spec, simp add: times_divide_eq) -apply (drule_tac x = u in spec, auto, arith) +apply (drule_tac x = u in spec, auto) apply (subgoal_tac "\f u - f x - f' x * (u - x)\ = \f x - f u - f' x * (x - u)\") apply (rule order_trans) apply (auto simp add: abs_le_interval_iff)