aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Linearize.v
diff options
context:
space:
mode:
authorxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2008-03-19 09:53:00 +0000
committerxleroy <xleroy@fca1b0fc-160b-0410-b1d3-a4f43f01ea2e>2008-03-19 09:53:00 +0000
commit22d8a1d40e38d1ca15d16fdc0aafca8d6228ecae (patch)
tree5850b2eb1d8c7b317fa3e239f4218230b188dedc /backend/Linearize.v
parentf85ac5c25d9dbefed72dda18c1d56e2391668c58 (diff)
downloadcompcert-kvx-22d8a1d40e38d1ca15d16fdc0aafca8d6228ecae.tar.gz
compcert-kvx-22d8a1d40e38d1ca15d16fdc0aafca8d6228ecae.zip
Nettoyages doc
git-svn-id: https://yquem.inria.fr/compcert/svn/compcert/trunk@566 fca1b0fc-160b-0410-b1d3-a4f43f01ea2e
Diffstat (limited to 'backend/Linearize.v')
-rw-r--r--backend/Linearize.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/backend/Linearize.v b/backend/Linearize.v
index 42330ed9..de372cc5 100644
--- a/backend/Linearize.v
+++ b/backend/Linearize.v
@@ -63,7 +63,7 @@ Open Scope error_monad_scope.
In this file, we present linearization in a way that clearly
separates the heuristic part (choosing an order for the basic blocks)
- from the actual code transformation parts. We proceed in three passes:
+ from the actual code transformation parts. We proceed in two passes:
- Choosing an order for the nodes. This returns an enumeration of CFG
nodes stating that they must be laid out in the order shown in the
list.
@@ -110,11 +110,11 @@ Definition reachable (f: LTL.function) : PMap.t bool :=
Parameter enumerate_aux: LTL.function -> PMap.t bool -> list node.
-(** Now comes the validation of an enumeration a posteriori. *)
+(** Now comes the a posteriori validation of a node enumeration. *)
Module Nodeset := FSetAVL.Make(OrderedPositive).
-(** Build a Nodeset.t from a list of nodes, checking that the list
+(** Build a [Nodeset.t] from a list of nodes, checking that the list
contains no duplicates. *)
Fixpoint nodeset_of_list (l: list node) (s: Nodeset.t)