doc-src/TutorialI/Inductive/Mutual.thy
changeset 17914 99ead7a7eb42
parent 12815 1f073030b97a
child 19389 0d57259fea82
--- a/doc-src/TutorialI/Inductive/Mutual.thy	Wed Oct 19 17:21:53 2005 +0200
+++ b/doc-src/TutorialI/Inductive/Mutual.thy	Wed Oct 19 21:52:07 2005 +0200
@@ -1,4 +1,4 @@
-(*<*)theory Mutual = Main:(*>*)
+(*<*)theory Mutual imports Main begin(*>*)
 
 subsection{*Mutually Inductive Definitions*}