--- a/src/Doc/Codegen/Setup.thy Fri Sep 20 19:07:10 2024 +0200
+++ b/src/Doc/Codegen/Setup.thy Fri Sep 20 19:51:08 2024 +0200
@@ -11,12 +11,12 @@
ML_file \<open>../more_antiquote.ML\<close>
no_syntax (output)
- "_constrain" :: "logic => type => logic" ("_::_" [4, 0] 3)
- "_constrain" :: "prop' => type => prop'" ("_::_" [4, 0] 3)
+ "_constrain" :: "logic => type => logic" (\<open>_::_\<close> [4, 0] 3)
+ "_constrain" :: "prop' => type => prop'" (\<open>_::_\<close> [4, 0] 3)
syntax (output)
- "_constrain" :: "logic => type => logic" ("_ :: _" [4, 0] 3)
- "_constrain" :: "prop' => type => prop'" ("_ :: _" [4, 0] 3)
+ "_constrain" :: "logic => type => logic" (\<open>_ :: _\<close> [4, 0] 3)
+ "_constrain" :: "prop' => type => prop'" (\<open>_ :: _\<close> [4, 0] 3)
declare [[default_code_width = 74]]