diff -r b8ca12f6681a -r 1f2051f41335 doc-src/IsarImplementation/Thy/Logic.thy --- a/doc-src/IsarImplementation/Thy/Logic.thy Sun Oct 25 21:35:46 2009 +0100 +++ b/doc-src/IsarImplementation/Thy/Logic.thy Mon Oct 26 08:54:20 2009 +0100 @@ -322,9 +322,9 @@ @{index_ML fastype_of: "term -> typ"} \\ @{index_ML lambda: "term -> term -> term"} \\ @{index_ML betapply: "term * term -> term"} \\ - @{index_ML Sign.declare_const: "Properties.T -> (binding * typ) * mixfix -> + @{index_ML Sign.declare_const: "(binding * typ) * mixfix -> theory -> term * theory"} \\ - @{index_ML Sign.add_abbrev: "string -> Properties.T -> binding * term -> + @{index_ML Sign.add_abbrev: "string -> binding * term -> theory -> (term * term) * theory"} \\ @{index_ML Sign.const_typargs: "theory -> string * typ -> typ list"} \\ @{index_ML Sign.const_instance: "theory -> string * typ list -> typ"} \\ @@ -370,11 +370,11 @@ "t u"}, with topmost @{text "\"}-conversion if @{text "t"} is an abstraction. - \item @{ML Sign.declare_const}~@{text "properties ((c, \), mx)"} + \item @{ML Sign.declare_const}~@{text "((c, \), mx)"} declares a new constant @{text "c :: \"} with optional mixfix syntax. - \item @{ML Sign.add_abbrev}~@{text "print_mode properties (c, t)"} + \item @{ML Sign.add_abbrev}~@{text "print_mode (c, t)"} introduces a new term abbreviation @{text "c \ t"}. \item @{ML Sign.const_typargs}~@{text "thy (c, \)"} and @{ML