src/HOL/Taylor.thy
changeset 44890 22f665a2e91c
parent 28952 15a4b2cf8c34
child 56193 c726ecfb22b6
--- a/src/HOL/Taylor.thy	Sun Sep 11 22:56:05 2011 +0200
+++ b/src/HOL/Taylor.thy	Mon Sep 12 07:55:43 2011 +0200
@@ -50,8 +50,8 @@
     let ?H = "x + c"
     from X have "c<?H & ?H<b \<and> f b = (\<Sum>m = 0..<n. diff m c / real (fact m) * (b - c) ^ m) +
       diff n ?H / real (fact n) * (b - c) ^ n"
-      by fastsimp
-    thus ?thesis by fastsimp
+      by fastforce
+    thus ?thesis by fastforce
   qed
 qed
 
@@ -90,8 +90,8 @@
     let ?H = "x + c"
     from X have "a<?H & ?H<c \<and> f a = (\<Sum>m = 0..<n. diff m c / real (fact m) * (a - c) ^ m) +
       diff n ?H / real (fact n) * (a - c) ^ n"
-      by fastsimp
-    thus ?thesis by fastsimp
+      by fastforce
+    thus ?thesis by fastforce
   qed
 qed
 
@@ -107,7 +107,7 @@
   note INIT
   moreover from DERIV and INTERV
   have "\<forall>m t. m < n \<and> x \<le> t \<and> t \<le> b \<longrightarrow> DERIV (diff m) t :> diff (Suc m) t"
-    by fastsimp
+    by fastforce
   moreover note True
   moreover from INTERV have "c \<le> b" by simp
   ultimately have EX: "\<exists>t>x. t < c \<and> f x =
@@ -120,7 +120,7 @@
   note INIT
   moreover from DERIV and INTERV
   have "\<forall>m t. m < n \<and> a \<le> t \<and> t \<le> x \<longrightarrow> DERIV (diff m) t :> diff (Suc m) t"
-    by fastsimp
+    by fastforce
   moreover from INTERV have "a \<le> c" by arith
   moreover from False and INTERV have "c < x" by arith
   ultimately have EX: "\<exists>t>c. t < x \<and> f x =