src/Doc/IsarImplementation/ML.thy
changeset 56199 8e8d28ed7529
parent 55838 e120a15b0ee6
child 56303 4cc3f4db3447
equal deleted inserted replaced
56198:21dd034523e5 56199:8e8d28ed7529
   625 
   625 
   626 text %mlref {*
   626 text %mlref {*
   627   \begin{mldecls}
   627   \begin{mldecls}
   628   @{index_ML ML_Context.the_generic_context: "unit -> Context.generic"} \\
   628   @{index_ML ML_Context.the_generic_context: "unit -> Context.generic"} \\
   629   @{index_ML "Context.>>": "(Context.generic -> Context.generic) -> unit"} \\
   629   @{index_ML "Context.>>": "(Context.generic -> Context.generic) -> unit"} \\
   630   @{index_ML bind_thms: "string * thm list -> unit"} \\
   630   @{index_ML ML_Thms.bind_thms: "string * thm list -> unit"} \\
   631   @{index_ML bind_thm: "string * thm -> unit"} \\
   631   @{index_ML ML_Thms.bind_thm: "string * thm -> unit"} \\
   632   \end{mldecls}
   632   \end{mldecls}
   633 
   633 
   634   \begin{description}
   634   \begin{description}
   635 
   635 
   636   \item @{ML "ML_Context.the_generic_context ()"} refers to the theory
   636   \item @{ML "ML_Context.the_generic_context ()"} refers to the theory
   640   until actual run-time.
   640   until actual run-time.
   641 
   641 
   642   \item @{ML "Context.>>"}~@{text f} applies context transformation
   642   \item @{ML "Context.>>"}~@{text f} applies context transformation
   643   @{text f} to the implicit context of the ML toplevel.
   643   @{text f} to the implicit context of the ML toplevel.
   644 
   644 
   645   \item @{ML bind_thms}~@{text "(name, thms)"} stores a list of
   645   \item @{ML ML_Thms.bind_thms}~@{text "(name, thms)"} stores a list of
   646   theorems produced in ML both in the (global) theory context and the
   646   theorems produced in ML both in the (global) theory context and the
   647   ML toplevel, associating it with the provided name.  Theorems are
   647   ML toplevel, associating it with the provided name.  Theorems are
   648   put into a global ``standard'' format before being stored.
   648   put into a global ``standard'' format before being stored.
   649 
   649 
   650   \item @{ML bind_thm} is similar to @{ML bind_thms} but refers to a
   650   \item @{ML ML_Thms.bind_thm} is similar to @{ML ML_Thms.bind_thms} but refers to a
   651   singleton fact.
   651   singleton fact.
   652 
   652 
   653   \end{description}
   653   \end{description}
   654 
   654 
   655   It is important to note that the above functions are really
   655   It is important to note that the above functions are really