src/Benchmarks/Quickcheck_Benchmark/Needham_Schroeder_Base.thy
changeset 81091 c007e6d9941d
parent 81019 dd59daa3c37a
child 81261 0c9075bdff38
--- a/src/Benchmarks/Quickcheck_Benchmark/Needham_Schroeder_Base.thy	Mon Sep 30 23:32:26 2024 +0200
+++ b/src/Benchmarks/Quickcheck_Benchmark/Needham_Schroeder_Base.thy	Tue Oct 01 20:39:16 2024 +0200
@@ -28,8 +28,6 @@
 
 syntax
   "_MTuple" :: "['a, args] \<Rightarrow> 'a * 'b"  (\<open>(\<open>indent=2 notation=\<open>mixfix message tuple\<close>\<close>\<lbrace>_,/ _\<rbrace>)\<close>)
-syntax_consts
-  MPair
 translations
   "\<lbrace>x, y, z\<rbrace>" \<rightleftharpoons> "\<lbrace>x, \<lbrace>y, z\<rbrace>\<rbrace>"
   "\<lbrace>x, y\<rbrace>" \<rightleftharpoons> "CONST MPair x y"