doc-src/Codegen/Thy/Setup.thy
author bulwahn
Fri, 21 Oct 2011 11:17:14 +0200
changeset 45231 d85a2fdc586c
parent 43564 9864182c6bad
child 46517 9d2e682a68eb
permissions -rw-r--r--
replacing code_inline by code_unfold, removing obsolete code_unfold, code_inline del now that the ancient code generator is removed

theory Setup
imports
  Complex_Main
  More_List RBT Dlist List_Cset Mapping
uses
  "../../antiquote_setup.ML"
  "../../more_antiquote.ML"
begin

setup {*
  Antiquote_Setup.setup #>
  More_Antiquote.setup #>
let
  val typ = Simple_Syntax.read_typ;
in
  Sign.del_modesyntax_i (Symbol.xsymbolsN, false)
   [("_constrain", typ "logic => type => logic", Mixfix ("_\<Colon>_", [4, 0], 3)),
    ("_constrain", typ "prop' => type => prop'", Mixfix ("_\<Colon>_", [4, 0], 3))] #>
  Sign.add_modesyntax_i (Symbol.xsymbolsN, false)
   [("_constrain", typ "logic => type => logic", Mixfix ("_ \<Colon>  _", [4, 0], 3)),
    ("_constrain", typ "prop' => type => prop'", Mixfix ("_ \<Colon> _", [4, 0], 3))]
end
*}

setup {* Code_Target.set_default_code_width 74 *}

declare [[names_unique = false]]

end