got rid of deepen_tac
authorpaulson
Fri, 20 Sep 2002 11:49:06 +0200
changeset 13572 1681c5b58766
parent 13571 d76a798281f4
child 13573 37b22343c35a
got rid of deepen_tac
src/HOL/GroupTheory/Sylow.ML
--- a/src/HOL/GroupTheory/Sylow.ML	Fri Sep 20 11:48:35 2002 +0200
+++ b/src/HOL/GroupTheory/Sylow.ML	Fri Sep 20 11:49:06 2002 +0200
@@ -267,9 +267,9 @@
 
 Goal "(%C:{*H*}. M1 #> (@g. g \\<in> (G .<cr>) \\<and> H #> g = C)) \\<in> {* H *} \\<rightarrow> M";
 by (simp_tac (simpset() addsimps [setrcos_eq]) 1);
-by (deepen_tac (claset() addIs [someI2] 
+by (fast_tac (claset() addIs [someI2] 
             addSIs [restrictI, RelM_equiv, M_in_quot,
-                    M1_RelM_rcosetGM1g RSN (4, EquivElemClass),M1_in_M]) 0 1); 
+                    [RelM_equiv,M_in_quot,asm_rl,M1_RelM_rcosetGM1g] MRS EquivElemClass, M1_in_M]) 1);
 qed "setrcos_H_funcset_M";
 
 Goal "\\<exists>g \\<in> {* H *}\\<rightarrow>M. inj_on g ({* H *})";