diff -r 646bdc51eb7d -r 137c242e7277 doc-src/IsarImplementation/Thy/logic.thy --- a/doc-src/IsarImplementation/Thy/logic.thy Thu Oct 04 12:32:58 2007 +0200 +++ b/doc-src/IsarImplementation/Thy/logic.thy Thu Oct 04 13:26:34 2007 +0200 @@ -327,7 +327,7 @@ @{index_ML lambda: "term -> term -> term"} \\ @{index_ML betapply: "term * term -> term"} \\ @{index_ML Sign.add_consts_i: "(string * typ * mixfix) list -> theory -> theory"} \\ - @{index_ML Sign.add_abbrev: "string -> bstring * term -> theory -> (term * term) * theory"} \\ + @{index_ML Sign.add_abbrev: "string -> Markup.property list -> bstring * 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"} \\ \end{mldecls} @@ -375,7 +375,7 @@ \item @{ML Sign.add_consts_i}~@{text "[(c, \, mx), \]"} declares a new constant @{text "c :: \"} with optional mixfix syntax. - \item @{ML Sign.add_abbrev}~@{text "print_mode (c, t)"} + \item @{ML Sign.add_abbrev}~@{text "print_mode properties (c, t)"} introduces a new term abbreviation @{text "c \ t"}. \item @{ML Sign.const_typargs}~@{text "thy (c, \)"} and @{ML