diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Library/Monad_Syntax.thy --- a/src/HOL/Library/Monad_Syntax.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Library/Monad_Syntax.thy Fri Sep 20 19:51:08 2024 +0200 @@ -15,10 +15,10 @@ \ consts - bind :: "'a \ ('b \ 'c) \ 'd" (infixl "\" 54) + bind :: "'a \ ('b \ 'c) \ 'd" (infixl \\\ 54) notation (ASCII) - bind (infixl ">>=" 54) + bind (infixl \>>=\ 54) abbreviation (do_notation) @@ -26,25 +26,25 @@ where "bind_do \ bind" notation (output) - bind_do (infixl "\" 54) + bind_do (infixl \\\ 54) notation (ASCII output) - bind_do (infixl ">>=" 54) + bind_do (infixl \>>=\ 54) nonterminal do_binds and do_bind syntax - "_do_block" :: "do_binds \ 'a" ("do {//(2 _)//}" [12] 62) - "_do_bind" :: "[pttrn, 'a] \ do_bind" ("(2_ \/ _)" 13) - "_do_let" :: "[pttrn, 'a] \ do_bind" ("(2let _ =/ _)" [1000, 13] 13) - "_do_then" :: "'a \ do_bind" ("_" [14] 13) - "_do_final" :: "'a \ do_binds" ("_") - "_do_cons" :: "[do_bind, do_binds] \ do_binds" ("_;//_" [13, 12] 12) - "_thenM" :: "['a, 'b] \ 'c" (infixl "\" 54) + "_do_block" :: "do_binds \ 'a" (\do {//(2 _)//}\ [12] 62) + "_do_bind" :: "[pttrn, 'a] \ do_bind" (\(2_ \/ _)\ 13) + "_do_let" :: "[pttrn, 'a] \ do_bind" (\(2let _ =/ _)\ [1000, 13] 13) + "_do_then" :: "'a \ do_bind" (\_\ [14] 13) + "_do_final" :: "'a \ do_binds" (\_\) + "_do_cons" :: "[do_bind, do_binds] \ do_binds" (\_;//_\ [13, 12] 12) + "_thenM" :: "['a, 'b] \ 'c" (infixl \\\ 54) syntax (ASCII) - "_do_bind" :: "[pttrn, 'a] \ do_bind" ("(2_ <-/ _)" 13) - "_thenM" :: "['a, 'b] \ 'c" (infixl ">>" 54) + "_do_bind" :: "[pttrn, 'a] \ do_bind" (\(2_ <-/ _)\ 13) + "_thenM" :: "['a, 'b] \ 'c" (infixl \>>\ 54) syntax_consts "_do_block" "_do_cons" "_do_bind" "_do_then" \ bind and