From e1e0f4f7f3c549fd3d5677b67c6b13ed687e6f12 Mon Sep 17 00:00:00 2001 From: Hugo Herbelin Date: Tue, 3 Jun 2014 17:15:40 +0200 Subject: Make standard library independent of the names generated by induction/elim over a dependent elimination principle for Prop arguments. --- theories/MSets/MSetEqProperties.v | 3 +-- 1 file changed, 1 insertion(+), 2 deletions(-) (limited to 'theories/MSets') diff --git a/theories/MSets/MSetEqProperties.v b/theories/MSets/MSetEqProperties.v index 843b9aaa7..ae20edc87 100644 --- a/theories/MSets/MSetEqProperties.v +++ b/theories/MSets/MSetEqProperties.v @@ -819,8 +819,7 @@ Proof. intros. rewrite for_all_exists in H; auto. rewrite negb_true_iff in H. -elim (@for_all_mem_4 (fun x =>negb (f x)) Comp' s);intros;auto. -elim p;intros. +destruct (@for_all_mem_4 (fun x =>negb (f x)) Comp' s) as (x,[]); auto. exists x;split;auto. rewrite <-negb_false_iff; auto. Qed. -- cgit v1.2.3