src/HOL/Decision_Procs/Approximation_Bounds.thy
changeset 70097 4005298550a6
parent 69597 ff784d5a5bfb
child 70347 e5cd5471c18a
--- a/src/HOL/Decision_Procs/Approximation_Bounds.thy	Tue Apr 09 21:05:48 2019 +0100
+++ b/src/HOL/Decision_Procs/Approximation_Bounds.thy	Wed Apr 10 13:34:55 2019 +0100
@@ -34,7 +34,7 @@
     by auto
   show ?thesis
     unfolding sum_distrib_left shift_pow uminus_add_conv_diff [symmetric] sum_negf[symmetric]
-    sum_head_upt_Suc[OF zero_less_Suc]
+    sum.atLeast_Suc_lessThan[OF zero_less_Suc]
     sum.reindex[OF inj_Suc, unfolded comp_def, symmetric, of "\<lambda> n. (-1)^n  *a n * x^n"] by auto
 qed