commented out unsound "lfp"/"gfp" handling + fixed set output syntax;
the "lfp"/"gfp" bug can be reproduced by looking for a counterexample to
lemma "(A \<union> B)^+ = A^+ \<union> B^+"
Refute incorrectly finds a countermodel for cardinality 1 (the smallest
counterexample requires cardinality 2).
\input{style}
\hyphenation{Isabelle}
\begin{document}
\title{Miscellaneous Isabelle/Isar examples for Higher-Order Logic}
\author{Markus Wenzel \\ \url{http://www.in.tum.de/~wenzelm/} \\[2ex]
With contributions by Gertrud Bauer and Tobias Nipkow}
\maketitle
\begin{abstract}
Isar offers a high-level proof (and theory) language for Isabelle.
We give various examples of Isabelle/Isar proof developments,
ranging from simple demonstrations of certain language features to a
bit more advanced applications. The ``real'' applications of
Isabelle/Isar are found elsewhere.
\end{abstract}
\tableofcontents
\parindent 0pt \parskip 0.5ex
\input{session}
\nocite{isabelle-isar-ref,Wenzel:1999:TPHOL}
\bibliographystyle{abbrv}
\bibliography{root}
\end{document}