src/HOL/Deriv.thy
changeset 44890 22f665a2e91c
parent 44568 e6f291cb5810
child 44921 58eef4843641
--- a/src/HOL/Deriv.thy	Sun Sep 11 22:56:05 2011 +0200
+++ b/src/HOL/Deriv.thy	Mon Sep 12 07:55:43 2011 +0200
@@ -745,7 +745,7 @@
     proof (rule ccontr)
       assume "\<not> (\<exists>x. a \<le> x \<and> x \<le> b \<and> f x = M)"
       with M1 have M3: "\<forall>x. a \<le> x & x \<le> b --> f x < M"
-        by (fastsimp simp add: linorder_not_le [symmetric])
+        by (fastforce simp add: linorder_not_le [symmetric])
       hence "\<forall>x. a \<le> x & x \<le> b --> isCont (%x. inverse (M - f x)) x"
         by (auto simp add: con)
       from isCont_bounded [OF le this]