diff -r 4159e1523ad8 -r 99ead7a7eb42 doc-src/TutorialI/Inductive/AB.thy --- a/doc-src/TutorialI/Inductive/AB.thy Wed Oct 19 17:21:53 2005 +0200 +++ b/doc-src/TutorialI/Inductive/AB.thy Wed Oct 19 21:52:07 2005 +0200 @@ -1,4 +1,4 @@ -(*<*)theory AB = Main:(*>*) +(*<*)theory AB imports Main begin(*>*) section{*Case Study: A Context Free Grammar*}