Expand description
Defines how flux represents refinement types internally. Definitions in this module are used
during refinement type checking. A couple of important differences between definitions in this
module and in crate::fhir
are:
- Types in this module use debruijn indices to represent local binders.
- Data structures are interned so they can be cheaply cloned.
Re-exports§
pub use normalize::NormalizeInfo;
pub use normalize::NormalizedDefns;
pub use normalize::local_deps;
pub use crate::fhir::InferMode;
pub use SortInfer::*;
pub use flux_rustc_bridge::ty::Region::*;
Modules§
- binder 🔒
- canonicalize
- A canonical type is a type where all existentials and constraint predicates are hoisted to
the top level. For example, the canonical version of
∃a. {∃b. i32[a + b] | b > 0}
is∃a,b. {i32[a + b] | b > 0}
. - expr 🔒
- fold
- This modules follows the implementation of folding in rustc. For more information read the
documentation in
rustc_middle::ty::fold
. - normalize
- pretty 🔒
- refining
- Refining is the process of generating a refined version of a rust type.
- region_
matching - subst
Macros§
Structs§
- AdtDef
- AdtDef
Data - AdtSort
Def - The definition of the data sort automatically generated for a struct or enum.
- AdtSort
DefData 🔒 - AdtSort
Variant - Alias
Reft - AliasTy
- Assoc
Refinements - Binder
- Bound
Reft - Bound
Region - BvSize
Vid - A bit vector size vvariable id
- Clause
- Const
- Coroutine
Oblig Predicate - ESpan
- EVid
- Existential variable id
- Early
Binder - Early
Reft Param - Existential
Projection - Existential
Trait Ref - Expr
- FnOutput
- FnSig
- FnTrait
Predicate - Func
Sort - Generic
Param Def - Generic
Predicates - Generics
- Invariant
- KVar
- In theory a kvar is just an unknown predicate that can use some variables in scope. In practice, fixpoint makes a difference between the first and the rest of the arguments, the first one being the kvar’s self argument. Fixpoint will only instantiate qualifiers that use the self argument. Flux generalizes the self argument to be a list. We call the rest of the arguments the scope.
- KVid
- Lambda
- A lambda abstraction with an elaborated output sort. We need the output sort of lambdas for encoding into fixpoint
- Local
Table InContext - Local
Table InContext Mut - Name
- NumVid
- A numeric vvariable id
- Outlives
Predicate - Param
Sort ParamSort
is used for polymorphic sorts (Set
,Map
, etc.) and bit-vector size parameters. They should occur “bound” under aPolyFuncSort
or anAdtSortDef
. We assume there’s a single binder and aParamSort
represents a variable as an index into the list of variables bound by that binder, i.e., the representation doesnt’t support higher-ranked sorts.- Path
- Poly
Func Sort - A polymorphic function sort parametric over sorts or bit-vector sizes.
- Projection
Predicate - Qualifier
- Real
- Refine
Param - Refinement
Generics - SortVid
- A sort vvariable id
- Subset
Ty - A subset type is a simplified version of a type that has the form
{b[e] | p}
whereb
is aBaseTy
,e
a refinement index, andp
a predicate. - Trait
Predicate - Trait
Ref - Ty
- Variant
Sig - Wfck
Results - AdtFlags
- Bound
Var - Const
Vid - A
const
variable ID. - Debruijn
Index - A De Bruijn index is a standard means of representing regions (and perhaps later types) in a higher-ranked setting. In particular, imagine a type like this:
- Early
Param Region - Late
Param Region - The parameter representation of late-bound function parameters, “some region
at least as big as the scope
fr.scope
”. - Param
Const - ParamTy
- Region
Vid - A region variable ID.
- Scalar
Int - The raw bytes of a simple value.
- TyVid
- A type variable ID.
- Variant
Idx - The source-order index of a variant in a type.
Enums§
- Aggregate
Kind - Alias
Kind - BaseTy
- BinOp
- Bound
Reft Kind - Bound
Variable Kind - BvSize
- The size of a bit-vector
- Clause
Kind - Coercion
- Const
Kind - Constant
- Constant
Info - Ctor
- Ensures
- Existential
Predicate - Expr
Kind - Field
Proj - Generic
Arg - Generic
Param DefKind - Hole
Kind - The position where a hole appears. This determines how it will be inferred. This is related
to, but not the same as, an
InferMode
. - Loc
- NumVar
Value - Opaqueness
- Option-like enum to explicitly mark that we don’t have information about an ADT because it was
annotated with
#[flux::opaque]
. Note that only structs can be marked as opaque. - PtrKind
- Region
- Sort
- SortArg
- An argument for a generic parameter in a
Sort
which can be either a generic sort or a generic bit-vector size. - Sort
Ctor - Sort
Infer - A placeholder for a sort that needs to be inferred
- Sort
Param Kind - See
PolyFuncSort
- TyKind
- TyOr
Base - TyOr
Ctor - UnOp
- Var
- Bound
Region Kind - Closure
Kind - Represents the various closure traits in the language. This
will determine the type of the environment (
self
, in the desugaring) argument that the closure expects. - FloatTy
- IntTy
- Late
Param Region Kind - When liberating bound regions, we map their
BoundRegionKind
to this as we need to track the index of anonymous regions. We otherwise end up liberating multiple bound regions to the same late-bound region. - Mutability
- UintTy
Constants§
- SELF_
PARAM_ TY - FIRST_
VARIANT - Equivalent to
VariantIdx(0)
. - INNERMOST
Statics§
Traits§
Functions§
- int_
invariants 🔒 - slice_
invariants 🔒 - returns the same invariants as for
usize
which is the length of a slice - uint_
invariants 🔒
Type Aliases§
- Bound
Variable Kinds - Clauses
- Generic
Args - Item
Local Map - List
- Poly
Existential Predicate - Poly
Existential Trait Ref - Poly
FnSig - Poly
Projection Predicate - Poly
Trait Predicate - Poly
Trait Ref - Poly
Variant - Poly
Variants - Refine
Args - Region
Outlives Predicate - Subset
TyCtor - A type constructor meant to be used as generic a argument of kind base. This is just an alias
to
Binder<SubsetTy>
, but we expect the binder to have a single bound variable of the sort of the underlying base type. - TyCtor
- Type
Outlives Predicate