aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init/Logic.v
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 /theories/Init/Logic.v
parenteb863af14628cd13ceb455c406937c717c8d3ee5 (diff)
Supporting "at occs" as a short-hand for "in |- * at occs" in "destruct".
Diffstat (limited to 'theories/Init/Logic.v')
-rw-r--r--theories/Init/Logic.v3
1 files changed, 1 insertions, 2 deletions
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.