src/HOL/Nat_Numeral.thy
changeset 31002 bc4117fe72ab
parent 30960 fec1a04b7220
child 31014 79f0858d9d49
--- a/src/HOL/Nat_Numeral.thy	Mon Apr 27 10:11:44 2009 +0200
+++ b/src/HOL/Nat_Numeral.thy	Mon Apr 27 10:11:46 2009 +0200
@@ -396,10 +396,10 @@
   by (simp add: power_Suc) 
 
 lemma power_even_eq: "(a::'a::recpower) ^ (2*n) = (a^n)^2"
-by (subst mult_commute) (simp add: power_mult)
+  by (subst mult_commute) (simp add: power_mult)
 
 lemma power_odd_eq: "(a::int) ^ Suc(2*n) = a * (a^n)^2"
-by (simp add: power_even_eq) 
+  by (simp add: power_even_eq)
 
 lemma power_minus_even [simp]:
   "(-a) ^ (2*n) = (a::'a::{comm_ring_1,recpower}) ^ (2*n)"