src/HOL/Power.thy
changeset 17149 e2b19c92ef51
parent 16796 140f1e0ea846
child 21199 2d83f93c3580
--- a/src/HOL/Power.thy	Fri Aug 26 08:42:52 2005 +0200
+++ b/src/HOL/Power.thy	Fri Aug 26 10:01:06 2005 +0200
@@ -351,6 +351,13 @@
 apply (erule dvd_imp_le, simp)
 done
 
+lemma power_diff:
+  assumes nz: "a ~= 0"
+  shows "n <= m ==> (a::'a::{recpower, field}) ^ (m-n) = (a^m) / (a^n)"
+  by (induct m n rule: diff_induct)
+    (simp_all add: power_Suc nonzero_mult_divide_cancel_left nz)
+
+
 text{*ML bindings for the general exponentiation theorems*}
 ML
 {*