aboutsummaryrefslogtreecommitdiffstats
path: root/backend/LICM.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-01 14:45:25 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-01 14:45:25 +0200
commita3d40b88608b8b5e7e615346ea1c33198355cbbc (patch)
tree1c8b4c022d94ff4dfd164aaf4bfa738a6b5828ba /backend/LICM.v
parent6379f6291eea909426f074db67837b04a1dec9ae (diff)
downloadcompcert-kvx-a3d40b88608b8b5e7e615346ea1c33198355cbbc.tar.gz
compcert-kvx-a3d40b88608b8b5e7e615346ea1c33198355cbbc.zip
clearer types
Diffstat (limited to 'backend/LICM.v')
-rw-r--r--backend/LICM.v5
1 files changed, 4 insertions, 1 deletions
diff --git a/backend/LICM.v b/backend/LICM.v
index 1b5334ba..d45eef43 100644
--- a/backend/LICM.v
+++ b/backend/LICM.v
@@ -6,4 +6,7 @@ Require Inject.
Definition gen_injections (f : function) (max_pc : node) (max_reg : reg):
PTree.t (list Inject.inj_instr) := PTree.empty (list Inject.inj_instr).
-Definition transf_program := Inject.transf_program gen_injections.
+Opaque gen_injections.
+
+Definition transf_program : program -> res program :=
+ Inject.transf_program gen_injections.