src/Doc/Implementation/Proof.thy
changeset 60642 48dd1cefb4ae
parent 59902 6afbe5a99139
child 60695 757549b4bbe6
equal deleted inserted replaced
60641:f6e8293747fd 60642:48dd1cefb4ae
   106   @{index_ML Variable.declare_term: "term -> Proof.context -> Proof.context"} \\
   106   @{index_ML Variable.declare_term: "term -> Proof.context -> Proof.context"} \\
   107   @{index_ML Variable.declare_constraints: "term -> Proof.context -> Proof.context"} \\
   107   @{index_ML Variable.declare_constraints: "term -> Proof.context -> Proof.context"} \\
   108   @{index_ML Variable.export: "Proof.context -> Proof.context -> thm list -> thm list"} \\
   108   @{index_ML Variable.export: "Proof.context -> Proof.context -> thm list -> thm list"} \\
   109   @{index_ML Variable.polymorphic: "Proof.context -> term list -> term list"} \\
   109   @{index_ML Variable.polymorphic: "Proof.context -> term list -> term list"} \\
   110   @{index_ML Variable.import: "bool -> thm list -> Proof.context ->
   110   @{index_ML Variable.import: "bool -> thm list -> Proof.context ->
   111   (((ctyp * ctyp) list * (cterm * cterm) list) * thm list) * Proof.context"} \\
   111   ((((indexname * sort) * ctyp) list * ((indexname * typ) * cterm) list) * thm list) * Proof.context"} \\
   112   @{index_ML Variable.focus: "term -> Proof.context ->
   112   @{index_ML Variable.focus: "term -> Proof.context ->
   113   ((string * (string * typ)) list * term) * Proof.context"} \\
   113   ((string * (string * typ)) list * term) * Proof.context"} \\
   114   \end{mldecls}
   114   \end{mldecls}
   115 
   115 
   116   \begin{description}
   116   \begin{description}