Skip to content

Commit

Permalink
Run $FSTAR/.scripts/remove_all_unused_opens.sh .
Browse files Browse the repository at this point in the history
  • Loading branch information
mtzguido committed Feb 18, 2025
1 parent 55fac43 commit dac35ec
Show file tree
Hide file tree
Showing 159 changed files with 2 additions and 268 deletions.
2 changes: 0 additions & 2 deletions lib/common/Pulse.Lib.Core.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -19,8 +19,6 @@ open FStar.Ghost
open PulseCore.FractionalPermission
open PulseCore.Observability
open FStar.PCM
module G = FStar.Ghost
module Set = FStar.Set
module T = FStar.Tactics.V2
open Pulse.Lib.Dv {}
open FStar.ExtractAs
Expand Down
1 change: 0 additions & 1 deletion lib/core/Pulse.Lib.Core.fst
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,6 @@ module Pulse.Lib.Core
module I = PulseCore.InstantiatedSemantics
module A = PulseCore.Atomic
module T = FStar.Tactics.V2
module F = FStar.FunctionalExtensionality
open PulseCore.InstantiatedSemantics
open PulseCore.FractionalPermission
open PulseCore.Observability
Expand Down
1 change: 0 additions & 1 deletion lib/core/PulseCore.Action.fst
Original file line number Diff line number Diff line change
Expand Up @@ -367,7 +367,6 @@ let exists_equiv (#a:_) (#p:a -> slprop)
let pf = FStar.Squash.return_squash pf in
I.slprop_equiv_elim (op_exists_Star p) (exists* x. p x)

module T = FStar.Tactics
let fresh_invariant ctx p = fun #ictx -> ITA.fresh_invariant ictx p ctx

let inames_live_inv (i:iref) (p:slprop) = fun #ictx -> ITA.inames_live_inv ictx i p
Expand Down
2 changes: 0 additions & 2 deletions lib/core/PulseCore.Action.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -16,9 +16,7 @@

module PulseCore.Action

module S = FStar.Set
module I = PulseCore.InstantiatedSemantics
module PP = PulseCore.Preorder
module Sep = PulseCore.IndirectionTheorySep
open FStar.PCM
open FStar.Ghost
Expand Down
1 change: 0 additions & 1 deletion lib/core/PulseCore.Atomic.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -334,7 +334,6 @@ val buy1 ()
// References
////////////////////////////////////////////////////////////////////////
open FStar.PCM
module PP = PulseCore.Preorder

val pts_to_not_null
(#a:Type u#1)
Expand Down
2 changes: 0 additions & 2 deletions lib/core/PulseCore.CompactHeapSig.fst
Original file line number Diff line number Diff line change
Expand Up @@ -2,8 +2,6 @@ module PulseCore.CompactHeapSig
open FStar.Ghost
open FStar.PCM
open PulseCore.HeapSig
module H2 = PulseCore.Heap2
module ST = PulseCore.HoareStateMonad
module CM = FStar.Algebra.CommMonoid
open FStar.Tactics.Typeclasses

Expand Down
2 changes: 0 additions & 2 deletions lib/core/PulseCore.Heap.fst
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,6 @@ module PulseCore.Heap
module F = FStar.FunctionalExtensionality
open FStar.FunctionalExtensionality
open FStar.PCM
module Frac = PulseCore.FractionalPermission
module PP = PulseCore.Preorder

#set-options "--fuel 1 --ifuel 1"
Expand Down Expand Up @@ -270,7 +269,6 @@ let join_empty_inverse (m0 m1:heap)
////////////////////////////////////////////////////////////////////////////////
let slprop = p:(heap ^-> prop) { heap_prop_is_affine p }

module W = FStar.WellFounded


let interp (p:slprop u#a) (m:heap u#a)
Expand Down
1 change: 0 additions & 1 deletion lib/core/PulseCore.Heap.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -16,7 +16,6 @@
module PulseCore.Heap
open FStar.Ghost
open FStar.PCM
module Frac = PulseCore.FractionalPermission

/// This module defines the behavior of a structured heap where each memory cell is governed by
/// a partial commutative monoid. This PCM structure is reused for the entire heap as it is possible
Expand Down
2 changes: 0 additions & 2 deletions lib/core/PulseCore.Heap2.fst
Original file line number Diff line number Diff line change
Expand Up @@ -3,8 +3,6 @@ module F = FStar.FunctionalExtensionality
open FStar.FunctionalExtensionality
open FStar.PCM
open PulseCore.Tags
module Frac = PulseCore.FractionalPermission
module PP = PulseCore.Preorder
module H = PulseCore.Heap

noeq
Expand Down
2 changes: 0 additions & 2 deletions lib/core/PulseCore.HeapSig.fst
Original file line number Diff line number Diff line change
@@ -1,8 +1,6 @@
module PulseCore.HeapSig
open FStar.Ghost
open FStar.PCM
module H2 = PulseCore.Heap2
module ST = PulseCore.HoareStateMonad
module CM = FStar.Algebra.CommMonoid

let star_commutative #h p q =
Expand Down
3 changes: 0 additions & 3 deletions lib/core/PulseCore.IndirectionTheoryActions.fst
Original file line number Diff line number Diff line change
Expand Up @@ -14,10 +14,7 @@
limitations under the License.
*)
module PulseCore.IndirectionTheoryActions
module F = FStar.FunctionalExtensionality
module T = FStar.Tactics
module PM = PulseCore.MemoryAlt
module HST = PulseCore.HoareStateMonad
open FStar.Ghost

let pm_sep_laws () : squash (
Expand Down
2 changes: 0 additions & 2 deletions lib/core/PulseCore.IndirectionTheoryActions.fsti
Original file line number Diff line number Diff line change
@@ -1,6 +1,4 @@
module PulseCore.IndirectionTheoryActions
module F = FStar.FunctionalExtensionality
module T = FStar.Tactics
module PM = PulseCore.MemoryAlt
module HST = PulseCore.HoareStateMonad
open PulseCore.IndirectionTheorySep
Expand Down
2 changes: 0 additions & 2 deletions lib/core/PulseCore.IndirectionTheorySep.fst
Original file line number Diff line number Diff line change
Expand Up @@ -19,8 +19,6 @@ open PulseCore.KnotInstantiation
open FStar.FunctionalExtensionality
module F = FStar.FunctionalExtensionality
module PM = PulseCore.MemoryAlt
module HS = PulseCore.HeapSig
module IT = PulseCore.IndirectionTheory
open FStar.Ghost {erased, hide, reveal}

let timeless_heap_le (a b: timeless_heap_sig.mem) : prop =
Expand Down
3 changes: 0 additions & 3 deletions lib/core/PulseCore.InstantiatedSemantics.fst
Original file line number Diff line number Diff line change
Expand Up @@ -17,8 +17,6 @@ module PulseCore.InstantiatedSemantics

module Sem = PulseCore.Semantics
module Sep = PulseCore.IndirectionTheorySep
module ITA = PulseCore.IndirectionTheoryActions
module U = FStar.Universe
module F = FStar.FunctionalExtensionality

open PulseCore.IndirectionTheorySep
Expand Down Expand Up @@ -80,7 +78,6 @@ let slprop_equiv_elim p q = ()
let slprop_equiv_unit p = unsquash ()
let slprop_equiv_comm p1 p2 = unsquash ()
let slprop_equiv_assoc p1 p2 p3 = unsquash ()
module T = FStar.Tactics.V2
let slprop_equiv_exists
(#a:Type)
(p q: a -> slprop)
Expand Down
2 changes: 0 additions & 2 deletions lib/core/PulseCore.KnotInstantiation.fst
Original file line number Diff line number Diff line change
Expand Up @@ -18,8 +18,6 @@ module PulseCore.KnotInstantiation
open PulseCore.IndirectionTheory
open FStar.FunctionalExtensionality
module F = FStar.FunctionalExtensionality
module PM = PulseCore.MemoryAlt
module HS = PulseCore.HeapSig
module IT = PulseCore.IndirectionTheory
open FStar.Ghost {erased, hide, reveal}

Expand Down
3 changes: 0 additions & 3 deletions lib/core/PulseCore.MemoryAlt.fst
Original file line number Diff line number Diff line change
Expand Up @@ -17,9 +17,7 @@
module PulseCore.MemoryAlt
open FStar.Ghost
open FStar.PCM
module PST = PulseCore.HoareStateMonad
module U = FStar.Universe
module S = FStar.Set
module CM = FStar.Algebra.CommMonoid
module H = PulseCore.HeapSig
module E = PulseCore.HeapExtension
Expand Down Expand Up @@ -169,7 +167,6 @@ let star (p1 p2:slprop u#a)
: slprop u#a
= sig.star p1 p2

module F = FStar.FunctionalExtensionality
let h_exists (#a:Type u#b) (f: (a -> slprop u#a))
: slprop u#a
= H.exists_ #sig #a (fun x -> reveal_slprop (f x))
Expand Down
1 change: 0 additions & 1 deletion lib/core/PulseCore.MemoryAlt.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -19,7 +19,6 @@ open FStar.Ghost
open FStar.PCM
module PST = PulseCore.HoareStateMonad
module U = FStar.Universe
module S = FStar.Set
module CM = FStar.Algebra.CommMonoid
/// This module adds memory invariants to the heap to expose the
/// final interface for Pulse's PCM-based memory model.
Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.AnchoredReference.fst
Original file line number Diff line number Diff line change
Expand Up @@ -24,7 +24,6 @@ open PulseCore.Preorder
open Pulse.Lib.FractionalAnchoredPreorder
module FRAP = Pulse.Lib.FractionalAnchoredPreorder
module GPR = Pulse.Lib.GhostPCMReference
module U32 = FStar.UInt32
module T = FStar.Tactics

let carrier (#a:Type0) (#p:preorder a) (#anc:anchor_rel p)
Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.AnchoredReference.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -22,7 +22,6 @@ open FStar.Preorder
open Pulse.Lib.FractionalAnchoredPreorder
#lang-pulse

module U32 = FStar.UInt32
module T = FStar.Tactics

[@@erasable]
Expand Down
2 changes: 0 additions & 2 deletions lib/pulse/lib/Pulse.Lib.Array.fst
Original file line number Diff line number Diff line change
Expand Up @@ -16,7 +16,6 @@

module Pulse.Lib.Array
#lang-pulse
module PM = Pulse.Main
open Pulse.Lib.Core
open Pulse.Lib.Reference
open Pulse.Lib.Array.Core
Expand All @@ -26,7 +25,6 @@ module US = FStar.SizeT
module U8 = FStar.UInt8
open Pulse.Lib.BoundedIntegers
module A = Pulse.Lib.Array.Core
module R = Pulse.Lib.Reference

#set-options "--print_implicits"

Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.BigReference.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,6 @@ module Pulse.Lib.BigReference
open Pulse.Lib.Core
open PulseCore.FractionalPermission
open FStar.Ghost
module U32 = FStar.UInt32
module T = FStar.Tactics
val ref ([@@@unused]a:Type u#2) : Type u#0

Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.Box.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -22,7 +22,6 @@ open PulseCore.FractionalPermission
open Pulse.Lib.Core
open Pulse.Class.PtsTo

module U32 = FStar.UInt32
module T = FStar.Tactics.V2

module R = Pulse.Lib.Reference
Expand Down
3 changes: 0 additions & 3 deletions lib/pulse/lib/Pulse.Lib.Deque.fst
Original file line number Diff line number Diff line change
Expand Up @@ -5,9 +5,6 @@ open Pulse.Lib.Pervasives
open Pulse.Lib.Stick.Util
open FStar.List.Tot
open Pulse.Lib.Trade
module T = FStar.Tactics
module I = Pulse.Lib.Stick.Util
module FA = Pulse.Lib.Forall.Util
module Box = Pulse.Lib.Box

noeq
Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.DequeRef.fst
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ module Pulse.Lib.DequeRef
open Pulse.Lib.Pervasives
open Pulse.Lib.Deque
module B = Pulse.Lib.Box
module DQ = Pulse.Lib.Deque
open FStar.List.Tot

let dq (t:Type0) = B.box (deque t)
Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.HashTable.Type.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,6 @@ module Pulse.Lib.HashTable.Type

open Pulse.Lib.Pervasives
module V = Pulse.Lib.Vec
module R = Pulse.Lib.Reference
module SZ = FStar.SizeT

open Pulse.Lib.HashTable.Spec
Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.HashTable.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -21,7 +21,6 @@ open Pulse.Lib.HashTable.Spec
open Pulse.Lib.HashTable.Type

module V = Pulse.Lib.Vec
module R = Pulse.Lib.Reference
module SZ = FStar.SizeT
module PHT = Pulse.Lib.HashTable.Spec

Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.HigherReference.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -19,7 +19,6 @@ open Pulse.Lib.Core
open PulseCore.FractionalPermission
open FStar.Ghost
open Pulse.Class.PtsTo
module U32 = FStar.UInt32
module T = FStar.Tactics
val ref ([@@@unused]a:Type u#1) : Type u#0

Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.LinkedList.fst
Original file line number Diff line number Diff line change
Expand Up @@ -19,7 +19,6 @@ module Pulse.Lib.LinkedList
open Pulse.Lib.Pervasives
open Pulse.Lib.Stick.Util
open FStar.List.Tot
module T = FStar.Tactics
module I = Pulse.Lib.Stick.Util
module FA = Pulse.Lib.Forall.Util

Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.MonotonicGhostRef.fst
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,6 @@ open Pulse.Lib.GhostPCMReference
open FStar.Preorder
module GR = Pulse.Lib.GhostPCMReference
module FP = Pulse.Lib.PCM.FractionalPreorder
module PP = PulseCore.Preorder


let mref (#t:Type) (p:preorder t) = GR.gref (FP.fp_pcm p)
Expand Down
3 changes: 0 additions & 3 deletions lib/pulse/lib/Pulse.Lib.MonotonicGhostRef.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -3,9 +3,6 @@ module Pulse.Lib.MonotonicGhostRef
open Pulse.Lib.Pervasives
open Pulse.Lib.GhostPCMReference
open FStar.Preorder
module GR = Pulse.Lib.GhostPCMReference
module FP = Pulse.Lib.PCM.FractionalPreorder
module PP = PulseCore.Preorder

let as_prop (t:Type0) = t <==> True

Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.PCM.FractionalPreorder.fst
Original file line number Diff line number Diff line change
Expand Up @@ -21,7 +21,6 @@ open FStar.Preorder
open PulseCore.Preorder
open PulseCore.FractionalPermission

module L = FStar.List.Tot

type pcm_carrier (#a:Type u#a) (p:preorder a) : Type u#a = option perm & hist p

Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.Primitives.fst
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,6 @@
module Pulse.Lib.Primitives
#lang-pulse

module B = Pulse.Lib.Box

friend Pulse.Lib.Box

Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.SeqMatch.fst
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,6 @@ open Pulse.Lib.OnRange
open Pulse.Lib.Stick.Util

module Seq = FStar.Seq
module SZ = FStar.SizeT

(* `seq_list_match` describes how to match a sequence of low-level
values (the low-level contents of an array) with a list of high-level
Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.SeqMatch.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,6 @@ include Pulse.Lib.Pervasives
open Pulse.Lib.Stick

module Seq = FStar.Seq
module SZ = FStar.SizeT

(* `seq_list_match` describes how to match a sequence of low-level
values (the low-level contents of an array) with a list of high-level
Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.Swap.Array.fst
Original file line number Diff line number Diff line change
Expand Up @@ -16,7 +16,6 @@

module Pulse.Lib.Swap.Array
#lang-pulse
module R = Pulse.Lib.Reference
module Prf = Pulse.Lib.Swap.Spec
open Pulse.Lib.Swap.Common
#set-options "--fuel 2 --ifuel 1"
Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/Pulse.Lib.Swap.Slice.fst
Original file line number Diff line number Diff line change
Expand Up @@ -16,7 +16,6 @@

module Pulse.Lib.Swap.Slice
#lang-pulse
module R = Pulse.Lib.Reference
module Prf = Pulse.Lib.Swap.Spec
open Pulse.Lib.Swap.Common
#set-options "--fuel 2 --ifuel 1"
Expand Down
2 changes: 0 additions & 2 deletions lib/pulse/lib/Pulse.Lib.Task.fst
Original file line number Diff line number Diff line change
Expand Up @@ -30,8 +30,6 @@ open Pulse.Lib.SpinLock
module RTC = FStar.ReflexiveTransitiveClosure
module FRAP = Pulse.Lib.FractionalAnchoredPreorder
module AR = Pulse.Lib.AnchoredReference
module Big = Pulse.Lib.BigReference
module Ghost = Pulse.Lib.GhostReference

noeq
type task_state : Type0 =
Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/pledge/Pulse.Lib.Shift.fst
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,6 @@ open FStar.Ghost
open Pulse.Class.Duplicable
open Pulse.Lib.Pervasives

module T = FStar.Tactics

let shift_elim_t is hyp extra concl : Type u#4 =
unit -> stt_ghost unit is (extra ** hyp) (fun _ -> concl)
Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/pledge/Pulse.Lib.SmallTrade.fst
Original file line number Diff line number Diff line change
Expand Up @@ -21,7 +21,6 @@ open FStar.Ghost
open Pulse.Lib.Core
open Pulse.Lib.Pervasives

module T = FStar.Tactics

type small_slprop = v:slprop { timeless v }

Expand Down
1 change: 0 additions & 1 deletion lib/pulse/lib/pledge/Pulse.Lib.Trade.fst
Original file line number Diff line number Diff line change
Expand Up @@ -19,7 +19,6 @@ module Pulse.Lib.Trade

open Pulse.Lib.Pervasives

module T = FStar.Tactics

let trade_elim_t is hyp extra concl : Type u#4 =
unit -> stt_ghost unit is (extra ** hyp) (fun _ -> concl)
Expand Down
2 changes: 0 additions & 2 deletions pulse2rust/src/Pulse2Rust.Deps.fst
Original file line number Diff line number Diff line change
Expand Up @@ -30,9 +30,7 @@ open RustBindings
open FStarC.Class.Setlike

module S = FStarC.Extraction.ML.Syntax
module EUtil = FStarC.Extraction.ML.Util

module UEnv = FStarC.Extraction.ML.UEnv

let empty_defs : reachable_defs = RBSet.empty ()
let singleton (p:S.mlpath) : reachable_defs = singleton (S.string_of_mlpath p)
Expand Down
2 changes: 0 additions & 2 deletions pulse2rust/src/Pulse2Rust.Deps.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -27,9 +27,7 @@ open Pulse2Rust.Extract
open RustBindings

module S = FStarC.Extraction.ML.Syntax
module EUtil = FStarC.Extraction.ML.Util

module UEnv = FStarC.Extraction.ML.UEnv

val empty_defs : reachable_defs

Expand Down
2 changes: 0 additions & 2 deletions pulse2rust/src/Pulse2Rust.Env.fst
Original file line number Diff line number Diff line change
Expand Up @@ -26,9 +26,7 @@ open Pulse2Rust.Rust.Syntax

open RustBindings

module S = FStarC.Extraction.ML.Syntax

module UEnv = FStarC.Extraction.ML.UEnv

let fail (s:string) =
failwith (format1 "Pulse to Rust extraction failed: %s" s)
Expand Down
Loading

0 comments on commit dac35ec

Please sign in to comment.