src/HOL/Transitive_Closure.thy
changeset 61424 c3658c18b7bc
parent 61378 3e04c9ca001a
child 61681 ca53150406c9
--- a/src/HOL/Transitive_Closure.thy	Tue Oct 13 09:21:14 2015 +0200
+++ b/src/HOL/Transitive_Closure.thy	Tue Oct 13 09:21:15 2015 +0200
@@ -898,7 +898,7 @@
 lemma rtranclp_imp_Sup_relpowp:
   assumes "(P^**) x y"
   shows "(\<Squnion>n. P ^^ n) x y"
-  using assms and rtrancl_imp_UN_relpow [to_pred] by blast
+  using assms and rtrancl_imp_UN_relpow [of "(x, y)", to_pred] by simp
 
 lemma relpow_imp_rtrancl:
   assumes "p \<in> R ^^ n"
@@ -918,7 +918,7 @@
 lemma relpowp_imp_rtranclp:
   assumes "(P ^^ n) x y"
   shows "(P^**) x y"
-  using assms and relpow_imp_rtrancl [to_pred] by blast
+  using assms and relpow_imp_rtrancl [of "(x, y)", to_pred] by simp
 
 lemma rtrancl_is_UN_relpow:
   "R^* = (\<Union>n. R ^^ n)"