src/HOL/Library/RType.thy
changeset 28228 7ebe8dc06cbb
parent 28084 a05ca48ef263
child 28335 25326092cf9a
--- a/src/HOL/Library/RType.thy	Tue Sep 16 09:21:22 2008 +0200
+++ b/src/HOL/Library/RType.thy	Tue Sep 16 09:21:24 2008 +0200
@@ -6,7 +6,7 @@
 header {* Reflecting Pure types into HOL *}
 
 theory RType
-imports Plain "~~/src/HOL/List" "~~/src/HOL/Code_Message" "~~/src/HOL/Code_Index" (* import all 'special code' types *)
+imports Plain "~~/src/HOL/List" "~~/src/HOL/Library/Code_Message"
 begin
 
 datatype "rtype" = RType message_string "rtype list"