diff -r 2dba15d3c402 -r 0c5eb47e2696 src/HOL/Decision_Procs/Approximation_Bounds.thy --- 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)"