src/HOL/Decision_Procs/Commutative_Ring.thy
changeset 52658 1e7896c7f781
parent 48891 c0eafbd55de3
child 53077 a1b3784f8129
--- a/src/HOL/Decision_Procs/Commutative_Ring.thy	Mon Jul 15 10:42:12 2013 +0200
+++ b/src/HOL/Decision_Procs/Commutative_Ring.thy	Mon Jul 15 11:29:19 2013 +0200
@@ -271,7 +271,7 @@
       with 1 have "\<And>P. Ipol ls (pow l P) = Ipol ls P ^ l" by simp
       moreover
       note Suc `even l` even_nat_plus_one_div_two
-      ultimately show ?thesis by (auto simp add: mul_ci power_Suc even_pow)
+      ultimately show ?thesis by (auto simp add: mul_ci even_pow)
     next
       assume "odd l"
       {
@@ -286,7 +286,7 @@
           have two_times: "2 * (w div 2) = w"
             by (simp only: numerals even_nat_div_two_times_two [OF `even w`])
           have "Ipol ls P * Ipol ls P = Ipol ls P ^ Suc (Suc 0)"
-            by (simp add: power_Suc)
+            by simp
           then have "Ipol ls P * Ipol ls P = Ipol ls P ^ 2"
             by (simp add: numerals)
           with Suc show ?thesis