aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Structures
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-13 14:38:26 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2016-04-27 21:55:48 +0200
commit3a2753bedf43a8c7306b1b3fc9cb37aafb78ad7a (patch)
tree4bf6607f8a29238bac0d87775d74f2105a1b9384 /theories/Structures
parent8c74d3e5578caeb5c62ba462528d9972c1de17f1 (diff)
Temporary hack to compensate missing comma while re-printing tactic
"exists c1, c2".
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 cee3d63f0..ece8db5b7 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), x; auto.
+ exists (snd x); exists x; auto.
Qed.
Lemma In_nil {elt} k : In k (@nil (key*elt)) <-> False.