src/HOL/Integ/Parity.thy
changeset 14443 75910c7557c5
parent 14436 77017c49c004
child 14450 3d2529f48b07
--- a/src/HOL/Integ/Parity.thy	Mon Mar 08 11:11:58 2004 +0100
+++ b/src/HOL/Integ/Parity.thy	Mon Mar 08 11:12:06 2004 +0100
@@ -249,6 +249,11 @@
      "odd x ==> (-1::'a::{number_ring,ringpower})^x = -1"
   by (rule neg_one_even_odd_power [THEN conjunct2, THEN mp], assumption)
 
+lemma neg_power_if:
+     "(-x::'a::{ring,ringpower}) ^ n = 
+      (if even n then (x ^ n) else -(x ^ n))"
+  by (induct n, simp_all split: split_if_asm add: power_Suc) 
+
 
 subsection {* Miscellaneous *}