Skip to content

Commit

Permalink
Run `.scripts/remove_all_unused_opens.sh src/ ulib/ doc/ tests/ examp…
Browse files Browse the repository at this point in the history
…les/ contrib/`
  • Loading branch information
mtzguido committed Feb 14, 2025
1 parent 69287dd commit 9b7eb79
Show file tree
Hide file tree
Showing 162 changed files with 0 additions and 288 deletions.
3 changes: 0 additions & 3 deletions contrib/CoreCrypto/ml/Tests.ml
Original file line number Diff line number Diff line change
@@ -1,6 +1,3 @@
(* The original "Bytes" module from OCaml. *)
module B = Bytes

(* This brings [Platform.Bytes] into scope. *)
open CoreCrypto
open Platform
Expand Down
3 changes: 0 additions & 3 deletions doc/book/code/ContextPollution.fst
Original file line number Diff line number Diff line change
Expand Up @@ -3,9 +3,6 @@ module ContextPollution
let warmup (x:bool { x == true }) = assert x

//SNIPPET_START: context_test1$
module T = FStar.Tactics
module B = LowStar.Buffer
module SA = Steel.Array
open FStar.Seq

#push-options "--query_stats"
Expand Down
1 change: 0 additions & 1 deletion doc/book/code/exercises/Part3.Typeclasses.fst
Original file line number Diff line number Diff line change
@@ -1,5 +1,4 @@
module Part3.Typeclasses
module TC = FStar.Tactics.Typeclasses

