diff options
author | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2008-04-27 11:16:15 +0000 |
---|---|---|
committer | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2008-04-27 11:16:15 +0000 |
commit | e961ace331ec961dcec0e2525d7b9142d04b5154 (patch) | |
tree | 08ffca7a4fdb28b5a79f3409d8478deecb099c3d /theories/Lists | |
parent | fc10282837971f8f0648841d944dd64b11d3a3db (diff) |
- Fix bug in unification not taking into account the right meta
substitution. Makes unification succeed a bit more often, hence auto
works better in some cases.
- Backtrack the changes of auto using Hint Unfold to do more delta and add
a new tactic "new auto" which does that, for compatibility.
The first fix may have a big impact on the contribs, whereas the second
should make them compile again... we'll see.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10855 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists')
-rw-r--r-- | theories/Lists/List.v | 4 |
1 files changed, 1 insertions, 3 deletions
diff --git a/theories/Lists/List.v b/theories/Lists/List.v index 5ab27cfc7..78a2db534 100644 --- a/theories/Lists/List.v +++ b/theories/Lists/List.v @@ -686,8 +686,7 @@ Section ListOps. rewrite app_nth1; auto. rewrite (minus_plus_simpl_l_reverse (length l) n 1). replace (1 + length l) with (S (length l)); auto with arith. - rewrite <- minus_Sn_m; auto with arith; simpl. - apply IHl; auto. + rewrite <- minus_Sn_m; auto with arith. rewrite rev_length; auto. Qed. @@ -1363,7 +1362,6 @@ End Fold_Right_Recursor. destruct n; destruct d; simpl; auto. destruct a; destruct (split l); simpl; auto. destruct a; destruct (split l); simpl in *; auto. - rewrite IHl; simpl; auto. Qed. Lemma split_length_l : forall (l:list (A*B)), |