doc-src/IsarAdvanced/Codegen/Thy/Codegen.thy
changeset 27103 d8549f4d900b
parent 27025 c1f9fb015ea5
child 27557 151731493264
equal deleted inserted replaced
27102:a98cd7450204 27103:d8549f4d900b
     5 theory Codegen
     5 theory Codegen
     6 imports Main
     6 imports Main
     7 uses "../../../antiquote_setup.ML"
     7 uses "../../../antiquote_setup.ML"
     8 begin
     8 begin
     9 
     9 
    10 ML {*
    10 ML {* CodeTarget.code_width := 74 *}
    11 CodeTarget.target_code_width := 74;
       
    12 *}
       
    13 
    11 
    14 (*>*)
    12 (*>*)
    15 
    13 
    16 chapter {* Code generation from Isabelle theories *}
    14 chapter {* Code generation from Isabelle theories *}
    17 
    15