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

Tweak closed proof in heap_lang/tests.

parent 2c6727dc
No related branches found
No related tags found
No related merge requests found
...@@ -80,25 +80,18 @@ Section LiftingTests. ...@@ -80,25 +80,18 @@ Section LiftingTests.
End LiftingTests. End LiftingTests.
Section ClosedProofs. Section ClosedProofs.
Definition Σ : iFunctorG := λ _, authF (constF heapRA). Definition Σ : iFunctorG := λ _, authF (constF heapRA).
Notation iProp := (iPropG heap_lang Σ).
Local Instance : inG heap_lang Σ (authRA heapRA). Instance: authG heap_lang Σ heapRA.
Proof. by exists 1%nat. Qed. Proof. split; try apply _. by exists 1%nat. Qed.
(* TODO: Why do I even have to explicitly do this? *)
Local Instance : authG heap_lang Σ heapRA.
Proof. split; by apply _. Qed.
Local Notation iProp := (iPropG heap_lang Σ).
Lemma heap_e_hoare σ : {{ ownP σ : iProp }} heap_e @ {{ λ v, v = '2 }}. Lemma heap_e_hoare σ : {{ ownP σ : iProp }} heap_e @ {{ λ v, v = '2 }}.
Proof. Proof.
apply ht_alt. rewrite (heap_alloc nroot); last by rewrite nclose_nroot. apply ht_alt. rewrite (heap_alloc nroot); last by rewrite nclose_nroot.
apply wp_strip_pvs, exist_elim=>?. rewrite and_elim_l. apply wp_strip_pvs, exist_elim=> ?. rewrite and_elim_l.
rewrite -heap_e_spec; first by eauto with I. by rewrite nclose_nroot. rewrite -heap_e_spec; first by eauto with I. by rewrite nclose_nroot.
Qed. Qed.
Print Assumptions heap_e_hoare. Print Assumptions heap_e_hoare.
End ClosedProofs.
End ClosedProofs.
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