--- a/doc-src/TutorialI/Misc/Option2.thy Fri Jun 17 11:35:35 2005 +0200
+++ b/doc-src/TutorialI/Misc/Option2.thy Fri Jun 17 16:12:49 2005 +0200
@@ -1,5 +1,5 @@
(*<*)
-theory Option2 = Main:
+theory Option2 imports Main begin
hide const None Some
hide type option
(*>*)