aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Structures
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 22:13:03 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 22:13:03 +0200
commit18512ba12400e30858ae19e5ef69b9590b96de06 (patch)
treed85d73110a1eb95b8873375cee0bd35821996657 /theories/Structures
parent3011cbfb224b3b2dfb72afd05094614b97a2128b (diff)
Revert "Temporary hack to compensate missing comma while re-printing tactic"
Diffstat (limited to 'theories/Structures')
-rw-r--r--theories/Structures/EqualitiesFacts.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Structures/EqualitiesFacts.v b/theories/Structures/EqualitiesFacts.v
index ece8db5b7..cee3d63f0 100644
--- a/theories/Structures/EqualitiesFacts.v
+++ b/theories/Structures/EqualitiesFacts.v
@@ -110,7 +110,7 @@ Module KeyDecidableType(D:DecidableType).
unfold In, MapsTo.
setoid_rewrite Exists_exists; setoid_rewrite InA_alt.
firstorder.
- exists (snd x); exists x; auto.
+ exists (snd x), x; auto.
Qed.
Lemma In_nil {elt} k : In k (@nil (key*elt)) <-> False.