add lemma power_eq_imp_eq_base
authorhuffman
Sun, 13 May 2007 19:15:36 +0200
changeset 22955 48dc37776d1e
parent 22954 372e3471fca2
child 22956 617140080e6a
add lemma power_eq_imp_eq_base
src/HOL/Power.thy
--- 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*}