diff -r f4112721a4b9 -r a9a4baa7779f Quotient-Paper/Paper.thy --- a/Quotient-Paper/Paper.thy Tue Jan 24 17:43:07 2012 +0000 +++ b/Quotient-Paper/Paper.thy Tue Jan 31 16:26:36 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}