diff --git a/theories/logatom/flat_combiner/flat.v b/theories/logatom/flat_combiner/flat.v
index dd2182925d8a83fd8f5b6f56a64007690259b712..f6fdf2b7334ca2fbfa1ec198837f5320d8aa789a 100644
--- a/theories/logatom/flat_combiner/flat.v
+++ b/theories/logatom/flat_combiner/flat.v
@@ -219,8 +219,8 @@ Section proof.
     ⊢ WP try_srv lk #s {{ Φ }}.
   Proof.
     iIntros "(#? & #? & HΦ)". wp_lam. wp_pures.
-    wp_bind (try_acquire _). iApply (try_acquire_spec with "[]"); first done.
-    iNext. iIntros ([]); last by (iIntros; wp_if).
+    wp_apply (try_acquire_spec with "[]"); first done.
+    iIntros ([]); last by (iIntros; wp_if).
     iIntros "[Hlocked [Ho2 HR]]".
     wp_if. wp_bind (! _)%E.
     iInv N as "H" "Hclose".
@@ -255,14 +255,14 @@ Section proof.
     + iDestruct "Hp" as (f x) "(>Hp & Hs')".
       wp_load. iMod ("Hclose" with "[Hp Hs']").
       { iNext. iFrame. iRight. iLeft. iExists f, x. iFrame. }
-      iModIntro. wp_match. wp_bind (try_srv _ _). iApply try_srv_spec=>//.
+      iModIntro. wp_match. wp_apply try_srv_spec=>//.
       iFrame "#". wp_seq. iApply ("IH" with "Ho3"); eauto.
     + iDestruct "Hp" as (f x) "(Hp & Hx & Ho2 & Ho4)".
       wp_load. iMod ("Hclose" with "[-Ho3 HΦ]") as "_".
       { iNext. (* FIXME: iFrame here divergses, with an enormous TC trace *)
         iRight. iRight. iLeft. iExists f, x. iFrame. }
       iModIntro. wp_match.
-      wp_bind (try_srv _ _). iApply try_srv_spec=>//.
+      wp_apply try_srv_spec=>//.
       iFrame "#". wp_seq. iApply ("IH" with "Ho3"); eauto.
     + iDestruct "Hp" as (x y) "[>Hp Hs']".
       iDestruct "Hs'" as (Q) "(>Hx & HoQ & HQ & >Ho1 & >Ho4)".
@@ -276,19 +276,19 @@ Section proof.
   Proof using Type* N.
     iIntros (R Φ) "HR HΦ".
     iMod (own_alloc (Excl ())) as (γr) "Ho2"; first done.
-    wp_lam. wp_bind (newlock _).
-    iApply (newlock_spec (own γr (Excl ()) ∗ R)%I with "[$Ho2 $HR]")=>//.
-    iNext. iIntros (lk γlk) "#Hlk".
-    wp_let. wp_bind (new_stack _).
-    iApply (new_bag_spec N (p_inv' R γm γr))=>//.
-    iNext. iIntros (s) "#Hss".
+    wp_lam.
+    wp_apply (newlock_spec (own γr (Excl ()) ∗ R)%I with "[$Ho2 $HR]")=>//.
+    iIntros (lk γlk) "#Hlk".
+    wp_let.
+    wp_apply (new_bag_spec N (p_inv' R γm γr))=>//.
+    iIntros (s) "#Hss".
     wp_pures. iModIntro. iApply "HΦ".
     iModIntro. iIntros (f). wp_pures.
     iIntros "!> !>" (P Q x) "#Hf !>".
-    iIntros (Φ') "Hp HΦ'". wp_pures. wp_bind (install _ _ _).
-    iApply (install_spec R P Q f x γm γr s with "[Hp]")=>//.
+    iIntros (Φ') "Hp HΦ'". wp_pures.
+    wp_apply (install_spec R P Q f x γm γr s with "[Hp]")=>//.
     { iFrame. iFrame "#". }
-    iNext. iIntros (p [[[[γx γ1] γ3] γ4] γq]) "[(Ho3 & Hx & HoQ) #?]".
+    iIntros (p [[[[γx γ1] γ3] γ4] γq]) "[(Ho3 & Hx & HoQ) #?]".
     wp_let. wp_bind (loop _ _ _).
     iApply (loop_spec with "[-Hx HoQ HΦ']")=>//.
     { iFrame "#". iFrame. }