class printable (a:Type) =
{
Expand Down
3 changes: 0 additions & 3 deletions doc/old/tutorial/code/exercises/LowStar.Ex3.fst
Original file line number Diff line number Diff line change
Expand Up @@ -27,9 +27,6 @@ open FStar.Integers
/// we don't end up referring to FStar.ST by accident.
module B = LowStar.Buffer
module HS = FStar.HyperStack
module M = LowStar.Modifies
module ST = FStar.HyperStack.ST
module S = FStar.Seq

/// This brings into scope the ``!*`` and ``*=`` operators, which are
/// specifically designed to operate on buffers of size 1, i.e. on pointers.
Expand Down
1 change: 0 additions & 1 deletion doc/old/tutorial/code/solutions/Ex12a1.Cap.fst
Original file line number Diff line number Diff line change
Expand Up @@ -23,7 +23,6 @@ open Platform.Bytes

module ACLs = Ex12a.ACLs
module MAC = Ex12.MAC
module SHA1 = Ex12.SHA1

// In Platform.Bytes: val utf8: s:string -> Tot bytes

Expand Down
2 changes: 0 additions & 2 deletions doc/old/tutorial/code/solutions/LowStar.Ex3.fst
Original file line number Diff line number Diff line change
Expand Up @@ -24,8 +24,6 @@ open FStar.Integers
module B = LowStar.Buffer
module HS = FStar.HyperStack
module M = LowStar.Modifies
module ST = FStar.HyperStack.ST
module S = FStar.Seq

/// This brings into scope the ``!*`` and ``*=`` operators, which are
/// specifically designed to operate on buffers of size 1, i.e. on pointers.
Expand Down
1 change: 0 additions & 1 deletion examples/crypto/HyE.AE.fst
Original file line number Diff line number Diff line change
Expand Up @@ -26,7 +26,6 @@ module CC = CoreCrypto
module B = Platform.Bytes

open HyE.Plain
module Plain = HyE.Plain

noeq type key : Type0 =
| Key: #region:erid -> raw:aes_key -> log:mlog_t region -> key
Expand Down
1 change: 0 additions & 1 deletion examples/crypto/HyE.AE.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -22,7 +22,6 @@ open HyE.Ideal

open Platform.Bytes
open CoreCrypto
module CC = CoreCrypto
module B = Platform.Bytes

open HyE.Plain
Expand Down
2 changes: 0 additions & 2 deletions examples/crypto/HyE.HCCA2.fst
Original file line number Diff line number Diff line change
Expand Up @@ -21,8 +21,6 @@ open HyE.PlainPKE
open Platform.Bytes
open FStar.HyperStack

module B = Platform.Bytes
module P = HyE.Plain
module C = HyE.CCA2
module A = HyE.AE
module RSA = HyE.RSA
Expand Down
1 change: 0 additions & 1 deletion examples/crypto/HyE.HCCA2.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -21,7 +21,6 @@ open HyE.PlainPKE
open Platform.Bytes
open FStar.HyperStack

module B = Platform.Bytes
module P = HyE.Plain
module C = HyE.CCA2
module A = HyE.AE
Expand Down
1 change: 0 additions & 1 deletion examples/crypto/HyE.RSA.fst
Original file line number Diff line number Diff line change
Expand Up @@ -32,7 +32,6 @@ open FStar.List.Tot
open Platform.Bytes
open CoreCrypto

module B = Platform.Bytes

assume type pkey
assume type skey
Expand Down
1 change: 0 additions & 1 deletion examples/crypto/OPLSS.Log.fst
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,6 @@ open FStar.HyperStack
module HS = FStar.HyperStack
module HST = FStar.HyperStack.ST
module B = LowStar.Monotonic.Buffer
module L = FStar.List.Tot

let grows (#a:Type)
: Preorder.preorder (seq a)
Expand Down
3 changes: 0 additions & 3 deletions examples/crypto/OPLSS.fst
Original file line number Diff line number Diff line change
@@ -1,8 +1,5 @@
module OPLSS
module UInt8 = FStar.UInt8
module HS = FStar.HyperStack
module ST = FStar.HyperStack.ST
module B = LowStar.Monotonic.Buffer
let bytes = Seq.seq UInt8.t
let lbytes l = b:bytes{Seq.length b = l}

Expand Down
1 change: 0 additions & 1 deletion examples/data_structures/LowStar.Lens.Buffer.fst
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,6 @@ open LowStar.Lens
open FStar.HyperStack.ST
module B = LowStar.Buffer
module HS = FStar.HyperStack
module HST = FStar.HyperStack.ST
open FStar.Integers

let mk #a #p #q (b:B.mbuffer a p q) (f:flavor b) (snap:HS.mem{B.live snap b})
Expand Down
1 change: 0 additions & 1 deletion examples/data_structures/LowStar.Lens.Tuple2.fst
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,6 @@ module LowStar.Lens.Tuple2
open LowStar.Lens
open FStar.HyperStack.ST
module B = LowStar.Buffer
module HS = FStar.HyperStack
module HST = FStar.HyperStack.ST
module LB = LowStar.Lens.Buffer

Expand Down
1 change: 0 additions & 1 deletion examples/data_structures/LowStar.Lens.fst
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,6 @@ module LowStar.Lens
open FStar.HyperStack.ST
module B = LowStar.Buffer
module HS = FStar.HyperStack
module HST = FStar.HyperStack.ST

let mods (l:hs_lens 'a 'b) (h:HS.mem) =
B.modifies (as_loc l.footprint) l.snapshot h /\
Expand Down
1 change: 0 additions & 1 deletion examples/data_structures/LowStar.Lens.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,6 @@ module LowStar.Lens
open FStar.HyperStack.ST
module B = LowStar.Buffer
module HS = FStar.HyperStack
module HST = FStar.HyperStack.ST

(* This module provides a more abstract way of verifying Low*
programs.
Expand Down
1 change: 0 additions & 1 deletion examples/dm4free/FStar.DM4F.Heap.fsti
Original file line number Diff line number Diff line change
Expand Up @@ -18,7 +18,6 @@ module FStar.DM4F.Heap
open FStar.Classical
open FStar.Set

module F = FStar.FunctionalExtensionality

(* Heap is a tuple of a source of freshness (the no. of the next
reference to be allocated) and a mapping of allocated raw
Expand Down
1 change: 0 additions & 1 deletion examples/doublylinkedlist/DoublyLinkedListIface.fst
Original file line number Diff line number Diff line change
Expand Up @@ -26,7 +26,6 @@ module DLL = DoublyLinkedList

module HS = FStar.HyperStack
module HST = FStar.HyperStack.ST
module G = FStar.Ghost
module L = FStar.List.Pure
module B = LowStar.Buffer

Expand Down
2 changes: 0 additions & 2 deletions examples/doublylinkedlist/Example.fst
Original file line number Diff line number Diff line change
Expand Up @@ -16,10 +16,8 @@

module Example

module HS = FStar.HyperStack
module HST = FStar.HyperStack.ST
module B = LowStar.Buffer
module DLL = DoublyLinkedListIface
module L = FStar.List.Tot

open DoublyLinkedListIface
Expand Down
1 change: 0 additions & 1 deletion examples/dsls/stlc/STLC.Infer.fst
Original file line number Diff line number Diff line change
Expand Up @@ -17,7 +17,6 @@
module STLC.Infer
module T = FStar.Tactics.V2
module R = FStar.Reflection.V2
module L = FStar.List.Tot
module RT = FStar.Reflection.Typing
open STLC.Core

Expand Down
1 change: 0 additions & 1 deletion examples/generic/Interop.fst
Original file line number Diff line number Diff line change
Expand Up @@ -11,7 +11,6 @@ module Interop
open FStar.FunctionalExtensionality
open FStar.Integers
open FStar.HyperStack.ST
module M = FStar.Map
module HS = FStar.HyperStack

(* A primitive to update the state monolithically with the result of a ghost function *)
Expand Down
3 changes: 0 additions & 3 deletions examples/interactive/FStar.InteractiveHelpers.ParseTest.fst
Original file line number Diff line number Diff line change
@@ -1,8 +1,5 @@
module FStar.InteractiveHelpers.ParseTest

module HS = FStar.HyperStack
module ST = FStar.HyperStack.ST
module B = LowStar.Buffer

open FStar.List
open FStar.Tactics.V2
Expand Down
1 change: 0 additions & 1 deletion examples/interactive/FStar.InteractiveHelpers.Tutorial.fst
Original file line number Diff line number Diff line change
Expand Up @@ -16,7 +16,6 @@ open FStar.InteractiveHelpers.Tutorial.Definitions
/// will need to restart the F* mode), which means that if you intend to use the
/// extended mode while working on a file, you have to make sure F* will load
/// FStar.InteractiveHelpers:
module FI = FStar.InteractiveHelpers
/// alternatively if you're not afraid of shadowing:
/// open FStar.InteractiveHelpers

Expand Down
1 change: 0 additions & 1 deletion examples/kv_parsing/EnumParsing.fst
Original file line number Diff line number Diff line change
Expand Up @@ -31,7 +31,6 @@ open FStar.HyperStack
open FStar.HyperStack.ST

module U8 = FStar.UInt8
module U16 = FStar.UInt16
module U32 = FStar.UInt32

(*! Pure model *)
Expand Down
2 changes: 0 additions & 2 deletions examples/kv_parsing/Parsing.fst
Original file line number Diff line number Diff line change
Expand Up @@ -31,9 +31,7 @@ module C = C
open C.Loops

module U8 = FStar.UInt8
module U16 = FStar.UInt16
module U32 = FStar.UInt32
module Cast = FStar.Int.Cast

type byte = U8.t
let bytes = seq byte
Expand Down
2 changes: 0 additions & 2 deletions examples/kv_parsing/PureEncoder.fst
Original file line number Diff line number Diff line change
Expand Up @@ -16,9 +16,7 @@
module PureEncoder

open FStar.Seq
module U16 = FStar.UInt16
module U32 = FStar.UInt32
module Cast = FStar.Int.Cast
module List = FStar.List.Tot

open KeyValue
Expand Down
3 changes: 0 additions & 3 deletions examples/kv_parsing/PureParser.fst
Original file line number Diff line number Diff line change
Expand Up @@ -21,10 +21,7 @@ open IntegerParsing

open FStar.Seq
open FStar.Krml.Endianness
module U8 = FStar.UInt8
module U16 = FStar.UInt16
module U32 = FStar.UInt32
module Cast = FStar.Int.Cast

(*** Spec-level pure parsing to values *)

Expand Down
2 changes: 0 additions & 2 deletions examples/kv_parsing/Serializer.fst
Original file line number Diff line number Diff line change
Expand Up @@ -20,9 +20,7 @@ open FStar.HyperStack
open FStar.HyperStack.ST
open FStar.Ghost
module B = FStar.Buffer
module U16 = FStar.UInt16
module U32 = FStar.UInt32
module Cast = FStar.Int.Cast

open KeyValue
open Slice
Expand Down
3 changes: 0 additions & 3 deletions examples/kv_parsing/Serializing.fst
Original file line number Diff line number Diff line change
Expand Up @@ -29,10 +29,7 @@ open FStar.Ghost
module C = C
open C.Loops

module U8 = FStar.UInt8
module U16 = FStar.UInt16
module U32 = FStar.UInt32
module Cast = FStar.Int.Cast

(* Note the lack of definitions around encoding, the pure specification for serialization.
Expand Down
2 changes: 0 additions & 2 deletions examples/kv_parsing/ValidatedAccess.fst
Original file line number Diff line number Diff line change
Expand Up @@ -31,9 +31,7 @@ open C.Loops

module B = FStar.Buffer

module U16 = FStar.UInt16
module U32 = FStar.UInt32
module I32 = FStar.Int32
module Cast = FStar.Int.Cast

(*** API to access validated but unparsed key-value buffer *)
Expand Down
2 changes: 0 additions & 2 deletions examples/kv_parsing/ValidatedParser.fst
Original file line number Diff line number Diff line change
Expand Up @@ -29,9 +29,7 @@ open FStar.HyperStack.ST

module B = FStar.Buffer

module U16 = FStar.UInt16
module U32 = FStar.UInt32
module Cast = FStar.Int.Cast

(*** API using validated but unparsed key-value buffer *)

Expand Down
3 changes: 0 additions & 3 deletions examples/kv_parsing/Validator.fst
Original file line number Diff line number Diff line change
Expand Up @@ -29,11 +29,8 @@ module C = C
// special karamel support for looping
open C.Loops

module B = FStar.Buffer

module U16 = FStar.UInt16
module U32 = FStar.UInt32
module Cast = FStar.Int.Cast

(*** Stateful validation of input buffer *)

Expand Down
1 change: 0 additions & 1 deletion examples/kv_parsing/VectorParsing.fst
Original file line number Diff line number Diff line change
Expand Up @@ -32,7 +32,6 @@ open C.Loops

module B = FStar.Buffer

module U8 = FStar.UInt8
module U16 = FStar.UInt16
module U32 = FStar.UInt32
module Cast = FStar.Int.Cast
Expand Down
3 changes: 0 additions & 3 deletions examples/layeredeffects/AlgForAll.fst
Original file line number Diff line number Diff line change
@@ -1,9 +1,6 @@
module AlgForAll

open FStar.Calc
module FE = FStar.FunctionalExtensionality
module F = FStar.FunctionalExtensionality
module W = FStar.WellFounded
module T = FStar.Tactics.V2
module ID5 = ID5
open Alg
Expand Down
3 changes: 0 additions & 3 deletions examples/layeredeffects/AlgHeap.fst
Original file line number Diff line number Diff line change
Expand Up @@ -5,10 +5,7 @@ module AlgHeap
open FStar.Tactics.V2
open FStar.List.Tot
open FStar.Universe
module L = Lattice
module Ghost = FStar.Ghost
module Map = FStar.Map
module T = FStar.Tactics.V2

type loc = int
type state = Map.t loc int
Expand Down
3 changes: 0 additions & 3 deletions examples/layeredeffects/AlgWP.fst
Original file line number Diff line number Diff line change
Expand Up @@ -7,9 +7,6 @@ WP from intensional information about the operations in the tree. *)

open FStar.List.Tot
open FStar.Calc
module FE = FStar.FunctionalExtensionality
module F = FStar.FunctionalExtensionality
module W = FStar.WellFounded
module T = FStar.Tactics.V2
// #show-options
module ID5 = ID5
Expand Down
3 changes: 0 additions & 3 deletions examples/layeredeffects/GenericPartialDM4A.fst
Original file line number Diff line number Diff line change
Expand Up @@ -3,9 +3,6 @@ module GenericPartialDM4A
open FStar.Tactics.V2
open FStar.Calc
open FStar.FunctionalExtensionality
module F = FStar.FunctionalExtensionality
module W = FStar.WellFounded
module T = FStar.Tactics.V2
open FStar.Preorder

// m is a monad.
Expand Down
3 changes: 0 additions & 3 deletions examples/layeredeffects/GenericTotalDM4A.fst
Original file line number Diff line number Diff line change
Expand Up @@ -3,9 +3,6 @@ module GenericTotalDM4A
open FStar.Tactics.V2
open FStar.Calc
open FStar.FunctionalExtensionality
module F = FStar.FunctionalExtensionality
module W = FStar.WellFounded
module T = FStar.Tactics.V2
open FStar.Preorder

// m is a monad.
Expand Down
1 change: 0 additions & 1 deletion examples/layeredeffects/HoareST.fst
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,6 @@ open FStar.Heap
open FStar.ST

module P = FStar.Preorder
module ST = FStar.ST

/// ST effect implemented as a layered effect over STATE

Expand Down
1 change: 0 additions & 1 deletion examples/layeredeffects/HoareSTPolyBind.fst
Original file line number Diff line number Diff line change
Expand Up @@ -20,7 +20,6 @@ open FStar.Heap
open FStar.ST

module P = FStar.Preorder
module ST = FStar.ST


/// ST effect implemented as a layered effect over STATE
Expand Down
1 change: 0 additions & 1 deletion examples/layeredeffects/ID3.fst
Original file line number Diff line number Diff line change
Expand Up @@ -71,7 +71,6 @@ sub_effect PURE ~> ID = lift_pure_nd
val test_f : unit -> ID int (as_pure_wp (fun p -> p 5 /\ p 3))
let test_f () = 3

module T = FStar.Tactics.V2

let l () : int =
reify (test_f ())
Expand Down
3 changes: 0 additions & 3 deletions examples/layeredeffects/ND.fst
Original file line number Diff line number Diff line change
Expand Up @@ -7,9 +7,6 @@ open FStar.List.Tot
open FStar.Calc

open FStar.FunctionalExtensionality
module F = FStar.FunctionalExtensionality
module W = FStar.WellFounded
module T = FStar.Tactics.V2

// m is a monad. In this particular example, lists
val m (a : Type u#a) : Type u#a
Expand Down
1 change: 0 additions & 1 deletion examples/layeredeffects/Z3EncodingIssue.fst
Original file line number Diff line number Diff line change
Expand Up @@ -38,7 +38,6 @@ open FStar.Integers

open FStar.HyperStack.ST

module HS = FStar.HyperStack

module B = LowStar.Buffer

Expand Down
Loading

0 comments on commit 9b7eb79

Please sign in to comment.