aboutsummaryrefslogtreecommitdiffstats
path: root/lib/Lattice.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2007-03-05 08:56:59 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2007-03-05 08:56:59 +0000
commit89dad2d42af874babb1e3179607aca3b92377616 (patch)
tree658b6179e39a23b504fe673de34ab34d56d6bf2c /lib/Lattice.v
parent4d0036dbe756e00627b7185ce8a69984405e062c (diff)
downloadcompcert-kvx-89dad2d42af874babb1e3179607aca3b92377616.tar.gz
compcert-kvx-89dad2d42af874babb1e3179607aca3b92377616.zip
Commentaires
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@184 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'lib/Lattice.v')
-rw-r--r--lib/Lattice.v8
1 files changed, 4 insertions, 4 deletions
diff --git a/lib/Lattice.v b/lib/Lattice.v
index 7ef1b9e1..f796367d 100644
--- a/lib/Lattice.v
+++ b/lib/Lattice.v
@@ -6,10 +6,10 @@ Require Import FSets.
(** * Signatures of semi-lattices *)
-(** A semi-lattice is a type [t] equipped with a decidable equality [eq],
- a partial order [ge], a smallest element [bot], and an upper
- bound operation [lub]. Note that we do not demand that [lub] computes
- the least upper bound. *)
+(** A semi-lattice is a type [t] equipped with an equivalence relation [eq],
+ a boolean equivalence test [beq], a partial order [ge], a smallest element
+ [bot], and an upper bound operation [lub].
+ Note that we do not demand that [lub] computes the least upper bound. *)
Module Type SEMILATTICE.