diff -r a5d3730043c2 -r 7d5ad23b8245 src/Doc/ProgProve/Basics.thy --- a/src/Doc/ProgProve/Basics.thy Mon Jun 10 08:39:48 2013 -0400 +++ b/src/Doc/ProgProve/Basics.thy Mon Jun 10 16:04:18 2013 +0200 @@ -9,7 +9,7 @@ \section{Basics} -\subsection{Types, Terms and Formulae} +\subsection{Types, Terms and Formulas} \label{sec:TypesTermsForms} HOL is a typed logic whose type system resembles that of functional @@ -58,7 +58,7 @@ Terms may also contain @{text "\"}-abstractions. For example, @{term "\x. x"} is the identity function. -\concept{Formulae} are terms of type @{text bool}. +\concept{Formulas} are terms of type @{text bool}. There are the basic constants @{term True} and @{term False} and the usual logical connectives (in decreasing order of precedence): @{text"\"}, @{text"\"}, @{text"\"}, @{text"\"}. @@ -133,7 +133,7 @@ The textual definition of a theory follows a fixed syntax with keywords like \isacommand{begin} and \isacommand{datatype}. Embedded in this syntax are -the types and formulae of HOL. To distinguish the two levels, everything +the types and formulas of HOL. To distinguish the two levels, everything HOL-specific (terms and types) must be enclosed in quotation marks: \texttt{"}\dots\texttt{"}. To lessen this burden, quotation marks around a single identifier can be dropped. When Isabelle prints a syntax error