doc-src/TutorialI/Rules/Primes.thy
changeset 16417 9bc16273c2d4
parent 11234 6902638af59e
child 22097 7ee0529c5674
--- a/doc-src/TutorialI/Rules/Primes.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/doc-src/TutorialI/Rules/Primes.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -3,7 +3,7 @@
 
 (*Euclid's algorithm 
   This material now appears AFTER that of Forward.thy *)
-theory Primes = Main:
+theory Primes imports Main begin
 consts
   gcd     :: "nat*nat \<Rightarrow> nat"