doc-src/IsarRef/Thy/Spec.thy
changeset 28758 4ce896a30f88
parent 28757 7f7002ad6289
child 28760 cbc435f7b16b
equal deleted inserted replaced
28757:7f7002ad6289 28758:4ce896a30f88
   806     @{command_def "ML"} & : & \isarkeep{theory~|~local{\dsh}theory} \\
   806     @{command_def "ML"} & : & \isarkeep{theory~|~local{\dsh}theory} \\
   807     @{command_def "ML_prf"} & : & \isarkeep{proof} \\
   807     @{command_def "ML_prf"} & : & \isarkeep{proof} \\
   808     @{command_def "ML_val"} & : & \isartrans{\cdot}{\cdot} \\
   808     @{command_def "ML_val"} & : & \isartrans{\cdot}{\cdot} \\
   809     @{command_def "ML_command"} & : & \isartrans{\cdot}{\cdot} \\
   809     @{command_def "ML_command"} & : & \isartrans{\cdot}{\cdot} \\
   810     @{command_def "setup"} & : & \isartrans{theory}{theory} \\
   810     @{command_def "setup"} & : & \isartrans{theory}{theory} \\
       
   811     @{index_ML bind_thms: "string * thm list -> unit"} \\
       
   812     @{index_ML bind_thm: "string * thm -> unit"} \\
   811   \end{matharray}
   813   \end{matharray}
   812 
   814 
   813   \begin{rail}
   815   \begin{rail}
   814     'use' name
   816     'use' name
   815     ;
   817     ;
   850   \item [@{command "setup"}~@{text "text"}] changes the current theory
   852   \item [@{command "setup"}~@{text "text"}] changes the current theory
   851   context by applying @{text "text"}, which refers to an ML expression
   853   context by applying @{text "text"}, which refers to an ML expression
   852   of type @{ML_type [source=false] "theory -> theory"}.  This enables
   854   of type @{ML_type [source=false] "theory -> theory"}.  This enables
   853   to initialize any object-logic specific tools and packages written
   855   to initialize any object-logic specific tools and packages written
   854   in ML, for example.
   856   in ML, for example.
       
   857 
       
   858   \item @{ML bind_thms}~@{text "(name, thms)"} stores a list of
       
   859   theorems produced in ML both in the theory context and the ML
       
   860   toplevel, associating it with the provided name.  Theorems are put
       
   861   into a global ``standard'' format before being stored.
       
   862 
       
   863   \item @{ML bind_thm} is similar to @{ML bind_thms} but refers to a
       
   864   singleton theorem.
   855   
   865   
   856   \end{descr}
   866   \end{descr}
   857 *}
   867 *}
   858 
   868 
   859 
   869