more inner-syntax markup;
authorwenzelm
Fri, 25 Oct 2024 16:03:58 +0200
changeset 81261 0c9075bdff38
parent 81260 ff60c3b565da
child 81262 d912f97aaa86
more inner-syntax markup;
src/Benchmarks/Quickcheck_Benchmark/Needham_Schroeder_Base.thy
src/Doc/Tutorial/Protocol/Message.thy
--- a/src/Benchmarks/Quickcheck_Benchmark/Needham_Schroeder_Base.thy	Fri Oct 25 15:48:40 2024 +0200
+++ b/src/Benchmarks/Quickcheck_Benchmark/Needham_Schroeder_Base.thy	Fri Oct 25 16:03:58 2024 +0200
@@ -28,6 +28,8 @@
 
 syntax
   "_MTuple" :: "['a, args] \<Rightarrow> 'a * 'b"  (\<open>(\<open>indent=2 notation=\<open>mixfix message tuple\<close>\<close>\<lbrace>_,/ _\<rbrace>)\<close>)
+syntax_consts
+  "_MTuple" \<rightleftharpoons> MPair
 translations
   "\<lbrace>x, y, z\<rbrace>" \<rightleftharpoons> "\<lbrace>x, \<lbrace>y, z\<rbrace>\<rbrace>"
   "\<lbrace>x, y\<rbrace>" \<rightleftharpoons> "CONST MPair x y"
--- a/src/Doc/Tutorial/Protocol/Message.thy	Fri Oct 25 15:48:40 2024 +0200
+++ b/src/Doc/Tutorial/Protocol/Message.thy	Fri Oct 25 16:03:58 2024 +0200
@@ -81,6 +81,8 @@
 text\<open>Concrete syntax: messages appear as \<open>\<lbrace>A,B,NA\<rbrace>\<close>, etc...\<close>
 syntax
   "_MTuple" :: "['a, args] \<Rightarrow> 'a * 'b"  ("(\<open>indent=2 notation=\<open>mixfix message tuple\<close>\<close>\<lbrace>_,/ _\<rbrace>)")
+syntax_consts
+  "_MTuple" \<rightleftharpoons> MPair
 translations
   "\<lbrace>x, y, z\<rbrace>" \<rightleftharpoons> "\<lbrace>x, \<lbrace>y, z\<rbrace>\<rbrace>"
   "\<lbrace>x, y\<rbrace>" \<rightleftharpoons> "CONST MPair x y"