From 76adb57c72fccb4f3e416bd7f3927f4fff72178b Mon Sep 17 00:00:00 2001 From: Hugo Herbelin Date: Sun, 1 Jun 2014 10:26:26 +0200 Subject: Making those proofs which depend on names generated for the arguments in Prop of constructors of inductive types independent of these names. Incidentally upgraded/simplified a couple of proofs, mainly in Reals. This prepares to the next commit about using names based on H for such hypotheses in Prop. --- theories/MSets/MSetWeakList.v | 4 ++-- 1 file changed, 2 insertions(+), 2 deletions(-) (limited to 'theories/MSets') diff --git a/theories/MSets/MSetWeakList.v b/theories/MSets/MSetWeakList.v index 9743e358f..372acd56a 100644 --- a/theories/MSets/MSetWeakList.v +++ b/theories/MSets/MSetWeakList.v @@ -217,10 +217,10 @@ Module MakeRaw (X:DecidableType) <: WRawSets X. Proof. induction s; simpl; intros. intuition; inv; auto. - destruct X.eq_dec; inv; rewrite !InA_cons, ?IHs; intuition. + destruct X.eq_dec as [|Hnot]; inv; rewrite !InA_cons, ?IHs; intuition. elim H. setoid_replace a with y; eauto. elim H3. setoid_replace x with y; eauto. - elim n. eauto. + elim Hnot. eauto. Qed. Global Instance remove_ok s x `(Ok s) : Ok (remove x s). -- cgit v1.2.3