src/HOL/TLA/README.html
author nipkow
Mon, 09 Feb 1998 14:40:59 +0100
changeset 4612 26764de50c74
parent 3849 3ea10bfd329d
child 5383 74c2da44d144
permissions -rw-r--r--
Used THEN_ALL_NEW.

<HTML><HEAD><TITLE>HOL/TLA/README</TITLE></HEAD><BODY bgcolor="white">

<H3>TLA: A formalization of TLA in HOL</H3>

Author:     Stephan Merz<BR>
Copyright   1997 Universit&auml;t M&uuml;nchen<P>

The distribution contains a representation of Lamport's
<A HREF="http://www.research.digital.com/SRC/personal/Leslie_Lamport/tla/tla.html">
Temporal Logic of Actions</A>
in Isabelle/HOL.

<p>

The encoding is mainly oriented towards practical verification
examples. It does not contain a formalization of TLA's semantics,
although it could be an interesting exercise to add such a formalization
to the existing representation. Instead, it is based on a 
<A HREF="http://www4.informatik.tu-muenchen.de/~merz/papers/ptla.ps">complete axiomatization</A>
of the "raw" (stuttering-sensitive) variant of propositional TLA. 
There is also a
<A HREF="http://www4.informatik.tu-muenchen.de/~merz/papers/IsaTLADesign.ps">design note</A> 
that explains the basic setup and use of the prover.

<p>

The distribution includes the following examples:
<UL>
  <li> a verification of Lamport's <quote>increment</quote> example
  (subdirectory inc),<P>

  <li> a proof that two buffers in a row implement a single buffer
  (subdirectory buffer), and<P>

   <li> the verification of Broy and Lamport's RPC-Memory example. For details see:<BR>

        Mart&iacute;n Abadi, Leslie Lamport, and Stephan Merz: 
        <A HREF="http://www4.informatik.tu-muenchen.de/~merz/papers/RPCMemory.html">
        A TLA Solution to the RPC-Memory Specification Problem</A>.
        In: <i>Formal System Specification</i>, LNCS 1169, 1996, 21-69.
</UL>

If you use Isabelle/TLA and have any comments, suggestions or contributions,
please contact <A HREF="mailto:merz@informatik.uni-muenchen.de">Stephan Merz</A>.

</BODY></HTML>