src/HOL/Hoare/README.html
author nipkow
Wed, 14 Oct 1998 15:26:31 +0200
changeset 5646 7c2ddbaf8b8c
parent 1715 7cbff1da8578
child 5647 4e8837255b87
permissions -rw-r--r--
New many-sorted version.

<HTML><HEAD><TITLE>HOL/Hoare/ReadMe</TITLE></HEAD><BODY>

<H2>Hoare Logic for a Simple WHILE Language</H2>

<H1>The language and logic<H1>

This directory contains an implementation of Hoare logic for a simple WHILE
language. The  are
<UL>
<LI> SKIP
<LI> _ := _
<LI> _ ; _
<LI> <kbd>IF _ THEN _ ELSE _ FI<kbd>
<LI> WHILE _ INV {_} DO _ OD
</UL>
Note that each WHILE-loop must be annotated with an invariant.
<P>

After loading theory Hoare, you can state goals of the form
<PRE>
|- VARS x y ... . {P} prog {Q}
</PRE>
where <kbd>prog</kbd> is a program in the above language, <kbd>P</kbd> is the
precondition, <kbd>Q</kbd> the postcondition, and <kbd>x y ...<kbd> is the
list of all <i>program variables</i> in <kbd>prog</kbd>. The latter list must
be nonempty and it must include all variables that occur on the left-hand
side of an assignment in <kbd>prof</kbd>. Example:
<PRE>
|- VARS x. {x = a} x := x+1 {x = a+1}
</PRE>
The (normal) variable <kbd>a</kbd> is merely used to record the initial
value of <kbd>x</kbd> and is not a program variable. Pre and postconditions
can be arbitrary HOL formulae mentioning both program variables and normal
variables.
<P>

The implementation hides reasoning in Hoare logic completely and provides a
tactic hoare_tac for generating the verification conditions in ordinary
logic:
<PRE>
by(hoare_tac tac i);
</PRE>
applies the tactic to subgoal <kbd>i</kbd> and applies the parameter
<kbd>tac</kbd> to all generated verification conditions. A typical call is
<PRE>
by(hoare_tac Asm_full_simp_tac 1);
</PRE>
which, given the example goal above, solves it completely.
<P>

IMPORTANT:
This is a logic of partial correctness. You can only prove that your program
does the right thing <i>if</i> it terminates, but not <i>that</i> it
terminates.

<H1>Notes on the implementation</H1>

This directory contains a sugared shallow semantic embedding of Hoare logic
for a while language. The implementation closely follows<P>


Mike Gordon.
<cite>Mechanizing Programming Logics in Higher Order Logic.</cite><BR>
University of Cambridge, Computer Laboratory, TR 145, 1988.<P>

published as<P>

Mike Gordon.
<cite>Mechanizing Programming Logics in Higher Order Logic.</cite><BR>
In
<cite>Current Trends in Hardware Verification and Automated Theorem Proving
</cite>,<BR>
edited by G. Birtwistle and P.A. Subrahmanyam, Springer-Verlag, 1989. 
<P>

At the top level, it provides a tactic <B>hoare_tac</B>, which transforms a
goal
<BLOCKQUOTE>
<KBD>{P} prog {Q}</KBD>
</BLOCKQUOTE>
into a set of HOL-level verification conditions.
<DL>
<DT>Syntax:
<DD> the letters a-z are interpreted as program variables,
     all other identifiers as mathematical variables.<P>
</DL>
The pre/post conditions can be arbitrary HOL formulae including program
variables. The program text should only refer to program variables.
<P>
<B>Note</B>: Program variables are typed in the same way as HOL
variables. Although you can write programs over arbitrary types, all
program variables in a particular program must be of the same type!
</BODY></HTML>