From f028cdebe044bb357570727669c3eeded2355e71 Mon Sep 17 00:00:00 2001 From: Ralf Jung <jung@mpi-sws.org> Date: Wed, 8 Nov 2017 10:01:08 +0100 Subject: [PATCH] bump iris --- opam | 2 +- theories/lang/lang.v | 2 +- theories/lang/races.v | 2 +- theories/lang/tactics.v | 2 +- 4 files changed, 4 insertions(+), 4 deletions(-) diff --git a/opam b/opam index d80a8a36..b1661244 100644 --- a/opam +++ b/opam @@ -11,5 +11,5 @@ build: [make "-j%{jobs}%"] install: [make "install"] remove: [ "sh" "-c" "rm -rf '%{lib}%/coq/user-contrib/lrust'" ] depends: [ - "coq-iris" { (= "dev.2017-11-04.0") | (= "dev") } + "coq-iris" { (= "dev.2017-11-07.2") | (= "dev") } ] diff --git a/theories/lang/lang.v b/theories/lang/lang.v index bd1dc084..ff076bd1 100644 --- a/theories/lang/lang.v +++ b/theories/lang/lang.v @@ -638,7 +638,7 @@ Proof. apply: (irreducible_fill (K:=ectx_language.fill K)); first done. apply prim_head_irreducible; unfold stuck_term. - inversion 1. - - apply ectxi_language_sub_values. + - apply ectxi_language_sub_redexes_are_values. intros [] ??; simplify_eq/=; eauto; discriminate_list. Qed. diff --git a/theories/lang/races.v b/theories/lang/races.v index 8fa7a547..bc7399c1 100644 --- a/theories/lang/races.v +++ b/theories/lang/races.v @@ -76,7 +76,7 @@ Lemma next_access_head_reductible_ctx e σ σ' a l K : Proof. intros Hhead Hred. apply prim_head_reducible. - eapply (reducible_fill (K:=ectx_language.fill K)), Hred. destruct Hhead; eauto. - - apply ectxi_language_sub_values. intros [] ? ->; inversion Hhead; eauto. + - apply ectxi_language_sub_redexes_are_values. intros [] ? ->; inversion Hhead; eauto. Qed. Definition head_reduce_not_to_stuck (e : expr) (σ : state) := diff --git a/theories/lang/tactics.v b/theories/lang/tactics.v index e890b488..91f72245 100644 --- a/theories/lang/tactics.v +++ b/theories/lang/tactics.v @@ -160,7 +160,7 @@ Proof. destruct e; simpl; try done; repeat (case_match; try done); inversion 1; try (apply val_irreducible; rewrite ?language.to_of_val; naive_solver eauto); []. rewrite -[stuck_term](fill_empty). apply stuck_irreducible. - - apply ectxi_language_sub_values=> /= Ki e' Hfill. + - apply ectxi_language_sub_redexes_are_values=> /= Ki e' Hfill. revert He. destruct e; simpl; try done; repeat (case_match; try done); rewrite ?bool_decide_spec; destruct Ki; inversion Hfill; subst; clear Hfill; -- GitLab