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

Remove obsolete FIXME.

parent 610698ec
No related branches found
No related tags found
No related merge requests found
...@@ -101,8 +101,7 @@ Section heap. ...@@ -101,8 +101,7 @@ Section heap.
Proof. Proof.
intros. rewrite -{1}(from_to_heap σ). etrans. intros. rewrite -{1}(from_to_heap σ). etrans.
{ rewrite [ownP _]later_intro. { rewrite [ownP _]later_intro.
apply (auth_alloc (ownP of_heap) N E (to_heap σ)); last done. apply (auth_alloc (ownP of_heap) N E); auto using to_heap_valid. }
apply to_heap_valid. }
apply pvs_mono, exist_elim=> γ. apply pvs_mono, exist_elim=> γ.
rewrite -(exist_intro (HeapG _ _ γ)) /heap_ctx; apply and_mono_r. rewrite -(exist_intro (HeapG _ _ γ)) /heap_ctx; apply and_mono_r.
rewrite /heap_mapsto /heap_name. rewrite /heap_mapsto /heap_name.
...@@ -110,8 +109,7 @@ Section heap. ...@@ -110,8 +109,7 @@ Section heap.
{ rewrite big_sepM_empty; apply True_intro. } { rewrite big_sepM_empty; apply True_intro. }
rewrite to_heap_insert big_sepM_insert //. rewrite to_heap_insert big_sepM_insert //.
rewrite (map_insert_singleton_op (to_heap σ)); rewrite (map_insert_singleton_op (to_heap σ));
last rewrite lookup_fmap Hl; auto. last by rewrite lookup_fmap Hl; auto.
(* FIXME: investigate why we have to unfold auth_own here. *)
by rewrite auth_own_op IH. by rewrite auth_own_op IH.
Qed. Qed.
......
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