src/HOL/Transitive_Closure.thy
changeset 31970 ccaadfcf6941
parent 31690 cc37bf07f9bb
child 32215 87806301a813
--- a/src/HOL/Transitive_Closure.thy	Thu Jul 09 17:33:22 2009 +0200
+++ b/src/HOL/Transitive_Closure.thy	Thu Jul 09 17:34:59 2009 +0200
@@ -737,6 +737,9 @@
 lemma rel_pow_add: "R ^^ (m+n) = R^^n O R^^m"
 by(induct n) auto
 
+lemma rel_pow_commute: "R O R ^^ n = R ^^ n O R"
+  by (induct n) (simp, simp add: O_assoc [symmetric])
+
 lemma rtrancl_imp_UN_rel_pow:
   assumes "p \<in> R^*"
   shows "p \<in> (\<Union>n. R ^^ n)"