--- a/CookBook/Intro.thy Wed Sep 17 19:20:37 2008 -0400
+++ b/CookBook/Intro.thy Tue Sep 30 03:30:40 2008 -0400
@@ -7,7 +7,7 @@
text {*
The purpose of this cookbook is to guide the reader through the
- first steps in Isabelle programming, and to provide recipes for
+ first steps of Isabelle programming, and to provide recipes for
solving common problems.
*}
@@ -17,7 +17,7 @@
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 Standard ML, the programming language in which
- most of Isabelle is implemented. If you are unfamiliar with any of
+ most of Isabelle is implemented. If you are unfamiliar with either of
these two subjects, you should first work through the Isabelle/HOL
tutorial \cite{isa-tutorial} and Paulson's book on Standard ML
\cite{paulson-ml2}.