src/HOL/Analysis/Complex_Transcendental.thy
changeset 64267 b9a1486e79be
parent 64240 eabf80376aab
child 64287 d85d88722745
--- a/src/HOL/Analysis/Complex_Transcendental.thy	Sun Oct 16 22:43:51 2016 +0200
+++ b/src/HOL/Analysis/Complex_Transcendental.thy	Mon Oct 17 11:46:22 2016 +0200
@@ -597,7 +597,7 @@
 text\<open>32-bit Approximation to e\<close>
 lemma e_approx_32: "\<bar>exp(1) - 5837465777 / 2147483648\<bar> \<le> (inverse(2 ^ 32)::real)"
   using Taylor_exp [of 1 14] exp_le
-  apply (simp add: setsum_distrib_right in_Reals_norm Re_exp atMost_nat_numeral fact_numeral)
+  apply (simp add: sum_distrib_right in_Reals_norm Re_exp atMost_nat_numeral fact_numeral)
   apply (simp only: pos_le_divide_eq [symmetric], linarith)
   done