(reverted to previous version)
authorhaftmann
Tue, 18 Sep 2007 11:06:22 +0200
changeset 24629 65947eb930fa
parent 24628 33137422d7fd
child 24630 351a308ab58d
(reverted to previous version)
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) \<Rightarrow> 'a"} & ${\mid} x {\mid}$\\
 @{text"\<le>"} & @{text "('a::ord) \<Rightarrow> 'a \<Rightarrow> bool"} & (infixl 50) \\
 @{text"<"} & @{text "('a::ord) \<Rightarrow> 'a \<Rightarrow> bool"} & (infixl 50) \\
-%@{term Least} & @{text "('a::ord \<Rightarrow> bool) \<Rightarrow> 'a"} &
-%@{text LEAST}$~x.~P$
+@{term min} &  @{text "('a::ord) \<Rightarrow> 'a \<Rightarrow> 'a"} \\
+@{term max} &  @{text "('a::ord) \<Rightarrow> 'a \<Rightarrow> 'a"} \\
+@{term Least} & @{text "('a::ord \<Rightarrow> bool) \<Rightarrow> '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}