src/HOL/Library/Multiset.thy
changeset 23281 e26ec695c9b3
parent 22316 f662831459de
child 23373 ead82c82da9e
--- a/src/HOL/Library/Multiset.thy	Wed Jun 06 19:12:40 2007 +0200
+++ b/src/HOL/Library/Multiset.thy	Wed Jun 06 19:12:59 2007 +0200
@@ -786,11 +786,11 @@
   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"
+    "multiset_of [x\<leftarrow>xs. P x] + multiset_of [x\<leftarrow>xs. \<not>P x] = multiset_of xs"
   by (induct xs) (auto simp: union_ac)
 
 lemma count_filter:
-    "count (multiset_of xs) x = length [y \<in> xs. y = x]"
+    "count (multiset_of xs) x = length [y \<leftarrow> xs. y = x]"
   by (induct xs) auto