src/Doc/Implementation/Local_Theory.thy
changeset 63402 f199837304d7
parent 61854 38b049cd3aad
child 63403 a962f349c8c9
equal deleted inserted replaced
63400:249fa34faba2 63402:f199837304d7
    89 \<close>
    89 \<close>
    90 
    90 
    91 text %mlref \<open>
    91 text %mlref \<open>
    92   \begin{mldecls}
    92   \begin{mldecls}
    93   @{index_ML_type local_theory: Proof.context} \\
    93   @{index_ML_type local_theory: Proof.context} \\
    94   @{index_ML Named_Target.init: "string -> theory -> local_theory"} \\[1ex]
    94   @{index_ML Named_Target.init: "(local_theory -> local_theory) -> string ->
       
    95     theory -> local_theory"} \\[1ex]
    95   @{index_ML Local_Theory.define: "(binding * mixfix) * (Attrib.binding * term) ->
    96   @{index_ML Local_Theory.define: "(binding * mixfix) * (Attrib.binding * term) ->
    96     local_theory -> (term * (string * thm)) * local_theory"} \\
    97     local_theory -> (term * (string * thm)) * local_theory"} \\
    97   @{index_ML Local_Theory.note: "Attrib.binding * thm list ->
    98   @{index_ML Local_Theory.note: "Attrib.binding * thm list ->
    98     local_theory -> (string * thm list) * local_theory"} \\
    99     local_theory -> (string * thm list) * local_theory"} \\
    99   \end{mldecls}
   100   \end{mldecls}