Skip to content

Commit

Permalink
Merge pull request #2407 from FStarLang/aseem_cancellable_lock
Browse files Browse the repository at this point in the history
A Steel library for cancellable locks
  • Loading branch information
nikswamy authored Dec 11, 2021
2 parents 17ecea9 + eba0599 commit f3ac827
Show file tree
Hide file tree
Showing 2 changed files with 139 additions and 0 deletions.
72 changes: 72 additions & 0 deletions ulib/experimental/Steel.ST.CancellableSpinLock.fst
Original file line number Diff line number Diff line change
@@ -0,0 +1,72 @@
(*
Copyright 2021 Microsoft Research
Licensed under the Apache License, Version 2.0 (the "License");
you may not use this file except in compliance with the License.
You may obtain a copy of the License at
http://www.apache.org/licenses/LICENSE-2.0
Unless required by applicable law or agreed to in writing, software
distributed under the License is distributed on an "AS IS" BASIS,
WITHOUT WARRANTIES OR CONDITIONS OF ANY KIND, either express or implied.
See the License for the specific language governing permissions and
limitations under the License.
Author: Aseem Rastogi
*)

module Steel.ST.CancellableSpinLock

open Steel.ST.Effect
open Steel.ST.Util
open Steel.FractionalPermission
open Steel.ST.Reference
open Steel.ST.SpinLock

module G = FStar.Ghost

[@@__reduce__]
let lock_inv_pred (r:ref bool) (v:vprop) : bool -> vprop =
fun b -> pts_to r full_perm b `star` (if b then v else emp)

[@@__reduce__]
let lock_inv (r:ref bool) (v:vprop) : vprop = exists_ (lock_inv_pred r v)

noeq
type cancellable_lock (v:vprop) = {
lref : ref bool;
llock : lock (lock_inv lref v)
}

let new_cancellable_lock v =
let r = alloc true in
intro_exists true (lock_inv_pred r v);
let l = new_lock (lock_inv r v) in
return ({lref = r; llock = l})

[@__reduce__]
let can_release #v c = pts_to c.lref full_perm true

let acquire #v c =
acquire c.llock;
let b_erased = elim_exists () in
let b = read c.lref in
if b
then begin
rewrite (if b_erased then v else emp) v;
rewrite (v `star` can_release c)
(maybe_acquired b c)
end
else begin
intro_exists (G.reveal b_erased) (lock_inv_pred c.lref v);
release c.llock;
rewrite emp (maybe_acquired b c)
end;
return b

let release #v c =
intro_exists true (lock_inv_pred c.lref v);
release c.llock

let cancel c = free c.lref
67 changes: 67 additions & 0 deletions ulib/experimental/Steel.ST.CancellableSpinLock.fsti
Original file line number Diff line number Diff line change
@@ -0,0 +1,67 @@
(*
Copyright 2021 Microsoft Research
Licensed under the Apache License, Version 2.0 (the "License");
you may not use this file except in compliance with the License.
You may obtain a copy of the License at
http://www.apache.org/licenses/LICENSE-2.0
Unless required by applicable law or agreed to in writing, software
distributed under the License is distributed on an "AS IS" BASIS,
WITHOUT WARRANTIES OR CONDITIONS OF ANY KIND, either express or implied.
See the License for the specific language governing permissions and
limitations under the License.
Author: Aseem Rastogi
*)

module Steel.ST.CancellableSpinLock

open Steel.ST.Effect

/// This module provides a cancellable spinlock Steel library
///
/// As with Steel.ST.SpinLock, a cancellable spinlock guards
/// a separation logic assertion
///
/// However, it allows for the cases when the client is not able
/// to maintain the assertion
///
/// At that point, the client may just cancel the lock


/// The lock type that guards the assertion `v`

val cancellable_lock (v:vprop) : Type0

/// A cancellable lock can be created by providing `v`

val new_cancellable_lock (v:vprop)
: STT (cancellable_lock v) v (fun _ -> emp)


/// `can_release` is the permission to release the lock
///
/// Acquiring the lock, if it succeeds, provides `v`, the protected assertion
/// and `can_release`

val can_release (#v:vprop) (c:cancellable_lock v) : vprop

let maybe_acquired (b:bool) (#v:vprop) (c:cancellable_lock v)
= if b then (v `star` can_release c) else emp

val acquire (#v:vprop) (c:cancellable_lock v)
: STT bool emp (fun b -> maybe_acquired b c)


/// The client may provide `v` and `can_release` to release the lock

val release (#v:vprop) (c:cancellable_lock v)
: STT unit (v `star` can_release c) (fun _ -> emp)

/// If the client is no longer able to maintain `v`,
/// they may just cancel the lock by providing `can_release`

val cancel (#v:vprop) (c:cancellable_lock v)
: STT unit (can_release c) (fun _ -> emp)

0 comments on commit f3ac827

Please sign in to comment.