doc-src/IsarAdvanced/Codegen/Thy/Codegen.thy
changeset 20948 9b9910b82645
child 21058 a32d357dfd70
equal deleted inserted replaced
20947:bc827aa5015e 20948:9b9910b82645
       
     1 
       
     2 (* $Id$ *)
       
     3 
       
     4 theory Codegen
       
     5 imports Main
       
     6 begin
       
     7 
       
     8 chapter {* Code generation from Isabelle theories *}
       
     9 
       
    10 section {* Introduction *}
       
    11 
       
    12 text {*
       
    13   \cite{isa-tutorial}
       
    14 *} (* add graphics here *)
       
    15 
       
    16 section {* Basics *}
       
    17 
       
    18 subsection {* Invoking the code generator *}
       
    19 
       
    20 subsection {* Theorem selection *}
       
    21 
       
    22 (* print_codethms, code func, default setup code nofunc *)
       
    23 
       
    24 subsection {* Type classes *}
       
    25 
       
    26 subsection {* Preprocessing *}
       
    27 
       
    28 (* preprocessing, print_codethms () *)
       
    29 
       
    30 subsection {* Incremental code generation *}
       
    31 
       
    32 (* print_codethms (\<dots>) *)
       
    33 
       
    34 
       
    35 section {* Customizing serialization  *}
       
    36 
       
    37 section {* Recipes and advanced topics *}
       
    38 
       
    39 (* understanding the type game, reflexive equations, code inline code_constsubst, code_abstype*)
       
    40 
       
    41 section {* ML interfaces *}
       
    42 
       
    43 subsection {* codegen\_data.ML *}
       
    44 
       
    45 subsection {* Implementing code generator applications *}
       
    46 
       
    47 end