Skip to content
Snippets Groups Projects
Commit 49b14e9f authored by Simon Spies's avatar Simon Spies
Browse files

tweak

parent ff2e9d17
No related branches found
No related tags found
No related merge requests found
Pipeline #110408 passed
...@@ -166,7 +166,7 @@ Section open_example. ...@@ -166,7 +166,7 @@ Section open_example.
Definition example : expr := Definition example : expr :=
let: "n" := external_code #() in let: "n" := external_code #() in
for: "n" do for: "n" do
enqueue q (λ: <>, print "Hello World!"). enqueue q (λ: <>, print #42).
Lemma for_zero e: Lemma for_zero e:
sbi_emp_valid (WP (for: #0 do e)%V [{ v, v = #() }])%I. sbi_emp_valid (WP (for: #0 do e)%V [{ v, v = #() }])%I.
...@@ -189,7 +189,7 @@ Section open_example. ...@@ -189,7 +189,7 @@ Section open_example.
Qed. Qed.
Lemma example_spec `{FiniteBoundedExistential SI}: Lemma example_spec `{FiniteBoundedExistential SI}:
queue N q $ (omul (one: ordA SI)) SEQ external_code #() [{ v, n: nat, v = #n }] ( s: string, SEQ print s [{ _, True }]) queue N q $ (omul (one: ordA SI)) SEQ external_code #() [{ v, n: nat, v = #n }] ( n: Z, SEQ print #n [{ _, True }])
SEQ example [{ _, True }]. SEQ example [{ _, True }].
Proof. Proof.
iIntros "(#Q & Hc & Hwp & #Hprint) Hna". rewrite /example. iIntros "(#Q & Hc & Hwp & #Hprint) Hna". rewrite /example.
......
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