src/HOL/NumberTheory/Int2.thy
changeset 20217 25b068a99d2b
parent 19670 2e4a143c73c5
child 21404 eb85850d3eb7
--- a/src/HOL/NumberTheory/Int2.thy	Wed Jul 26 13:31:07 2006 +0200
+++ b/src/HOL/NumberTheory/Int2.thy	Wed Jul 26 19:23:04 2006 +0200
@@ -191,7 +191,7 @@
   have "x * x ^ nat (p - 2) = x ^ (nat (p - 2) + 1)"
     by auto
   also from prems have "nat (p - 2) + 1 = nat (p - 2 + 1)"
-    by (simp only: nat_add_distrib, auto)
+    by (simp only: nat_add_distrib)
   also have "p - 2 + 1 = p - 1" by arith
   finally have "[x * x ^ nat (p - 2) = x ^ nat (p - 1)] (mod p)"
     by (rule ssubst, auto)