src/ZF/Finite.ML
changeset 2033 639de962ded4
parent 1956 589af052bcd4
child 2469 b50b8c0eec01
--- a/src/ZF/Finite.ML	Thu Sep 26 12:50:48 1996 +0200
+++ b/src/ZF/Finite.ML	Thu Sep 26 15:14:23 1996 +0200
@@ -73,7 +73,7 @@
 \       !!x y. [| x: A;  y: Fin(A);  x:y;  P(y) |] ==> P(y-{x}) \
 \    |] ==> c<=b --> P(b-c)";
 by (rtac (major RS Fin_induct) 1);
-by (rtac (Diff_cons RS ssubst) 2);
+by (stac Diff_cons 2);
 by (ALLGOALS (asm_simp_tac (Fin_ss addsimps (prems@[Diff_0, cons_subset_iff, 
                                 Diff_subset RS Fin_subset]))));
 qed "Fin_0_induct_lemma";