doc-src/TutorialI/Recdef/Induction.thy
changeset 16417 9bc16273c2d4
parent 11458 09a6c44a48ea
--- a/doc-src/TutorialI/Recdef/Induction.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/doc-src/TutorialI/Recdef/Induction.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -1,5 +1,5 @@
 (*<*)
-theory Induction = examples + simplification:;
+theory Induction imports examples simplification begin;
 (*>*)
 
 text{*