src/HOL/Library/Permutation.thy
changeset 44890 22f665a2e91c
parent 40122 1d8ad2ff3e01
child 50037 f2a32197a33a
--- a/src/HOL/Library/Permutation.thy	Sun Sep 11 22:56:05 2011 +0200
+++ b/src/HOL/Library/Permutation.thy	Mon Sep 12 07:55:43 2011 +0200
@@ -153,7 +153,7 @@
 lemma perm_distinct_iff: "xs <~~> ys ==> distinct xs = distinct ys"
   apply (induct pred: perm)
      apply simp_all
-   apply fastsimp
+   apply fastforce
   apply (metis perm_set_eq)
   done
 
@@ -171,7 +171,7 @@
     apply (metis Cons Cons_eq_appendI distinct.simps(2)
       distinct_remdups distinct_remdups_id perm_append_swap perm_distinct_iff)
    apply (subgoal_tac "set (a#list) = set (ysa@a#zs) & distinct (a#list) & distinct (ysa@a#zs)")
-    apply (fastsimp simp add: insert_ident)
+    apply (fastforce simp add: insert_ident)
    apply (metis distinct_remdups set_remdups)
    apply (subgoal_tac "length (remdups xs) < Suc (length xs)")
    apply simp