CookBook/Intro.thy
changeset 106 bdd82350cf22
parent 102 5e309df58557
child 107 258ce361ba1b
equal deleted inserted replaced
105:f49dc7e96235 106:bdd82350cf22
     6 
     6 
     7 chapter {* Introduction *}
     7 chapter {* Introduction *}
     8 
     8 
     9 text {*
     9 text {*
    10   If your next project requires you to program on the ML-level of Isabelle,
    10   If your next project requires you to program on the ML-level of Isabelle,
    11   then this Cookbook is for you. It will guide you through the first steps of
    11   then this tutorial is for you. It will guide you through the first steps of
    12   Isabelle programming, and also explain tricks of the trade. The best way to
    12   Isabelle programming, and also explain tricks of the trade. The best way to
    13   get to know the ML-level of Isabelle is by experimenting with the many code
    13   get to know the ML-level of Isabelle is by experimenting with the many code
    14   examples included in the Cookbook. The code is as far as possible checked
    14   examples included in the tutorial. The code is as far as possible checked
    15   against recent versions of Isabelle.  If something does not work, then
    15   against recent versions of Isabelle.  If something does not work, then
    16   please let us know. If you have comments, criticism or like to add to the
    16   please let us know. If you have comments, criticism or like to add to the
    17   Cookbook, feel free---you are most welcome!
    17   tutorial, feel free---you are most welcome!
    18 *}
    18 *}
    19 
    19 
    20 section {* Intended Audience and Prior Knowledge *}
    20 section {* Intended Audience and Prior Knowledge *}
    21 
    21 
    22 text {* 
    22 text {* 
    23   This Cookbook targets readers who already know how to use Isabelle for
    23   This tutorial targets readers who already know how to use Isabelle for
    24   writing theories and proofs. We also assume that readers are familiar with
    24   writing theories and proofs. We also assume that readers are familiar with
    25   the functional programming language ML, the language in which most of
    25   the functional programming language ML, the language in which most of
    26   Isabelle is implemented. If you are unfamiliar with either of these two
    26   Isabelle is implemented. If you are unfamiliar with either of these two
    27   subjects, you should first work through the Isabelle/HOL tutorial
    27   subjects, you should first work through the Isabelle/HOL tutorial
    28   \cite{isa-tutorial} or Paulson's book on ML \cite{paulson-ml2}.
    28   \cite{isa-tutorial} or Paulson's book on ML \cite{paulson-ml2}.
    66 
    66 
    67 section {* Typographic Conventions *}
    67 section {* Typographic Conventions *}
    68 
    68 
    69 text {*
    69 text {*
    70 
    70 
    71   All ML-code in this Cookbook is typeset in highlighted boxes, like the following 
    71   All ML-code in this tutorial is typeset in highlighted boxes, like the following 
    72   ML-expression:
    72   ML-expression:
    73 
    73 
    74   \begin{isabelle}
    74   \begin{isabelle}
    75   \begin{graybox}
    75   \begin{graybox}
    76   \isacommand{ML}~@{text "\<verbopen>"}\isanewline
    76   \isacommand{ML}~@{text "\<verbopen>"}\isanewline