diff options
author | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2009-01-18 18:01:12 +0000 |
---|---|---|
committer | msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7> | 2009-01-18 18:01:12 +0000 |
commit | 05b31844f683c3bc81b371c94be5cc6f6f4edf61 (patch) | |
tree | ea983b637b98a8971b5ae978abc48228814b200b /theories | |
parent | cb738f93e74b2d11bc5a67e75cf5f6f07e676d77 (diff) |
Various little fixes:
- allow a new line after a (** printing *) directive in coqdoc so as not
to output spurious new lines.
- never directly unify the lemma with an evar in setoid_rewrite (they
act as opaque constants).
- Fix a useless dependency introduced by tauto which splits a record in
SetoidList.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11799 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r-- | theories/Lists/SetoidList.v | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Lists/SetoidList.v b/theories/Lists/SetoidList.v index 886c95aad..aed4a3bca 100644 --- a/theories/Lists/SetoidList.v +++ b/theories/Lists/SetoidList.v @@ -687,7 +687,7 @@ destruct (eqA_dec x a). left; auto. destruct IHl. left; auto. -right; red; inversion_clear 1; tauto. +right; red; inversion_clear 1; contradiction. Qed. Fixpoint removeA (x : A) (l : list A){struct l} : list A := |