src/HOL/Power.thy
changeset 35828 46cfc4b8112e
parent 35216 7641e8d831d2
child 36349 39be26d1bc28
--- a/src/HOL/Power.thy	Wed Mar 17 19:37:44 2010 +0100
+++ b/src/HOL/Power.thy	Thu Mar 18 12:58:52 2010 +0100
@@ -334,7 +334,7 @@
   "abs ((-a) ^ n) = abs (a ^ n)"
   by (simp add: power_abs)
 
-lemma zero_less_power_abs_iff [simp, noatp]:
+lemma zero_less_power_abs_iff [simp, no_atp]:
   "0 < abs a ^ n \<longleftrightarrow> a \<noteq> 0 \<or> n = 0"
 proof (induct n)
   case 0 show ?case by simp