Skip to content
Snippets Groups Projects
Commit 005a0803 authored by Ralf Jung's avatar Ralf Jung
Browse files

update dependencies

parent 3b1c1e1c
No related branches found
No related tags found
No related merge requests found
Pipeline #86933 passed
......@@ -8,7 +8,7 @@ dev-repo: "git+https://gitlab.mpi-sws.org/iris/examples.git"
synopsis: "A collection of case studies for Iris -- not meant to be used as a dependency of anything"
depends: [
"coq-iris-heap-lang" { (= "dev.2023-06-30.0.7e865892") | (= "dev") }
"coq-iris-heap-lang" { (= "dev.2023-07-25.2.621d76cf") | (= "dev") }
"coq-autosubst" { = "dev" }
]
......
......@@ -21,8 +21,7 @@ Local Existing Instance entails_po.
Lemma clProp_bi_mixin :
BiMixin
clProp_entails clProp_emp clProp_pure clProp_and clProp_or clProp_impl
(@clProp_forall) (@clProp_exist) clProp_sep clProp_wand
clProp_persistently.
(@clProp_forall) (@clProp_exist) clProp_sep clProp_wand.
Proof.
split.
- exact: entails_po.
......@@ -35,7 +34,6 @@ Proof.
- exact: exist_ne.
- exact: and_ne.
- exact: impl_ne.
- solve_proper.
- exact: pure_intro.
- exact: pure_elim'.
- exact: and_elim_l.
......@@ -71,6 +69,15 @@ Proof.
apply impl_intro_r.
- (* (P ⊢ Q -∗ R) → P ∗ Q ⊢ R *)
apply impl_elim_l'.
Qed.
Lemma clProp_bi_persistently_mixin :
BiPersistentlyMixin
clProp_entails clProp_emp clProp_and
(@clProp_exist) clProp_sep clProp_persistently.
Proof.
split.
- solve_proper.
- (* (P ⊢ Q) → <pers> P ⊢ <pers> Q *)
done.
- (* <pers> P ⊢ <pers> <pers> P *)
......@@ -95,7 +102,9 @@ Proof. by eapply bi_later_mixin_id, clProp_bi_mixin. Qed.
Canonical Structure clPropI : bi :=
{| bi_ofe_mixin := ofe_mixin_of clProp;
bi_bi_mixin := clProp_bi_mixin; bi_bi_later_mixin := clProp_bi_later_mixin |}.
bi_bi_mixin := clProp_bi_mixin;
bi_bi_persistently_mixin := clProp_bi_persistently_mixin;
bi_bi_later_mixin := clProp_bi_later_mixin |}.
Lemma clProp_plainly_mixin : BiPlainlyMixin clPropI clProp_plainly.
Proof.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Finish editing this message first!
Please register or to comment