aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2017-12-18 18:57:34 +0100
committerGravatar Maxime Dénès <mail@maximedenes.fr>2017-12-18 18:57:34 +0100
commit6af0969228e57c611e5a0876efe613055de342cd (patch)
treecfeb33115bb53bc41c588cf75dc70ef515eceff9 /test-suite
parent3690e568a36f8b418ec9c253a3188403f53021ba (diff)
parent6734614d8ace6860e3deb1861611ba4b012cfae1 (diff)
Merge PR #6380: Add tactics to reset and display the Ltac profile
Diffstat (limited to 'test-suite')
-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.