aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/6378.v
diff options
context:
space:
mode:
authorGravatar Jason Gross <jgross@mit.edu>2017-12-11 02:23:10 -0500
committerGravatar Jason Gross <jgross@mit.edu>2017-12-14 12:05:50 -0500
commit40aca595dd8e26373bfa4f6b6d4cd7d43a933210 (patch)
tree3fef33ca12ba2bab8ce0efacf6cec6f640b3497c /test-suite/bugs/closed/6378.v
parentb270ad686075e5579dc3826fafdc324ea339785c (diff)
Add tactics to reset and display the Ltac profile
This is useful for tactics that run a bunch of tests and need to display the profile for each of them.
Diffstat (limited to 'test-suite/bugs/closed/6378.v')
-rw-r--r--test-suite/bugs/closed/6378.v14
1 files changed, 14 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/6378.v b/test-suite/bugs/closed/6378.v
index d0ef090d0..68ae7961d 100644
--- a/test-suite/bugs/closed/6378.v
+++ b/test-suite/bugs/closed/6378.v
@@ -1,4 +1,18 @@
+Require Import Coq.ZArith.ZArith.
+Ltac profile_constr tac :=
+ let dummy := match goal with _ => reset ltac profile; start ltac profiling end in
+ let ret := match goal with _ => tac () end in
+ let dummy := match goal with _ => stop ltac profiling; show ltac profile end in
+ pose 1.
+
+Ltac slow _ := eval vm_compute in (Z.div_eucl, Z.div_eucl, Z.div_eucl, Z.div_eucl, Z.div_eucl).
+
Goal True.
start ltac profiling.
+ reset ltac profile.
+ reset ltac profile.
stop ltac profiling.
+ time profile_constr slow.
+ show ltac profile cutoff 0.
+ show ltac profile "slow".
Abort.