changeset 517 | d8c376662bb4 |
parent 489 | 1343540ed715 |
child 565 | cecd7a941885 |
516:fb6c29a90003 | 517:d8c376662bb4 |
---|---|
1 theory Ind_Intro |
1 theory Ind_Intro |
2 imports "../Base" |
2 imports "../Base" |
3 begin |
3 begin |
4 |
4 |
5 (*<*) |
|
6 setup{* |
|
7 open_file_with_prelude |
|
8 "Ind_Package_Code.thy" |
|
9 ["theory Ind_Package", "imports Main", "begin"] |
|
10 *} |
|
11 (*>*) |
|
12 |
5 |
13 chapter {* How to Write a Definitional Package\label{chp:package} *} |
6 chapter {* How to Write a Definitional Package\label{chp:package} *} |
14 |
7 |
15 text {* |
8 text {* |
16 \begin{flushright} |
9 \begin{flushright} |