src/Doc/Implementation/Proof.thy
changeset 74240 36774e8af3db
parent 73764 35d8132633c6
child 74266 612b7e0d6721
equal deleted inserted replaced
74239:914a214e110e 74240:36774e8af3db
    99   @{define_ML Variable.declare_term: "term -> Proof.context -> Proof.context"} \\
    99   @{define_ML Variable.declare_term: "term -> Proof.context -> Proof.context"} \\
   100   @{define_ML Variable.declare_constraints: "term -> Proof.context -> Proof.context"} \\
   100   @{define_ML Variable.declare_constraints: "term -> Proof.context -> Proof.context"} \\
   101   @{define_ML Variable.export: "Proof.context -> Proof.context -> thm list -> thm list"} \\
   101   @{define_ML Variable.export: "Proof.context -> Proof.context -> thm list -> thm list"} \\
   102   @{define_ML Variable.polymorphic: "Proof.context -> term list -> term list"} \\
   102   @{define_ML Variable.polymorphic: "Proof.context -> term list -> term list"} \\
   103   @{define_ML Variable.import: "bool -> thm list -> Proof.context ->
   103   @{define_ML Variable.import: "bool -> thm list -> Proof.context ->
   104   ((((indexname * sort) * ctyp) list * ((indexname * typ) * cterm) list) * thm list)
   104   ((ctyp Term_Subst.TVars.table * cterm Term_Subst.Vars.table) * thm list)
   105     * Proof.context"} \\
   105     * Proof.context"} \\
   106   @{define_ML Variable.focus: "binding list option -> term -> Proof.context ->
   106   @{define_ML Variable.focus: "binding list option -> term -> Proof.context ->
   107   ((string * (string * typ)) list * term) * Proof.context"} \\
   107   ((string * (string * typ)) list * term) * Proof.context"} \\
   108   \end{mldecls}
   108   \end{mldecls}
   109 
   109