src/HOL/Library/Primes.thy
changeset 15140 322485b816ac
parent 15131 c69542757a4d
child 15628 9f912f8fd2df
--- a/src/HOL/Library/Primes.thy	Tue Aug 17 11:00:24 2004 +0200
+++ b/src/HOL/Library/Primes.thy	Wed Aug 18 11:09:40 2004 +0200
@@ -7,7 +7,7 @@
 header {* The Greatest Common Divisor and Euclid's algorithm *}
 
 theory Primes
-import Main
+imports Main
 begin
 
 text {*