diff --git a/coq-reloc.opam b/coq-reloc.opam
index 9889dc8f1cf24affab0285caf48291ed0596d31f..c8eab3026905789384732d44b65f7f76552607ce 100644
--- a/coq-reloc.opam
+++ b/coq-reloc.opam
@@ -6,7 +6,7 @@ bug-reports: "https://gitlab.mpi-sws.org/dfrumin/reloc/issues"
 dev-repo: "git+https://gitlab.mpi-sws.org/dfrumin/reloc.git"
 
 depends: [
-  "coq-iris-heap-lang" { (= "dev.2022-06-28.0.b337ca8c") | (= "dev") }
+  "coq-iris-heap-lang" { (= "dev.2022-07-05.1.a32f36a9") | (= "dev") }
   "coq-autosubst" { = "dev" }
 ]
 
diff --git a/theories/logic/adequacy.v b/theories/logic/adequacy.v
index 0bddd0758964129c1bbaf15cb02960ecffa0c9c8..cf630f393f2f654614a414d2c7479b966b45faac 100644
--- a/theories/logic/adequacy.v
+++ b/theories/logic/adequacy.v
@@ -24,7 +24,7 @@ Lemma refines_adequate Σ `{relocPreG Σ}
             ∧ P v v').
 Proof.
   intros HA Hlog.
-  eapply (heap_adequacy Σ _); iIntros (Hinv) "_".
+  eapply (heap_adequacy Σ _); iIntros (Hinv ?) "_".
   iMod (own_alloc (● (to_tpool [e'], to_heap (heap σ))
     ⋅ ◯ ((to_tpool [e'] : tpoolUR, ∅) : cfgUR)))
     as (γc) "[Hcfg1 Hcfg2]".