From 84cbc09bd1400f732a6c70e8a840e4c13d018478 Mon Sep 17 00:00:00 2001 From: Matthieu Sozeau Date: Thu, 17 Oct 2013 14:55:57 +0200 Subject: Correct rebase on STM code. Thanks to E. Tassi for help on dealing with latent universes. Now the universes in the type of a definition/lemma are eagerly added to the environment so that later proofs can be checked independently of the original (delegated) proof body. - Fixed firstorder, ring to work correctly with universe polymorphism. - Changed constr_of_global to raise an anomaly if side effects would be lost by turning a polymorphic constant into a constr. - Fix a non-termination issue in solve_evar_evar. - --- theories/MSets/MSetGenTree.v | 3 ++- 1 file changed, 2 insertions(+), 1 deletion(-) (limited to 'theories/MSets') diff --git a/theories/MSets/MSetGenTree.v b/theories/MSets/MSetGenTree.v index 3142d97ca..6164e6e93 100644 --- a/theories/MSets/MSetGenTree.v +++ b/theories/MSets/MSetGenTree.v @@ -962,7 +962,8 @@ 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. - setoid_rewrite elements_spec1; firstorder. + do 2 setoid_rewrite elements_spec1. (*FIXME due to regression in rewrite *) + firstorder. Qed. Definition lt (s1 s2 : tree) : Prop := -- cgit v1.2.3