remove unused intermediate lemma
authorhuffman
Tue, 29 May 2012 11:30:13 +0200
changeset 48011 391439b10100
parent 48010 0da831254551
child 48012 b6e5e86a7303
remove unused intermediate lemma
src/HOL/Library/Multiset.thy
--- a/src/HOL/Library/Multiset.thy	Tue May 29 11:13:00 2012 +0200
+++ b/src/HOL/Library/Multiset.thy	Tue May 29 11:30:13 2012 +0200
@@ -539,14 +539,6 @@
 
 subsection {* Induction and case splits *}
 
-lemma setsum_decr:
-  "finite F ==> (0::nat) < f a ==>
-    setsum (f (a := f a - 1)) F = (if a\<in>F then setsum f F - 1 else setsum f F)"
-apply (induct rule: finite_induct)
- apply auto
-apply (drule_tac a = a in mk_disjoint_insert, auto)
-done
-
 theorem multiset_induct [case_names empty add, induct type: multiset]:
   assumes empty: "P {#}"
   assumes add: "\<And>M x. P M \<Longrightarrow> P (M + {#x#})"