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

Frame preserving updates only from steps ≠ 0.

parent 2ccdb104
No related branches found
No related tags found
No related merge requests found
...@@ -129,7 +129,7 @@ Lemma wsat_update_gst n E σ r rf m1 (P : iGst Λ Σ → Prop) : ...@@ -129,7 +129,7 @@ Lemma wsat_update_gst n E σ r rf m1 (P : iGst Λ Σ → Prop) :
wsat (S n) E σ (r rf) m2, wsat (S n) E σ (update_gst m2 r rf) P m2. wsat (S n) E σ (r rf) m2, wsat (S n) E σ (update_gst m2 r rf) P m2.
Proof. Proof.
intros [mf Hr] Hup [rs [(?&?&?) HE Hwld]]. intros [mf Hr] Hup [rs [(?&?&?) HE Hwld]].
destruct (Hup (mf gst (rf big_opM rs)) (S n)) as (m2&?&Hval'). destruct (Hup (mf gst (rf big_opM rs)) n) as (m2&?&Hval').
{ by rewrite /= (associative _ m1) -Hr (associative _). } { by rewrite /= (associative _ m1) -Hr (associative _). }
exists m2; split; [exists rs; split; split_ands'; auto|done]. exists m2; split; [exists rs; split; split_ands'; auto|done].
Qed. Qed.
......
...@@ -142,11 +142,11 @@ Class CMRAMonotone {A B : cmraT} (f : A → B) := { ...@@ -142,11 +142,11 @@ Class CMRAMonotone {A B : cmraT} (f : A → B) := {
(** * Frame preserving updates *) (** * Frame preserving updates *)
Definition cmra_updateP {A : cmraT} (x : A) (P : A Prop) := z n, Definition cmra_updateP {A : cmraT} (x : A) (P : A Prop) := z n,
{n} (x z) y, P y {n} (y z). {S n} (x z) y, P y {S n} (y z).
Instance: Params (@cmra_updateP) 3. Instance: Params (@cmra_updateP) 3.
Infix "⇝:" := cmra_updateP (at level 70). Infix "⇝:" := cmra_updateP (at level 70).
Definition cmra_update {A : cmraT} (x y : A) := z n, Definition cmra_update {A : cmraT} (x y : A) := z n,
{n} (x z) {n} (y z). {S n} (x z) {S n} (y z).
Infix "⇝" := cmra_update (at level 70). Infix "⇝" := cmra_update (at level 70).
Instance: Params (@cmra_update) 3. Instance: Params (@cmra_update) 3.
...@@ -393,15 +393,12 @@ Section discrete. ...@@ -393,15 +393,12 @@ Section discrete.
Qed. Qed.
Definition discreteRA : cmraT := Definition discreteRA : cmraT :=
CMRAT (cofe_mixin A) discrete_cmra_mixin discrete_extend_mixin. CMRAT (cofe_mixin A) discrete_cmra_mixin discrete_extend_mixin.
Lemma discrete_updateP (x : discreteRA) (P : A Prop) `{!Inhabited (sig P)} : Lemma discrete_updateP (x : discreteRA) (P : A Prop) :
( z, (x z) y, P y (y z)) x ⇝: P. ( z, (x z) y, P y (y z)) x ⇝: P.
Proof. Proof. intros Hvalid z n; apply Hvalid. Qed.
intros Hvalid z [|n]; [|apply Hvalid].
by destruct (_ : Inhabited (sig P)) as [[y ?]]; exists y.
Qed.
Lemma discrete_update (x y : discreteRA) : Lemma discrete_update (x y : discreteRA) :
( z, (x z) (y z)) x y. ( z, (x z) (y z)) x y.
Proof. intros Hvalid z [|n]; [done|apply Hvalid]. Qed. Proof. intros Hvalid z n; apply Hvalid. Qed.
End discrete. End discrete.
(** ** CMRA for the unit type *) (** ** CMRA for the unit type *)
...@@ -477,7 +474,7 @@ Section prod. ...@@ -477,7 +474,7 @@ Section prod.
Lemma prod_update x y : x.1 y.1 x.2 y.2 x y. Lemma prod_update x y : x.1 y.1 x.2 y.2 x y.
Proof. intros ?? z n [??]; split; simpl in *; auto. Qed. Proof. intros ?? z n [??]; split; simpl in *; auto. Qed.
Lemma prod_updateP (P : A * B Prop) P1 P2 x : Lemma prod_updateP (P : A * B Prop) P1 P2 x :
x.1 ⇝: P1 x.2 ⇝: P2 ( y, P1 (y.1) P2 (y.2) P y) x ⇝: P. x.1 ⇝: P1 x.2 ⇝: P2 ( a b, P1 a P2 b P (a,b)) x ⇝: P.
Proof. Proof.
intros Hx1 Hx2 HP z n [??]; simpl in *. intros Hx1 Hx2 HP z n [??]; simpl in *.
destruct (Hx1 (z.1) n) as (a&?&?), (Hx2 (z.2) n) as (b&?&?); auto. destruct (Hx1 (z.1) n) as (a&?&?), (Hx2 (z.2) n) as (b&?&?); auto.
......
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