src/HOL/Induct/Comb.thy
changeset 16563 a92f96951355
parent 16417 9bc16273c2d4
child 16588 8de758143786
--- a/src/HOL/Induct/Comb.thy	Fri Jun 24 16:21:01 2005 +0200
+++ b/src/HOL/Induct/Comb.thy	Fri Jun 24 17:25:10 2005 +0200
@@ -95,9 +95,9 @@
     "[| diamond(r);  (x,y) \<in> r^* |] ==>   
           \<forall>y'. (x,y') \<in> r --> (\<exists>z. (y',z) \<in> r^* & (y,z) \<in> r)"
 apply (unfold diamond_def)
-apply (erule rtrancl_induct, blast, clarify)
-apply (drule spec, drule mp, assumption)
-apply (blast intro: rtrancl_trans [OF _ r_into_rtrancl])
+apply (erule rtrancl_induct)
+apply (meson rtrancl_refl)
+apply (meson rtrancl_trans r_into_rtrancl)
 done
 
 lemma diamond_rtrancl: "diamond(r) ==> diamond(r^*)"
@@ -210,7 +210,7 @@
 lemma parcontract_subset_reduce: "parcontract <= contract^*"
 apply (rule subsetI)
 apply (simp only: split_tupled_all)
-apply (erule parcontract.induct , blast+)
+apply (erule parcontract.induct, blast+)
 done
 
 lemma reduce_eq_parreduce: "contract^* = parcontract^*"