--- a/src/HOL/WF.ML Wed May 22 18:32:37 1996 +0200
+++ b/src/HOL/WF.ML Thu May 23 14:37:06 1996 +0200
@@ -27,7 +27,7 @@
\ !!x.[| ! y. (y,x): r --> P(y) |] ==> P(x) \
\ |] ==> P(a)";
by (rtac (major RS spec RS mp RS spec) 1);
-by (fast_tac (HOL_cs addEs prems) 1);
+by (fast_tac (!claset addEs prems) 1);
qed "wf_induct";
(*Perform induction on i, then prove the wf(r) subgoal using prems. *)
@@ -38,9 +38,9 @@
val prems = goal WF.thy "[| wf(r); (a,x):r; (x,a):r |] ==> P";
by (subgoal_tac "! x. (a,x):r --> (x,a):r --> P" 1);
-by (fast_tac (HOL_cs addIs prems) 1);
+by (fast_tac (!claset addIs prems) 1);
by (wf_ind_tac "a" prems 1);
-by (fast_tac set_cs 1);
+by (Fast_tac 1);
qed "wf_asym";
val prems = goal WF.thy "[| wf(r); (a,a): r |] ==> P";
@@ -58,8 +58,8 @@
by (res_inst_tac [("a","x")] (prem RS wf_induct) 1);
by (rtac (impI RS allI) 1);
by (etac tranclE 1);
-by (fast_tac HOL_cs 1);
-by (fast_tac HOL_cs 1);
+by (Fast_tac 1);
+by (Fast_tac 1);
qed "wf_trancl";