From 90bc7991937882aea4c9130e10b4b89a8a09734f Mon Sep 17 00:00:00 2001 From: Ralf Jung <jung@mpi-sws.org> Date: Tue, 5 Jul 2022 19:21:58 -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 3fa8f5e8..98f70f36 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-06-28.0.b337ca8c") | (= "dev") } + "coq-iris" { (= "dev.2022-07-05.1.a32f36a9") | (= "dev") } ] build: [make "-j%{jobs}%"] diff --git a/theories/lang/adequacy.v b/theories/lang/adequacy.v index ec4b64cd..ec935cd6 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 _ _); iIntros (??). + intros Hwp; eapply (wp_adequacy_lc _ _); 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