--- a/src/Doc/Codegen/Setup.thy Tue Oct 08 23:31:06 2024 +0200
+++ b/src/Doc/Codegen/Setup.thy Wed Oct 09 13:06:55 2024 +0200
@@ -10,13 +10,7 @@
ML_file \<open>../antiquote_setup.ML\<close>
ML_file \<open>../more_antiquote.ML\<close>
-no_syntax (output)
- "_constrain" :: "logic => type => logic" (\<open>_::_\<close> [4, 0] 3)
- "_constrain" :: "prop' => type => prop'" (\<open>_::_\<close> [4, 0] 3)
-
-syntax (output)
- "_constrain" :: "logic => type => logic" (\<open>_ :: _\<close> [4, 0] 3)
- "_constrain" :: "prop' => type => prop'" (\<open>_ :: _\<close> [4, 0] 3)
+unbundle constrain_space_syntax
declare [[default_code_width = 74]]