changeset 346 | 0fea8b7a14a1 |
parent 295 | 24c68350d059 |
child 489 | 1343540ed715 |
--- a/ProgTutorial/Package/Ind_Intro.thy Mon Oct 12 17:07:17 2009 +0200 +++ b/ProgTutorial/Package/Ind_Intro.thy Tue Oct 13 22:57:25 2009 +0200 @@ -1,7 +1,15 @@ theory Ind_Intro -imports Main +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} *} text {*