src/HOL/Library/Multiset.thy
changeset 15630 cc3776f004e2
parent 15402 97204f3b4705
child 15867 5c63b6c2f4a5
--- a/src/HOL/Library/Multiset.thy	Fri Mar 25 17:47:11 2005 +0100
+++ b/src/HOL/Library/Multiset.thy	Sat Mar 26 00:00:56 2005 +0100
@@ -742,7 +742,7 @@
 lemma set_of_multiset_of[simp]: "set_of(multiset_of x) = set x"
  by (induct_tac x, auto) 
 
-lemma multset_of_append[simp]: 
+lemma multiset_of_append[simp]: 
   "multiset_of (xs @ ys) = multiset_of xs + multiset_of ys"
   by (rule_tac x=ys in spec, induct_tac xs, auto simp: union_ac) 
 
@@ -778,6 +778,9 @@
   apply simp
   done
 
+lemma multiset_of_compl_union[simp]:
+ "multiset_of [x\<in>xs. P x] + multiset_of [x\<in>xs. \<not>P x] = multiset_of xs"
+  by (induct xs) (auto simp: union_ac)
 
 subsection {* Pointwise ordering induced by count *}