src/Doc/Implementation/Integration.thy
changeset 62847 1bd1d8492931
parent 61854 38b049cd3aad
child 62947 3374f3ffb2ec
equal deleted inserted replaced
62846:3c576c7f9731 62847:1bd1d8492931
   150 \<close>
   150 \<close>
   151 
   151 
   152 text %mlref \<open>
   152 text %mlref \<open>
   153   \begin{mldecls}
   153   \begin{mldecls}
   154   @{index_ML use_thy: "string -> unit"} \\
   154   @{index_ML use_thy: "string -> unit"} \\
   155   @{index_ML use_thys: "string list -> unit"} \\[0.5ex]
       
   156   @{index_ML Thy_Info.get_theory: "string -> theory"} \\
   155   @{index_ML Thy_Info.get_theory: "string -> theory"} \\
   157   @{index_ML Thy_Info.remove_thy: "string -> unit"} \\
   156   @{index_ML Thy_Info.remove_thy: "string -> unit"} \\
   158   @{index_ML Thy_Info.register_thy: "theory -> unit"} \\
   157   @{index_ML Thy_Info.register_thy: "theory -> unit"} \\
   159   \end{mldecls}
   158   \end{mldecls}
   160 
   159 
   161   \<^descr> @{ML use_thy}~\<open>A\<close> ensures that theory \<open>A\<close> is fully up-to-date wrt.\ the
   160   \<^descr> @{ML use_thy}~\<open>A\<close> ensures that theory \<open>A\<close> is fully up-to-date wrt.\ the
   162   external file store; outdated ancestors are reloaded on demand.
   161   external file store; outdated ancestors are reloaded on demand.
   163 
       
   164   \<^descr> @{ML use_thys} is similar to @{ML use_thy}, but handles several theories
       
   165   simultaneously. Thus it acts like processing the import header of a theory,
       
   166   without performing the merge of the result. By loading a whole sub-graph of
       
   167   theories, the intrinsic parallelism can be exploited by the system to
       
   168   speedup loading.
       
   169 
       
   170   This variant is used by default in @{tool build} @{cite "isabelle-system"}.
       
   171 
   162 
   172   \<^descr> @{ML Thy_Info.get_theory}~\<open>A\<close> retrieves the theory value presently
   163   \<^descr> @{ML Thy_Info.get_theory}~\<open>A\<close> retrieves the theory value presently
   173   associated with name \<open>A\<close>. Note that the result might be outdated wrt.\ the
   164   associated with name \<open>A\<close>. Note that the result might be outdated wrt.\ the
   174   file-system content.
   165   file-system content.
   175 
   166