src/ZF/UNITY/Union.thy
changeset 80754 701912f5645a
parent 76217 8655344f1cf6
child 80761 bc936d3d8b45
--- a/src/ZF/UNITY/Union.thy	Fri Aug 23 22:47:51 2024 +0200
+++ b/src/ZF/UNITY/Union.thy	Fri Aug 23 23:14:39 2024 +0200
@@ -43,11 +43,12 @@
 syntax
   "_JOIN1"  :: "[pttrns, i] \<Rightarrow> i"     (\<open>(3\<Squnion>_./ _)\<close> 10)
   "_JOIN"   :: "[pttrn, i, i] \<Rightarrow> i"   (\<open>(3\<Squnion>_ \<in> _./ _)\<close> 10)
-
 translations
   "\<Squnion>x \<in> A. B" == "CONST JOIN(A, (\<lambda>x. B))"
   "\<Squnion>x y. B"   == "\<Squnion>x. \<Squnion>y. B"
   "\<Squnion>x. B"     == "CONST JOIN(CONST state, (\<lambda>x. B))"
+syntax_consts
+  "_JOIN1" "_JOIN" == JOIN
 
 
 subsection\<open>SKIP\<close>