src/HOL/Library/Multiset.thy
changeset 51161 6ed12ae3b3e1
parent 51143 0a2371e7ced3
child 51548 757fa47af981
--- a/src/HOL/Library/Multiset.thy	Fri Feb 15 11:47:33 2013 +0100
+++ b/src/HOL/Library/Multiset.thy	Fri Feb 15 11:47:34 2013 +0100
@@ -5,7 +5,7 @@
 header {* (Finite) multisets *}
 
 theory Multiset
-imports Main DAList
+imports Main DAList (* FIXME too specific dependency for a generic theory *)
 begin
 
 subsection {* The type of multisets *}