equal
deleted
inserted
replaced
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 ((ctyp Term_Subst.TVars.table * cterm Term_Subst.Vars.table) * thm list) |
104 ((ctyp TVars.table * cterm 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 |