aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--theories/Lists/PolyList.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Lists/PolyList.v b/theories/Lists/PolyList.v
index 9638d4a21..00983c1cf 100644
--- a/theories/Lists/PolyList.v
+++ b/theories/Lists/PolyList.v
@@ -561,7 +561,7 @@ Save.
Lemma in_prod : (A:Set)(B:Set)(l:(list A))(l':(list B))
(x:A)(y:B)(In x l)->(In y l')->(In (x,y) (list_prod l l')).
Induction l;
-[ Simpl; Tauto
+[ Tauto
| Simpl; Intros; Apply in_or_app; Elim H0; Clear H0;
[ Left; Rewrite H0; Apply in_prod_aux; Assumption
| Right; Auto]