src/HOL/Power.thy
changeset 22955 48dc37776d1e
parent 22853 7f000a385606
child 22957 82a799ae7579
--- a/src/HOL/Power.thy	Sun May 13 18:16:49 2007 +0200
+++ b/src/HOL/Power.thy	Sun May 13 19:15:36 2007 +0200
@@ -319,6 +319,11 @@
       ==> a = (b::'a::{ordered_semidom,recpower})"
 by (blast intro: power_le_imp_le_base order_antisym order_eq_refl sym)
 
+lemma power_eq_imp_eq_base:
+  fixes a b :: "'a::{ordered_semidom,recpower}"
+  shows "\<lbrakk>a ^ n = b ^ n; 0 \<le> a; 0 \<le> b; 0 < n\<rbrakk> \<Longrightarrow> a = b"
+by (cases n, simp_all, rule power_inject_base)
+
 
 subsection{*Exponentiation for the Natural Numbers*}