aboutsummaryrefslogtreecommitdiffstats
path: root/backend/Profiling.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-08 12:36:24 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-08 12:36:24 +0200
commit3c30567c452f030267d0fb09465adf8d7b44a90d (patch)
tree59d1eb891066a97580d83b60cdb160030d5ae114 /backend/Profiling.v
parent1972df30827022dcb39110cddf9032eaa3dc61b9 (diff)
downloadcompcert-kvx-3c30567c452f030267d0fb09465adf8d7b44a90d.tar.gz
compcert-kvx-3c30567c452f030267d0fb09465adf8d7b44a90d.zip
installed Profiling (not finished)
Diffstat (limited to 'backend/Profiling.v')
-rw-r--r--backend/Profiling.v23
1 files changed, 11 insertions, 12 deletions
diff --git a/backend/Profiling.v b/backend/Profiling.v
index 4995c507..1840af6e 100644
--- a/backend/Profiling.v
+++ b/backend/Profiling.v
@@ -4,7 +4,7 @@ Require Import Memory Registers Op RTL.
Local Open Scope positive.
-Parameter fundef_id : fundef -> Z.
+Parameter function_id : function -> Z.
Parameter branch_id : Z -> node -> Z.
Section PER_FUNCTION_ID.
@@ -47,20 +47,19 @@ Section PER_FUNCTION_ID.
| Icond cond args ifso ifnot expected => true
| _ => false
end) prog)).
-
- Definition transf_function (f : function) : function :=
- let max_pc := max_pc_function f in
- let conditions := gen_conditions (fn_code f) in
- {| fn_sig := f.(fn_sig);
- fn_params := f.(fn_params);
- fn_stacksize := f.(fn_stacksize);
- fn_code := snd (inject_l (fn_code f) (Pos.succ max_pc) conditions);
- fn_entrypoint := f.(fn_entrypoint) |}.
-
End PER_FUNCTION_ID.
+Definition transf_function (f : function) : function :=
+ let max_pc := max_pc_function f in
+ let conditions := gen_conditions (fn_code f) in
+ {| fn_sig := f.(fn_sig);
+ fn_params := f.(fn_params);
+ fn_stacksize := f.(fn_stacksize);
+ fn_code := snd (inject_l (function_id f) (fn_code f) (Pos.succ max_pc) conditions);
+ fn_entrypoint := f.(fn_entrypoint) |}.
+
Definition transf_fundef (fd: fundef) : fundef :=
- AST.transf_fundef (transf_function (fundef_id fd)) fd.
+ AST.transf_fundef transf_function fd.
Definition transf_program (p: program) : program :=
transform_program transf_fundef p.