aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-02 17:02:32 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-02 19:58:03 +0100
commit78717e3cdc53fda4f41bfa41f13872083413abc0 (patch)
tree2e69726fd968a34c03f88a99d7f4207cd6c77d99
parenteb863af14628cd13ceb455c406937c717c8d3ee5 (diff)
Supporting "at occs" as a short-hand for "in |- * at occs" in "destruct".
-rw-r--r--parsing/g_tactic.ml44
-rw-r--r--theories/Init/Logic.v3
2 files changed, 4 insertions, 3 deletions
diff --git a/parsing/g_tactic.ml4 b/parsing/g_tactic.ml4
index a57720755..e6f2af32b 100644
--- a/parsing/g_tactic.ml4
+++ b/parsing/g_tactic.ml4
@@ -395,7 +395,9 @@ GEXTEND Gram
| -> {onhyps=None; concl_occs=AllOccurrences} ] ]
;
opt_clause:
- [ [ "in"; cl = in_clause -> Some cl | -> None ] ]
+ [ [ "in"; cl = in_clause -> Some cl
+ | "at"; occs = occs_nums -> Some {onhyps=Some[]; concl_occs=occs}
+ | -> None ] ]
;
concl_occ:
[ [ "*"; occs = occs -> occs
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index 6e8a405e0..a7ed3c7f7 100644
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -467,8 +467,7 @@ Proof.
intros.
unfold f_equal.
rewrite <- (eq_trans_sym_inv_l (Hf a)).
- pattern (f a) at 1 2 3 4 5 7 8, (Hf a) at 1 2.
- destruct (Hf a).
+ destruct (Hf a) at 1 2.
destruct (Hf a).
reflexivity.
Defined.