src/HOL/IMP/Machines.thy
changeset 32235 8f9b8d14fc9f
parent 31970 ccaadfcf6941
child 42174 d0be2722ce9f
--- a/src/HOL/IMP/Machines.thy	Mon Jul 27 17:36:30 2009 +0200
+++ b/src/HOL/IMP/Machines.thy	Mon Jul 27 21:47:41 2009 +0200
@@ -6,7 +6,7 @@
   "((x,z) \<in> R ^^ n) = (n=0 \<and> z=x \<or> (\<exists>m y. n = Suc m \<and> (x,y) \<in> R \<and> (y,z) \<in> R ^^ m))"
 apply(rule iffI)
  apply(blast elim:rel_pow_E2)
-apply (fastsimp simp add:gr0_conv_Suc rel_pow_commute)
+apply (auto simp: rel_pow_commute[symmetric])
 done
 
 subsection "Instructions"