diff --git a/theories/typing/lib/smallvec/smallvec_basic.v b/theories/typing/lib/smallvec/smallvec_basic.v
index e1f0911630c27bb8bd6b32bdd4b9b054c2e21ed0..58598751a2ce0455e1017a0b4e2343032f76783b 100644
--- a/theories/typing/lib/smallvec/smallvec_basic.v
+++ b/theories/typing/lib/smallvec/smallvec_basic.v
@@ -109,9 +109,8 @@ Section smallvec_basic.
     typed_val (smallvec_new n ty) (fn(∅) → smallvec n ty) (λ post _, post []).
   Proof.
     eapply type_fn; [apply _|]=> _ ???. simpl_subst.
-    iIntros (???) "_ #TIME _ _ _ Na L C _ Obs".
-    iMod persistent_time_receipt_0 as "⧖". wp_bind (new _).
-    iApply (wp_persistent_time_receipt with "TIME ⧖"); [done|].
+    iIntros (???) "_ #TIME _ _ _ Na L C _ Obs". iMod persistent_time_receipt_0 as "⧖".
+    wp_bind (new _). iApply (wp_persistent_time_receipt with "TIME ⧖"); [done|].
     iApply wp_new; [done..|]. iIntros "!>" (r).
     rewrite !Nat2Z.id/= !heap_mapsto_vec_cons !shift_loc_assoc.
     iIntros "[† (↦₀ & ↦₁ & ↦₂ & ↦₃ & ↦ex)] ⧖". wp_seq. wp_write.
@@ -120,7 +119,7 @@ Section smallvec_basic.
     iExists _, _. do 2 (iSplit; [done|]). rewrite/= freeable_sz_full.
     iFrame "†". iNext. rewrite split_mt_smallvec. iExists true, _, 0, 0, [#].
     rewrite/= !heap_mapsto_vec_cons !shift_loc_assoc heap_mapsto_vec_nil.
-    iFrame "↦₀ ↦₁ ↦₂ ↦₃". do 2 (iSplit; [done|]). iExists _. iFrame.
+    iFrame "↦₀ ↦₁ ↦₂ ↦₃". do 2 (iSplit; [done|]). iExists _. iFrame "↦ex".
     by rewrite repeat_length.
   Qed.
 
diff --git a/theories/typing/lib/vec/vec_basic.v b/theories/typing/lib/vec/vec_basic.v
index 865c9c4092fd53298b45d1428bc2f6c550d385c3..da20c4f287fea37d396f345549cbb8085ba0d855 100644
--- a/theories/typing/lib/vec/vec_basic.v
+++ b/theories/typing/lib/vec/vec_basic.v
@@ -87,11 +87,10 @@ Section vec_basic.
     typed_val vec_new (fn(∅) → vec_ty ty) (λ post _, post []).
   Proof.
     eapply type_fn; [apply _|]=> _ ???. simpl_subst.
-    iIntros (???) "_ #TIME _ _ _ Na L C _ Obs".
-    wp_apply wp_new; [done..|]. iIntros (r).
-    rewrite !heap_mapsto_vec_cons shift_loc_assoc. iIntros "[† (↦₀ & ↦₁ & ↦₂ &_)]".
-    wp_seq. iMod persistent_time_receipt_0 as "⧖". wp_bind (new _).
-    iApply (wp_persistent_time_receipt with "TIME ⧖"); [done|].
+    iIntros (???) "_ #TIME _ _ _ Na L C _ Obs". wp_apply wp_new; [done..|].
+    iIntros (r). rewrite !heap_mapsto_vec_cons shift_loc_assoc.
+    iIntros "[† (↦₀ & ↦₁ & ↦₂ &_)]". wp_seq. iMod persistent_time_receipt_0 as "⧖".
+    wp_bind (new _). iApply (wp_persistent_time_receipt with "TIME ⧖"); [done|].
     iApply wp_new; [done..|]. iIntros "!>" (l) "[†' _] ⧖". wp_bind (_ <- _)%E.
     iApply (wp_persistent_time_receipt with "TIME ⧖"); [done|]. wp_write.
     iIntros "⧖". wp_seq. wp_op. wp_write. wp_op. wp_write. do 2 wp_seq.
@@ -100,7 +99,7 @@ Section vec_basic.
     iExists _, _. do 2 (iSplit; [done|]). rewrite/= freeable_sz_full split_mt_vec'.
     iFrame "†". iNext. iExists _, 0, 0, [#]=>/=. iSplit; [done|].
     rewrite !heap_mapsto_vec_cons heap_mapsto_vec_nil shift_loc_assoc.
-    iFrame "↦₀ ↦₁ ↦₂ †'". iSplit; [by iNext|]. iExists []. by rewrite heap_mapsto_vec_nil.
+    iFrame "↦₀ ↦₁ ↦₂ †'". iSplit; [done|]. iExists []. by rewrite heap_mapsto_vec_nil.
   Qed.
 
   Definition vec_drop {𝔄} (ty: type 𝔄) : val :=