aboutsummaryrefslogtreecommitdiffstats
path: root/driver/Compopts.v
diff options
context:
space:
mode:
Diffstat (limited to 'driver/Compopts.v')
-rw-r--r--driver/Compopts.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/driver/Compopts.v b/driver/Compopts.v
index 9c6448b7..4f86901b 100644
--- a/driver/Compopts.v
+++ b/driver/Compopts.v
@@ -62,3 +62,7 @@ Parameter thumb: unit -> bool.
(** Flag -g. For insertion of debugging information. *)
Parameter debug: 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.