src/HOL/Library/Code_Message.thy
changeset 27487 c8a6ce181805
parent 27368 9f90ac19e32b
child 28054 2b84d34c5d02
--- a/src/HOL/Library/Code_Message.thy	Fri Jul 04 16:33:08 2008 +0200
+++ b/src/HOL/Library/Code_Message.thy	Mon Jul 07 08:47:17 2008 +0200
@@ -5,7 +5,7 @@
 header {* Monolithic strings (message strings) for code generation *}
 
 theory Code_Message
-imports Plain List
+imports Plain "~~/src/HOL/List"
 begin
 
 subsection {* Datatype of messages *}