From 63e065c76e9ba032fdec4f8586250e45c3593203 Mon Sep 17 00:00:00 2001 From: Ralf Jung <jung@mpi-sws.org> Date: Tue, 5 Jul 2022 19:36:33 -0400 Subject: [PATCH] update dependencies for later credits --- coq-actris.opam | 2 +- theories/logrel/term_typing_judgment.v | 2 +- 2 files changed, 2 insertions(+), 2 deletions(-) diff --git a/coq-actris.opam b/coq-actris.opam index 0bece13..fe376fb 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 9075dff..d07bdcd 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. -- GitLab