doc-src/IsarImplementation/Thy/logic.thy
changeset 21324 a5089fc012b5
parent 20929 cd2a6d00ec47
child 21827 0b1d07f79c1e
equal deleted inserted replaced
21323:74ab7c0980c7 21324:a5089fc012b5
   326   @{index_ML fastype_of: "term -> typ"} \\
   326   @{index_ML fastype_of: "term -> typ"} \\
   327   @{index_ML lambda: "term -> term -> term"} \\
   327   @{index_ML lambda: "term -> term -> term"} \\
   328   @{index_ML betapply: "term * term -> term"} \\
   328   @{index_ML betapply: "term * term -> term"} \\
   329   @{index_ML Sign.add_consts_i: "(string * typ * mixfix) list -> theory -> theory"} \\
   329   @{index_ML Sign.add_consts_i: "(string * typ * mixfix) list -> theory -> theory"} \\
   330   @{index_ML Sign.add_abbrevs: "string * bool ->
   330   @{index_ML Sign.add_abbrevs: "string * bool ->
   331   ((string * mixfix) * term) list -> theory -> theory"} \\
   331   ((string * mixfix) * term) list -> theory -> (term * term) list * theory"} \\
   332   @{index_ML Sign.const_typargs: "theory -> string * typ -> typ list"} \\
   332   @{index_ML Sign.const_typargs: "theory -> string * typ -> typ list"} \\
   333   @{index_ML Sign.const_instance: "theory -> string * typ list -> typ"} \\
   333   @{index_ML Sign.const_instance: "theory -> string * typ list -> typ"} \\
   334   \end{mldecls}
   334   \end{mldecls}
   335 
   335 
   336   \begin{description}
   336   \begin{description}