aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Relations
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-07 18:41:42 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-07 18:41:42 +0000
commitf0c4286a9edf07d3638742257b8c39487e47d44a (patch)
tree3f4314d1244df441a10c5d02a1887015ca570b13 /theories/Relations
parente5643982202eeddf2c4fb7808d5c530a87009e89 (diff)
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
Diffstat (limited to 'theories/Relations')
-rwxr-xr-xtheories/Relations/Relations.v2
1 files changed, 1 insertions, 1 deletions
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)