Skip to content
Snippets Groups Projects
Commit 1f9c5efc authored by Ralf Jung's avatar Ralf Jung
Browse files

add test for iAuIntro errors (status quo)

parent 62798412
No related branches found
No related tags found
No related merge requests found
......@@ -12,6 +12,17 @@
AACC << ∀ (v0 : val) (q : Qp), l ↦{q} v0 ABORT l ↦ v >> @ ⊤, ∅
<< l ↦{q} v0, COMM Q -∗ Q >>
"non_laterable"
: string
The command has indeed failed with message:
Tactic failure: iAuIntro: not all spatial assumptions are laterable.
The command has indeed failed with message:
Tactic failure: wp_apply: cannot apply
(<<< ∀ (v : val) (q : Qp), ?Goal ↦{q} v >>>
! #?Goal @ ⊤
<<< ?Goal ↦{q} v, RET v >>>).
"printing"
: string
1 subgoal
Σ : gFunctors
......
......@@ -17,7 +17,24 @@ Section tests.
Qed.
End tests.
(* Test if we get reasonable error messages with non-laterable assertions in the context. *)
Section error.
Context `{!heapG Σ} {aheap: atomic_heap Σ}.
Import atomic_heap.notation.
Check "non_laterable".
Lemma non_laterable (P : iProp Σ) (l : loc) :
P -∗ WP !#l {{ _, True }}.
Proof.
iIntros "HP". wp_apply load_spec. Fail iAuIntro.
Restart.
iIntros "HP". Fail awp_apply load_spec.
Abort.
End error.
(* Test if AWP and the AU obtained from AWP print. *)
Check "printing".
Section printing.
Context `{!heapG Σ}.
......
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