src/HOL/Power.thy
changeset 58410 6d46ad54a2ab
parent 58157 c376c43c346c
child 58437 8d124c73c37a
--- a/src/HOL/Power.thy	Sun Sep 21 16:56:06 2014 +0200
+++ b/src/HOL/Power.thy	Sun Sep 21 16:56:11 2014 +0200
@@ -214,7 +214,7 @@
   by (rule power_minus_Bit0)
 
 lemma power_minus1_even [simp]:
-  "-1 ^ (2*n) = 1"
+  "(- 1) ^ (2*n) = 1"
 proof (induct n)
   case 0 show ?case by simp
 next
@@ -222,7 +222,7 @@
 qed
 
 lemma power_minus1_odd:
-  "-1 ^ Suc (2*n) = -1"
+  "(- 1) ^ Suc (2*n) = -1"
   by simp
 
 lemma power_minus_even [simp]: