equal
deleted
inserted
replaced
13 is transformed by a sequence of transitions (commands) within a theory body. |
13 is transformed by a sequence of transitions (commands) within a theory body. |
14 This is a pure value with pure functions acting on it in a timeless and |
14 This is a pure value with pure functions acting on it in a timeless and |
15 stateless manner. Historically, the sequence of transitions was wrapped up |
15 stateless manner. Historically, the sequence of transitions was wrapped up |
16 as sequential command loop, such that commands are applied one-by-one. In |
16 as sequential command loop, such that commands are applied one-by-one. In |
17 contemporary Isabelle/Isar, processing toplevel commands usually works in |
17 contemporary Isabelle/Isar, processing toplevel commands usually works in |
18 parallel in multi-threaded Isabelle/ML \cite{Wenzel:2009,Wenzel:2013:ITP}. |
18 parallel in multi-threaded Isabelle/ML @{cite "Wenzel:2009" and |
|
19 "Wenzel:2013:ITP"}. |
19 *} |
20 *} |
20 |
21 |
21 |
22 |
22 subsection {* Toplevel state *} |
23 subsection {* Toplevel state *} |
23 |
24 |
180 theories simultaneously. Thus it acts like processing the import header of a |
181 theories simultaneously. Thus it acts like processing the import header of a |
181 theory, without performing the merge of the result. By loading a whole |
182 theory, without performing the merge of the result. By loading a whole |
182 sub-graph of theories, the intrinsic parallelism can be exploited by the |
183 sub-graph of theories, the intrinsic parallelism can be exploited by the |
183 system to speedup loading. |
184 system to speedup loading. |
184 |
185 |
185 This variant is used by default in @{tool build} \cite{isabelle-sys}. |
186 This variant is used by default in @{tool build} @{cite "isabelle-sys"}. |
186 |
187 |
187 \item @{ML Thy_Info.get_theory}~@{text A} retrieves the theory value |
188 \item @{ML Thy_Info.get_theory}~@{text A} retrieves the theory value |
188 presently associated with name @{text A}. Note that the result might be |
189 presently associated with name @{text A}. Note that the result might be |
189 outdated wrt.\ the file-system content. |
190 outdated wrt.\ the file-system content. |
190 |
191 |