src/HOL/Library/Multiset.thy
changeset 68990 a319e3c522ba
parent 68988 93546c85374a
child 68992 8f7d3241ed68
--- a/src/HOL/Library/Multiset.thy	Thu Sep 13 15:15:50 2018 +0200
+++ b/src/HOL/Library/Multiset.thy	Thu Sep 13 16:15:05 2018 +0200
@@ -1890,9 +1890,6 @@
 lemma union_mset_compl[simp]: "\<forall>x. P x = (\<not> Q x) \<Longrightarrow> filter_mset P M + filter_mset Q M = M"
 by (induction M) simp_all
 
-lemma mset_compl_union: "mset [x\<leftarrow>xs. P x] + mset [x\<leftarrow>xs. \<not>P x] = mset xs"
-  by (induct xs) auto
-
 lemma nth_mem_mset: "i < length ls \<Longrightarrow> (ls ! i) \<in># mset ls"
 proof (induct ls arbitrary: i)
   case Nil