src/HOL/Transitive_Closure.thy
changeset 13867 1fdecd15437f
parent 13726 9550a6f4ed4a
child 14208 144f45277d5a
--- a/src/HOL/Transitive_Closure.thy	Mon Mar 17 17:37:48 2003 +0100
+++ b/src/HOL/Transitive_Closure.thy	Mon Mar 17 18:38:50 2003 +0100
@@ -341,13 +341,8 @@
   apply (blast intro: rtrancl_trans)
   done
 
-lemma irrefl_tranclI: "r^-1 \<inter> r^+ = {} ==> (x, x) \<notin> r^+"
-  apply (subgoal_tac "ALL y. (x, y) : r^+ --> x \<noteq> y")
-   apply fast
-  apply (intro strip)
-  apply (erule trancl_induct)
-   apply (auto intro: r_into_trancl)
-  done
+lemma irrefl_tranclI: "r^-1 \<inter> r^* = {} ==> (x, x) \<notin> r^+"
+by(blast elim: tranclE dest: trancl_into_rtrancl)
 
 lemma irrefl_trancl_rD: "!!X. ALL x. (x, x) \<notin> r^+ ==> (x, y) \<in> r ==> x \<noteq> y"
   by (blast dest: r_into_trancl)