src/CCL/Wfd.thy
changeset 47966 b8a94ed1646e
parent 47432 e1576d13e933
child 51798 ad3a241def73
--- a/src/CCL/Wfd.thy	Wed May 23 15:40:10 2012 +0200
+++ b/src/CCL/Wfd.thy	Wed May 23 15:57:12 2012 +0200
@@ -209,18 +209,18 @@
   apply (unfold Wfd_def)
   apply clarify
   apply (tactic {* wfd_strengthen_tac @{context} "%x. x:Nat" 1 *})
-   apply (fastsimp iff: NatPRXH)
+   apply (fastforce iff: NatPRXH)
   apply (erule Nat_ind)
-   apply (fastsimp iff: NatPRXH)+
+   apply (fastforce iff: NatPRXH)+
   done
 
 lemma ListPR_wf: "Wfd(ListPR(A))"
   apply (unfold Wfd_def)
   apply clarify
   apply (tactic {* wfd_strengthen_tac @{context} "%x. x:List (A)" 1 *})
-   apply (fastsimp iff: ListPRXH)
+   apply (fastforce iff: ListPRXH)
   apply (erule List_ind)
-   apply (fastsimp iff: ListPRXH)+
+   apply (fastforce iff: ListPRXH)+
   done