src/HOL/Decision_Procs/Approximation.thy
changeset 32642 026e7c6a6d08
parent 32441 0273a2f787ea
child 32650 34bfa2492298
--- a/src/HOL/Decision_Procs/Approximation.thy	Mon Sep 21 16:11:36 2009 +0200
+++ b/src/HOL/Decision_Procs/Approximation.thy	Tue Sep 22 15:36:55 2009 +0200
@@ -1904,7 +1904,7 @@
 	show "0 < real x * 2/3" using * by auto
 	show "real ?max + 1 \<le> real x * 2/3" using * up
 	  by (cases "0 < real x * real (lapprox_posrat prec 2 3) - 1",
-	      auto simp add: real_of_float_max)
+	      auto simp add: real_of_float_max min_max.sup_absorb1)
       qed
       finally have "real (?lb_horner (Float 1 -1)) + real (?lb_horner ?max)
 	\<le> ln (real x)"