src/HOL/Product_Type.thy
changeset 78801 42ae6e0ecfd4
parent 78799 807b249f1061
child 79492 c1b0f64eb865
--- a/src/HOL/Product_Type.thy	Thu Oct 19 17:06:39 2023 +0200
+++ b/src/HOL/Product_Type.thy	Thu Oct 19 21:38:09 2023 +0200
@@ -1304,7 +1304,7 @@
 ML_file \<open>Tools/set_comprehension_pointfree.ML\<close>
 
 simproc_setup passive set_comprehension ("Collect P") =
-  \<open>K Set_Comprehension_Pointfree.code_simproc\<close>
+  \<open>K Set_Comprehension_Pointfree.code_proc\<close>
 
 setup \<open>Code_Preproc.map_pre (fn ctxt => ctxt addsimprocs [\<^simproc>\<open>set_comprehension\<close>])\<close>