src/HOL/Library/Primes.thy
changeset 13187 e5434b822a96
parent 13032 1ec445c51931
child 14353 79f9fbef9106
--- a/src/HOL/Library/Primes.thy	Thu May 30 10:12:11 2002 +0200
+++ b/src/HOL/Library/Primes.thy	Thu May 30 10:12:52 2002 +0200
@@ -185,7 +185,6 @@
   apply (auto simp add: prime_def)
   apply (case_tac m)
    apply (auto dest!: dvd_imp_le)
-  apply arith
   done
 
 text {*