diff --git a/theories/heap_lang/lib/barrier/proof.v b/theories/heap_lang/lib/barrier/proof.v
index 41e84948d73841d2d7a1f7186fdc52768da86a64..dd3928187a6a0ecb1cac32eb022eb118dd80ae40 100644
--- a/theories/heap_lang/lib/barrier/proof.v
+++ b/theories/heap_lang/lib/barrier/proof.v
@@ -198,6 +198,4 @@ Lemma recv_mono l P1 P2 : (P1 ⊢ P2) → recv l P1 ⊢ recv l P2.
 Proof. iIntros (HP) "H". iApply (recv_weaken with "[] H"). iApply HP. Qed.
 End proof.
 
-SearchAbout _.
-
 Typeclasses Opaque barrier_ctx send recv.