shortened a proof
authorpaulson
Fri, 20 Sep 2002 11:49:38 +0200
changeset 13573 37b22343c35a
parent 13572 1681c5b58766
child 13574 f9796358e66f
shortened a proof
src/ZF/Induct/Comb.thy
--- a/src/ZF/Induct/Comb.thy	Fri Sep 20 11:49:06 2002 +0200
+++ b/src/ZF/Induct/Comb.thy	Fri Sep 20 11:49:38 2002 +0200
@@ -177,8 +177,8 @@
   apply (drule field_contract_eq [THEN equalityD1, THEN subsetD])
   apply (erule rtrancl_induct)
    apply (blast intro: reduction_rls)
-  apply (erule trans_rtrancl [THEN transD])
-  apply (blast intro: contract_combD2 reduction_rls)
+  apply (blast intro: trans_rtrancl [THEN transD] 
+                      contract_combD2 reduction_rls)
   done
 
 text {* Counterexample to the diamond property for @{text "-1->"}. *}