-
QF_BV/spear/wget_v1.10.2/src_wget_vc18197.smt2 smt2_eval_CVC4 FAIL
QF_BV/spear/wget_v1.10.2/src_wget_vc18755.smt2 smt2_eval_CVC4 FAIL
QF_BV/spear/wget_v1.10.2/src_wget_vc18756.smt2 smt2_eval_CVC4 FAIL…
-
This is related to #53. Here are some goals that are not solved by `cvc4` but produce simple subgoals:
```
From SMTCoq Require Import SMTCoq.
Require Import ZArith.
Notation "a ==? b" := (@eqb…
rafoo updated
2 years ago
-
Issuing:
`brew install cvc4/cvc4/cvc4 --HEAD --with-java-bindings`
ends up in failure with:
```
bash
-c
source /private/tmp/cvc4-20200727-69733-71pi7c/venv/bin/activate && ./configure.sh -…
-
[Installation instructions](https://github.com/ucsd-progsys/liquidhaskell/blob/develop/INSTALL.md) say that at least _one of_ `Z3`, `CVC4` or `MathSat` is required.
However, according to issue #131…
-
```coq
Require Import SMTCoq.SMTCoq.
Goal forall b1 b2, b1 = true -> b2 = true -> b1 = b2.
cvc4.
(* Error:
In nested Ltac calls to "cvc4" and "cvc4_bool", last call failed.
CVC4 returned sat…
-
For this formula, CVC4 without fmf-bound gives a result quickly, while CVC4 hangs using fmf-bound. It is likely a performance issue.
```
[581] % time cvc4 -q small.smt2
unsat
real 0m0.087s
user…
-
cryptol has the ability to `:set prover=any`. For the same reason that exists, it would be good to have multiple parallel solvers supported in saw. I'm not sure if it would be possible to have a par…
TomMD updated
4 weeks ago
-
My test file `Test.lhs` looks like this:
```
> module Test where
> {-@ hanoi :: Nat -> Nat @-}
> hanoi :: Int -> Int
> hanoi n | n == 1 = 1
> | otherwise = 2 * (hanoi (n - 1)) + 1
```…
-
Should the `nat_convert` tactic convert inequalities to boolean equalities that CVC4 understands? I can't find a way to solve this goal.
```coq
Goal forall a b c : nat,
a + b < c ->
b < …
-
```coq
Require Import SMTCoq.SMTCoq.
Goal True.
cvc4.
(* Error:
In nested Ltac calls to "cvc4" and "cvc4_bool", last call failed.
Anomaly
"Uncaught exception Failure("SExprParser: failed to…