Skip to content

Commit

Permalink
rlimit for higherarray
Browse files Browse the repository at this point in the history
  • Loading branch information
aseemr committed Mar 14, 2023
1 parent 862fe6e commit f6205dd
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions ulib/experimental/Steel.ST.HigherArray.fst
Original file line number Diff line number Diff line change
Expand Up @@ -645,6 +645,7 @@ let memcpy0
(pts_to a1 _ e0);
return ()

#push-options "--z3rlimit 50"
let blit0 (#t:_) (#p0:perm) (#s0 #s1:Ghost.erased (Seq.seq t))
(src:array t)
(idx_src: US.t)
Expand Down Expand Up @@ -677,6 +678,7 @@ let blit0 (#t:_) (#p0:perm) (#s0 #s1:Ghost.erased (Seq.seq t))
vpattern_rewrite #_ #_ #(merge _ _) (fun a -> pts_to a _ _) src;
vpattern_rewrite (pts_to src _) (Ghost.reveal s0);
noop ()
#pop-options

#pop-options

Expand Down

0 comments on commit f6205dd

Please sign in to comment.