diff --git a/coq-actris.opam b/coq-actris.opam
index 0bece13d0e64d9d7318fd271683d4e6200be9a40..fe376fb244a9cca0cbff2da22292b6e1854d541c 100644
--- a/coq-actris.opam
+++ b/coq-actris.opam
@@ -8,7 +8,7 @@ bug-reports: "https://gitlab.mpi-sws.org/iris/actris/issues"
 dev-repo: "git+https://gitlab.mpi-sws.org/iris/actris.git"
 
 depends: [
-  "coq-iris-heap-lang" { (= "dev.2022-06-28.0.b337ca8c") | (= "dev") }
+  "coq-iris-heap-lang" { (= "dev.2022-07-05.1.a32f36a9") | (= "dev") }
 ]
 
 build: [make "-j%{jobs}%"]
diff --git a/theories/logrel/term_typing_judgment.v b/theories/logrel/term_typing_judgment.v
index 9075dffb824090aac90491182ca1c3f4462b3d7a..d07bdcd40a957bf19c539489107a340f15cc6503 100644
--- a/theories/logrel/term_typing_judgment.v
+++ b/theories/logrel/term_typing_judgment.v
@@ -96,7 +96,7 @@ Lemma ltyped_safety `{heapGpreS Σ} e σ es σ' e' :
   rtc erased_step ([e], σ) (es, σ') → e' ∈ es →
   is_Some (to_val e') ∨ reducible e' σ'.
 Proof.
-  intros Hty. apply (heap_adequacy Σ NotStuck e σ (λ _, True))=> // ?.
+  intros Hty. apply (heap_adequacy Σ NotStuck e σ (λ _, True))=> // ??.
   destruct (Hty _) as (A & He). iIntros "_".
   iDestruct (He $!∅ with "[]") as "He"; first by rewrite /ctx_ltyped.
   iEval (rewrite -(subst_map_empty e)). iApply (wp_wand with "He"); auto.