diff -r beee83623cc9 -r 293b896b9c25 src/HOL/Relation_Power.thy --- a/src/HOL/Relation_Power.thy Mon Feb 23 13:55:36 2009 -0800 +++ b/src/HOL/Relation_Power.thy Mon Feb 23 16:25:52 2009 -0800 @@ -61,16 +61,16 @@ lemma funpow_swap1: "f((f^n) x) = (f^n)(f x)" proof - - have "f((f^n) x) = (f^(n+1)) x" by simp + have "f((f^n) x) = (f^(n+1)) x" unfolding One_nat_def by simp also have "\ = (f^n o f^1) x" by (simp only: funpow_add) - also have "\ = (f^n)(f x)" by simp + also have "\ = (f^n)(f x)" unfolding One_nat_def by simp finally show ?thesis . qed lemma rel_pow_1 [simp]: fixes R :: "('a*'a)set" shows "R^1 = R" - by simp + unfolding One_nat_def by simp lemma rel_pow_0_I: "(x,x) : R^0" by simp