src/Doc/Implementation/ML.thy
changeset 62876 507c90523113
parent 62505 9e2a65912111
child 62969 9f394a16c557
equal deleted inserted replaced
62875:5a0c06491974 62876:507c90523113
   614   instead.
   614   instead.
   615 \<close>
   615 \<close>
   616 
   616 
   617 text %mlref \<open>
   617 text %mlref \<open>
   618   \begin{mldecls}
   618   \begin{mldecls}
   619   @{index_ML ML_Context.the_generic_context: "unit -> Context.generic"} \\
   619   @{index_ML Context.the_generic_context: "unit -> Context.generic"} \\
   620   @{index_ML "Context.>>": "(Context.generic -> Context.generic) -> unit"} \\
   620   @{index_ML "Context.>>": "(Context.generic -> Context.generic) -> unit"} \\
   621   @{index_ML ML_Thms.bind_thms: "string * thm list -> unit"} \\
   621   @{index_ML ML_Thms.bind_thms: "string * thm list -> unit"} \\
   622   @{index_ML ML_Thms.bind_thm: "string * thm -> unit"} \\
   622   @{index_ML ML_Thms.bind_thm: "string * thm -> unit"} \\
   623   \end{mldecls}
   623   \end{mldecls}
   624 
   624 
   625     \<^descr> @{ML "ML_Context.the_generic_context ()"} refers to the theory context of
   625     \<^descr> @{ML "Context.the_generic_context ()"} refers to the theory context of
   626     the ML toplevel --- at compile time. ML code needs to take care to refer to
   626     the ML toplevel --- at compile time. ML code needs to take care to refer to
   627     @{ML "ML_Context.the_generic_context ()"} correctly. Recall that evaluation
   627     @{ML "Context.the_generic_context ()"} correctly. Recall that evaluation
   628     of a function body is delayed until actual run-time.
   628     of a function body is delayed until actual run-time.
   629 
   629 
   630     \<^descr> @{ML "Context.>>"}~\<open>f\<close> applies context transformation \<open>f\<close> to the implicit
   630     \<^descr> @{ML "Context.>>"}~\<open>f\<close> applies context transformation \<open>f\<close> to the implicit
   631     context of the ML toplevel.
   631     context of the ML toplevel.
   632 
   632