src/HOL/Power.thy
changeset 55718 34618f031ba9
parent 55096 916b2ac758f4
child 55811 aa1acc25126b
--- a/src/HOL/Power.thy	Mon Feb 24 13:52:48 2014 +0100
+++ b/src/HOL/Power.thy	Mon Feb 24 15:45:55 2014 +0000
@@ -610,6 +610,11 @@
 
 subsection {* Miscellaneous rules *}
 
+lemma self_le_power:
+  fixes x::"'a::linordered_semidom" 
+  shows "1 \<le> x \<Longrightarrow> 0 < n \<Longrightarrow> x \<le> x ^ n"
+  by (metis gr_implies_not0 le_eq_less_or_eq less_one nat_le_linear power_increasing power_one_right)
+
 lemma power_eq_if: "p ^ m = (if m=0 then 1 else p * (p ^ (m - 1)))"
   unfolding One_nat_def by (cases m) simp_all