Skip to content

Commit

Permalink
Merge pull request #3015 from mtzguido/no-encode-if-admit
Browse files Browse the repository at this point in the history
Do not encode to SMT if admitting queries
  • Loading branch information
mtzguido authored Aug 14, 2023
2 parents bdfe784 + f7429df commit 8808598
Show file tree
Hide file tree
Showing 2 changed files with 26 additions and 17 deletions.
38 changes: 22 additions & 16 deletions ocaml/fstar-lib/generated/FStar_SMTEncoding_Solver.ml

Some generated files are not rendered by default. Learn more about how customized files appear on GitHub.

5 changes: 4 additions & 1 deletion src/smtencoding/FStar.SMTEncoding.Solver.fst
Original file line number Diff line number Diff line change
Expand Up @@ -1220,6 +1220,9 @@ let disable_quake_for (f : unit -> 'a) : 'a =
(* Split queries if needed according to --split_queries option. Note:
sync SMT queries do not pass via this function. *)
let do_solve_maybe_split use_env_msg tcenv q : unit =
(* If we are admiting queries, don't do anything, and bail out
right now to save time/memory *)
if Options.admit_smt_queries () then () else begin
match Options.split_queries () with
| Options.No -> do_solve false false use_env_msg tcenv q
| Options.OnFailure ->
Expand All @@ -1234,7 +1237,7 @@ let do_solve_maybe_split use_env_msg tcenv q : unit =
| Options.Always ->
(* Set retrying=false so queries go through the full config list, etc. *)
split_and_solve false use_env_msg tcenv q
end
(* Attempt to discharge a VC through the SMT solver. Will
automatically retry increasing fuel as needed, and perform quake testing
(repeating the query to make sure it is robust). This function will
Expand Down

0 comments on commit 8808598

Please sign in to comment.