src/ZF/Induct/Multiset.thy
changeset 80761 bc936d3d8b45
parent 80754 701912f5645a
child 80917 2a77bc3b4eac
--- a/src/ZF/Induct/Multiset.thy	Sun Aug 25 15:02:19 2024 +0200
+++ b/src/ZF/Induct/Multiset.thy	Sun Aug 25 15:07:22 2024 +0200
@@ -75,9 +75,9 @@
 
 syntax
   "_MColl" :: "[pttrn, i, o] \<Rightarrow> i" (\<open>(1{# _ \<in> _./ _#})\<close>)
+syntax_consts "_MColl" \<rightleftharpoons> MCollect
 translations
   "{#x \<in> M. P#}" == "CONST MCollect(M, \<lambda>x. P)"
-syntax_consts "_MColl" \<rightleftharpoons> MCollect
 
   (* multiset orderings *)