aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/bteauto.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2016-06-16 14:20:10 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2016-06-16 18:21:08 +0200
commit0abade8ca36a68fbd90beb209de7647851416953 (patch)
tree8f7875f9505bb5e3d91e55d9f71786e11a8bb27c /test-suite/success/bteauto.v
parentb0c84990af22e52e659bd2469af95ad2f39a047e (diff)
Tentative fix of test-suite file to avoid loop
Looping on jenkins only, couldn't reproduce locally. To be investigated further.
Diffstat (limited to 'test-suite/success/bteauto.v')
-rw-r--r--test-suite/success/bteauto.v2
1 files changed, 0 insertions, 2 deletions
diff --git a/test-suite/success/bteauto.v b/test-suite/success/bteauto.v
index 21bb10fe1..590f6e191 100644
--- a/test-suite/success/bteauto.v
+++ b/test-suite/success/bteauto.v
@@ -58,8 +58,6 @@ Hint Cut [_* eq_trans eq_sym eq_trans] : core.
Goal forall x y z : nat, x = y -> z = y -> x = z.
Proof.
intros.
- Fail Timeout 1 eauto 10000.
-
typeclasses eauto with core.
Qed.