aboutsummaryrefslogtreecommitdiffstats
path: root/backend/RTL.v
diff options
context:
space:
mode:
authorXavier Leroy <xavier.leroy@inria.fr>2015-09-15 17:31:31 +0200
committerXavier Leroy <xavier.leroy@inria.fr>2015-09-15 17:31:31 +0200
commitd35426083623b2cb659d977f3c7f73dd6de4e383 (patch)
treeca06325030c37f427d0e9cb0281bc7e2fe0121c5 /backend/RTL.v
parentde40fce9c16ced8d23389cbcfc55ef6d99466fe8 (diff)
downloadcompcert-kvx-d35426083623b2cb659d977f3c7f73dd6de4e383.tar.gz
compcert-kvx-d35426083623b2cb659d977f3c7f73dd6de4e383.zip
Isuue #50: outdated comment on type RTL.function.
Diffstat (limited to 'backend/RTL.v')
-rw-r--r--backend/RTL.v3
1 files changed, 1 insertions, 2 deletions
diff --git a/backend/RTL.v b/backend/RTL.v
index 56a5efeb..3cd4335d 100644
--- a/backend/RTL.v
+++ b/backend/RTL.v
@@ -104,8 +104,7 @@ Record function: Type := mkfunction {
for its stack-allocated activation record. [fn_params] is the list
of registers that are bound to the values of arguments at call time.
[fn_entrypoint] is the node of the first instruction of the function
- in the CFG. [fn_code_wf] asserts that all instructions of the function
- have nodes no greater than [fn_nextpc]. *)
+ in the CFG. *)
Definition fundef := AST.fundef function.