diff -r 33137422d7fd -r 65947eb930fa doc-src/TutorialI/Misc/appendix.thy --- a/doc-src/TutorialI/Misc/appendix.thy Tue Sep 18 10:44:02 2007 +0200 +++ b/doc-src/TutorialI/Misc/appendix.thy Tue Sep 18 11:06:22 2007 +0200 @@ -1,7 +1,5 @@ (*<*) -theory appendix -imports Main -begin +theory appendix imports Main begin; (*>*) text{* @@ -24,10 +22,12 @@ @{term abs} & @{text "('a::minus) \ 'a"} & ${\mid} x {\mid}$\\ @{text"\"} & @{text "('a::ord) \ 'a \ bool"} & (infixl 50) \\ @{text"<"} & @{text "('a::ord) \ 'a \ bool"} & (infixl 50) \\ -%@{term Least} & @{text "('a::ord \ bool) \ 'a"} & -%@{text LEAST}$~x.~P$ +@{term min} & @{text "('a::ord) \ 'a \ 'a"} \\ +@{term max} & @{text "('a::ord) \ 'a \ 'a"} \\ +@{term Least} & @{text "('a::ord \ bool) \ 'a"} & +@{text LEAST}$~x.~P$ \end{tabular} -\caption{Algebraic symbols and operations in HOL} +\caption{Overloaded Constants in HOL} \label{tab:overloading} \end{center} \end{table}