diff -r aa8474398030 -r ad4d5365d9d8 src/HOL/Power.thy --- a/src/HOL/Power.thy Tue Oct 23 22:48:25 2007 +0200 +++ b/src/HOL/Power.thy Tue Oct 23 23:27:23 2007 +0200 @@ -140,7 +140,7 @@ done lemma power_eq_0_iff [simp]: - "(a^n = 0) = (a = (0::'a::{ring_1_no_zero_divisors,recpower}) & n\0)" + "(a^n = 0) = (a = (0::'a::{ring_1_no_zero_divisors,recpower}) & n>0)" apply (induct "n") apply (auto simp add: power_Suc zero_neq_one [THEN not_sym]) done @@ -342,7 +342,7 @@ lemma nat_one_le_power [simp]: "1 \ i ==> Suc 0 \ i^n" by (insert one_le_power [of i n], simp) -lemma nat_zero_less_power_iff [simp]: "(x^n = 0) = (x = (0::nat) & n\0)" +lemma nat_zero_less_power_iff [simp]: "(x^n > 0) = (x > (0::nat) | n=0)" by (induct "n", auto) text{*Valid for the naturals, but what if @{text"0