diff -r ff2a637a449e -r fc5066122e68 src/HOL/Metis_Examples/Message.thy --- a/src/HOL/Metis_Examples/Message.thy Fri Oct 18 11:44:05 2024 +0200 +++ b/src/HOL/Metis_Examples/Message.thy Fri Oct 18 14:20:09 2024 +0200 @@ -50,6 +50,8 @@ text\Concrete syntax: messages appear as \\A,B,NA\\, etc...\ syntax "_MTuple" :: "['a, args] \ 'a * 'b" (\(\indent=2 notation=\mixfix message tuple\\\_,/ _\)\) +syntax_consts + "_MTuple" \ MPair translations "\x, y, z\" \ "\x, \y, z\\" "\x, y\" \ "CONST MPair x y"