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