aboutsummaryrefslogtreecommitdiffstats
path: root/driver/Compopts.v
diff options
context:
space:
mode:
authorDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-08 17:02:45 +0200
committerDavid Monniaux <david.monniaux@univ-grenoble-alpes.fr>2020-04-08 17:02:45 +0200
commitc3f5f3dbd088091e3fab9f357b01693932d148f8 (patch)
treefee361b1e1cc616a1b9c412ae5cec7c9467dcf32 /driver/Compopts.v
parent96165dbec88ab4c951d99e64e51f5c55a1244137 (diff)
downloadcompcert-kvx-c3f5f3dbd088091e3fab9f357b01693932d148f8.tar.gz
compcert-kvx-c3f5f3dbd088091e3fab9f357b01693932d148f8.zip
reloading and exploiting seems to work
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 245322ef..98cbcc37 100644
--- a/driver/Compopts.v
+++ b/driver/Compopts.v
@@ -78,6 +78,9 @@ Parameter optim_forward_moves: unit -> bool.
(** Flag -fprofile-arcs. Add profiling logger. *)
Parameter profile_arcs : unit -> bool.
+(** Flag -fbranch_probabilities. Use profiling information if available *)
+Parameter branch_probabilities : 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.