aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/MSets
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-04-07 19:21:05 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-05-06 09:58:59 +0200
commit4cb7fe525a472928aee02d772458d28a2b71072a (patch)
tree5934260488727e9c06871ce775376535c252f721 /theories/MSets
parent2d6de8b102ea3cd05c5d193190faf787ccb84baa (diff)
- Fix arity handling in retyping (de Bruijn bug!)
- Enforce that no u <= Prop/Set can be added for u introduced by the user in Evd.process_constraints. (Needs to be enforced in the kernel as well, but that's the main entry point). - Fix a test-suite script and remove a regression comment, it's just as before now.
Diffstat (limited to 'theories/MSets')
-rw-r--r--theories/MSets/MSetGenTree.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/MSets/MSetGenTree.v b/theories/MSets/MSetGenTree.v
index 6164e6e93..2ec125427 100644
--- a/theories/MSets/MSetGenTree.v
+++ b/theories/MSets/MSetGenTree.v
@@ -962,7 +962,7 @@ Proof. firstorder. Qed.
Lemma eq_Leq : forall s s', eq s s' <-> L.eq (elements s) (elements s').
Proof.
unfold eq, Equal, L.eq; intros.
- do 2 setoid_rewrite elements_spec1. (*FIXME due to regression in rewrite *)
+ setoid_rewrite elements_spec1.
firstorder.
Qed.