diff -r 6968fd7507de -r bd602eb894ab Quotient-Paper/Paper.thy --- a/Quotient-Paper/Paper.thy Fri Feb 03 15:47:47 2012 +0000 +++ b/Quotient-Paper/Paper.thy Fri Feb 03 15:51:55 2012 +0000 @@ -428,7 +428,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 @@ -1284,7 +1284,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}