--- a/src/HOL/Library/AssocList.thy Thu Jun 26 10:06:54 2008 +0200
+++ b/src/HOL/Library/AssocList.thy Thu Jun 26 10:07:01 2008 +0200
@@ -6,7 +6,7 @@
header {* Map operations implemented on association lists*}
theory AssocList
-imports Map
+imports Plain Map
begin
text {*