aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--test-suite/success/unification.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/success/unification.v b/test-suite/success/unification.v
index ddf122e85..e5b6e4159 100644
--- a/test-suite/success/unification.v
+++ b/test-suite/success/unification.v
@@ -135,4 +135,4 @@ Goal (forall (A B : Set) (f : A -> B), (fun x => f x) = f) ->
forall (A B C : Set) (g : (A -> B) -> C) (f : A -> B), g (fun x => f x) = g f.
Proof.
intros.
- rewrite H.
+ rewrite H with (f:=f0).