src/HOL/Product_Type.thy
changeset 78799 807b249f1061
parent 78794 c74fd21af246
child 78801 42ae6e0ecfd4
--- a/src/HOL/Product_Type.thy	Thu Oct 19 11:30:16 2023 +0200
+++ b/src/HOL/Product_Type.thy	Thu Oct 19 16:31:17 2023 +0200
@@ -1303,9 +1303,8 @@
 
 ML_file \<open>Tools/set_comprehension_pointfree.ML\<close>
 
-simproc_setup set_comprehension ("Collect P") =
+simproc_setup passive set_comprehension ("Collect P") =
   \<open>K Set_Comprehension_Pointfree.code_simproc\<close>
-  (passive)
 
 setup \<open>Code_Preproc.map_pre (fn ctxt => ctxt addsimprocs [\<^simproc>\<open>set_comprehension\<close>])\<close>