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
¤ Dauer der Verarbeitung: 0.18 Sekunden
(vorverarbeitet)
¤
|
Haftungshinweis
Die Informationen auf dieser Webseite wurden
nach bestem Wissen sorgfältig zusammengestellt. Es wird jedoch weder Vollständigkeit, noch Richtigkeit,
noch Qualität der bereit gestellten Informationen zugesichert.
Bemerkung:
Die farbliche Syntaxdarstellung ist noch experimentell.
|