src/HOL/Map.thy
changeset 15140 322485b816ac
parent 15131 c69542757a4d
child 15251 bb6f072c8d10
--- a/src/HOL/Map.thy	Tue Aug 17 11:00:24 2004 +0200
+++ b/src/HOL/Map.thy	Wed Aug 18 11:09:40 2004 +0200
@@ -9,7 +9,7 @@
 header {* Maps *}
 
 theory Map
-import List
+imports List
 begin
 
 types ('a,'b) "~=>" = "'a => 'b option" (infixr 0)