src/ZF/UNITY/Union.thy
changeset 80761 bc936d3d8b45
parent 80754 701912f5645a
child 80917 2a77bc3b4eac
--- a/src/ZF/UNITY/Union.thy	Sun Aug 25 15:02:19 2024 +0200
+++ b/src/ZF/UNITY/Union.thy	Sun Aug 25 15:07:22 2024 +0200
@@ -43,12 +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)
+syntax_consts
+  "_JOIN1" "_JOIN" == JOIN
 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>