src/HOL/Library/Multiset.thy
changeset 47143 212f7a975d49
parent 46921 aa862ff8a8a9
child 47177 2fa00264392a
--- a/src/HOL/Library/Multiset.thy	Mon Mar 26 21:03:30 2012 +0200
+++ b/src/HOL/Library/Multiset.thy	Tue Mar 27 14:14:46 2012 +0200
@@ -1189,7 +1189,7 @@
 lemma Mempty_Bag [code]:
   "{#} = Bag (DAList.empty)"
   by (simp add: multiset_eq_iff alist.Alist_inverse DAList.empty_def)
-  
+
 lemma single_Bag [code]:
   "{#x#} = Bag (DAList.update x 1 DAList.empty)"
   by (simp add: multiset_eq_iff alist.Alist_inverse impl_of_update impl_of_empty)