src/HOL/HOLCF/Sprod.thy
changeset 81019 dd59daa3c37a
parent 80914 d97fdabd9e2b
child 81091 c007e6d9941d
--- a/src/HOL/HOLCF/Sprod.thy	Mon Sep 30 13:00:42 2024 +0200
+++ b/src/HOL/HOLCF/Sprod.thy	Mon Sep 30 20:30:59 2024 +0200
@@ -40,13 +40,10 @@
 definition ssplit :: "('a \<rightarrow> 'b \<rightarrow> 'c) \<rightarrow> ('a ** 'b) \<rightarrow> 'c"
   where "ssplit = (\<Lambda> f p. seq\<cdot>p\<cdot>(f\<cdot>(sfst\<cdot>p)\<cdot>(ssnd\<cdot>p)))"
 
-nonterminal stuple_args
 syntax
-  "" :: "logic \<Rightarrow> stuple_args"  (\<open>_\<close>)
-  "_stuple_args" :: "logic \<Rightarrow> stuple_args \<Rightarrow> stuple_args"  (\<open>_,/ _\<close>)
-  "_stuple" :: "[logic, stuple_args] \<Rightarrow> logic"  (\<open>(1'(:_,/ _:'))\<close>)
+  "_stuple" :: "[logic, args] \<Rightarrow> logic"  (\<open>(\<open>indent=1 notation=\<open>mixfix strict tuple\<close>\<close>'(:_,/ _:'))\<close>)
 syntax_consts
-  "_stuple_args" "_stuple" \<rightleftharpoons> spair
+  spair
 translations
   "(:x, y, z:)" \<rightleftharpoons> "(:x, (:y, z:):)"
   "(:x, y:)" \<rightleftharpoons> "CONST spair\<cdot>x\<cdot>y"