doc-src/IsarRef/Thy/Spec.thy
changeset 28758 4ce896a30f88
parent 28757 7f7002ad6289
child 28760 cbc435f7b16b
--- a/doc-src/IsarRef/Thy/Spec.thy	Thu Nov 13 21:40:00 2008 +0100
+++ b/doc-src/IsarRef/Thy/Spec.thy	Thu Nov 13 21:40:30 2008 +0100
@@ -808,6 +808,8 @@
     @{command_def "ML_val"} & : & \isartrans{\cdot}{\cdot} \\
     @{command_def "ML_command"} & : & \isartrans{\cdot}{\cdot} \\
     @{command_def "setup"} & : & \isartrans{theory}{theory} \\
+    @{index_ML bind_thms: "string * thm list -> unit"} \\
+    @{index_ML bind_thm: "string * thm -> unit"} \\
   \end{matharray}
 
   \begin{rail}
@@ -852,6 +854,14 @@
   of type @{ML_type [source=false] "theory -> theory"}.  This enables
   to initialize any object-logic specific tools and packages written
   in ML, for example.
+
+  \item @{ML bind_thms}~@{text "(name, thms)"} stores a list of
+  theorems produced in ML both in the theory context and the ML
+  toplevel, associating it with the provided name.  Theorems are put
+  into a global ``standard'' format before being stored.
+
+  \item @{ML bind_thm} is similar to @{ML bind_thms} but refers to a
+  singleton theorem.
   
   \end{descr}
 *}