src/HOL/Library/RType.thy
changeset 28228 7ebe8dc06cbb
parent 28084 a05ca48ef263
child 28335 25326092cf9a
equal deleted inserted replaced
28227:77221ee0f7b9 28228:7ebe8dc06cbb
     4 *)
     4 *)
     5 
     5 
     6 header {* Reflecting Pure types into HOL *}
     6 header {* Reflecting Pure types into HOL *}
     7 
     7 
     8 theory RType
     8 theory RType
     9 imports Plain "~~/src/HOL/List" "~~/src/HOL/Code_Message" "~~/src/HOL/Code_Index" (* import all 'special code' types *)
     9 imports Plain "~~/src/HOL/List" "~~/src/HOL/Library/Code_Message"
    10 begin
    10 begin
    11 
    11 
    12 datatype "rtype" = RType message_string "rtype list"
    12 datatype "rtype" = RType message_string "rtype list"
    13 
    13 
    14 class rtype =
    14 class rtype =