src/HOL/Finite_Set.thy
changeset 49764 9979d64b8016
parent 49758 718f10c8bbfc
child 49806 acb6fa98e310
--- a/src/HOL/Finite_Set.thy	Wed Oct 10 10:47:21 2012 +0200
+++ b/src/HOL/Finite_Set.thy	Wed Oct 10 10:47:43 2012 +0200
@@ -16,18 +16,7 @@
     emptyI [simp, intro!]: "finite {}"
   | insertI [simp, intro!]: "finite A \<Longrightarrow> finite (insert a A)"
 
-(* FIXME: move to Set theory *)
-ML_file "Tools/set_comprehension_pointfree.ML"
-
-simproc_setup finite_Collect ("finite (Collect P)") =
-  {* K Set_Comprehension_Pointfree.simproc *}
-
-(* FIXME: move to Set theory*)
-setup {*
-  Code_Preproc.map_pre (fn ss => ss addsimprocs
-    [Raw_Simplifier.make_simproc {name = "set comprehension", lhss = [@{cpat "Collect ?P"}],
-    proc = K Set_Comprehension_Pointfree.code_simproc, identifier = []}])
-*}
+simproc_setup finite_Collect ("finite (Collect P)") = {* K Set_Comprehension_Pointfree.simproc *}
 
 lemma finite_induct [case_names empty insert, induct set: finite]:
   -- {* Discharging @{text "x \<notin> F"} entails extra work. *}