Skip to content

Commit

Permalink
add --enum-inst option for cvc5
Browse files Browse the repository at this point in the history
  • Loading branch information
PratherConid committed Dec 4, 2024
1 parent 436da90 commit 8fc8cad
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Auto/Solver/SMT.lean
Original file line number Diff line number Diff line change
Expand Up @@ -108,7 +108,7 @@ def createSolver (name : SolverName) : MetaM SolverProc := do
| .none => throwError "{decl_name%} :: Unexpected error"
| .z3 => createAux "z3" #["-in", "-smt2", s!"-T:{tlim}"]
| .cvc4 => throwError "cvc4 is not supported"
| .cvc5 => createAux "cvc5" #[s!"--tlimit={tlim * 1000}", "--produce-models"]
| .cvc5 => createAux "cvc5" #[s!"--tlimit={tlim * 1000}", "--produce-models", "--enum-inst"]
where
createAux (path : String) (args : Array String) : MetaM SolverProc :=
IO.Process.spawn {stdin := .piped, stdout := .piped, stderr := .piped,
Expand Down

0 comments on commit 8fc8cad

Please sign in to comment.