From 215bbe5cddc7fae276fe50131dcff70bc1b7f6d9 Mon Sep 17 00:00:00 2001 From: msozeau Date: Wed, 5 Nov 2008 20:42:15 +0000 Subject: Port [rewrite] tactics to open terms. Currently no check that evars introduced by the lemma remain in the subgoals (i.e. it's really [erewrite]). git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11544 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/FSets/FSetEqProperties.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/FSets') diff --git a/theories/FSets/FSetEqProperties.v b/theories/FSets/FSetEqProperties.v index 41034ce85..9d47ef72c 100644 --- a/theories/FSets/FSetEqProperties.v +++ b/theories/FSets/FSetEqProperties.v @@ -73,7 +73,7 @@ Qed. Lemma is_empty_equal_empty: is_empty s = equal s empty. Proof. apply bool_1; split; intros. -rewrite <- (empty_is_empty_1 (s:=empty)); auto with set. +auto with set. rewrite <- is_empty_iff; auto with set. Qed. -- cgit v1.2.3