src/Doc/Implementation/Proof.thy
changeset 66663 49318345c332
parent 61854 38b049cd3aad
child 69597 ff784d5a5bfb
equal deleted inserted replaced
66650:bcea02893d17 66663:49318345c332
    99   @{index_ML Variable.declare_term: "term -> Proof.context -> Proof.context"} \\
    99   @{index_ML Variable.declare_term: "term -> Proof.context -> Proof.context"} \\
   100   @{index_ML Variable.declare_constraints: "term -> Proof.context -> Proof.context"} \\
   100   @{index_ML Variable.declare_constraints: "term -> Proof.context -> Proof.context"} \\
   101   @{index_ML Variable.export: "Proof.context -> Proof.context -> thm list -> thm list"} \\
   101   @{index_ML Variable.export: "Proof.context -> Proof.context -> thm list -> thm list"} \\
   102   @{index_ML Variable.polymorphic: "Proof.context -> term list -> term list"} \\
   102   @{index_ML Variable.polymorphic: "Proof.context -> term list -> term list"} \\
   103   @{index_ML Variable.import: "bool -> thm list -> Proof.context ->
   103   @{index_ML Variable.import: "bool -> thm list -> Proof.context ->
   104   ((((indexname * sort) * ctyp) list * ((indexname * typ) * cterm) list) * thm list) * Proof.context"} \\
   104   ((((indexname * sort) * ctyp) list * ((indexname * typ) * cterm) list) * thm list)
       
   105     * Proof.context"} \\
   105   @{index_ML Variable.focus: "binding list option -> term -> Proof.context ->
   106   @{index_ML Variable.focus: "binding list option -> term -> Proof.context ->
   106   ((string * (string * typ)) list * term) * Proof.context"} \\
   107   ((string * (string * typ)) list * term) * Proof.context"} \\
   107   \end{mldecls}
   108   \end{mldecls}
   108 
   109 
   109   \<^descr> @{ML Variable.add_fixes}~\<open>xs ctxt\<close> fixes term variables \<open>xs\<close>, returning
   110   \<^descr> @{ML Variable.add_fixes}~\<open>xs ctxt\<close> fixes term variables \<open>xs\<close>, returning