| changeset 80784 | 3d9e7746d9db |
| parent 80768 | c7723cc15de8 |
| child 80914 | d97fdabd9e2b |
--- a/src/HOL/Library/Monad_Syntax.thy Wed Aug 28 16:46:33 2024 +0200 +++ b/src/HOL/Library/Monad_Syntax.thy Wed Aug 28 19:40:07 2024 +0200 @@ -47,8 +47,7 @@ "_thenM" :: "['a, 'b] \<Rightarrow> 'c" (infixl ">>" 54) syntax_consts - "_do_block" "_do_cons" \<rightleftharpoons> bind_do and - "_do_bind" "_thenM" \<rightleftharpoons> bind and + "_do_block" "_do_cons" "_do_bind" "_do_then" \<rightleftharpoons> bind and "_do_let" \<rightleftharpoons> Let translations