--- a/CookBook/Intro.thy Wed Dec 17 05:08:33 2008 +0000
+++ b/CookBook/Intro.thy Sat Jan 03 20:44:54 2009 +0000
@@ -9,13 +9,13 @@
The purpose of this Cookbook is to guide the reader through the
first steps of Isabelle programming, and to provide recipes for
solving common problems. The code provided in the Cookbook is
- checked against recent versions of Isabelle.
+ as far as possible checked against recent versions of Isabelle.
*}
section {* Intended Audience and Prior Knowledge *}
text {*
- This cookbook targets an audience who already knows how to use Isabelle
+ This Cookbook targets an audience who already knows how to use Isabelle
for writing theories and proofs. We also assume that readers are
familiar with the functional programming language ML, the language in
which most of Isabelle is implemented. If you are unfamiliar with either of