2019-02-23 08:24:07 -06:00
|
|
|
//! Methods for lowering the HIR to types. There are two main cases here:
|
|
|
|
//!
|
|
|
|
//! - Lowering a type reference like `&usize` or `Option<foo::bar::Baz>` to a
|
|
|
|
//! type: The entry point for this is `Ty::from_hir`.
|
|
|
|
//! - Building the type for an item: This happens through the `type_for_def` query.
|
|
|
|
//!
|
|
|
|
//! This usually involves resolving names, collecting generic arguments etc.
|
2019-04-09 15:04:59 -05:00
|
|
|
use std::iter;
|
2019-07-04 15:05:17 -05:00
|
|
|
use std::sync::Arc;
|
2019-02-23 08:24:07 -06:00
|
|
|
|
2019-07-04 15:05:17 -05:00
|
|
|
use super::{FnSig, GenericPredicate, Substs, TraitRef, Ty, TypeCtor};
|
2019-02-23 08:24:07 -06:00
|
|
|
use crate::{
|
2019-05-20 17:02:29 -05:00
|
|
|
adt::VariantDef,
|
2019-07-04 15:05:17 -05:00
|
|
|
generics::HasGenericParams,
|
|
|
|
generics::{GenericDef, WherePredicate},
|
|
|
|
nameres::Namespace,
|
|
|
|
path::{GenericArg, PathSegment},
|
|
|
|
resolve::{Resolution, Resolver},
|
2019-05-20 17:02:29 -05:00
|
|
|
ty::AdtDef,
|
2019-07-04 15:05:17 -05:00
|
|
|
type_ref::TypeRef,
|
|
|
|
BuiltinType, Const, Enum, EnumVariant, Function, HirDatabase, ModuleDef, Path, Static, Struct,
|
|
|
|
StructField, Trait, TypeAlias, Union,
|
2019-02-23 08:24:07 -06:00
|
|
|
};
|
|
|
|
|
|
|
|
impl Ty {
|
|
|
|
pub(crate) fn from_hir(db: &impl HirDatabase, resolver: &Resolver, type_ref: &TypeRef) -> Self {
|
|
|
|
match type_ref {
|
2019-03-21 16:20:03 -05:00
|
|
|
TypeRef::Never => Ty::simple(TypeCtor::Never),
|
2019-02-23 08:24:07 -06:00
|
|
|
TypeRef::Tuple(inner) => {
|
|
|
|
let inner_tys =
|
|
|
|
inner.iter().map(|tr| Ty::from_hir(db, resolver, tr)).collect::<Vec<_>>();
|
2019-05-04 12:07:25 -05:00
|
|
|
Ty::apply(
|
|
|
|
TypeCtor::Tuple { cardinality: inner_tys.len() as u16 },
|
|
|
|
Substs(inner_tys.into()),
|
|
|
|
)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
TypeRef::Path(path) => Ty::from_hir_path(db, resolver, path),
|
|
|
|
TypeRef::RawPtr(inner, mutability) => {
|
|
|
|
let inner_ty = Ty::from_hir(db, resolver, inner);
|
2019-03-21 16:20:03 -05:00
|
|
|
Ty::apply_one(TypeCtor::RawPtr(*mutability), inner_ty)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
TypeRef::Array(inner) => {
|
|
|
|
let inner_ty = Ty::from_hir(db, resolver, inner);
|
2019-03-21 16:20:03 -05:00
|
|
|
Ty::apply_one(TypeCtor::Array, inner_ty)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
TypeRef::Slice(inner) => {
|
|
|
|
let inner_ty = Ty::from_hir(db, resolver, inner);
|
2019-03-21 16:20:03 -05:00
|
|
|
Ty::apply_one(TypeCtor::Slice, inner_ty)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
TypeRef::Reference(inner, mutability) => {
|
|
|
|
let inner_ty = Ty::from_hir(db, resolver, inner);
|
2019-03-21 16:20:03 -05:00
|
|
|
Ty::apply_one(TypeCtor::Ref(*mutability), inner_ty)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
TypeRef::Placeholder => Ty::Unknown,
|
|
|
|
TypeRef::Fn(params) => {
|
2019-03-16 11:21:32 -05:00
|
|
|
let inner_tys =
|
2019-02-23 08:24:07 -06:00
|
|
|
params.iter().map(|tr| Ty::from_hir(db, resolver, tr)).collect::<Vec<_>>();
|
2019-03-16 12:14:41 -05:00
|
|
|
let sig = Substs(inner_tys.into());
|
2019-05-04 12:07:25 -05:00
|
|
|
Ty::apply(TypeCtor::FnPtr { num_args: sig.len() as u16 - 1 }, sig)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
TypeRef::Error => Ty::Unknown,
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
|
|
|
pub(crate) fn from_hir_path(db: &impl HirDatabase, resolver: &Resolver, path: &Path) -> Self {
|
|
|
|
// Resolve the path (in type namespace)
|
2019-06-08 10:38:14 -05:00
|
|
|
let resolution = resolver.resolve_path_without_assoc_items(db, path).take_types();
|
2019-02-23 08:24:07 -06:00
|
|
|
|
|
|
|
let def = match resolution {
|
|
|
|
Some(Resolution::Def(def)) => def,
|
|
|
|
Some(Resolution::LocalBinding(..)) => {
|
|
|
|
// this should never happen
|
|
|
|
panic!("path resolved to local binding in type ns");
|
|
|
|
}
|
|
|
|
Some(Resolution::GenericParam(idx)) => {
|
|
|
|
return Ty::Param {
|
|
|
|
idx,
|
2019-03-23 02:53:48 -05:00
|
|
|
// FIXME: maybe return name in resolution?
|
2019-02-23 08:24:07 -06:00
|
|
|
name: path
|
|
|
|
.as_ident()
|
|
|
|
.expect("generic param should be single-segment path")
|
|
|
|
.clone(),
|
|
|
|
};
|
|
|
|
}
|
|
|
|
Some(Resolution::SelfType(impl_block)) => {
|
|
|
|
return impl_block.target_ty(db);
|
|
|
|
}
|
|
|
|
None => return Ty::Unknown,
|
|
|
|
};
|
|
|
|
|
|
|
|
let typable: TypableDef = match def.into() {
|
|
|
|
None => return Ty::Unknown,
|
|
|
|
Some(it) => it,
|
|
|
|
};
|
|
|
|
let ty = db.type_for_def(typable, Namespace::Types);
|
|
|
|
let substs = Ty::substs_from_path(db, resolver, path, typable);
|
2019-02-24 10:25:41 -06:00
|
|
|
ty.subst(&substs)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
|
2019-02-23 15:59:01 -06:00
|
|
|
pub(super) fn substs_from_path_segment(
|
2019-02-23 08:24:07 -06:00
|
|
|
db: &impl HirDatabase,
|
|
|
|
resolver: &Resolver,
|
2019-02-23 15:59:01 -06:00
|
|
|
segment: &PathSegment,
|
2019-02-23 08:24:07 -06:00
|
|
|
resolved: TypableDef,
|
|
|
|
) -> Substs {
|
2019-05-19 08:08:16 -05:00
|
|
|
let def_generic: Option<GenericDef> = match resolved {
|
|
|
|
TypableDef::Function(func) => Some(func.into()),
|
|
|
|
TypableDef::Struct(s) => Some(s.into()),
|
2019-05-23 12:18:47 -05:00
|
|
|
TypableDef::Union(u) => Some(u.into()),
|
2019-05-19 08:08:16 -05:00
|
|
|
TypableDef::Enum(e) => Some(e.into()),
|
|
|
|
TypableDef::EnumVariant(var) => Some(var.parent_enum(db).into()),
|
|
|
|
TypableDef::TypeAlias(t) => Some(t.into()),
|
2019-05-30 06:05:35 -05:00
|
|
|
TypableDef::Const(_) | TypableDef::Static(_) | TypableDef::BuiltinType(_) => None,
|
2019-02-23 08:24:07 -06:00
|
|
|
};
|
2019-05-19 08:08:16 -05:00
|
|
|
substs_from_path_segment(db, resolver, segment, def_generic, false)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
2019-02-23 15:59:01 -06:00
|
|
|
|
|
|
|
/// Collect generic arguments from a path into a `Substs`. See also
|
|
|
|
/// `create_substs_for_ast_path` and `def_to_ty` in rustc.
|
|
|
|
pub(super) fn substs_from_path(
|
|
|
|
db: &impl HirDatabase,
|
|
|
|
resolver: &Resolver,
|
|
|
|
path: &Path,
|
|
|
|
resolved: TypableDef,
|
|
|
|
) -> Substs {
|
|
|
|
let last = path.segments.last().expect("path should have at least one segment");
|
|
|
|
let segment = match resolved {
|
2019-02-24 10:25:41 -06:00
|
|
|
TypableDef::Function(_)
|
|
|
|
| TypableDef::Struct(_)
|
2019-05-23 12:18:47 -05:00
|
|
|
| TypableDef::Union(_)
|
2019-02-24 10:25:41 -06:00
|
|
|
| TypableDef::Enum(_)
|
2019-02-25 01:27:47 -06:00
|
|
|
| TypableDef::Const(_)
|
2019-02-25 02:21:01 -06:00
|
|
|
| TypableDef::Static(_)
|
2019-05-30 06:05:35 -05:00
|
|
|
| TypableDef::TypeAlias(_)
|
|
|
|
| TypableDef::BuiltinType(_) => last,
|
2019-02-23 15:59:01 -06:00
|
|
|
TypableDef::EnumVariant(_) => {
|
|
|
|
// the generic args for an enum variant may be either specified
|
|
|
|
// on the segment referring to the enum, or on the segment
|
|
|
|
// referring to the variant. So `Option::<T>::None` and
|
|
|
|
// `Option::None::<T>` are both allowed (though the former is
|
|
|
|
// preferred). See also `def_ids_for_path_segments` in rustc.
|
|
|
|
let len = path.segments.len();
|
|
|
|
let segment = if len >= 2 && path.segments[len - 2].args_and_bindings.is_some() {
|
|
|
|
// Option::<T>::None
|
|
|
|
&path.segments[len - 2]
|
|
|
|
} else {
|
|
|
|
// Option::None::<T>
|
|
|
|
last
|
|
|
|
};
|
|
|
|
segment
|
|
|
|
}
|
|
|
|
};
|
|
|
|
Ty::substs_from_path_segment(db, resolver, segment, resolved)
|
|
|
|
}
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
|
2019-03-26 17:07:26 -05:00
|
|
|
pub(super) fn substs_from_path_segment(
|
|
|
|
db: &impl HirDatabase,
|
|
|
|
resolver: &Resolver,
|
|
|
|
segment: &PathSegment,
|
2019-05-19 08:08:16 -05:00
|
|
|
def_generic: Option<GenericDef>,
|
2019-03-26 17:07:26 -05:00
|
|
|
add_self_param: bool,
|
|
|
|
) -> Substs {
|
|
|
|
let mut substs = Vec::new();
|
2019-05-19 08:08:16 -05:00
|
|
|
let def_generics = def_generic.map(|def| def.generic_params(db)).unwrap_or_default();
|
|
|
|
|
2019-03-26 17:07:26 -05:00
|
|
|
let parent_param_count = def_generics.count_parent_params();
|
2019-04-09 15:04:59 -05:00
|
|
|
substs.extend(iter::repeat(Ty::Unknown).take(parent_param_count));
|
2019-03-26 17:07:26 -05:00
|
|
|
if add_self_param {
|
|
|
|
// FIXME this add_self_param argument is kind of a hack: Traits have the
|
|
|
|
// Self type as an implicit first type parameter, but it can't be
|
|
|
|
// actually provided in the type arguments
|
2019-04-09 15:04:59 -05:00
|
|
|
// (well, actually sometimes it can, in the form of type-relative paths: `<Foo as Default>::default()`)
|
2019-03-26 17:07:26 -05:00
|
|
|
substs.push(Ty::Unknown);
|
|
|
|
}
|
|
|
|
if let Some(generic_args) = &segment.args_and_bindings {
|
|
|
|
// if args are provided, it should be all of them, but we can't rely on that
|
2019-04-09 15:04:59 -05:00
|
|
|
let self_param_correction = if add_self_param { 1 } else { 0 };
|
|
|
|
let param_count = def_generics.params.len() - self_param_correction;
|
2019-03-26 17:07:26 -05:00
|
|
|
for arg in generic_args.args.iter().take(param_count) {
|
|
|
|
match arg {
|
|
|
|
GenericArg::Type(type_ref) => {
|
|
|
|
let ty = Ty::from_hir(db, resolver, type_ref);
|
|
|
|
substs.push(ty);
|
|
|
|
}
|
|
|
|
}
|
|
|
|
}
|
|
|
|
}
|
|
|
|
// add placeholders for args that were not provided
|
|
|
|
let supplied_params = substs.len();
|
|
|
|
for _ in supplied_params..def_generics.count_params_including_parent() {
|
|
|
|
substs.push(Ty::Unknown);
|
|
|
|
}
|
|
|
|
assert_eq!(substs.len(), def_generics.count_params_including_parent());
|
2019-05-19 08:08:16 -05:00
|
|
|
|
|
|
|
// handle defaults
|
|
|
|
if let Some(def_generic) = def_generic {
|
|
|
|
let default_substs = db.generic_defaults(def_generic);
|
|
|
|
assert_eq!(substs.len(), default_substs.len());
|
|
|
|
|
2019-05-20 04:48:58 -05:00
|
|
|
for (i, default_ty) in default_substs.iter().enumerate() {
|
|
|
|
if substs[i] == Ty::Unknown {
|
|
|
|
substs[i] = default_ty.clone();
|
2019-05-19 08:08:16 -05:00
|
|
|
}
|
2019-05-20 04:48:58 -05:00
|
|
|
}
|
2019-05-19 08:08:16 -05:00
|
|
|
}
|
|
|
|
|
2019-05-20 04:48:58 -05:00
|
|
|
Substs(substs.into())
|
2019-03-26 17:07:26 -05:00
|
|
|
}
|
|
|
|
|
|
|
|
impl TraitRef {
|
2019-05-05 07:21:00 -05:00
|
|
|
pub(crate) fn from_path(
|
2019-03-26 17:07:26 -05:00
|
|
|
db: &impl HirDatabase,
|
|
|
|
resolver: &Resolver,
|
2019-05-05 07:21:00 -05:00
|
|
|
path: &Path,
|
2019-03-31 13:02:16 -05:00
|
|
|
explicit_self_ty: Option<Ty>,
|
2019-03-26 17:07:26 -05:00
|
|
|
) -> Option<Self> {
|
2019-06-08 10:38:14 -05:00
|
|
|
let resolved = match resolver.resolve_path_without_assoc_items(db, &path).take_types()? {
|
2019-03-26 17:07:26 -05:00
|
|
|
Resolution::Def(ModuleDef::Trait(tr)) => tr,
|
|
|
|
_ => return None,
|
|
|
|
};
|
2019-03-31 13:02:16 -05:00
|
|
|
let mut substs = Self::substs_from_path(db, resolver, path, resolved);
|
|
|
|
if let Some(self_ty) = explicit_self_ty {
|
|
|
|
// FIXME this could be nicer
|
|
|
|
let mut substs_vec = substs.0.to_vec();
|
|
|
|
substs_vec[0] = self_ty;
|
|
|
|
substs.0 = substs_vec.into();
|
|
|
|
}
|
2019-03-26 17:07:26 -05:00
|
|
|
Some(TraitRef { trait_: resolved, substs })
|
|
|
|
}
|
|
|
|
|
2019-05-05 07:21:00 -05:00
|
|
|
pub(crate) fn from_hir(
|
|
|
|
db: &impl HirDatabase,
|
|
|
|
resolver: &Resolver,
|
|
|
|
type_ref: &TypeRef,
|
|
|
|
explicit_self_ty: Option<Ty>,
|
|
|
|
) -> Option<Self> {
|
|
|
|
let path = match type_ref {
|
|
|
|
TypeRef::Path(path) => path,
|
|
|
|
_ => return None,
|
|
|
|
};
|
|
|
|
TraitRef::from_path(db, resolver, path, explicit_self_ty)
|
|
|
|
}
|
|
|
|
|
2019-03-26 17:07:26 -05:00
|
|
|
fn substs_from_path(
|
|
|
|
db: &impl HirDatabase,
|
|
|
|
resolver: &Resolver,
|
|
|
|
path: &Path,
|
|
|
|
resolved: Trait,
|
|
|
|
) -> Substs {
|
|
|
|
let segment = path.segments.last().expect("path should have at least one segment");
|
2019-05-19 08:08:16 -05:00
|
|
|
substs_from_path_segment(db, resolver, segment, Some(resolved.into()), true)
|
2019-03-26 17:07:26 -05:00
|
|
|
}
|
2019-04-20 05:34:36 -05:00
|
|
|
|
|
|
|
pub(crate) fn for_trait(db: &impl HirDatabase, trait_: Trait) -> TraitRef {
|
|
|
|
let substs = Substs::identity(&trait_.generic_params(db));
|
|
|
|
TraitRef { trait_, substs }
|
|
|
|
}
|
2019-05-05 07:21:00 -05:00
|
|
|
|
|
|
|
pub(crate) fn for_where_predicate(
|
|
|
|
db: &impl HirDatabase,
|
|
|
|
resolver: &Resolver,
|
|
|
|
pred: &WherePredicate,
|
|
|
|
) -> Option<TraitRef> {
|
|
|
|
let self_ty = Ty::from_hir(db, resolver, &pred.type_ref);
|
|
|
|
TraitRef::from_path(db, resolver, &pred.trait_ref, Some(self_ty))
|
|
|
|
}
|
2019-03-26 17:07:26 -05:00
|
|
|
}
|
|
|
|
|
2019-02-23 08:24:07 -06:00
|
|
|
/// Build the declared type of an item. This depends on the namespace; e.g. for
|
|
|
|
/// `struct Foo(usize)`, we have two types: The type of the struct itself, and
|
|
|
|
/// the constructor function `(usize) -> Foo` which lives in the values
|
|
|
|
/// namespace.
|
|
|
|
pub(crate) fn type_for_def(db: &impl HirDatabase, def: TypableDef, ns: Namespace) -> Ty {
|
|
|
|
match (def, ns) {
|
|
|
|
(TypableDef::Function(f), Namespace::Values) => type_for_fn(db, f),
|
2019-05-20 17:02:29 -05:00
|
|
|
(TypableDef::Struct(s), Namespace::Types) => type_for_adt(db, s),
|
2019-02-23 08:24:07 -06:00
|
|
|
(TypableDef::Struct(s), Namespace::Values) => type_for_struct_constructor(db, s),
|
2019-05-20 17:02:29 -05:00
|
|
|
(TypableDef::Enum(e), Namespace::Types) => type_for_adt(db, e),
|
2019-02-23 08:24:07 -06:00
|
|
|
(TypableDef::EnumVariant(v), Namespace::Values) => type_for_enum_variant_constructor(db, v),
|
2019-05-23 12:18:47 -05:00
|
|
|
(TypableDef::Union(u), Namespace::Types) => type_for_adt(db, u),
|
2019-02-24 14:36:49 -06:00
|
|
|
(TypableDef::TypeAlias(t), Namespace::Types) => type_for_type_alias(db, t),
|
2019-02-25 01:27:47 -06:00
|
|
|
(TypableDef::Const(c), Namespace::Values) => type_for_const(db, c),
|
2019-02-25 02:21:01 -06:00
|
|
|
(TypableDef::Static(c), Namespace::Values) => type_for_static(db, c),
|
2019-05-30 06:05:35 -05:00
|
|
|
(TypableDef::BuiltinType(t), Namespace::Types) => type_for_builtin(t),
|
2019-02-23 08:24:07 -06:00
|
|
|
|
|
|
|
// 'error' cases:
|
|
|
|
(TypableDef::Function(_), Namespace::Types) => Ty::Unknown,
|
2019-05-23 12:18:47 -05:00
|
|
|
(TypableDef::Union(_), Namespace::Values) => Ty::Unknown,
|
2019-02-23 08:24:07 -06:00
|
|
|
(TypableDef::Enum(_), Namespace::Values) => Ty::Unknown,
|
|
|
|
(TypableDef::EnumVariant(_), Namespace::Types) => Ty::Unknown,
|
2019-02-24 14:36:49 -06:00
|
|
|
(TypableDef::TypeAlias(_), Namespace::Values) => Ty::Unknown,
|
2019-02-25 01:27:47 -06:00
|
|
|
(TypableDef::Const(_), Namespace::Types) => Ty::Unknown,
|
2019-02-25 02:21:01 -06:00
|
|
|
(TypableDef::Static(_), Namespace::Types) => Ty::Unknown,
|
2019-05-30 06:05:35 -05:00
|
|
|
(TypableDef::BuiltinType(_), Namespace::Values) => Ty::Unknown,
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
}
|
|
|
|
|
2019-03-16 11:29:55 -05:00
|
|
|
/// Build the signature of a callable item (function, struct or enum variant).
|
|
|
|
pub(crate) fn callable_item_sig(db: &impl HirDatabase, def: CallableDef) -> FnSig {
|
|
|
|
match def {
|
|
|
|
CallableDef::Function(f) => fn_sig_for_fn(db, f),
|
|
|
|
CallableDef::Struct(s) => fn_sig_for_struct_constructor(db, s),
|
|
|
|
CallableDef::EnumVariant(e) => fn_sig_for_enum_variant_constructor(db, e),
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
2019-02-23 08:24:07 -06:00
|
|
|
/// Build the type of a specific field of a struct or enum variant.
|
|
|
|
pub(crate) fn type_for_field(db: &impl HirDatabase, field: StructField) -> Ty {
|
|
|
|
let parent_def = field.parent_def(db);
|
|
|
|
let resolver = match parent_def {
|
|
|
|
VariantDef::Struct(it) => it.resolver(db),
|
|
|
|
VariantDef::EnumVariant(it) => it.parent_enum(db).resolver(db),
|
|
|
|
};
|
|
|
|
let var_data = parent_def.variant_data(db);
|
|
|
|
let type_ref = &var_data.fields().unwrap()[field.id].type_ref;
|
|
|
|
Ty::from_hir(db, &resolver, type_ref)
|
|
|
|
}
|
|
|
|
|
2019-07-09 14:34:23 -05:00
|
|
|
pub(crate) fn trait_env(
|
|
|
|
db: &impl HirDatabase,
|
|
|
|
resolver: &Resolver,
|
|
|
|
) -> Arc<super::TraitEnvironment> {
|
2019-06-29 12:14:52 -05:00
|
|
|
let predicates = resolver
|
|
|
|
.where_predicates_in_scope()
|
|
|
|
.map(|pred| {
|
|
|
|
TraitRef::for_where_predicate(db, &resolver, pred)
|
|
|
|
.map_or(GenericPredicate::Error, GenericPredicate::Implemented)
|
|
|
|
})
|
|
|
|
.collect::<Vec<_>>();
|
|
|
|
|
2019-07-09 14:34:23 -05:00
|
|
|
Arc::new(super::TraitEnvironment { predicates })
|
2019-06-29 12:14:52 -05:00
|
|
|
}
|
|
|
|
|
2019-05-05 07:21:00 -05:00
|
|
|
/// Resolve the where clause(s) of an item with generics.
|
2019-07-06 09:41:04 -05:00
|
|
|
pub(crate) fn generic_predicates_query(
|
2019-05-05 07:21:00 -05:00
|
|
|
db: &impl HirDatabase,
|
|
|
|
def: GenericDef,
|
|
|
|
) -> Arc<[GenericPredicate]> {
|
|
|
|
let resolver = def.resolver(db);
|
2019-07-06 09:41:04 -05:00
|
|
|
let predicates = resolver
|
|
|
|
.where_predicates_in_scope()
|
2019-05-05 07:21:00 -05:00
|
|
|
.map(|pred| {
|
|
|
|
TraitRef::for_where_predicate(db, &resolver, pred)
|
|
|
|
.map_or(GenericPredicate::Error, GenericPredicate::Implemented)
|
|
|
|
})
|
|
|
|
.collect::<Vec<_>>();
|
|
|
|
predicates.into()
|
|
|
|
}
|
|
|
|
|
2019-05-19 08:08:16 -05:00
|
|
|
/// Resolve the default type params from generics
|
2019-07-06 09:41:04 -05:00
|
|
|
pub(crate) fn generic_defaults_query(db: &impl HirDatabase, def: GenericDef) -> Substs {
|
2019-05-19 08:08:16 -05:00
|
|
|
let resolver = def.resolver(db);
|
|
|
|
let generic_params = def.generic_params(db);
|
|
|
|
|
|
|
|
let defaults = generic_params
|
|
|
|
.params_including_parent()
|
|
|
|
.into_iter()
|
|
|
|
.map(|p| {
|
|
|
|
p.default.as_ref().map_or(Ty::Unknown, |path| Ty::from_hir_path(db, &resolver, path))
|
|
|
|
})
|
|
|
|
.collect::<Vec<_>>();
|
|
|
|
|
|
|
|
Substs(defaults.into())
|
|
|
|
}
|
|
|
|
|
2019-03-16 11:21:32 -05:00
|
|
|
fn fn_sig_for_fn(db: &impl HirDatabase, def: Function) -> FnSig {
|
2019-06-18 12:07:35 -05:00
|
|
|
let data = def.data(db);
|
2019-03-16 11:21:32 -05:00
|
|
|
let resolver = def.resolver(db);
|
2019-06-18 12:07:35 -05:00
|
|
|
let params = data.params().iter().map(|tr| Ty::from_hir(db, &resolver, tr)).collect::<Vec<_>>();
|
|
|
|
let ret = Ty::from_hir(db, &resolver, data.ret_type());
|
2019-03-16 11:21:32 -05:00
|
|
|
FnSig::from_params_and_return(params, ret)
|
|
|
|
}
|
|
|
|
|
2019-02-23 08:24:07 -06:00
|
|
|
/// Build the declared type of a function. This should not need to look at the
|
|
|
|
/// function body.
|
|
|
|
fn type_for_fn(db: &impl HirDatabase, def: Function) -> Ty {
|
|
|
|
let generics = def.generic_params(db);
|
2019-04-20 05:34:36 -05:00
|
|
|
let substs = Substs::identity(&generics);
|
2019-03-21 16:20:03 -05:00
|
|
|
Ty::apply(TypeCtor::FnDef(def.into()), substs)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
|
2019-02-25 01:27:47 -06:00
|
|
|
/// Build the declared type of a const.
|
|
|
|
fn type_for_const(db: &impl HirDatabase, def: Const) -> Ty {
|
2019-06-18 12:07:35 -05:00
|
|
|
let data = def.data(db);
|
2019-02-25 01:27:47 -06:00
|
|
|
let resolver = def.resolver(db);
|
|
|
|
|
2019-06-18 12:07:35 -05:00
|
|
|
Ty::from_hir(db, &resolver, data.type_ref())
|
2019-02-25 01:27:47 -06:00
|
|
|
}
|
|
|
|
|
2019-02-25 02:21:01 -06:00
|
|
|
/// Build the declared type of a static.
|
|
|
|
fn type_for_static(db: &impl HirDatabase, def: Static) -> Ty {
|
2019-06-18 12:07:35 -05:00
|
|
|
let data = def.data(db);
|
2019-02-25 02:21:01 -06:00
|
|
|
let resolver = def.resolver(db);
|
|
|
|
|
2019-06-18 12:07:35 -05:00
|
|
|
Ty::from_hir(db, &resolver, data.type_ref())
|
2019-02-25 02:21:01 -06:00
|
|
|
}
|
|
|
|
|
2019-05-30 06:05:35 -05:00
|
|
|
/// Build the declared type of a static.
|
|
|
|
fn type_for_builtin(def: BuiltinType) -> Ty {
|
|
|
|
Ty::simple(match def {
|
|
|
|
BuiltinType::Char => TypeCtor::Char,
|
|
|
|
BuiltinType::Bool => TypeCtor::Bool,
|
|
|
|
BuiltinType::Str => TypeCtor::Str,
|
|
|
|
BuiltinType::Int(ty) => TypeCtor::Int(ty.into()),
|
|
|
|
BuiltinType::Float(ty) => TypeCtor::Float(ty.into()),
|
|
|
|
})
|
|
|
|
}
|
|
|
|
|
2019-03-16 11:21:32 -05:00
|
|
|
fn fn_sig_for_struct_constructor(db: &impl HirDatabase, def: Struct) -> FnSig {
|
2019-02-23 08:24:07 -06:00
|
|
|
let var_data = def.variant_data(db);
|
|
|
|
let fields = match var_data.fields() {
|
|
|
|
Some(fields) => fields,
|
2019-03-16 11:21:32 -05:00
|
|
|
None => panic!("fn_sig_for_struct_constructor called on unit struct"),
|
2019-02-23 08:24:07 -06:00
|
|
|
};
|
|
|
|
let resolver = def.resolver(db);
|
2019-03-16 11:21:32 -05:00
|
|
|
let params = fields
|
2019-02-23 08:24:07 -06:00
|
|
|
.iter()
|
|
|
|
.map(|(_, field)| Ty::from_hir(db, &resolver, &field.type_ref))
|
|
|
|
.collect::<Vec<_>>();
|
2019-05-20 17:02:29 -05:00
|
|
|
let ret = type_for_adt(db, def);
|
2019-03-16 11:21:32 -05:00
|
|
|
FnSig::from_params_and_return(params, ret)
|
|
|
|
}
|
|
|
|
|
|
|
|
/// Build the type of a tuple struct constructor.
|
|
|
|
fn type_for_struct_constructor(db: &impl HirDatabase, def: Struct) -> Ty {
|
|
|
|
let var_data = def.variant_data(db);
|
|
|
|
if var_data.fields().is_none() {
|
2019-05-20 17:02:29 -05:00
|
|
|
return type_for_adt(db, def); // Unit struct
|
2019-03-16 11:21:32 -05:00
|
|
|
}
|
|
|
|
let generics = def.generic_params(db);
|
2019-04-20 05:34:36 -05:00
|
|
|
let substs = Substs::identity(&generics);
|
2019-03-21 16:20:03 -05:00
|
|
|
Ty::apply(TypeCtor::FnDef(def.into()), substs)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
|
2019-03-16 11:21:32 -05:00
|
|
|
fn fn_sig_for_enum_variant_constructor(db: &impl HirDatabase, def: EnumVariant) -> FnSig {
|
2019-02-23 08:24:07 -06:00
|
|
|
let var_data = def.variant_data(db);
|
|
|
|
let fields = match var_data.fields() {
|
|
|
|
Some(fields) => fields,
|
2019-03-16 11:21:32 -05:00
|
|
|
None => panic!("fn_sig_for_enum_variant_constructor called for unit variant"),
|
2019-02-23 08:24:07 -06:00
|
|
|
};
|
|
|
|
let resolver = def.parent_enum(db).resolver(db);
|
2019-03-16 11:21:32 -05:00
|
|
|
let params = fields
|
2019-02-23 08:24:07 -06:00
|
|
|
.iter()
|
|
|
|
.map(|(_, field)| Ty::from_hir(db, &resolver, &field.type_ref))
|
|
|
|
.collect::<Vec<_>>();
|
2019-03-16 11:21:32 -05:00
|
|
|
let generics = def.parent_enum(db).generic_params(db);
|
2019-04-20 05:34:36 -05:00
|
|
|
let substs = Substs::identity(&generics);
|
2019-05-20 17:02:29 -05:00
|
|
|
let ret = type_for_adt(db, def.parent_enum(db)).subst(&substs);
|
2019-03-16 11:21:32 -05:00
|
|
|
FnSig::from_params_and_return(params, ret)
|
|
|
|
}
|
|
|
|
|
|
|
|
/// Build the type of a tuple enum variant constructor.
|
|
|
|
fn type_for_enum_variant_constructor(db: &impl HirDatabase, def: EnumVariant) -> Ty {
|
|
|
|
let var_data = def.variant_data(db);
|
|
|
|
if var_data.fields().is_none() {
|
2019-05-20 17:02:29 -05:00
|
|
|
return type_for_adt(db, def.parent_enum(db)); // Unit variant
|
2019-03-16 11:21:32 -05:00
|
|
|
}
|
|
|
|
let generics = def.parent_enum(db).generic_params(db);
|
2019-04-20 05:34:36 -05:00
|
|
|
let substs = Substs::identity(&generics);
|
2019-03-21 16:20:03 -05:00
|
|
|
Ty::apply(TypeCtor::FnDef(def.into()), substs)
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
|
2019-05-20 17:02:29 -05:00
|
|
|
fn type_for_adt(db: &impl HirDatabase, adt: impl Into<AdtDef> + HasGenericParams) -> Ty {
|
|
|
|
let generics = adt.generic_params(db);
|
|
|
|
Ty::apply(TypeCtor::Adt(adt.into()), Substs::identity(&generics))
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
|
|
|
|
2019-02-24 14:36:49 -06:00
|
|
|
fn type_for_type_alias(db: &impl HirDatabase, t: TypeAlias) -> Ty {
|
2019-02-24 10:25:41 -06:00
|
|
|
let generics = t.generic_params(db);
|
|
|
|
let resolver = t.resolver(db);
|
|
|
|
let type_ref = t.type_ref(db);
|
2019-04-20 05:34:36 -05:00
|
|
|
let substs = Substs::identity(&generics);
|
2019-05-12 10:53:44 -05:00
|
|
|
let inner = Ty::from_hir(db, &resolver, &type_ref.unwrap_or(TypeRef::Error));
|
2019-02-24 10:25:41 -06:00
|
|
|
inner.subst(&substs)
|
|
|
|
}
|
|
|
|
|
2019-02-23 08:24:07 -06:00
|
|
|
#[derive(Clone, Copy, Debug, PartialEq, Eq, Hash)]
|
|
|
|
pub enum TypableDef {
|
|
|
|
Function(Function),
|
|
|
|
Struct(Struct),
|
2019-05-23 12:18:47 -05:00
|
|
|
Union(Union),
|
2019-02-23 08:24:07 -06:00
|
|
|
Enum(Enum),
|
|
|
|
EnumVariant(EnumVariant),
|
2019-02-24 14:36:49 -06:00
|
|
|
TypeAlias(TypeAlias),
|
2019-02-25 01:27:47 -06:00
|
|
|
Const(Const),
|
2019-02-25 02:21:01 -06:00
|
|
|
Static(Static),
|
2019-05-30 06:05:35 -05:00
|
|
|
BuiltinType(BuiltinType),
|
2019-02-23 08:24:07 -06:00
|
|
|
}
|
2019-05-30 06:05:35 -05:00
|
|
|
impl_froms!(
|
|
|
|
TypableDef: Function,
|
|
|
|
Struct,
|
|
|
|
Union,
|
|
|
|
Enum,
|
|
|
|
EnumVariant,
|
|
|
|
TypeAlias,
|
|
|
|
Const,
|
|
|
|
Static,
|
|
|
|
BuiltinType
|
|
|
|
);
|
2019-02-23 08:24:07 -06:00
|
|
|
|
|
|
|
impl From<ModuleDef> for Option<TypableDef> {
|
|
|
|
fn from(def: ModuleDef) -> Option<TypableDef> {
|
|
|
|
let res = match def {
|
|
|
|
ModuleDef::Function(f) => f.into(),
|
|
|
|
ModuleDef::Struct(s) => s.into(),
|
2019-05-23 12:18:47 -05:00
|
|
|
ModuleDef::Union(u) => u.into(),
|
2019-02-23 08:24:07 -06:00
|
|
|
ModuleDef::Enum(e) => e.into(),
|
|
|
|
ModuleDef::EnumVariant(v) => v.into(),
|
2019-02-24 14:36:49 -06:00
|
|
|
ModuleDef::TypeAlias(t) => t.into(),
|
2019-02-25 01:27:47 -06:00
|
|
|
ModuleDef::Const(v) => v.into(),
|
2019-02-25 02:21:01 -06:00
|
|
|
ModuleDef::Static(v) => v.into(),
|
2019-05-30 06:05:35 -05:00
|
|
|
ModuleDef::BuiltinType(t) => t.into(),
|
2019-02-25 02:21:01 -06:00
|
|
|
ModuleDef::Module(_) | ModuleDef::Trait(_) => return None,
|
2019-02-23 08:24:07 -06:00
|
|
|
};
|
|
|
|
Some(res)
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
|
|
|
#[derive(Clone, Copy, Debug, PartialEq, Eq, Hash)]
|
|
|
|
pub enum CallableDef {
|
|
|
|
Function(Function),
|
|
|
|
Struct(Struct),
|
|
|
|
EnumVariant(EnumVariant),
|
|
|
|
}
|
|
|
|
impl_froms!(CallableDef: Function, Struct, EnumVariant);
|
2019-07-06 10:43:13 -05:00
|
|
|
|
|
|
|
impl From<CallableDef> for GenericDef {
|
|
|
|
fn from(def: CallableDef) -> GenericDef {
|
|
|
|
match def {
|
|
|
|
CallableDef::Function(f) => f.into(),
|
|
|
|
CallableDef::Struct(s) => s.into(),
|
|
|
|
CallableDef::EnumVariant(e) => e.into(),
|
|
|
|
}
|
|
|
|
}
|
|
|
|
}
|