src/Doc/Implementation/Integration.thy
changeset 82680 f7f8bb1c28ce
parent 76987 4c275405faae
equal deleted inserted replaced
82679:1dd29afaddda 82680:f7f8bb1c28ce
   151 text %mlref \<open>
   151 text %mlref \<open>
   152   \begin{mldecls}
   152   \begin{mldecls}
   153   @{define_ML use_thy: "string -> unit"} \\
   153   @{define_ML use_thy: "string -> unit"} \\
   154   @{define_ML Thy_Info.get_theory: "string -> theory"} \\
   154   @{define_ML Thy_Info.get_theory: "string -> theory"} \\
   155   @{define_ML Thy_Info.remove_thy: "string -> unit"} \\
   155   @{define_ML Thy_Info.remove_thy: "string -> unit"} \\
   156   @{define_ML Thy_Info.register_thy: "theory -> unit"} \\
       
   157   \end{mldecls}
   156   \end{mldecls}
   158 
   157 
   159   \<^descr> \<^ML>\<open>use_thy\<close>~\<open>A\<close> ensures that theory \<open>A\<close> is fully up-to-date wrt.\ the
   158   \<^descr> \<^ML>\<open>use_thy\<close>~\<open>A\<close> ensures that theory \<open>A\<close> is fully up-to-date wrt.\ the
   160   external file store; outdated ancestors are reloaded on demand.
   159   external file store; outdated ancestors are reloaded on demand.
   161 
   160 
   163   associated with name \<open>A\<close>. Note that the result might be outdated wrt.\ the
   162   associated with name \<open>A\<close>. Note that the result might be outdated wrt.\ the
   164   file-system content.
   163   file-system content.
   165 
   164 
   166   \<^descr> \<^ML>\<open>Thy_Info.remove_thy\<close>~\<open>A\<close> deletes theory \<open>A\<close> and all descendants from
   165   \<^descr> \<^ML>\<open>Thy_Info.remove_thy\<close>~\<open>A\<close> deletes theory \<open>A\<close> and all descendants from
   167   the theory database.
   166   the theory database.
   168 
       
   169   \<^descr> \<^ML>\<open>Thy_Info.register_thy\<close>~\<open>text thy\<close> registers an existing theory value
       
   170   with the theory loader database and updates source version information
       
   171   according to the file store.
       
   172 \<close>
   167 \<close>
   173 
   168 
   174 end
   169 end