src/CCL/Set.thy
changeset 81011 6d34c2bedaa3
parent 80917 2a77bc3b4eac
child 81091 c007e6d9941d
--- a/src/CCL/Set.thy	Sun Sep 29 21:40:37 2024 +0200
+++ b/src/CCL/Set.thy	Sun Sep 29 21:57:47 2024 +0200
@@ -20,7 +20,7 @@
 syntax
   "_Coll" :: "[idt, o] \<Rightarrow> 'a set"  (\<open>(\<open>indent=1 notation=\<open>mixfix Collect\<close>\<close>{_./ _})\<close>)
 syntax_consts
-  "_Coll" == Collect
+  Collect
 translations
   "{x. P}" == "CONST Collect(\<lambda>x. P)"