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

FP update for auth without fragment.

parent e059aa12
No related branches found
No related tags found
No related merge requests found
......@@ -191,11 +191,17 @@ Proof.
exists bf2. rewrite -assoc.
apply (Hab' _ (Some _)); auto. by rewrite /= assoc.
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.
Lemma auth_update_no_frag af b : ~l~> b @ Some af af ~~> (b af) b.
Proof.
intros. rewrite -{1}(left_id _ _ af) -{1}(right_id _ _ ( _)).
by apply auth_update.
Qed.
End cmra.
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