src/HOL/Typerep.thy
changeset 31048 ac146fc38b51
parent 31031 cbec39ebf8f2
child 31137 cd3aafc1c631
--- a/src/HOL/Typerep.thy	Wed May 06 16:01:05 2009 +0200
+++ b/src/HOL/Typerep.thy	Wed May 06 16:01:06 2009 +0200
@@ -1,11 +1,9 @@
-(*  Title:      HOL/Typerep.thy
-    Author:     Florian Haftmann, TU Muenchen
-*)
+(* Author: Florian Haftmann, TU Muenchen *)
 
 header {* Reflecting Pure types into HOL *}
 
 theory Typerep
-imports Plain List Code_Message
+imports Plain String
 begin
 
 datatype typerep = Typerep message_string "typerep list"
@@ -42,7 +40,7 @@
 struct
 
 fun mk f (Type (tyco, tys)) =
-      @{term Typerep} $ Message_String.mk tyco
+      @{term Typerep} $ HOLogic.mk_message_string tyco
         $ HOLogic.mk_list @{typ typerep} (map (mk f) tys)
   | mk f (TFree v) =
       f v;