diff -r 883248dcf3f8 -r 9429f2e7d16a doc-src/TutorialI/Misc/appendix.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/doc-src/TutorialI/Misc/appendix.thy Mon Jan 29 19:24:17 2001 +0100 @@ -0,0 +1,37 @@ +(*<*) +theory appendix = Main:; +(*>*) + +text{* +\begin{table}[htbp] +\begin{center} +\begin{tabular}{lll} +Constant & Type & Syntax \\ +\hline +@{term 0} & @{text "'a::zero"} \\ +@{text"+"} & @{text "('a::plus) \ 'a \ 'a"} & (infixl 65) \\ +@{text"-"} & @{text "('a::minus) \ 'a \ 'a"} & (infixl 65) \\ +@{text"-"} & @{text "('a::minus) \ 'a"} \\ +@{text"*"} & @{text "('a::times) \ 'a \ 'a"} & (infixl 70) \\ +@{text div} & @{text "('a::div) \ 'a \ 'a"} & (infixl 70) \\ +@{text mod} & @{text "('a::div) \ 'a \ 'a"} & (infixl 70) \\ +@{text dvd} & @{text "('a::times) \ 'a \ bool"} & (infixl 50) \\ +@{text"/"} & @{text "('a::inverse) \ 'a \ 'a"} & (infixl 70) \\ +@{text"^"} & @{text "('a::power) \ nat \ 'a"} & (infixr 80) \\ +@{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 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{Overloaded Constants in HOL} +\label{tab:overloading} +\end{center} +\end{table} +*} + +(*<*) +end +(*>*)