src/Doc/Codegen/Setup.thy
author wenzelm
Wed, 09 Sep 2015 14:47:41 +0200
changeset 61143 5f898411ce87
parent 59378 065f349852e6
child 61670 301e0b4ecd45
permissions -rw-r--r--
eliminated \<Colon> from syntax of constraints;

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"

no_syntax (output)
  "_constrain" :: "logic => type => logic"  ("_::_" [4, 0] 3)
  "_constrain" :: "prop' => type => prop'"  ("_::_" [4, 0] 3)

syntax (output)
  "_constrain" :: "logic => type => logic"  ("_ :: _" [4, 0] 3)
  "_constrain" :: "prop' => type => prop'"  ("_ :: _" [4, 0] 3)

declare [[default_code_width = 74]]

declare [[names_unique = false]]

end