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

tweak tests a bit

parent bc0339ec
No related branches found
No related tags found
No related merge requests found
......@@ -550,10 +550,12 @@ Section lock_gen.
"l" <- #42;;
release "lock".
Lemma wp_lock_client_spin `{!heapGS Σ, !lockG Σ} :
(* Making sure that using [spin_lockG] here works, not just [lockG]. *)
Lemma wp_lock_client_spin `{!heapGS Σ, !spin_lockG Σ} :
WP lock_client_spin {{ _, True }}.
Proof.
unfold lock_client_spin. wp_alloc l as "Hl".
unfold lock_client_spin. simpl. Show. (* should show no spin_lock.<something> *)
wp_alloc l as "Hl".
wp_smart_apply (newlock_spec ( n : Z, l #n) with "[Hl]")
as (lk γ) "#Hlock"; first by eauto.
wp_smart_apply (acquire_spec with "Hlock") as "(Hlocked & %v & Hloc)".
......@@ -562,7 +564,7 @@ Section lock_gen.
Qed.
End lock_gen.
(** Making sure we the [lockG] conditions are resolved when using adequacy. For
(** Making sure that the [lockG/spin_lockG] conditions are resolved when using adequacy. For
the generic client, we need to instantiate it with a specific lock for that to
make sense. *)
Section lock_adequacy.
......
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