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

FP update for auth without frame.

parent 24c28e2c
No related branches found
No related tags found
No related merge requests found
...@@ -183,8 +183,7 @@ Lemma auth_both_op a b : Auth (Excl' a) b ≡ ● a ⋅ ◯ b. ...@@ -183,8 +183,7 @@ Lemma auth_both_op a b : Auth (Excl' a) b ≡ ● a ⋅ ◯ b.
Proof. by rewrite /op /auth_op /= left_id. Qed. Proof. by rewrite /op /auth_op /= left_id. Qed.
Lemma auth_update a af b : Lemma auth_update a af b :
a ~l~> b @ Some af a ~l~> b @ Some af (a af) a ~~> (b af) b.
(a af) a ~~> (b af) b.
Proof. Proof.
intros [Hab Hab']; apply cmra_total_update. intros [Hab Hab']; apply cmra_total_update.
move=> n [[[?|]|] bf1] // =>-[[bf2 Ha] ?]; do 2 red; simpl in *. move=> n [[[?|]|] bf1] // =>-[[bf2 Ha] ?]; do 2 red; simpl in *.
...@@ -192,6 +191,11 @@ Proof. ...@@ -192,6 +191,11 @@ Proof.
exists bf2. rewrite -assoc. exists bf2. rewrite -assoc.
apply (Hab' _ (Some _)); auto. by rewrite /= assoc. apply (Hab' _ (Some _)); auto. by rewrite /= assoc.
Qed. Qed.
Lemma auth_update_no_frame a b : a ~l~> b @ Some a a ~~> b b.
Proof.
intros. rewrite -{1}(right_id _ _ a) -{1}(right_id _ _ b).
by apply auth_update.
Qed.
End cmra. End cmra.
Arguments authR : clear implicits. Arguments authR : clear implicits.
......
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