src/HOL/Decision_Procs/Approximation_Bounds.thy
changeset 66280 0c5eb47e2696
parent 65582 a1bc1b020cf2
child 66453 cc19f7ca2ed6
--- a/src/HOL/Decision_Procs/Approximation_Bounds.thy	Sat Jul 15 14:54:13 2017 +0100
+++ b/src/HOL/Decision_Procs/Approximation_Bounds.thy	Sat Jul 15 16:27:10 2017 +0100
@@ -339,7 +339,7 @@
         show ?thesis by auto
       qed
       hence "sqrt (2 powr (?E mod 2)) < sqrt (2 * 2)"
-        by (auto simp del: real_sqrt_four)
+        by (intro real_sqrt_less_mono) auto
       hence E_mod_pow: "sqrt (2 powr (?E mod 2)) < 2" by auto
 
       have E_eq: "2 powr ?E = 2 powr (?E div 2 + ?E div 2 + ?E mod 2)"