src/HOL/Finite_Set.thy
changeset 48128 bf172a5929bb
parent 48122 f479f36ed2ff
parent 48125 602dc0215954
child 48175 fea68365c975
--- a/src/HOL/Finite_Set.thy	Mon Jun 25 16:03:21 2012 +0200
+++ b/src/HOL/Finite_Set.thy	Mon Jun 25 18:21:18 2012 +0200
@@ -21,13 +21,13 @@
 use "Tools/set_comprehension_pointfree.ML"
 
 simproc_setup finite_Collect ("finite (Collect P)") =
-  {* Set_Comprehension_Pointfree.simproc *}
+  {* 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 = Set_Comprehension_Pointfree.code_simproc, identifier = []}])
+    proc = K Set_Comprehension_Pointfree.code_simproc, identifier = []}])
 *}
 
 lemma finite_induct [case_names empty insert, induct set: finite]:
@@ -872,7 +872,7 @@
     case (insert x F) then show ?case apply -
     apply (simp add: subset_insert_iff, clarify)
     apply (subgoal_tac "finite C")
-      prefer 2 apply (blast dest: finite_subset [COMP swap_prems_rl])
+      prefer 2 apply (blast dest: finite_subset [rotated])
     apply (subgoal_tac "C = insert x (C - {x})")
       prefer 2 apply blast
     apply (erule ssubst)
@@ -1524,7 +1524,7 @@
   apply - apply (erule finite_induct) apply simp
   apply (simp add: subset_insert_iff, clarify)
   apply (subgoal_tac "finite C")
-  prefer 2 apply (blast dest: finite_subset [COMP swap_prems_rl])
+  prefer 2 apply (blast dest: finite_subset [rotated])
   apply (subgoal_tac "C = insert x (C - {x})")
   prefer 2 apply blast
   apply (erule ssubst)