TLA: A formalization of TLA in HOL
Author: Stephan Merz
Copyright 1997 Universität München
The distribution contains a representation of Lamport's
Temporal Logic of Actions
in Isabelle/HOL.
The encoding is mainly oriented towards practical verification
examples. It does not contain a formalization of TLA's semantics;
instead, it is based on a
complete axiomatization of the "raw"
(stuttering-sensitive) variant of propositional TLA. It is
accompanied by a
design note that explains the basic
setup and use of the prover.
The distribution includes the following examples:
- a verification of Lamport's
increment
example
(subdirectory inc),
- a proof that two buffers in a row implement a single buffer
(subdirectory buffer), and
- the verification of Broy and Lamport's RPC-Memory example. For details see:
Martín Abadi, Leslie Lamport, and Stephan Merz:
A TLA Solution to the RPC-Memory Specification Problem.
In: Formal System Specification, LNCS 1169, 1996, 21-69.
If you use Isabelle/TLA and have any comments, suggestions or contributions,
please contact Stephan Merz.