New lemma
authornipkow
Mon, 08 Jun 2009 08:52:18 +0200
changeset 31501 2a60c9b951e0
parent 31500 eced346b2231
child 31503 cca1281e6384
New lemma
src/HOL/SetInterval.thy
--- a/src/HOL/SetInterval.thy	Mon Jun 08 00:26:57 2009 +0200
+++ b/src/HOL/SetInterval.thy	Mon Jun 08 08:52:18 2009 +0200
@@ -833,6 +833,13 @@
 apply (simp add: atLeastLessThanSuc_atLeastAtMost[symmetric] algebra_simps)
 done
 
+lemma setsum_ub_add_nat: assumes "(m::nat) \<le> n + 1"
+  shows "setsum f {m..n + p} = setsum f {m..n} + setsum f {n + 1..n + p}"
+proof-
+  have "{m .. n+p} = {m..n} \<union> {n+1..n+p}" using `m \<le> n+1` by auto
+  thus ?thesis by (auto simp: ivl_disj_int setsum_Un_disjoint
+    atLeastSucAtMost_greaterThanAtMost)
+qed
 
 lemma setsum_add_nat_ivl: "\<lbrakk> m \<le> n; n \<le> p \<rbrakk> \<Longrightarrow>
   setsum f {m..<n} + setsum f {n..<p} = setsum f {m..<p::nat}"