src/Doc/Codegen/Setup.thy
author wenzelm
Fri, 18 Feb 2022 23:10:33 +0100
changeset 75102 678fae02f9b3
parent 69605 a96320074298
child 80914 d97fdabd9e2b
permissions -rw-r--r--
improved support for Java Chromium Embedded Framework (JCEF): works on x86_64-linux and x86_64-windows with jdk-15 (not jdk-17), does not work on arm64 and darwin;

theory Setup
imports
  Complex_Main
  "HOL-Library.Dlist"
  "HOL-Library.RBT"
  "HOL-Library.Mapping"
  "HOL-Library.IArray"
begin

ML_file \<open>../antiquote_setup.ML\<close>
ML_file \<open>../more_antiquote.ML\<close>

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