aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Relations
diff options
context:
space:
mode:
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)