aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar delahaye <delahaye@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-24 00:42:52 +0000
committerGravatar delahaye <delahaye@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-24 00:42:52 +0000
commit2e68487cf52e6a853cdd61bce22e7836afdd3821 (patch)
tree3deff16b72cec5bfb841ecd38930ff12f5a1c9a5 /theories
parentb8949a0d69b5d7b2cf8759e5c4580ae0bb6a73fa (diff)
Petite simplif due au nouveau Tauto
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@939 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-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]