doc-src/IsarImplementation/Thy/logic.thy
changeset 29581 b3b33e0298eb
parent 29008 d863c103ded0
child 29615 24a58ae5dc0e
equal deleted inserted replaced
29580:117b88da143c 29581:b3b33e0298eb
   321   \end{mldecls}
   321   \end{mldecls}
   322   \begin{mldecls}
   322   \begin{mldecls}
   323   @{index_ML fastype_of: "term -> typ"} \\
   323   @{index_ML fastype_of: "term -> typ"} \\
   324   @{index_ML lambda: "term -> term -> term"} \\
   324   @{index_ML lambda: "term -> term -> term"} \\
   325   @{index_ML betapply: "term * term -> term"} \\
   325   @{index_ML betapply: "term * term -> term"} \\
   326   @{index_ML Sign.declare_const: "Properties.T -> (Binding.T * typ) * mixfix ->
   326   @{index_ML Sign.declare_const: "Properties.T -> (binding * typ) * mixfix ->
   327   theory -> term * theory"} \\
   327   theory -> term * theory"} \\
   328   @{index_ML Sign.add_abbrev: "string -> Properties.T -> Binding.T * term ->
   328   @{index_ML Sign.add_abbrev: "string -> Properties.T -> binding * term ->
   329   theory -> (term * term) * theory"} \\
   329   theory -> (term * term) * theory"} \\
   330   @{index_ML Sign.const_typargs: "theory -> string * typ -> typ list"} \\
   330   @{index_ML Sign.const_typargs: "theory -> string * typ -> typ list"} \\
   331   @{index_ML Sign.const_instance: "theory -> string * typ list -> typ"} \\
   331   @{index_ML Sign.const_instance: "theory -> string * typ list -> typ"} \\
   332   \end{mldecls}
   332   \end{mldecls}
   333 
   333