aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-08-01 14:39:51 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-08-05 19:52:20 +0200
commit99be46eb50213d1f35dfc4d30f35760ad5e75621 (patch)
tree9893c47cf1778fdeede3c2f6e1ec13539ca9ca14 /theories/Lists
parent69aff8116b4878671daf73cc7ccf713aac0c0e6d (diff)
More proofs independent of the names generated by induction/elim over
a dependent elimination principle for Prop arguments.
Diffstat (limited to 'theories/Lists')
-rw-r--r--theories/Lists/ListSet.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Lists/ListSet.v b/theories/Lists/ListSet.v
index 03c2222aa..f02c1d13f 100644
--- a/theories/Lists/ListSet.v
+++ b/theories/Lists/ListSet.v
@@ -116,7 +116,7 @@ Section first_definitions.
simple induction x; simpl; intros.
apply H0; red; trivial.
case (Aeq_dec a a0); auto with datatypes.
- intro; apply H; intros; auto.
+ intro Hneg; apply H; intros; auto.
apply H1; red; intro.
case H3; auto.
Qed.