aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/complexity/injection.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/complexity/injection.v')
-rw-r--r--test-suite/complexity/injection.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/complexity/injection.v b/test-suite/complexity/injection.v
index eb01133e7..db2d9c53f 100644
--- a/test-suite/complexity/injection.v
+++ b/test-suite/complexity/injection.v
@@ -110,4 +110,4 @@ Lemma test: forall n1 w1 n2 w2, mk_world n1 w1 = mk_world n2 w2 ->
n1 = n2.
Proof.
intros.
-Time injection H.
+Timeout 10 Time injection H.