Skip to content

Commit

Permalink
Fix brittle proof.
Browse files Browse the repository at this point in the history
  • Loading branch information
gebner authored and mtzguido committed Sep 26, 2024
1 parent 87a9ba9 commit f661c50
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion ulib/LowStar.Monotonic.Buffer.fst
Original file line number Diff line number Diff line change
Expand Up @@ -1877,7 +1877,8 @@ let blit #a #rrel1 #rrel2 #rel1 #rel2 src idx_src dst idx_dst len =
g_upd_seq_as_seq dst (Seq.slice s2' 0 (U32.v length2)) h //for modifies clause
| _, _ -> ()

#push-options "--z3rlimit 128 --max_fuel 0 --max_ifuel 1 --initial_ifuel 1 --z3cliopt smt.qi.EAGER_THRESHOLD=4"
#restart-solver
#push-options "--z3rlimit 256 --max_fuel 0 --max_ifuel 1 --initial_ifuel 1 --z3cliopt smt.qi.EAGER_THRESHOLD=4"
let fill' (#t:Type) (#rrel #rel: srel t)
(b: mbuffer t rrel rel)
(z:t)
Expand Down

0 comments on commit f661c50

Please sign in to comment.