doc-src/IsarImplementation/Thy/Logic.thy
changeset 39821 bf164c153d10
parent 39281 148b78fb70d8
child 39832 1080dee73a53
equal deleted inserted replaced
39820:cd691e2c7a1a 39821:bf164c153d10
   550   @{index_ML Thm.implies_intr: "cterm -> thm -> thm"} \\
   550   @{index_ML Thm.implies_intr: "cterm -> thm -> thm"} \\
   551   @{index_ML Thm.implies_elim: "thm -> thm -> thm"} \\
   551   @{index_ML Thm.implies_elim: "thm -> thm -> thm"} \\
   552   @{index_ML Thm.generalize: "string list * string list -> int -> thm -> thm"} \\
   552   @{index_ML Thm.generalize: "string list * string list -> int -> thm -> thm"} \\
   553   @{index_ML Thm.instantiate: "(ctyp * ctyp) list * (cterm * cterm) list -> thm -> thm"} \\
   553   @{index_ML Thm.instantiate: "(ctyp * ctyp) list * (cterm * cterm) list -> thm -> thm"} \\
   554   @{index_ML Thm.add_axiom: "binding * term -> theory -> (string * thm) * theory"} \\
   554   @{index_ML Thm.add_axiom: "binding * term -> theory -> (string * thm) * theory"} \\
   555   @{index_ML Thm.add_oracle: "binding * ('a -> cterm) -> theory
   555   @{index_ML Thm.add_oracle: "binding * ('a -> cterm) -> theory ->
   556   -> (string * ('a -> thm)) * theory"} \\
   556   (string * ('a -> thm)) * theory"} \\
   557   @{index_ML Thm.add_def: "bool -> bool -> binding * term -> theory -> (string * thm) * theory"} \\
   557   @{index_ML Thm.add_def: "bool -> bool -> binding * term -> theory ->
       
   558   (string * thm) * theory"} \\
   558   \end{mldecls}
   559   \end{mldecls}
   559   \begin{mldecls}
   560   \begin{mldecls}
   560   @{index_ML Theory.add_deps: "string -> string * typ -> (string * typ) list -> theory -> theory"} \\
   561   @{index_ML Theory.add_deps: "string -> string * typ -> (string * typ) list ->
       
   562   theory -> theory"} \\
   561   \end{mldecls}
   563   \end{mldecls}
   562 
   564 
   563   \begin{description}
   565   \begin{description}
   564 
   566 
   565   \item @{ML_type ctyp} and @{ML_type cterm} represent certified types
   567   \item @{ML_type ctyp} and @{ML_type cterm} represent certified types