summaryrefslogtreecommitdiff
path: root/test-suite/bugs/opened/shouldnotfail/1338.v-disabled
blob: f383d534407c927639515d73238d11001d68e150 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
Require Import Omega.

Goal forall x, 0 <= x -> x <= 20 -> 
x <> 0  
  -> x <> 1 -> x <> 2 -> x <> 3 -> x <>4 -> x <> 5 -> x <> 6 -> x <> 7 -> x <> 8
-> x <> 9 -> x <> 10 
  -> x <> 11 -> x <> 12 -> x <> 13 -> x <> 14 -> x <> 15 -> x <> 16 -> x <> 17
-> x <> 18 -> x <> 19 -> x <> 20 -> False.
Proof.
  intros.
  omega.
Qed.