doc-src/IsarAdvanced/Codegen/Thy/Setup.thy
author haftmann
Mon, 22 Sep 2008 13:56:04 +0200
changeset 28315 d3cf88fe77bc
parent 28213 b52f9205a02d
child 28419 f65e8b318581
permissions -rw-r--r--
generic quickcheck framework

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

ML_val {* Code_Target.code_width := 74 *}

end