--- a/src/HOL/Library/Primes.thy Mon Aug 16 14:21:54 2004 +0200
+++ b/src/HOL/Library/Primes.thy Mon Aug 16 14:22:27 2004 +0200
@@ -6,7 +6,9 @@
header {* The Greatest Common Divisor and Euclid's algorithm *}
-theory Primes = Main:
+theory Primes
+import Main
+begin
text {*
See \cite{davenport92}.