src/HOL/Transcendental.thy
changeset 63365 5340fb6633d0
parent 63295 52792bb9126e
child 63367 6c731c8b7f03
--- a/src/HOL/Transcendental.thy	Sat Jul 02 08:41:05 2016 +0200
+++ b/src/HOL/Transcendental.thy	Sat Jul 02 08:41:05 2016 +0200
@@ -272,7 +272,8 @@
     have "?s sums y" using sums_if'[OF \<open>f sums y\<close>] .
     from this[unfolded sums_def, THEN LIMSEQ_Suc]
     have "(\<lambda> n. if even n then f (n div 2) else 0) sums y"
-      by (simp add: lessThan_Suc_eq_insert_0 image_iff setsum.reindex if_eq sums_def cong del: if_cong)
+      by (simp add: lessThan_Suc_eq_insert_0 setsum_atLeast1_atMost_eq image_Suc_lessThan
+        if_eq sums_def cong del: if_cong)
   }
   from sums_add[OF g_sums this] show ?thesis unfolding if_sum .
 qed