doc-src/TutorialI/Misc/prime_def.thy
changeset 16417 9bc16273c2d4
parent 11457 279da0358aa9
--- a/doc-src/TutorialI/Misc/prime_def.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/doc-src/TutorialI/Misc/prime_def.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -1,5 +1,5 @@
 (*<*)
-theory prime_def = Main:;
+theory prime_def imports Main begin;
 consts prime :: "nat \<Rightarrow> bool"
 (*>*)
 text{*