src/HOL/Code_Eval.thy
changeset 28952 15a4b2cf8c34
parent 28661 a287d0e8aa9d
child 28965 1de908189869
equal deleted inserted replaced
28948:1860f016886d 28952:15a4b2cf8c34
     4 *)
     4 *)
     5 
     5 
     6 header {* Term evaluation using the generic code generator *}
     6 header {* Term evaluation using the generic code generator *}
     7 
     7 
     8 theory Code_Eval
     8 theory Code_Eval
     9 imports Plain "~~/src/HOL/Library/RType"
     9 imports Plain Typerep
    10 begin
    10 begin
    11 
    11 
    12 subsection {* Term representation *}
    12 subsection {* Term representation *}
    13 
    13 
    14 subsubsection {* Terms and class @{text term_of} *}
    14 subsubsection {* Terms and class @{text term_of} *}