src/Doc/Codegen/Setup.thy
author paulson <lp15@cam.ac.uk>
Wed, 18 Mar 2015 14:13:27 +0000
changeset 59741 5b762cd73a8e
parent 59378 065f349852e6
child 61143 5f898411ce87
permissions -rw-r--r--
Lots of new material on complex-valued functions. Modified simplification of (x/n)^k

theory Setup
imports
  Complex_Main
  "~~/src/Tools/Permanent_Interpretation"
  "~~/src/HOL/Library/Dlist"
  "~~/src/HOL/Library/RBT"
  "~~/src/HOL/Library/Mapping"
  "~~/src/HOL/Library/IArray"
begin

ML_file "../antiquote_setup.ML"
ML_file "../more_antiquote.ML"

setup \<open>
let
  val typ = Simple_Syntax.read_typ;
in
  Sign.del_syntax (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_syntax (Symbol.xsymbolsN, false)
   [("_constrain", typ "logic => type => logic", Mixfix ("_ \<Colon>  _", [4, 0], 3)),
    ("_constrain", typ "prop' => type => prop'", Mixfix ("_ \<Colon> _", [4, 0], 3))]
end
\<close>

declare [[default_code_width = 74]]

declare [[names_unique = false]]

end