src/HOL/README.html
author kleing
Mon, 19 Apr 2004 09:31:00 +0200
changeset 14626 dfb8d2977263
parent 14543 0e266a5dd6e3
child 15283 f21466450330
permissions -rw-r--r--
renamed HOL-Import-HOL to HOL4, added to images target

<html>

<!-- $Id$ -->

<head><title>HOL/README</title></head>

<body>

<h2>HOL: Higher-Order Logic</h2>

These are the main sources of the Isabelle system for Higher-Order Logic.

<p>

There are also several example sessions:
<dl>

<dt>Algebra
<dd>rings and univariate polynomials

<dt>Auth
<dd>a new approach to verifying authentication protocols

<dt>AxClasses
<dd>a few basic examples of using axiomatic type classes

<dt>BCV
<dd>generic model of bytecode verification, i.e. data-flow analysis
for assembly languages with subtypes

<dt>HOL-Complex
<dd>a development of the complex numbers, the reals, and the hyper-reals,
which are used in non-standard analysis (builds the image HOL-Complex)

<dt>HOL-Complex-HahnBanach
<dd>the Hahn-Banach theorem for real vector spaces (in Isabelle/Isar)

<dt>HOL-Complex-ex
<dd>miscellaneous real ans complex number examples

<dt>Hoare
<dd>verification of imperative programs (verification conditions are
generated automatically from pre/post conditions and loop invariants)

<dt>IMP
<dd>mechanization of a large part of a semantics text by Glynn Winskel

<dt>IMPP
<dd>extension of IMP with local variables and mutually recursive
procedures

<dt>IOA
<dd>a simple theory of Input/Output Automata

<dt>Induct
<dd>examples of (co)inductive definitions

<dt>Isar_examples
<dd>several introductory examples using Isabelle/Isar

<dt>Lambda
<dd>fundamental properties of lambda-calculus (Church-Rosser and termination)

<dt>Lattice
<dd>lattices and order structures (in Isabelle/Isar)

<dt>MicroJava
<dd>formalization of a fragment of Java, together with a corresponding
virtual machine and a specification of its bytecode verifier and a
lightweight bytecode verifier, including proofs of type-safety.

<dt>Modelcheck
<dd>basic setup for integration of some model checkers in Isabelle/HOL

<dt>NumberTheory
<dd>fundamental Theorem of Arithmetic, Chinese Remainder Theorem,
Fermat/Euler Theorem, Wilson's Theorem

<dt>Prolog
<dd>a (bare-bones) implementation of Lambda-Prolog

<dt>Subst
<dd>defines a theory of substitution and unification.

<dt>TLA
<dd>Lamport's Temporal Logic of Actions (with separate example sessions)

<dt>UNITY
<dd>Chandy and Misra's UNITY formalism

<dt>W0
<dd>a precursor of MiniML, without let-expressions

<dt>ex
<dd>miscellaneous examples

</dl>

Useful references on Higher-Order Logic:

<ul>

<li>P. B. Andrews,<br>
An Introduction to Mathematical Logic and Type Theory<br>
(Academic Press, 1986).

<li>A. Church,<br>
A Formulation of the Simple Theory of Types<br>
(Journal of Symbolic Logic, 1940).

<li>M. J. C. Gordon and T. F. Melham (editors),<br>
Introduction to HOL: A theorem proving environment for higher order logic<br>
(Cambridge University Press, 1993).

<li>J. Lambek and P. J. Scott,<br>
Introduction to Higher Order Categorical Logic<br>
(Cambridge University Press, 1986).

</ul>

</body>
</html>