From f0c4286a9edf07d3638742257b8c39487e47d44a Mon Sep 17 00:00:00 2001 From: herbelin Date: Mon, 7 Apr 2003 18:41:42 +0000 Subject: Nommage explicite des hypotheses introduites quand le nom existe aussi comme global git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3861 85f007b7-540e-0410-9357-904b9bb8a0f7 --- theories/Relations/Relations.v | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) (limited to 'theories/Relations') diff --git a/theories/Relations/Relations.v b/theories/Relations/Relations.v index 86627c8b3..f792e4c2a 100755 --- a/theories/Relations/Relations.v +++ b/theories/Relations/Relations.v @@ -15,7 +15,7 @@ Require Export Operators_Properties. Lemma inverse_image_of_equivalence : (A,B:Set)(f:A->B) (r:(relation B))(equivalence B r)->(equivalence A [x,y:A](r (f x) (f y))). Intros; Split; Elim H; Red; Auto. -Intros; Apply equiv_trans with (f y); Assumption. +Intros _ equiv_trans _ x y z H0 H1; Apply equiv_trans with (f y); Assumption. Qed. Lemma inverse_image_of_eq : (A,B:Set)(f:A->B) -- cgit v1.2.3