--- a/src/Doc/Tutorial/Protocol/Message.thy Fri Sep 20 19:07:10 2024 +0200
+++ b/src/Doc/Tutorial/Protocol/Message.thy Fri Sep 20 19:51:08 2024 +0200
@@ -81,9 +81,9 @@
text\<open>Concrete syntax: messages appear as \<open>\<lbrace>A,B,NA\<rbrace>\<close>, etc...\<close>
nonterminal mtuple_args
syntax
- "" :: "'a \<Rightarrow> mtuple_args" ("_")
- "_MTuple_args" :: "'a \<Rightarrow> mtuple_args \<Rightarrow> mtuple_args" ("_,/ _")
- "_MTuple" :: "['a, mtuple_args] \<Rightarrow> 'a * 'b" ("(2\<lbrace>_,/ _\<rbrace>)")
+ "" :: "'a \<Rightarrow> mtuple_args" (\<open>_\<close>)
+ "_MTuple_args" :: "'a \<Rightarrow> mtuple_args \<Rightarrow> mtuple_args" (\<open>_,/ _\<close>)
+ "_MTuple" :: "['a, mtuple_args] \<Rightarrow> 'a * 'b" (\<open>(2\<lbrace>_,/ _\<rbrace>)\<close>)
syntax_consts
"_MTuple_args" "_MTuple" \<rightleftharpoons> MPair
translations