src/HOL/Multivariate_Analysis/ex/Approximations.thy
changeset 61945 1135b8de26c3
parent 61694 6571c78c9667
child 62085 5b7758af429e
--- a/src/HOL/Multivariate_Analysis/ex/Approximations.thy	Mon Dec 28 01:26:34 2015 +0100
+++ b/src/HOL/Multivariate_Analysis/ex/Approximations.thy	Mon Dec 28 01:28:28 2015 +0100
@@ -24,7 +24,7 @@
 qed
 
 (*32-bit approximation. SLOW simplification steps: big calculations with the rewriting engine*)
-lemma pi_approx_32: "abs(pi - 13493037705/4294967296) \<le> inverse(2 ^ 32)"
+lemma pi_approx_32: "\<bar>pi - 13493037705/4294967296\<bar> \<le> inverse(2 ^ 32)"
   apply (simp only: abs_diff_le_iff)
   apply (rule sin_pi6_straddle, simp_all)
    using Taylor_sin [of "1686629713/3221225472" 11]