doc-src/IsarAdvanced/Codegen/Thy/Setup.thy
author haftmann
Thu, 25 Sep 2008 09:28:08 +0200
changeset 28350 715163ec93c0
parent 28213 b52f9205a02d
child 28419 f65e8b318581
permissions -rw-r--r--
non left-linear equations for nbe

theory Setup
imports Main
uses "../../../antiquote_setup.ML"
begin

ML_val {* Code_Target.code_width := 74 *}

end