From 89dad2d42af874babb1e3179607aca3b92377616 Mon Sep 17 00:00:00 2001 From: xleroy Date: Mon, 5 Mar 2007 08:56:59 +0000 Subject: Commentaires git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@184 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e --- lib/Lattice.v | 8 ++++---- 1 file changed, 4 insertions(+), 4 deletions(-) (limited to 'lib/Lattice.v') 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. -- cgit