diff -r d90869a85f60 -r 2b949a3bfaac src/Pure/Pure.thy --- a/src/Pure/Pure.thy Tue Oct 08 23:31:06 2024 +0200 +++ b/src/Pure/Pure.thy Wed Oct 09 13:06:55 2024 +0200 @@ -1575,6 +1575,20 @@ qed qed + +section \Misc\ + +bundle constrain_space_syntax \ \type constraints with spacing\ +begin +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) +end + + declare [[ML_write_global = false]] ML_command \\<^assert> (not (can ML_command \() handle _ => ()\))\