aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Unusedglob.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-21 22:08:07 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-21 22:08:07 +0200
commit9cc12b684ee6833971c9549aa76cc683ba931090 (patch)
treec3c602e334aea87be90e9d6b4988df225554e454 /backend/Unusedglob.v
parentb17a25bae0f9580caadfa5f795a3c12a050075f5 (diff)
downloadcompcert-kvx-9cc12b684ee6833971c9549aa76cc683ba931090.tar.gz
compcert-kvx-9cc12b684ee6833971c9549aa76cc683ba931090.zip
begin scripting the Compiler.v file
Diffstat (limited to 'backend/Unusedglob.v')
-rw-r--r--backend/Unusedglob.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/backend/Unusedglob.v b/backend/Unusedglob.v
index 93ca7af4..3b8e19ad 100644
--- a/backend/Unusedglob.v
+++ b/backend/Unusedglob.v
@@ -126,7 +126,7 @@ Fixpoint filter_globdefs (used: IS.t) (accu defs: list (ident * globdef fundef u
Definition global_defined (p: program) (pm: prog_map) (id: ident) : bool :=
match pm!id with Some _ => true | None => ident_eq id (prog_main p) end.
-Definition transform_program (p: program) : res program :=
+Definition transf_program (p: program) : res program :=
let pm := prog_defmap p in
match used_globals p pm with
| None => Error (msg "Unusedglob: analysis failed")