aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-02-23 11:20:26 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2018-02-28 19:44:38 +0100
commitaa95d82692684a416d7a1c25fce38b4eca1e49c9 (patch)
treebd595bb73c79052cab616e9d75f1a24590dadc5e /theories
parentccb7bd2948e9bd84997f3461257b2ce1c7ad3e6a (diff)
Uniform spacing layout in Tactics.v.
Diffstat (limited to 'theories')
-rw-r--r--theories/Init/Tactics.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/theories/Init/Tactics.v b/theories/Init/Tactics.v
index 287b44fd0..c36494c9e 100644
--- a/theories/Init/Tactics.v
+++ b/theories/Init/Tactics.v
@@ -253,6 +253,7 @@ Tactic Notation "dependent" "induction" ident(H) :=
writing a version of [inversion] / [dependent destruction] which
does not lose information, i.e., does not turn a goal which is
provable into one which requires axiom K / UIP. *)
+
Ltac simpl_proj_exist_in H :=
repeat match type of H with
| context G[proj1_sig (exist _ ?x ?p)]
@@ -308,6 +309,7 @@ Ltac inversion_sigma_step :=
Ltac inversion_sigma := repeat inversion_sigma_step.
(** A version of [time] that works for constrs *)
+
Ltac time_constr tac :=
let eval_early := match goal with _ => restart_timer end in
let ret := tac () in