diff -r 6968fd7507de -r bd602eb894ab Quotient-Paper-jv/Paper.thy --- a/Quotient-Paper-jv/Paper.thy Fri Feb 03 15:47:47 2012 +0000 +++ b/Quotient-Paper-jv/Paper.thy Fri Feb 03 15:51:55 2012 +0000 @@ -325,7 +325,7 @@ of \emph{aggregate equivalence relation}, \emph{respectfulness} and \emph{preservation} from Homeier \cite{Homeier05}. - {\bf EXAMPLE BY HUFFMAN ABOUT @{thm map_concat}} + {\bf EXAMPLE BY HUFFMAN @{thm map_concat_fset[no_vars]}} In addition we are able to clearly specify what is involved in the lifting process (this was only hinted at in \cite{Homeier05} and @@ -437,7 +437,7 @@ \begin{definition}[Bounded $\forall$ and $\lambda$]\label{def:babs} @{text "\x \ S. P x"} holds if for all @{text x}, @{text "x \ S"} implies @{text "P x"}; - and @{text "(\x \ S. f x) = f x"} provided @{text "x \ S"}. + and @{text "(\x \ S. f x) x = f x"} provided @{text "x \ S"}. \end{definition} The central definition in Homeier's work \cite{Homeier05} relates equivalence @@ -1294,7 +1294,7 @@ \begin{isabelle}\ \ \ \ \ % \begin{tabular}{@ {}l} - \isacommand{fun}~~@{text "int_rel :: (nat \ nat) \ (nat \ nat) \ (nat \ nat)"}\\ + \isacommand{fun}~~@{text "int_rel :: (nat \ nat) \ (nat \ nat) \ bool"}\\ \isacommand{where}~~@{text "int_rel (m, n) (p, q) = (m + q = n + p)"} \end{tabular} \end{isabelle}