aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Lists/SetoidList.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-05-23 18:17:38 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-05-23 18:17:38 +0000
commitc0f26dd0ebae4bad9a8850a198f0126ea4656e73 (patch)
tree9e35faa7547ec7061d6c9b523b700046c7d80043 /theories/Lists/SetoidList.v
parent582b5147cb79267ce79c03718cb3575826dc831c (diff)
Changement de précédence de l'argument du by de assert; conséquences sur les .v
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@8853 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Lists/SetoidList.v')
-rw-r--r--theories/Lists/SetoidList.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/theories/Lists/SetoidList.v b/theories/Lists/SetoidList.v
index f9b28be3a..76d6ff112 100644
--- a/theories/Lists/SetoidList.v
+++ b/theories/Lists/SetoidList.v
@@ -160,7 +160,7 @@ Proof.
inversion_clear H0.
constructor; auto.
intro.
- assert (ltA x x) by eapply SortA_InfA_InA; eauto.
+ assert (ltA x x) by (eapply SortA_InfA_InA; eauto).
elim (ltA_not_eqA H3); auto.
Qed.
@@ -330,11 +330,11 @@ destruct (H3 y); clear H3.
destruct H6; intuition.
swap H4; apply InA_eqA with y; auto.
destruct H0.
-assert (InA y (x' :: s')) by rewrite H3; auto.
+assert (InA y (x' :: s')) by (rewrite H3; auto).
inversion_clear H6; auto.
elim H1; apply eqA_trans with y; auto.
destruct H0.
-assert (InA y (x' :: s')) by rewrite H3; auto.
+assert (InA y (x' :: s')) by (rewrite H3; auto).
inversion_clear H7; auto.
elim H6; auto.
Qed.