# HG changeset patch
# User nipkow
# Date 1115052412 -7200
# Node ID 5df57194d064bed5916095e3069d4af5f5e34f6e
# Parent 5f0c8a3f022654caa0a3a148e6cb72c63f460bfd
*** empty log message ***
diff -r 5f0c8a3f0226 -r 5df57194d064 src/HOL/README.html
--- a/src/HOL/README.html Mon May 02 18:29:29 2005 +0200
+++ b/src/HOL/README.html Mon May 02 18:46:52 2005 +0200
@@ -29,24 +29,21 @@
AxClasses
a few basic examples of using axiomatic type classes
-BCV
-generic model of bytecode verification, i.e. data-flow analysis
-for assembly languages with subtypes
-
-HOL-Complex
+Complex
a development of the complex numbers, the reals, and the hyper-reals,
which are used in non-standard analysis (builds the image HOL-Complex)
-HOL-Complex-HahnBanach
-the Hahn-Banach theorem for real vector spaces (in Isabelle/Isar)
-
-HOL-Complex-ex
-miscellaneous real ans complex number examples
-
Hoare
verification of imperative programs (verification conditions are
generated automatically from pre/post conditions and loop invariants)
+HoareParallel
+verification of shared-variable imperative programs a la Owicki-Gries.
+(verification conditions are generated automatically)
+
+Hyperreal
+Nonstandard analysis. Builds on Real and is part of Complex.
+
IMP
mechanization of a large part of a semantics text by Glynn Winskel
@@ -54,12 +51,15 @@
extension of IMP with local variables and mutually recursive
procedures
-IOA
-a simple theory of Input/Output Automata
+Import
+theories imported from other (HOL) theorem provers.
Induct
examples of (co)inductive definitions
+IOA
+a simple theory of Input/Output Automata
+
Isar_examples
several introductory examples using Isabelle/Isar
@@ -69,23 +69,41 @@
Lattice
lattices and order structures (in Isabelle/Isar)
+Library
+A collection of generic theories
+
+Matrix
+two-dimensional matrices
+
MicroJava
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.
+lightweight bytecode verifier, including proofs of type-safety
Modelcheck
basic setup for integration of some model checkers in Isabelle/HOL
+NanoJava
+Haore Logic for a tiny fragment of Java
+
NumberTheory
fundamental Theorem of Arithmetic, Chinese Remainder Theorem,
-Fermat/Euler Theorem, Wilson's Theorem
+Fermat/Euler Theorem, Wilson's Theorem, Quadratic Reciprocity
Prolog
a (bare-bones) implementation of Lambda-Prolog
+Real
+the real numbers, part of Complex
+
+Real/HahnBanach
+the Hahn-Banach theorem for real vector spaces (in Isabelle/Isar)
+
+SET-Protocol
+verification of the SET Protocol
+
Subst
-defines a theory of substitution and unification.
+a theory of substitution and unification.
TLA
Lamport's Temporal Logic of Actions (with separate example sessions)