aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Init
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-02 22:11:54 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-02 22:23:20 +0100
commit844431761eaaf0c42d7daf3ae21de731aa230eee (patch)
tree1ad54331eb08d2b860bfaa1ae95e6a08ecec2771 /theories/Init
parent4df1ddc6d6bd0707396337869b663b4c8f930f60 (diff)
Improving elimination with indices, getting rid of intrusive residual
local definitions...
Diffstat (limited to 'theories/Init')
-rw-r--r--theories/Init/Logic.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Init/Logic.v b/theories/Init/Logic.v
index a7ed3c7f7..a7a1fd97c 100644
--- a/theories/Init/Logic.v
+++ b/theories/Init/Logic.v
@@ -483,7 +483,7 @@ Proof.
destruct (eq_id_comm_l f Hfsymf (f a)).
destruct (eq_id_comm_l f Hfsymf a).
unfold Hfsymf.
- destruct (Hf a). simpl. unfold a0; clear a0.
+ destruct (Hf a). simpl.
rewrite eq_trans_refl_l.
reflexivity.
Defined.