Skip to content
Snippets Groups Projects
Commit 7d9516fc authored by Robbert Krebbers's avatar Robbert Krebbers
Browse files

Bump gpfsl.

parent 7c6d21c6
No related branches found
No related tags found
No related merge requests found
Pipeline #16436 failed
......@@ -10,5 +10,5 @@ build: [make "-j%{jobs}%"]
install: [make "install"]
remove: [ "sh" "-c" "rm -rf '%{lib}%/coq/user-contrib/lrust'" ]
depends: [
"coq-gpfsl" { (= "dev.2019-04-25.0.8e1ed3d2") | (= "dev") }
"coq-gpfsl" { (= "dev.2019-05-02.0.92f26ecd") | (= "dev") }
]
......@@ -218,7 +218,7 @@ Proof.
iAssert ([ map] γ↦_ f, Φ γ V)%I with "[HP]" as "HP'".
{ rewrite -big_sepM_later -monPred_at_big_sepM. iNext. by iRewrite "HeqP" in "HP". }
iCombine "Hf" "HP'" as "Hf".
rewrite -big_sepM_sepM big_opM_fmap; iApply (fupd_big_sepM _ _ f).
rewrite -big_sepM_sep big_opM_fmap; iApply (fupd_big_sepM _ _ f).
iApply (@big_sepM_impl with "[$Hf]").
iAlways; iIntros (γ b' ?) "[(Hγ' & #$ & #$) HΦ]".
iInv N as (b) "[>Hγ _]" "Hclose".
......
......@@ -301,7 +301,7 @@ Proof. rewrite /lft_dead. iDestruct 1 as (Λ V') "[% H']". set_solver. Qed.
(* Fractional and AsFractional instances *)
Global Instance lft_tok_fractional κ : Fractional (λ q, q.[κ])%I.
Proof.
intros p q. rewrite /lft_tok -big_sepMS_sepMS. apply big_sepMS_proper=>Λ ?.
intros p q. rewrite /lft_tok -big_sepMS_sep. apply big_sepMS_proper=>Λ ?.
iSplit.
- iIntros "H". iDestruct "H" as (V') "[#? H] ".
(* FIXME : the Proper instance for singleton cannot be found automatically here. *)
......@@ -321,7 +321,7 @@ Proof. split. done. apply _. Qed.
Lemma lft_tok_split_obj `{LatBottom Lat bot} q1 q2 κ :
(q1 + q2).[κ] -∗ q1.[κ] <obj> q2.[κ].
Proof.
rewrite /lft_tok. rewrite -monPred_objectively_big_sepMS_entails -big_sepMS_sepMS.
rewrite /lft_tok. rewrite -monPred_objectively_big_sepMS_entails -big_sepMS_sep.
apply big_sepMS_mono=>// Λ ?. iStartProof (iProp _). iDestruct 1 as (V) "[#? H]".
rewrite (fin_maps.singleton_proper Λ _ (Cinl (_, to_latT V to_latT bot))); last first.
{ rewrite lat_op_join' right_id //. } rewrite -pair_op -Cinl_op -op_singleton.
......
......@@ -60,7 +60,7 @@ Section lft_contexts.
Global Arguments llctx_interp _ _%Qp.
Global Instance llctx_interp_fractional L :
Fractional (llctx_interp L).
Proof. intros ??. rewrite -big_sepL_sepL. by setoid_rewrite <-fractional. Qed.
Proof. intros ??. rewrite -big_sepL_sep. by setoid_rewrite <-fractional. Qed.
Global Instance llctx_interp_as_fractional L q :
AsFractional (llctx_interp L q) (llctx_interp L) q.
Proof. split. done. apply _. Qed.
......
0% Loading or .
You are about to add 0 people to the discussion. Proceed with caution.
Please register or to comment