diff -r fb6c29a90003 -r d8c376662bb4 ProgTutorial/Package/Ind_Intro.thy --- a/ProgTutorial/Package/Ind_Intro.thy Mon Apr 30 12:36:32 2012 +0100 +++ b/ProgTutorial/Package/Ind_Intro.thy Mon Apr 30 14:43:52 2012 +0100 @@ -2,13 +2,6 @@ imports "../Base" begin -(*<*) -setup{* -open_file_with_prelude - "Ind_Package_Code.thy" - ["theory Ind_Package", "imports Main", "begin"] -*} -(*>*) chapter {* How to Write a Definitional Package\label{chp:package} *}