--- a/src/HOL/Imperative_HOL/Overview.thy Fri Sep 20 19:07:10 2024 +0200
+++ b/src/HOL/Imperative_HOL/Overview.thy Fri Sep 20 19:51:08 2024 +0200
@@ -9,12 +9,12 @@
(* type constraints with spacing *)
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)
(*>*)
text \<open>