src/HOL/Series.thy
changeset 68127 137d5d0112bb
parent 68064 b249fab48c76
child 68499 d4312962161a
--- a/src/HOL/Series.thy	Wed May 09 07:48:54 2018 +0200
+++ b/src/HOL/Series.thy	Wed May 09 14:07:19 2018 +0100
@@ -115,24 +115,11 @@
   shows "f sums (\<Sum>n\<in>N. f n)"
 proof -
   have eq: "sum f {..<n + Suc (Max N)} = sum f N" for n
-  proof (cases "N = {}")
-    case True
-    with f have "f = (\<lambda>x. 0)" by auto
-    then show ?thesis by simp
-  next
-    case [simp]: False
-    show ?thesis
-    proof (safe intro!: sum.mono_neutral_right f)
-      fix i
-      assume "i \<in> N"
-      then have "i \<le> Max N" by simp
-      then show "i < n + Suc (Max N)" by simp
-    qed
-  qed
+    by (rule sum.mono_neutral_right) (auto simp: add_increasing less_Suc_eq_le f)
   show ?thesis
     unfolding sums_def
     by (rule LIMSEQ_offset[of _ "Suc (Max N)"])
-       (simp add: eq atLeast0LessThan del: add_Suc_right)
+      (simp add: eq atLeast0LessThan del: add_Suc_right)
 qed
 
 corollary sums_0: "(\<And>n. f n = 0) \<Longrightarrow> (f sums 0)"