18537
|
1 |
|
|
2 |
(* $Id$ *)
|
|
3 |
|
|
4 |
theory "proof" imports base begin
|
|
5 |
|
|
6 |
chapter {* Structured reasoning *}
|
|
7 |
|
|
8 |
section {* Proof context *}
|
|
9 |
|
20026
|
10 |
subsection {* Local variables *}
|
|
11 |
|
|
12 |
text %mlref {*
|
|
13 |
\begin{mldecls}
|
|
14 |
@{index_ML Variable.declare_term: "term -> Proof.context -> Proof.context"} \\
|
|
15 |
@{index_ML Variable.import: "bool -> thm list -> Proof.context -> thm list * Proof.context"} \\
|
|
16 |
@{index_ML Variable.export: "Proof.context -> Proof.context -> thm list -> thm list"} \\
|
|
17 |
@{index_ML Variable.trade: "Proof.context -> (thm list -> thm list) -> thm list -> thm list"} \\
|
|
18 |
@{index_ML Variable.monomorphic: "Proof.context -> term list -> term list"} \\
|
|
19 |
@{index_ML Variable.polymorphic: "Proof.context -> term list -> term list"} \\
|
|
20 |
\end{mldecls}
|
|
21 |
|
|
22 |
\begin{description}
|
|
23 |
|
|
24 |
\item @{ML Variable.declare_term} FIXME
|
|
25 |
|
|
26 |
\item @{ML Variable.import} FIXME
|
|
27 |
|
|
28 |
\item @{ML Variable.export} FIXME
|
|
29 |
|
|
30 |
\item @{ML Variable.trade} composes @{ML Variable.import} and @{ML
|
|
31 |
Variable.export}.
|
|
32 |
|
|
33 |
\item @{ML Variable.monomorphic} FIXME
|
|
34 |
|
|
35 |
\item @{ML Variable.polymorphic} FIXME
|
|
36 |
|
|
37 |
\end{description}
|
|
38 |
*}
|
|
39 |
|
18537
|
40 |
text FIXME
|
|
41 |
|
|
42 |
section {* Proof state *}
|
|
43 |
|
|
44 |
text {*
|
|
45 |
FIXME
|
|
46 |
|
|
47 |
\glossary{Proof state}{The whole configuration of a structured proof,
|
|
48 |
consisting of a \seeglossary{proof context} and an optional
|
|
49 |
\seeglossary{structured goal}. Internally, an Isar proof state is
|
|
50 |
organized as a stack to accomodate block structure of proof texts.
|
|
51 |
For historical reasons, a low-level \seeglossary{tactical goal} is
|
|
52 |
occasionally called ``proof state'' as well.}
|
|
53 |
|
|
54 |
\glossary{Structured goal}{FIXME}
|
|
55 |
|
|
56 |
\glossary{Goal}{See \seeglossary{tactical goal} or \seeglossary{structured goal}. \norefpage}
|
|
57 |
|
|
58 |
|
|
59 |
*}
|
|
60 |
|
|
61 |
section {* Methods *}
|
|
62 |
|
|
63 |
text FIXME
|
|
64 |
|
|
65 |
section {* Attributes *}
|
|
66 |
|
|
67 |
text FIXME
|
|
68 |
|
|
69 |
end
|