aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output-modulo-time/ltacprof.v
blob: d79451f0f79171c16042c1e647b8903deef24180 (plain)
1
2
3
4
5
6
7
8
(* -*- coq-prog-args: ("-emacs" "-profile-ltac") -*- *)
Ltac sleep' := do 100 (do 100 (do 100 idtac)).
Ltac sleep := sleep'.

Theorem x : True.
Proof.
  idtac. idtac. sleep. constructor.
Defined.