aboutsummaryrefslogtreecommitdiffstats
path: root/driver/Compopts.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-08 11:35:17 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-08 11:35:17 +0200
commit1972df30827022dcb39110cddf9032eaa3dc61b9 (patch)
tree37a7e62cbe08675ca56d2f734104bd2d164f74e0 /driver/Compopts.v
parent66f700d36891a90983bb97d245e04a2e97913c7d (diff)
downloadcompcert-kvx-1972df30827022dcb39110cddf9032eaa3dc61b9.tar.gz
compcert-kvx-1972df30827022dcb39110cddf9032eaa3dc61b9.zip
begin installing profiling
Diffstat (limited to 'driver/Compopts.v')
-rw-r--r--driver/Compopts.v3
1 files changed, 3 insertions, 0 deletions
diff --git a/driver/Compopts.v b/driver/Compopts.v
index 848657e5..245322ef 100644
--- a/driver/Compopts.v
+++ b/driver/Compopts.v
@@ -75,6 +75,9 @@ Parameter all_loads_nontrap: unit -> bool.
(** Flag -fforward-moves. Forward moves after CSE. *)
Parameter optim_forward_moves: unit -> bool.
+(** Flag -fprofile-arcs. Add profiling logger. *)
+Parameter profile_arcs : unit -> bool.
+
(* TODO is there a more appropriate place? *)
Require Import Coqlib.
Definition time {A B: Type} (name: string) (f: A -> B) : A -> B := f.