From 98949375345b93b85f7e7c4981cd29f8d0873cb7 Mon Sep 17 00:00:00 2001
From: Ralf Jung <jung@mpi-sws.org>
Date: Wed, 3 Aug 2022 17:55:45 -0400
Subject: [PATCH] update dependencies

---
 coq-lambda-rust.opam     | 2 +-
 theories/lang/adequacy.v | 2 +-
 2 files changed, 2 insertions(+), 2 deletions(-)

diff --git a/coq-lambda-rust.opam b/coq-lambda-rust.opam
index 10ef93e1..db0fc708 100644
--- a/coq-lambda-rust.opam
+++ b/coq-lambda-rust.opam
@@ -13,7 +13,7 @@ the type system, and safety proof for some Rust libraries.
 """
 
 depends: [
-  "coq-iris" { (= "dev.2022-07-27.1.d01b4bc8") | (= "dev") }
+  "coq-iris" { (= "dev.2022-08-03.0.949ab7bc") | (= "dev") }
 ]
 
 build: [make "-j%{jobs}%"]
diff --git a/theories/lang/adequacy.v b/theories/lang/adequacy.v
index ec935cd6..ec4b64cd 100644
--- a/theories/lang/adequacy.v
+++ b/theories/lang/adequacy.v
@@ -21,7 +21,7 @@ Definition lrust_adequacy Σ `{!lrustGpreS Σ} e σ φ :
   (∀ `{!lrustGS Σ}, True ⊢ WP e {{ v, ⌜φ v⌝ }}) →
   adequate NotStuck e σ (λ v _, φ v).
 Proof.
-  intros Hwp; eapply (wp_adequacy_lc _ _); iIntros (???).
+  intros Hwp; eapply (wp_adequacy _ _); iIntros (??).
   iMod (own_alloc (● to_heap σ)) as (vγ) "Hvγ".
   { apply (auth_auth_valid (to_heap _)), to_heap_valid. }
   iMod (own_alloc (● (∅ : heap_freeableUR))) as (fγ) "Hfγ";
-- 
GitLab