src/Doc/Implementation/Integration.thy
changeset 61477 e467ae7aa808
parent 61458 987533262fc2
child 61493 0debd22f0c0e
equal deleted inserted replaced
61476:1884c40f1539 61477:e467ae7aa808
     7 chapter \<open>System integration\<close>
     7 chapter \<open>System integration\<close>
     8 
     8 
     9 section \<open>Isar toplevel \label{sec:isar-toplevel}\<close>
     9 section \<open>Isar toplevel \label{sec:isar-toplevel}\<close>
    10 
    10 
    11 text \<open>
    11 text \<open>
    12   The Isar \emph{toplevel state} represents the outermost configuration that
    12   The Isar \<^emph>\<open>toplevel state\<close> represents the outermost configuration that
    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
   147 
   147 
   148 text \<open>
   148 text \<open>
   149   In batch mode and within dumped logic images, the theory database maintains
   149   In batch mode and within dumped logic images, the theory database maintains
   150   a collection of theories as a directed acyclic graph. A theory may refer to
   150   a collection of theories as a directed acyclic graph. A theory may refer to
   151   other theories as @{keyword "imports"}, or to auxiliary files via special
   151   other theories as @{keyword "imports"}, or to auxiliary files via special
   152   \emph{load commands} (e.g.\ @{command ML_file}). For each theory, the base
   152   \<^emph>\<open>load commands\<close> (e.g.\ @{command ML_file}). For each theory, the base
   153   directory of its own theory file is called \emph{master directory}: this is
   153   directory of its own theory file is called \<^emph>\<open>master directory\<close>: this is
   154   used as the relative location to refer to other files from that theory.
   154   used as the relative location to refer to other files from that theory.
   155 \<close>
   155 \<close>
   156 
   156 
   157 text %mlref \<open>
   157 text %mlref \<open>
   158   \begin{mldecls}
   158   \begin{mldecls}