doc-src/TutorialI/Types/Overloading2.thy
changeset 10654 458068404143
parent 10396 5ab08609e6c8
child 10696 76d7f6c9a14c
--- a/doc-src/TutorialI/Types/Overloading2.thy	Wed Dec 13 09:32:55 2000 +0100
+++ b/doc-src/TutorialI/Types/Overloading2.thy	Wed Dec 13 09:39:53 2000 +0100
@@ -37,11 +37,11 @@
 @{text"*"} & @{text "('a::times) \<Rightarrow> 'a \<Rightarrow> 'a"} & (infixl 70) \\
 @{text"^"} & @{text "('a::power) \<Rightarrow> nat \<Rightarrow> 'a"} & (infixr 80) \\
 @{text"-"} & @{text "('a::minus) \<Rightarrow> 'a"} \\
-@{term abs} &  @{text "('a::minus) \<Rightarrow> 'a"} \\
+@{term abs} &  @{text "('a::minus) \<Rightarrow> 'a"} & $\mid~\mid$\\
 @{text"\<le>"} & @{text "('a::ord) \<Rightarrow> 'a \<Rightarrow> bool"} & (infixl 50) \\
 @{text"<"} & @{text "('a::ord) \<Rightarrow> 'a \<Rightarrow> bool"} & (infixl 50) \\
 @{term min} &  @{text "('a::ord) \<Rightarrow> 'a \<Rightarrow> 'a"} \\
-@{term max} &  @{text "('a::ord) \<Rightarrow> 'a \<Rightarrow> 'a"} \\
+@{term max} &  @{text "('a::ord) \<Rightarrow> 'a \<Rightarrow> 'a"}
 \end{tabular}
 \caption{Overloaded constants in HOL}
 \label{tab:overloading}