doc-src/IsarAdvanced/Codegen/Thy/Setup.thy
changeset 28213 b52f9205a02d
child 28419 f65e8b318581
equal deleted inserted replaced
28212:44831b583999 28213:b52f9205a02d
       
     1 theory Setup
       
     2 imports Main
       
     3 uses "../../../antiquote_setup.ML"
       
     4 begin
       
     5 
       
     6 ML_val {* Code_Target.code_width := 74 *}
       
     7 
       
     8 end