equal
deleted
inserted
replaced
57 @{index_ML_type Toplevel.state} \\ |
57 @{index_ML_type Toplevel.state} \\ |
58 @{index_ML Toplevel.UNDEF: "exn"} \\ |
58 @{index_ML Toplevel.UNDEF: "exn"} \\ |
59 @{index_ML Toplevel.is_toplevel: "Toplevel.state -> bool"} \\ |
59 @{index_ML Toplevel.is_toplevel: "Toplevel.state -> bool"} \\ |
60 @{index_ML Toplevel.theory_of: "Toplevel.state -> theory"} \\ |
60 @{index_ML Toplevel.theory_of: "Toplevel.state -> theory"} \\ |
61 @{index_ML Toplevel.proof_of: "Toplevel.state -> Proof.state"} \\ |
61 @{index_ML Toplevel.proof_of: "Toplevel.state -> Proof.state"} \\ |
62 @{index_ML Toplevel.debug: "bool ref"} \\ |
62 @{index_ML Toplevel.debug: "bool Unsynchronized.ref"} \\ |
63 @{index_ML Toplevel.timing: "bool ref"} \\ |
63 @{index_ML Toplevel.timing: "bool Unsynchronized.ref"} \\ |
64 @{index_ML Toplevel.profiling: "int ref"} \\ |
64 @{index_ML Toplevel.profiling: "int Unsynchronized.ref"} \\ |
65 \end{mldecls} |
65 \end{mldecls} |
66 |
66 |
67 \begin{description} |
67 \begin{description} |
68 |
68 |
69 \item @{ML_type Toplevel.state} represents Isar toplevel states, |
69 \item @{ML_type Toplevel.state} represents Isar toplevel states, |
83 a theory or proof (!), otherwise raises @{ML Toplevel.UNDEF}. |
83 a theory or proof (!), otherwise raises @{ML Toplevel.UNDEF}. |
84 |
84 |
85 \item @{ML Toplevel.proof_of}~@{text "state"} selects the Isar proof |
85 \item @{ML Toplevel.proof_of}~@{text "state"} selects the Isar proof |
86 state if available, otherwise raises @{ML Toplevel.UNDEF}. |
86 state if available, otherwise raises @{ML Toplevel.UNDEF}. |
87 |
87 |
88 \item @{ML "set Toplevel.debug"} makes the toplevel print further |
88 \item @{ML "Toplevel.debug := true"} makes the toplevel print further |
89 details about internal error conditions, exceptions being raised |
89 details about internal error conditions, exceptions being raised |
90 etc. |
90 etc. |
91 |
91 |
92 \item @{ML "set Toplevel.timing"} makes the toplevel print timing |
92 \item @{ML "Toplevel.timing := true"} makes the toplevel print timing |
93 information for each Isar command being executed. |
93 information for each Isar command being executed. |
94 |
94 |
95 \item @{ML Toplevel.profiling}~@{verbatim ":="}~@{text "n"} controls |
95 \item @{ML Toplevel.profiling}~@{verbatim ":="}~@{text "n"} controls |
96 low-level profiling of the underlying {\ML} runtime system. For |
96 low-level profiling of the underlying {\ML} runtime system. For |
97 Poly/ML, @{text "n = 1"} means time and @{text "n = 2"} space |
97 Poly/ML, @{text "n = 1"} means time and @{text "n = 2"} space |