src/HOL/Library/Primes.thy
changeset 15131 c69542757a4d
parent 14706 71590b7733b7
child 15140 322485b816ac
--- 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}.