1
theory Setup
2
imports Complex_Main
3
uses "../../../antiquote_setup.ML" "../../../more_antiquote.ML"
4
begin
5
6
ML {* no_document use_thys
7
["Efficient_Nat", "Code_Char_chr", "Product_ord"] *}
8
9
ML_val {* Code_Target.code_width := 74 *}
10
11
end