doc-src/IsarRef/Thy/Spec.thy
changeset 39850 f4c614ece7ed
parent 39831 350857040d09
child 40079 07445603208a
--- a/doc-src/IsarRef/Thy/Spec.thy	Thu Oct 14 21:55:21 2010 +0100
+++ b/doc-src/IsarRef/Thy/Spec.thy	Fri Oct 15 19:19:41 2010 +0100
@@ -837,11 +837,6 @@
     @{command_def "attribute_setup"} & : & @{text "theory \<rightarrow> theory"} \\
   \end{matharray}
 
-  \begin{mldecls}
-    @{index_ML bind_thms: "string * thm list -> unit"} \\
-    @{index_ML bind_thm: "string * thm -> unit"} \\
-  \end{mldecls}
-
   \begin{rail}
     'use' name
     ;
@@ -918,20 +913,6 @@
           let val context' = context
           in context' end)) *}  "my declaration"
 
-text {*
-  \begin{description}
-
-  \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{description}
-*}
-
 
 section {* Primitive specification elements *}