2015-09-16 14:56:30 +00:00
|
|
|
/*
|
|
|
|
This file is part of cpp-ethereum.
|
|
|
|
|
|
|
|
cpp-ethereum is free software: you can redistribute it and/or modify
|
|
|
|
it under the terms of the GNU General Public License as published by
|
|
|
|
the Free Software Foundation, either version 3 of the License, or
|
|
|
|
(at your option) any later version.
|
|
|
|
|
|
|
|
cpp-ethereum is distributed in the hope that it will be useful,
|
|
|
|
but WITHOUT ANY WARRANTY; without even the implied warranty of
|
|
|
|
MERCHANTABILITY or FITNESS FOR A PARTICULAR PURPOSE. See the
|
|
|
|
GNU General Public License for more details.
|
|
|
|
|
|
|
|
You should have received a copy of the GNU General Public License
|
|
|
|
along with cpp-ethereum. If not, see <http://www.gnu.org/licenses/>.
|
|
|
|
*/
|
|
|
|
/**
|
|
|
|
* @author Christian <c@ethdev.com>
|
|
|
|
* @date 2015
|
|
|
|
* Type analyzer and checker.
|
|
|
|
*/
|
|
|
|
|
2015-10-20 22:21:52 +00:00
|
|
|
#include <libsolidity/analysis/TypeChecker.h>
|
2015-09-16 14:56:30 +00:00
|
|
|
#include <memory>
|
|
|
|
#include <boost/range/adaptor/reversed.hpp>
|
2015-10-20 22:21:52 +00:00
|
|
|
#include <libsolidity/ast/AST.h>
|
2016-03-01 21:56:39 +00:00
|
|
|
#include <libevmasm/Assembly.h> // needed for inline assembly
|
|
|
|
#include <libsolidity/inlineasm/AsmCodeGen.h>
|
2015-09-16 14:56:30 +00:00
|
|
|
|
|
|
|
using namespace std;
|
|
|
|
using namespace dev;
|
|
|
|
using namespace dev::solidity;
|
|
|
|
|
|
|
|
|
2016-06-06 17:36:19 +00:00
|
|
|
bool TypeChecker::checkTypeRequirements(ContractDefinition const& _contract)
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
|
|
|
try
|
|
|
|
{
|
|
|
|
visit(_contract);
|
|
|
|
}
|
2015-10-15 12:36:23 +00:00
|
|
|
catch (FatalError const&)
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
|
|
|
// We got a fatal error which required to stop further type checking, but we can
|
|
|
|
// continue normally from here.
|
|
|
|
if (m_errors.empty())
|
|
|
|
throw; // Something is weird here, rather throw again.
|
|
|
|
}
|
2015-10-16 12:52:01 +00:00
|
|
|
return Error::containsOnlyWarnings(m_errors);
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
|
|
|
TypePointer const& TypeChecker::type(Expression const& _expression) const
|
|
|
|
{
|
|
|
|
solAssert(!!_expression.annotation().type, "Type requested but not present.");
|
|
|
|
return _expression.annotation().type;
|
|
|
|
}
|
|
|
|
|
|
|
|
TypePointer const& TypeChecker::type(VariableDeclaration const& _variable) const
|
|
|
|
{
|
|
|
|
solAssert(!!_variable.annotation().type, "Type requested but not present.");
|
|
|
|
return _variable.annotation().type;
|
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(ContractDefinition const& _contract)
|
|
|
|
{
|
2015-11-19 17:02:04 +00:00
|
|
|
m_scope = &_contract;
|
|
|
|
|
2015-09-16 14:56:30 +00:00
|
|
|
// We force our own visiting order here.
|
2015-11-23 22:57:17 +00:00
|
|
|
//@TODO structs will be visited again below, but it is probably fine.
|
2015-09-16 14:56:30 +00:00
|
|
|
ASTNode::listAccept(_contract.definedStructs(), *this);
|
|
|
|
ASTNode::listAccept(_contract.baseContracts(), *this);
|
|
|
|
|
|
|
|
checkContractDuplicateFunctions(_contract);
|
|
|
|
checkContractIllegalOverrides(_contract);
|
|
|
|
checkContractAbstractFunctions(_contract);
|
|
|
|
checkContractAbstractConstructors(_contract);
|
|
|
|
|
|
|
|
FunctionDefinition const* function = _contract.constructor();
|
2016-09-06 01:50:47 +00:00
|
|
|
if (function) {
|
|
|
|
if (!function->returnParameters().empty())
|
|
|
|
typeError(function->returnParameterList()->location(), "Non-empty \"returns\" directive for constructor.");
|
|
|
|
if (function->isDeclaredConst())
|
|
|
|
typeError(function->location(), "Constructor cannot be defined as constant.");
|
2016-09-06 03:07:05 +00:00
|
|
|
if (function->visibility() != FunctionDefinition::Visibility::Public && function->visibility() != FunctionDefinition::Visibility::Internal)
|
|
|
|
typeError(function->location(), "Constructor must be public or internal.");
|
2016-09-06 01:50:47 +00:00
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
|
|
|
|
FunctionDefinition const* fallbackFunction = nullptr;
|
2015-11-23 22:57:17 +00:00
|
|
|
for (FunctionDefinition const* function: _contract.definedFunctions())
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
|
|
|
if (function->name().empty())
|
|
|
|
{
|
|
|
|
if (fallbackFunction)
|
|
|
|
{
|
2015-10-02 12:41:40 +00:00
|
|
|
auto err = make_shared<Error>(Error::Type::DeclarationError);
|
2015-09-16 14:56:30 +00:00
|
|
|
*err << errinfo_comment("Only one fallback function is allowed.");
|
2015-09-22 09:17:54 +00:00
|
|
|
m_errors.push_back(err);
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
else
|
|
|
|
{
|
2015-11-23 22:57:17 +00:00
|
|
|
fallbackFunction = function;
|
2016-08-25 21:53:03 +00:00
|
|
|
if (_contract.isLibrary())
|
|
|
|
typeError(fallbackFunction->location(), "Libraries cannot have fallback functions.");
|
2016-08-26 19:01:47 +00:00
|
|
|
if (fallbackFunction->isDeclaredConst())
|
|
|
|
typeError(fallbackFunction->location(), "Fallback function cannot be declared constant.");
|
2015-09-16 14:56:30 +00:00
|
|
|
if (!fallbackFunction->parameters().empty())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(fallbackFunction->parameterList().location(), "Fallback function cannot take parameters.");
|
2016-08-25 11:25:30 +00:00
|
|
|
if (!fallbackFunction->returnParameters().empty())
|
|
|
|
typeError(fallbackFunction->returnParameterList()->location(), "Fallback function cannot return values.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
}
|
|
|
|
if (!function->isImplemented())
|
|
|
|
_contract.annotation().isFullyImplemented = false;
|
|
|
|
}
|
|
|
|
|
2015-11-23 22:57:17 +00:00
|
|
|
ASTNode::listAccept(_contract.subNodes(), *this);
|
2015-09-16 14:56:30 +00:00
|
|
|
|
|
|
|
checkContractExternalTypeClashes(_contract);
|
|
|
|
// check for hash collisions in function signatures
|
|
|
|
set<FixedHash<4>> hashes;
|
|
|
|
for (auto const& it: _contract.interfaceFunctionList())
|
|
|
|
{
|
|
|
|
FixedHash<4> const& hash = it.first;
|
|
|
|
if (hashes.count(hash))
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_contract.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
string("Function signature hash collision for ") + it.second->externalSignature()
|
|
|
|
);
|
|
|
|
hashes.insert(hash);
|
|
|
|
}
|
|
|
|
|
|
|
|
if (_contract.isLibrary())
|
|
|
|
checkLibraryRequirements(_contract);
|
|
|
|
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::checkContractDuplicateFunctions(ContractDefinition const& _contract)
|
|
|
|
{
|
|
|
|
/// Checks that two functions with the same name defined in this contract have different
|
|
|
|
/// argument types and that there is at most one constructor.
|
|
|
|
map<string, vector<FunctionDefinition const*>> functions;
|
2015-11-23 22:57:17 +00:00
|
|
|
for (FunctionDefinition const* function: _contract.definedFunctions())
|
|
|
|
functions[function->name()].push_back(function);
|
2015-09-16 14:56:30 +00:00
|
|
|
|
|
|
|
// Constructor
|
|
|
|
if (functions[_contract.name()].size() > 1)
|
|
|
|
{
|
|
|
|
SecondarySourceLocation ssl;
|
|
|
|
auto it = ++functions[_contract.name()].begin();
|
|
|
|
for (; it != functions[_contract.name()].end(); ++it)
|
|
|
|
ssl.append("Another declaration is here:", (*it)->location());
|
|
|
|
|
2015-10-02 12:41:40 +00:00
|
|
|
auto err = make_shared<Error>(Error(Error::Type::DeclarationError));
|
2015-09-16 14:56:30 +00:00
|
|
|
*err <<
|
|
|
|
errinfo_sourceLocation(functions[_contract.name()].front()->location()) <<
|
|
|
|
errinfo_comment("More than one constructor defined.") <<
|
|
|
|
errinfo_secondarySourceLocation(ssl);
|
2015-09-22 09:17:54 +00:00
|
|
|
m_errors.push_back(err);
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
for (auto const& it: functions)
|
|
|
|
{
|
|
|
|
vector<FunctionDefinition const*> const& overloads = it.second;
|
|
|
|
for (size_t i = 0; i < overloads.size(); ++i)
|
|
|
|
for (size_t j = i + 1; j < overloads.size(); ++j)
|
|
|
|
if (FunctionType(*overloads[i]).hasEqualArgumentTypes(FunctionType(*overloads[j])))
|
|
|
|
{
|
2015-10-02 12:41:40 +00:00
|
|
|
auto err = make_shared<Error>(Error(Error::Type::DeclarationError));
|
2015-09-16 14:56:30 +00:00
|
|
|
*err <<
|
|
|
|
errinfo_sourceLocation(overloads[j]->location()) <<
|
|
|
|
errinfo_comment("Function with same name and arguments defined twice.") <<
|
|
|
|
errinfo_secondarySourceLocation(SecondarySourceLocation().append(
|
|
|
|
"Other declaration is here:", overloads[i]->location()));
|
2015-09-22 09:17:54 +00:00
|
|
|
m_errors.push_back(err);
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::checkContractAbstractFunctions(ContractDefinition const& _contract)
|
|
|
|
{
|
|
|
|
// Mapping from name to function definition (exactly one per argument type equality class) and
|
|
|
|
// flag to indicate whether it is fully implemented.
|
|
|
|
using FunTypeAndFlag = std::pair<FunctionTypePointer, bool>;
|
|
|
|
map<string, vector<FunTypeAndFlag>> functions;
|
|
|
|
|
|
|
|
// Search from base to derived
|
|
|
|
for (ContractDefinition const* contract: boost::adaptors::reverse(_contract.annotation().linearizedBaseContracts))
|
2015-11-23 22:57:17 +00:00
|
|
|
for (FunctionDefinition const* function: contract->definedFunctions())
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
2016-06-06 17:36:19 +00:00
|
|
|
// Take constructors out of overload hierarchy
|
|
|
|
if (function->isConstructor())
|
|
|
|
continue;
|
2015-09-16 14:56:30 +00:00
|
|
|
auto& overloads = functions[function->name()];
|
|
|
|
FunctionTypePointer funType = make_shared<FunctionType>(*function);
|
|
|
|
auto it = find_if(overloads.begin(), overloads.end(), [&](FunTypeAndFlag const& _funAndFlag)
|
|
|
|
{
|
|
|
|
return funType->hasEqualArgumentTypes(*_funAndFlag.first);
|
|
|
|
});
|
|
|
|
if (it == overloads.end())
|
|
|
|
overloads.push_back(make_pair(funType, function->isImplemented()));
|
|
|
|
else if (it->second)
|
|
|
|
{
|
|
|
|
if (!function->isImplemented())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(function->location(), "Redeclaring an already implemented function as abstract");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
else if (function->isImplemented())
|
|
|
|
it->second = true;
|
|
|
|
}
|
|
|
|
|
|
|
|
// Set to not fully implemented if at least one flag is false.
|
|
|
|
for (auto const& it: functions)
|
|
|
|
for (auto const& funAndFlag: it.second)
|
|
|
|
if (!funAndFlag.second)
|
|
|
|
{
|
|
|
|
_contract.annotation().isFullyImplemented = false;
|
|
|
|
return;
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::checkContractAbstractConstructors(ContractDefinition const& _contract)
|
|
|
|
{
|
|
|
|
set<ContractDefinition const*> argumentsNeeded;
|
|
|
|
// check that we get arguments for all base constructors that need it.
|
|
|
|
// If not mark the contract as abstract (not fully implemented)
|
|
|
|
|
|
|
|
vector<ContractDefinition const*> const& bases = _contract.annotation().linearizedBaseContracts;
|
|
|
|
for (ContractDefinition const* contract: bases)
|
|
|
|
if (FunctionDefinition const* constructor = contract->constructor())
|
|
|
|
if (contract != &_contract && !constructor->parameters().empty())
|
|
|
|
argumentsNeeded.insert(contract);
|
|
|
|
|
|
|
|
for (ContractDefinition const* contract: bases)
|
|
|
|
{
|
|
|
|
if (FunctionDefinition const* constructor = contract->constructor())
|
|
|
|
for (auto const& modifier: constructor->modifiers())
|
|
|
|
{
|
|
|
|
auto baseContract = dynamic_cast<ContractDefinition const*>(
|
|
|
|
&dereference(*modifier->name())
|
|
|
|
);
|
|
|
|
if (baseContract)
|
|
|
|
argumentsNeeded.erase(baseContract);
|
|
|
|
}
|
|
|
|
|
|
|
|
|
|
|
|
for (ASTPointer<InheritanceSpecifier> const& base: contract->baseContracts())
|
|
|
|
{
|
|
|
|
auto baseContract = dynamic_cast<ContractDefinition const*>(&dereference(base->name()));
|
|
|
|
solAssert(baseContract, "");
|
|
|
|
if (!base->arguments().empty())
|
|
|
|
argumentsNeeded.erase(baseContract);
|
|
|
|
}
|
|
|
|
}
|
|
|
|
if (!argumentsNeeded.empty())
|
|
|
|
_contract.annotation().isFullyImplemented = false;
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::checkContractIllegalOverrides(ContractDefinition const& _contract)
|
|
|
|
{
|
|
|
|
// TODO unify this at a later point. for this we need to put the constness and the access specifier
|
|
|
|
// into the types
|
|
|
|
map<string, vector<FunctionDefinition const*>> functions;
|
|
|
|
map<string, ModifierDefinition const*> modifiers;
|
|
|
|
|
|
|
|
// We search from derived to base, so the stored item causes the error.
|
|
|
|
for (ContractDefinition const* contract: _contract.annotation().linearizedBaseContracts)
|
|
|
|
{
|
2015-11-23 22:57:17 +00:00
|
|
|
for (FunctionDefinition const* function: contract->definedFunctions())
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
|
|
|
if (function->isConstructor())
|
|
|
|
continue; // constructors can neither be overridden nor override anything
|
|
|
|
string const& name = function->name();
|
|
|
|
if (modifiers.count(name))
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(modifiers[name]->location(), "Override changes function to modifier.");
|
2015-09-16 14:56:30 +00:00
|
|
|
FunctionType functionType(*function);
|
|
|
|
// function should not change the return type
|
|
|
|
for (FunctionDefinition const* overriding: functions[name])
|
|
|
|
{
|
|
|
|
FunctionType overridingType(*overriding);
|
|
|
|
if (!overridingType.hasEqualArgumentTypes(functionType))
|
|
|
|
continue;
|
|
|
|
if (
|
|
|
|
overriding->visibility() != function->visibility() ||
|
|
|
|
overriding->isDeclaredConst() != function->isDeclaredConst() ||
|
2016-08-26 18:37:10 +00:00
|
|
|
overriding->isPayable() != function->isPayable() ||
|
2015-09-16 14:56:30 +00:00
|
|
|
overridingType != functionType
|
|
|
|
)
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(overriding->location(), "Override changes extended function signature.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
2015-11-23 22:57:17 +00:00
|
|
|
functions[name].push_back(function);
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
2015-11-23 22:57:17 +00:00
|
|
|
for (ModifierDefinition const* modifier: contract->functionModifiers())
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
|
|
|
string const& name = modifier->name();
|
|
|
|
ModifierDefinition const*& override = modifiers[name];
|
|
|
|
if (!override)
|
2015-11-23 22:57:17 +00:00
|
|
|
override = modifier;
|
2015-09-16 14:56:30 +00:00
|
|
|
else if (ModifierType(*override) != ModifierType(*modifier))
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(override->location(), "Override changes modifier signature.");
|
2015-09-16 14:56:30 +00:00
|
|
|
if (!functions[name].empty())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(override->location(), "Override changes modifier to function.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::checkContractExternalTypeClashes(ContractDefinition const& _contract)
|
|
|
|
{
|
|
|
|
map<string, vector<pair<Declaration const*, FunctionTypePointer>>> externalDeclarations;
|
|
|
|
for (ContractDefinition const* contract: _contract.annotation().linearizedBaseContracts)
|
|
|
|
{
|
2015-11-23 22:57:17 +00:00
|
|
|
for (FunctionDefinition const* f: contract->definedFunctions())
|
2015-09-16 14:56:30 +00:00
|
|
|
if (f->isPartOfExternalInterface())
|
|
|
|
{
|
|
|
|
auto functionType = make_shared<FunctionType>(*f);
|
2016-01-15 17:11:05 +00:00
|
|
|
// under non error circumstances this should be true
|
2016-01-15 16:36:06 +00:00
|
|
|
if (functionType->interfaceFunctionType())
|
|
|
|
externalDeclarations[functionType->externalSignature()].push_back(
|
|
|
|
make_pair(f, functionType)
|
|
|
|
);
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
2015-11-23 22:57:17 +00:00
|
|
|
for (VariableDeclaration const* v: contract->stateVariables())
|
2015-09-16 14:56:30 +00:00
|
|
|
if (v->isPartOfExternalInterface())
|
|
|
|
{
|
|
|
|
auto functionType = make_shared<FunctionType>(*v);
|
2016-01-15 17:11:05 +00:00
|
|
|
// under non error circumstances this should be true
|
2016-01-15 16:36:06 +00:00
|
|
|
if (functionType->interfaceFunctionType())
|
|
|
|
externalDeclarations[functionType->externalSignature()].push_back(
|
|
|
|
make_pair(v, functionType)
|
|
|
|
);
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
}
|
|
|
|
for (auto const& it: externalDeclarations)
|
|
|
|
for (size_t i = 0; i < it.second.size(); ++i)
|
|
|
|
for (size_t j = i + 1; j < it.second.size(); ++j)
|
|
|
|
if (!it.second[i].second->hasEqualArgumentTypes(*it.second[j].second))
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
it.second[j].first->location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Function overload clash during conversion to external types for arguments."
|
|
|
|
);
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::checkLibraryRequirements(ContractDefinition const& _contract)
|
|
|
|
{
|
|
|
|
solAssert(_contract.isLibrary(), "");
|
|
|
|
if (!_contract.baseContracts().empty())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_contract.location(), "Library is not allowed to inherit.");
|
2015-09-16 14:56:30 +00:00
|
|
|
|
|
|
|
for (auto const& var: _contract.stateVariables())
|
|
|
|
if (!var->isConstant())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(var->location(), "Library cannot have non-constant state variables");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::endVisit(InheritanceSpecifier const& _inheritance)
|
|
|
|
{
|
|
|
|
auto base = dynamic_cast<ContractDefinition const*>(&dereference(_inheritance.name()));
|
|
|
|
solAssert(base, "Base contract not available.");
|
|
|
|
|
|
|
|
if (base->isLibrary())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_inheritance.location(), "Libraries cannot be inherited from.");
|
2015-09-16 14:56:30 +00:00
|
|
|
|
|
|
|
auto const& arguments = _inheritance.arguments();
|
2016-08-31 18:43:24 +00:00
|
|
|
TypePointers parameterTypes = ContractType(*base).newExpressionType()->parameterTypes();
|
2015-09-16 14:56:30 +00:00
|
|
|
if (!arguments.empty() && parameterTypes.size() != arguments.size())
|
2015-12-09 16:37:19 +00:00
|
|
|
{
|
2015-09-16 14:56:30 +00:00
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_inheritance.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Wrong argument count for constructor call: " +
|
|
|
|
toString(arguments.size()) +
|
|
|
|
" arguments given but expected " +
|
|
|
|
toString(parameterTypes.size()) +
|
|
|
|
"."
|
|
|
|
);
|
2015-12-09 16:37:19 +00:00
|
|
|
return;
|
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
|
|
|
|
for (size_t i = 0; i < arguments.size(); ++i)
|
|
|
|
if (!type(*arguments[i])->isImplicitlyConvertibleTo(*parameterTypes[i]))
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
arguments[i]->location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Invalid type for argument in constructor call. "
|
|
|
|
"Invalid implicit conversion from " +
|
|
|
|
type(*arguments[i])->toString() +
|
|
|
|
" to " +
|
|
|
|
parameterTypes[i]->toString() +
|
|
|
|
" requested."
|
2015-11-22 19:39:10 +00:00
|
|
|
);
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::endVisit(UsingForDirective const& _usingFor)
|
|
|
|
{
|
|
|
|
ContractDefinition const* library = dynamic_cast<ContractDefinition const*>(
|
|
|
|
_usingFor.libraryName().annotation().referencedDeclaration
|
|
|
|
);
|
|
|
|
if (!library || !library->isLibrary())
|
|
|
|
typeError(_usingFor.libraryName().location(), "Library name expected.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(StructDefinition const& _struct)
|
|
|
|
{
|
|
|
|
for (ASTPointer<VariableDeclaration> const& member: _struct.members())
|
|
|
|
if (!type(*member)->canBeStored())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(member->location(), "Type cannot be used in struct.");
|
2015-09-16 14:56:30 +00:00
|
|
|
|
|
|
|
// Check recursion, fatal error if detected.
|
|
|
|
using StructPointer = StructDefinition const*;
|
|
|
|
using StructPointersSet = set<StructPointer>;
|
|
|
|
function<void(StructPointer,StructPointersSet const&)> check = [&](StructPointer _struct, StructPointersSet const& _parents)
|
|
|
|
{
|
|
|
|
if (_parents.count(_struct))
|
2015-11-04 10:49:26 +00:00
|
|
|
fatalTypeError(_struct->location(), "Recursive struct definition.");
|
2015-09-16 14:56:30 +00:00
|
|
|
StructPointersSet parents = _parents;
|
|
|
|
parents.insert(_struct);
|
|
|
|
for (ASTPointer<VariableDeclaration> const& member: _struct->members())
|
|
|
|
if (type(*member)->category() == Type::Category::Struct)
|
|
|
|
{
|
|
|
|
auto const& typeName = dynamic_cast<UserDefinedTypeName const&>(*member->typeName());
|
|
|
|
check(&dynamic_cast<StructDefinition const&>(*typeName.annotation().referencedDeclaration), parents);
|
|
|
|
}
|
|
|
|
};
|
|
|
|
check(&_struct, StructPointersSet{});
|
|
|
|
|
|
|
|
ASTNode::listAccept(_struct.members(), *this);
|
|
|
|
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(FunctionDefinition const& _function)
|
|
|
|
{
|
2015-10-02 11:11:38 +00:00
|
|
|
bool isLibraryFunction = dynamic_cast<ContractDefinition const&>(*_function.scope()).isLibrary();
|
2016-08-26 18:37:10 +00:00
|
|
|
if (_function.isPayable())
|
|
|
|
{
|
|
|
|
if (isLibraryFunction)
|
|
|
|
typeError(_function.location(), "Library functions cannot be payable.");
|
|
|
|
if (!_function.isConstructor() && !_function.name().empty() && !_function.isPartOfExternalInterface())
|
|
|
|
typeError(_function.location(), "Internal functions cannot be payable.");
|
2016-09-06 08:58:56 +00:00
|
|
|
if (_function.isDeclaredConst())
|
|
|
|
typeError(_function.location(), "Functions cannot be constant and payable at the same time.");
|
2016-08-26 18:37:10 +00:00
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
for (ASTPointer<VariableDeclaration> const& var: _function.parameters() + _function.returnParameters())
|
|
|
|
{
|
|
|
|
if (!type(*var)->canLiveOutsideStorage())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(var->location(), "Type is required to live outside storage.");
|
2015-10-02 11:11:38 +00:00
|
|
|
if (_function.visibility() >= FunctionDefinition::Visibility::Public && !(type(*var)->interfaceType(isLibraryFunction)))
|
2015-11-04 10:49:26 +00:00
|
|
|
fatalTypeError(var->location(), "Internal type is not allowed for public or external functions.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
for (ASTPointer<ModifierInvocation> const& modifier: _function.modifiers())
|
|
|
|
visitManually(
|
|
|
|
*modifier,
|
|
|
|
_function.isConstructor() ?
|
2015-09-21 16:55:58 +00:00
|
|
|
dynamic_cast<ContractDefinition const&>(*_function.scope()).annotation().linearizedBaseContracts :
|
2015-09-16 14:56:30 +00:00
|
|
|
vector<ContractDefinition const*>()
|
|
|
|
);
|
|
|
|
if (_function.isImplemented())
|
|
|
|
_function.body().accept(*this);
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(VariableDeclaration const& _variable)
|
|
|
|
{
|
|
|
|
// Variables can be declared without type (with "var"), in which case the first assignment
|
|
|
|
// sets the type.
|
|
|
|
// Note that assignments before the first declaration are legal because of the special scoping
|
|
|
|
// rules inherited from JavaScript.
|
|
|
|
|
2015-10-08 16:01:12 +00:00
|
|
|
// type is filled either by ReferencesResolver directly from the type name or by
|
|
|
|
// TypeChecker at the VariableDeclarationStatement level.
|
2015-09-16 14:56:30 +00:00
|
|
|
TypePointer varType = _variable.annotation().type;
|
2015-10-08 16:01:12 +00:00
|
|
|
solAssert(!!varType, "Failed to infer variable type.");
|
2015-09-16 14:56:30 +00:00
|
|
|
if (_variable.isConstant())
|
|
|
|
{
|
|
|
|
if (!dynamic_cast<ContractDefinition const*>(_variable.scope()))
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_variable.location(), "Illegal use of \"constant\" specifier.");
|
2015-09-16 14:56:30 +00:00
|
|
|
if (!_variable.value())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_variable.location(), "Uninitialized \"constant\" variable.");
|
2015-10-08 16:01:12 +00:00
|
|
|
if (!varType->isValueType())
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
|
|
|
bool constImplemented = false;
|
|
|
|
if (auto arrayType = dynamic_cast<ArrayType const*>(varType.get()))
|
|
|
|
constImplemented = arrayType->isByteArray();
|
|
|
|
if (!constImplemented)
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_variable.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Illegal use of \"constant\" specifier. \"constant\" "
|
|
|
|
"is not yet implemented for this type."
|
|
|
|
);
|
|
|
|
}
|
|
|
|
}
|
2015-10-08 16:01:12 +00:00
|
|
|
if (_variable.value())
|
|
|
|
expectType(*_variable.value(), *varType);
|
2015-09-16 14:56:30 +00:00
|
|
|
if (!_variable.isStateVariable())
|
|
|
|
{
|
|
|
|
if (varType->dataStoredIn(DataLocation::Memory) || varType->dataStoredIn(DataLocation::CallData))
|
|
|
|
if (!varType->canLiveOutsideStorage())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_variable.location(), "Type " + varType->toString() + " is only valid in storage.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
else if (
|
|
|
|
_variable.visibility() >= VariableDeclaration::Visibility::Public &&
|
2015-10-02 11:11:38 +00:00
|
|
|
!FunctionType(_variable).interfaceFunctionType()
|
2015-09-16 14:56:30 +00:00
|
|
|
)
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_variable.location(), "Internal type is not allowed for public state variables.");
|
2015-09-16 14:56:30 +00:00
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::visitManually(
|
|
|
|
ModifierInvocation const& _modifier,
|
|
|
|
vector<ContractDefinition const*> const& _bases
|
|
|
|
)
|
|
|
|
{
|
|
|
|
std::vector<ASTPointer<Expression>> const& arguments = _modifier.arguments();
|
|
|
|
for (ASTPointer<Expression> const& argument: arguments)
|
|
|
|
argument->accept(*this);
|
|
|
|
_modifier.name()->accept(*this);
|
|
|
|
|
|
|
|
auto const* declaration = &dereference(*_modifier.name());
|
|
|
|
vector<ASTPointer<VariableDeclaration>> emptyParameterList;
|
|
|
|
vector<ASTPointer<VariableDeclaration>> const* parameters = nullptr;
|
|
|
|
if (auto modifierDecl = dynamic_cast<ModifierDefinition const*>(declaration))
|
|
|
|
parameters = &modifierDecl->parameters();
|
|
|
|
else
|
|
|
|
// check parameters for Base constructors
|
|
|
|
for (ContractDefinition const* base: _bases)
|
|
|
|
if (declaration == base)
|
|
|
|
{
|
|
|
|
if (auto referencedConstructor = base->constructor())
|
|
|
|
parameters = &referencedConstructor->parameters();
|
|
|
|
else
|
|
|
|
parameters = &emptyParameterList;
|
|
|
|
break;
|
|
|
|
}
|
|
|
|
if (!parameters)
|
2016-01-08 14:20:20 +00:00
|
|
|
{
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_modifier.location(), "Referenced declaration is neither modifier nor base class.");
|
2016-01-08 14:20:20 +00:00
|
|
|
return;
|
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
if (parameters->size() != arguments.size())
|
2016-02-11 16:10:35 +00:00
|
|
|
{
|
2015-09-16 14:56:30 +00:00
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_modifier.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Wrong argument count for modifier invocation: " +
|
|
|
|
toString(arguments.size()) +
|
|
|
|
" arguments given but expected " +
|
|
|
|
toString(parameters->size()) +
|
|
|
|
"."
|
|
|
|
);
|
2016-02-11 16:10:35 +00:00
|
|
|
return;
|
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
for (size_t i = 0; i < _modifier.arguments().size(); ++i)
|
|
|
|
if (!type(*arguments[i])->isImplicitlyConvertibleTo(*type(*(*parameters)[i])))
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
arguments[i]->location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Invalid type for argument in modifier invocation. "
|
|
|
|
"Invalid implicit conversion from " +
|
|
|
|
type(*arguments[i])->toString() +
|
|
|
|
" to " +
|
|
|
|
type(*(*parameters)[i])->toString() +
|
|
|
|
" requested."
|
|
|
|
);
|
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(EventDefinition const& _eventDef)
|
|
|
|
{
|
|
|
|
unsigned numIndexed = 0;
|
|
|
|
for (ASTPointer<VariableDeclaration> const& var: _eventDef.parameters())
|
|
|
|
{
|
|
|
|
if (var->isIndexed())
|
|
|
|
numIndexed++;
|
2015-10-07 14:40:54 +00:00
|
|
|
if (_eventDef.isAnonymous() && numIndexed > 4)
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_eventDef.location(), "More than 4 indexed arguments for anonymous event.");
|
2015-10-07 14:40:54 +00:00
|
|
|
else if (!_eventDef.isAnonymous() && numIndexed > 3)
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_eventDef.location(), "More than 3 indexed arguments for event.");
|
2015-09-16 14:56:30 +00:00
|
|
|
if (!type(*var)->canLiveOutsideStorage())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(var->location(), "Type is required to live outside storage.");
|
2015-10-02 11:11:38 +00:00
|
|
|
if (!type(*var)->interfaceType(false))
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(var->location(), "Internal type is not allowed as event parameter type.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
2016-03-01 21:56:39 +00:00
|
|
|
bool TypeChecker::visit(InlineAssembly const& _inlineAssembly)
|
|
|
|
{
|
|
|
|
// Inline assembly does not have its own type-checking phase, so we just run the
|
|
|
|
// code-generator and see whether it produces any errors.
|
|
|
|
// External references have already been resolved in a prior stage and stored in the annotation.
|
|
|
|
assembly::CodeGenerator codeGen(_inlineAssembly.operations(), m_errors);
|
|
|
|
codeGen.typeCheck([&](assembly::Identifier const& _identifier, eth::Assembly& _assembly, assembly::CodeGenerator::IdentifierContext _context) {
|
|
|
|
auto ref = _inlineAssembly.annotation().externalReferences.find(&_identifier);
|
|
|
|
if (ref == _inlineAssembly.annotation().externalReferences.end())
|
|
|
|
return false;
|
|
|
|
Declaration const* declaration = ref->second;
|
|
|
|
solAssert(!!declaration, "");
|
|
|
|
if (_context == assembly::CodeGenerator::IdentifierContext::RValue)
|
|
|
|
{
|
|
|
|
solAssert(!!declaration->type(), "Type of declaration required but not yet determined.");
|
|
|
|
unsigned pushes = 0;
|
|
|
|
if (dynamic_cast<FunctionDefinition const*>(declaration))
|
|
|
|
pushes = 1;
|
|
|
|
else if (auto var = dynamic_cast<VariableDeclaration const*>(declaration))
|
|
|
|
{
|
|
|
|
if (var->isConstant())
|
|
|
|
fatalTypeError(SourceLocation(), "Constant variables not yet implemented for inline assembly.");
|
|
|
|
if (var->isLocalVariable())
|
|
|
|
pushes = var->type()->sizeOnStack();
|
|
|
|
else if (var->type()->isValueType())
|
|
|
|
pushes = 1;
|
|
|
|
else
|
|
|
|
pushes = 2; // slot number, intra slot offset
|
|
|
|
}
|
|
|
|
else if (auto contract = dynamic_cast<ContractDefinition const*>(declaration))
|
|
|
|
{
|
|
|
|
if (!contract->isLibrary())
|
|
|
|
return false;
|
|
|
|
pushes = 1;
|
|
|
|
}
|
|
|
|
for (unsigned i = 0; i < pushes; ++i)
|
|
|
|
_assembly.append(u256(0)); // just to verify the stack height
|
|
|
|
}
|
|
|
|
else
|
|
|
|
{
|
|
|
|
// lvalue context
|
|
|
|
if (auto varDecl = dynamic_cast<VariableDeclaration const*>(declaration))
|
|
|
|
{
|
|
|
|
if (!varDecl->isLocalVariable())
|
|
|
|
return false; // only local variables are inline-assemlby lvalues
|
|
|
|
for (unsigned i = 0; i < declaration->type()->sizeOnStack(); ++i)
|
2016-04-04 11:41:35 +00:00
|
|
|
_assembly.append(Instruction::POP); // remove value just to verify the stack height
|
2016-03-01 21:56:39 +00:00
|
|
|
}
|
|
|
|
else
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
return true;
|
|
|
|
});
|
|
|
|
return false;
|
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
|
|
|
|
bool TypeChecker::visit(IfStatement const& _ifStatement)
|
|
|
|
{
|
|
|
|
expectType(_ifStatement.condition(), BoolType());
|
|
|
|
_ifStatement.trueStatement().accept(*this);
|
|
|
|
if (_ifStatement.falseStatement())
|
|
|
|
_ifStatement.falseStatement()->accept(*this);
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(WhileStatement const& _whileStatement)
|
|
|
|
{
|
|
|
|
expectType(_whileStatement.condition(), BoolType());
|
|
|
|
_whileStatement.body().accept(*this);
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(ForStatement const& _forStatement)
|
|
|
|
{
|
|
|
|
if (_forStatement.initializationExpression())
|
|
|
|
_forStatement.initializationExpression()->accept(*this);
|
|
|
|
if (_forStatement.condition())
|
|
|
|
expectType(*_forStatement.condition(), BoolType());
|
|
|
|
if (_forStatement.loopExpression())
|
|
|
|
_forStatement.loopExpression()->accept(*this);
|
|
|
|
_forStatement.body().accept(*this);
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::endVisit(Return const& _return)
|
|
|
|
{
|
|
|
|
if (!_return.expression())
|
|
|
|
return;
|
|
|
|
ParameterList const* params = _return.annotation().functionReturnParameters;
|
|
|
|
if (!params)
|
2015-10-12 21:02:35 +00:00
|
|
|
{
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_return.location(), "Return arguments not allowed.");
|
2015-10-12 21:02:35 +00:00
|
|
|
return;
|
|
|
|
}
|
|
|
|
TypePointers returnTypes;
|
|
|
|
for (auto const& var: params->parameters())
|
|
|
|
returnTypes.push_back(type(*var));
|
|
|
|
if (auto tupleType = dynamic_cast<TupleType const*>(type(*_return.expression()).get()))
|
|
|
|
{
|
|
|
|
if (tupleType->components().size() != params->parameters().size())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_return.location(), "Different number of arguments in return statement than in returns declaration.");
|
2015-10-12 21:02:35 +00:00
|
|
|
else if (!tupleType->isImplicitlyConvertibleTo(TupleType(returnTypes)))
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_return.expression()->location(),
|
2015-10-12 21:02:35 +00:00
|
|
|
"Return argument type " +
|
|
|
|
type(*_return.expression())->toString() +
|
|
|
|
" is not implicitly convertible to expected type " +
|
|
|
|
TupleType(returnTypes).toString(false) +
|
|
|
|
"."
|
|
|
|
);
|
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
else if (params->parameters().size() != 1)
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_return.location(), "Different number of arguments in return statement than in returns declaration.");
|
2015-09-16 14:56:30 +00:00
|
|
|
else
|
|
|
|
{
|
|
|
|
TypePointer const& expected = type(*params->parameters().front());
|
|
|
|
if (!type(*_return.expression())->isImplicitlyConvertibleTo(*expected))
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_return.expression()->location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Return argument type " +
|
|
|
|
type(*_return.expression())->toString() +
|
|
|
|
" is not implicitly convertible to expected type (type of first return variable) " +
|
|
|
|
expected->toString() +
|
|
|
|
"."
|
|
|
|
);
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
2015-10-08 16:01:12 +00:00
|
|
|
bool TypeChecker::visit(VariableDeclarationStatement const& _statement)
|
|
|
|
{
|
2015-10-09 17:35:41 +00:00
|
|
|
if (!_statement.initialValue())
|
2015-10-08 16:01:12 +00:00
|
|
|
{
|
2015-10-09 17:35:41 +00:00
|
|
|
// No initial value is only permitted for single variables with specified type.
|
|
|
|
if (_statement.declarations().size() != 1 || !_statement.declarations().front())
|
2015-11-04 10:49:26 +00:00
|
|
|
fatalTypeError(_statement.location(), "Assignment necessary for type detection.");
|
2015-10-09 17:35:41 +00:00
|
|
|
VariableDeclaration const& varDecl = *_statement.declarations().front();
|
|
|
|
if (!varDecl.annotation().type)
|
2015-11-04 10:49:26 +00:00
|
|
|
fatalTypeError(_statement.location(), "Assignment necessary for type detection.");
|
2015-10-12 21:02:35 +00:00
|
|
|
if (auto ref = dynamic_cast<ReferenceType const*>(type(varDecl).get()))
|
2015-10-09 17:35:41 +00:00
|
|
|
{
|
|
|
|
if (ref->dataStoredIn(DataLocation::Storage))
|
|
|
|
{
|
2015-10-15 09:10:55 +00:00
|
|
|
auto err = make_shared<Error>(Error::Type::Warning);
|
2015-10-09 17:35:41 +00:00
|
|
|
*err <<
|
|
|
|
errinfo_sourceLocation(varDecl.location()) <<
|
|
|
|
errinfo_comment("Uninitialized storage pointer. Did you mean '<type> memory " + varDecl.name() + "'?");
|
|
|
|
m_errors.push_back(err);
|
|
|
|
}
|
|
|
|
}
|
|
|
|
varDecl.accept(*this);
|
2015-10-08 16:01:12 +00:00
|
|
|
return false;
|
|
|
|
}
|
2015-10-09 17:35:41 +00:00
|
|
|
|
|
|
|
// Here we have an initial value and might have to derive some types before we can visit
|
|
|
|
// the variable declaration(s).
|
|
|
|
|
|
|
|
_statement.initialValue()->accept(*this);
|
2015-10-09 18:44:56 +00:00
|
|
|
TypePointers valueTypes;
|
2015-10-12 21:02:35 +00:00
|
|
|
if (auto tupleType = dynamic_cast<TupleType const*>(type(*_statement.initialValue()).get()))
|
2015-10-09 18:44:56 +00:00
|
|
|
valueTypes = tupleType->components();
|
|
|
|
else
|
2015-10-12 21:02:35 +00:00
|
|
|
valueTypes = TypePointers{type(*_statement.initialValue())};
|
2015-10-09 17:35:41 +00:00
|
|
|
|
2015-10-09 18:44:56 +00:00
|
|
|
// Determine which component is assigned to which variable.
|
2015-10-09 17:35:41 +00:00
|
|
|
// If numbers do not match, fill up if variables begin or end empty (not both).
|
2015-10-09 18:44:56 +00:00
|
|
|
vector<VariableDeclaration const*>& assignments = _statement.annotation().assignments;
|
|
|
|
assignments.resize(valueTypes.size(), nullptr);
|
|
|
|
vector<ASTPointer<VariableDeclaration>> const& variables = _statement.declarations();
|
2015-10-13 12:31:24 +00:00
|
|
|
if (variables.empty())
|
|
|
|
{
|
|
|
|
if (!valueTypes.empty())
|
|
|
|
fatalTypeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_statement.location(),
|
2015-10-13 12:31:24 +00:00
|
|
|
"Too many components (" +
|
|
|
|
toString(valueTypes.size()) +
|
|
|
|
") in value for variable assignment (0) needed"
|
|
|
|
);
|
|
|
|
}
|
|
|
|
else if (valueTypes.size() != variables.size() && !variables.front() && !variables.back())
|
2015-10-09 18:44:56 +00:00
|
|
|
fatalTypeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_statement.location(),
|
2015-10-09 18:44:56 +00:00
|
|
|
"Wildcard both at beginning and end of variable declaration list is only allowed "
|
|
|
|
"if the number of components is equal."
|
|
|
|
);
|
|
|
|
size_t minNumValues = variables.size();
|
2015-10-13 12:31:24 +00:00
|
|
|
if (!variables.empty() && (!variables.back() || !variables.front()))
|
2015-10-09 18:44:56 +00:00
|
|
|
--minNumValues;
|
|
|
|
if (valueTypes.size() < minNumValues)
|
|
|
|
fatalTypeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_statement.location(),
|
2015-10-09 18:44:56 +00:00
|
|
|
"Not enough components (" +
|
|
|
|
toString(valueTypes.size()) +
|
|
|
|
") in value to assign all variables (" +
|
|
|
|
toString(minNumValues) + ")."
|
|
|
|
);
|
|
|
|
if (valueTypes.size() > variables.size() && variables.front() && variables.back())
|
|
|
|
fatalTypeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_statement.location(),
|
2015-10-09 18:44:56 +00:00
|
|
|
"Too many components (" +
|
|
|
|
toString(valueTypes.size()) +
|
|
|
|
") in value for variable assignment (" +
|
|
|
|
toString(minNumValues) +
|
|
|
|
" needed)."
|
|
|
|
);
|
2015-10-13 12:31:24 +00:00
|
|
|
bool fillRight = !variables.empty() && (!variables.back() || variables.front());
|
2015-10-09 18:44:56 +00:00
|
|
|
for (size_t i = 0; i < min(variables.size(), valueTypes.size()); ++i)
|
|
|
|
if (fillRight)
|
|
|
|
assignments[i] = variables[i].get();
|
|
|
|
else
|
|
|
|
assignments[assignments.size() - i - 1] = variables[variables.size() - i - 1].get();
|
2015-10-09 17:35:41 +00:00
|
|
|
|
2015-10-09 18:44:56 +00:00
|
|
|
for (size_t i = 0; i < assignments.size(); ++i)
|
2015-10-09 17:35:41 +00:00
|
|
|
{
|
2015-10-09 18:44:56 +00:00
|
|
|
if (!assignments[i])
|
2015-10-09 17:35:41 +00:00
|
|
|
continue;
|
2015-10-09 18:44:56 +00:00
|
|
|
VariableDeclaration const& var = *assignments[i];
|
2015-10-09 17:35:41 +00:00
|
|
|
solAssert(!var.value(), "Value has to be tied to statement.");
|
2015-10-09 18:44:56 +00:00
|
|
|
TypePointer const& valueComponentType = valueTypes[i];
|
2015-10-09 17:35:41 +00:00
|
|
|
solAssert(!!valueComponentType, "");
|
|
|
|
if (!var.annotation().type)
|
|
|
|
{
|
|
|
|
// Infer type from value.
|
|
|
|
solAssert(!var.typeName(), "");
|
|
|
|
var.annotation().type = valueComponentType->mobileType();
|
2016-05-10 08:26:53 +00:00
|
|
|
if (!var.annotation().type)
|
2016-05-10 12:57:29 +00:00
|
|
|
{
|
2016-05-10 08:26:53 +00:00
|
|
|
if (valueComponentType->category() == Type::Category::RationalNumber)
|
|
|
|
fatalTypeError(
|
|
|
|
_statement.initialValue()->location(),
|
|
|
|
"Invalid rational " +
|
|
|
|
valueComponentType->toString() +
|
|
|
|
" (absolute value too large or divison by zero)."
|
|
|
|
);
|
|
|
|
else
|
|
|
|
solAssert(false, "");
|
2016-05-10 12:57:29 +00:00
|
|
|
}
|
2015-10-09 17:35:41 +00:00
|
|
|
var.accept(*this);
|
|
|
|
}
|
|
|
|
else
|
|
|
|
{
|
|
|
|
var.accept(*this);
|
|
|
|
if (!valueComponentType->isImplicitlyConvertibleTo(*var.annotation().type))
|
2016-05-05 22:47:08 +00:00
|
|
|
{
|
|
|
|
if (
|
|
|
|
valueComponentType->category() == Type::Category::RationalNumber &&
|
2016-05-10 12:30:24 +00:00
|
|
|
dynamic_cast<RationalNumberType const&>(*valueComponentType).isFractional() &&
|
2016-05-10 08:26:53 +00:00
|
|
|
valueComponentType->mobileType()
|
2016-05-05 22:47:08 +00:00
|
|
|
)
|
|
|
|
typeError(
|
|
|
|
_statement.location(),
|
|
|
|
"Type " +
|
|
|
|
valueComponentType->toString() +
|
|
|
|
" is not implicitly convertible to expected type " +
|
|
|
|
var.annotation().type->toString() +
|
|
|
|
". Try converting to type " +
|
|
|
|
valueComponentType->mobileType()->toString() +
|
|
|
|
" or use an explicit conversion."
|
|
|
|
);
|
|
|
|
else
|
|
|
|
typeError(
|
|
|
|
_statement.location(),
|
|
|
|
"Type " +
|
|
|
|
valueComponentType->toString() +
|
|
|
|
" is not implicitly convertible to expected type " +
|
|
|
|
var.annotation().type->toString() +
|
|
|
|
"."
|
|
|
|
);
|
|
|
|
}
|
2015-10-09 17:35:41 +00:00
|
|
|
}
|
2015-10-08 16:01:12 +00:00
|
|
|
}
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
2015-09-16 14:56:30 +00:00
|
|
|
void TypeChecker::endVisit(ExpressionStatement const& _statement)
|
|
|
|
{
|
2016-03-29 20:08:51 +00:00
|
|
|
if (type(_statement.expression())->category() == Type::Category::RationalNumber)
|
2016-05-10 08:26:53 +00:00
|
|
|
if (!dynamic_cast<RationalNumberType const&>(*type(_statement.expression())).mobileType())
|
2016-04-12 17:36:34 +00:00
|
|
|
typeError(_statement.expression().location(), "Invalid rational number.");
|
2016-06-21 12:36:23 +00:00
|
|
|
|
2016-06-24 14:41:17 +00:00
|
|
|
if (auto call = dynamic_cast<FunctionCall const*>(&_statement.expression()))
|
|
|
|
{
|
|
|
|
if (auto callType = dynamic_cast<FunctionType const*>(type(call->expression()).get()))
|
|
|
|
{
|
|
|
|
using Location = FunctionType::Location;
|
|
|
|
Location location = callType->location();
|
|
|
|
if (
|
|
|
|
location == Location::Bare ||
|
|
|
|
location == Location::BareCallCode ||
|
|
|
|
location == Location::BareDelegateCall ||
|
|
|
|
location == Location::Send
|
|
|
|
)
|
|
|
|
warning(_statement.location(), "Return value of low-level calls not used.");
|
|
|
|
}
|
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
2016-01-07 09:01:46 +00:00
|
|
|
bool TypeChecker::visit(Conditional const& _conditional)
|
2015-12-22 16:50:06 +00:00
|
|
|
{
|
2016-01-07 09:01:46 +00:00
|
|
|
expectType(_conditional.condition(), BoolType());
|
2015-12-23 16:12:41 +00:00
|
|
|
|
2016-01-11 07:08:28 +00:00
|
|
|
_conditional.trueExpression().accept(*this);
|
|
|
|
_conditional.falseExpression().accept(*this);
|
2016-01-07 09:01:46 +00:00
|
|
|
|
2016-01-11 16:00:14 +00:00
|
|
|
TypePointer trueType = type(_conditional.trueExpression())->mobileType();
|
|
|
|
TypePointer falseType = type(_conditional.falseExpression())->mobileType();
|
2016-01-07 09:01:46 +00:00
|
|
|
|
2016-01-11 16:00:14 +00:00
|
|
|
TypePointer commonType = Type::commonType(trueType, falseType);
|
2016-01-11 07:08:28 +00:00
|
|
|
if (!commonType)
|
2016-01-07 09:01:46 +00:00
|
|
|
{
|
2016-01-11 07:08:28 +00:00
|
|
|
typeError(
|
|
|
|
_conditional.location(),
|
|
|
|
"True expression's type " +
|
|
|
|
trueType->toString() +
|
|
|
|
" doesn't match false expression's type " +
|
|
|
|
falseType->toString() +
|
|
|
|
"."
|
|
|
|
);
|
|
|
|
// even we can't find a common type, we have to set a type here,
|
|
|
|
// otherwise the upper statement will not be able to check the type.
|
|
|
|
commonType = trueType;
|
|
|
|
}
|
2016-01-07 09:01:46 +00:00
|
|
|
|
2016-01-11 07:08:28 +00:00
|
|
|
_conditional.annotation().type = commonType;
|
2016-01-07 09:01:46 +00:00
|
|
|
|
2016-01-11 07:08:28 +00:00
|
|
|
if (_conditional.annotation().lValueRequested)
|
|
|
|
typeError(
|
|
|
|
_conditional.location(),
|
|
|
|
"Conditional expression as left value is not supported yet."
|
|
|
|
);
|
2016-01-07 09:01:46 +00:00
|
|
|
|
|
|
|
return false;
|
2015-12-22 16:50:06 +00:00
|
|
|
}
|
|
|
|
|
2015-09-16 14:56:30 +00:00
|
|
|
bool TypeChecker::visit(Assignment const& _assignment)
|
|
|
|
{
|
|
|
|
requireLValue(_assignment.leftHandSide());
|
|
|
|
TypePointer t = type(_assignment.leftHandSide());
|
|
|
|
_assignment.annotation().type = t;
|
2015-10-14 13:19:50 +00:00
|
|
|
if (TupleType const* tupleType = dynamic_cast<TupleType const*>(t.get()))
|
|
|
|
{
|
2015-10-15 14:02:00 +00:00
|
|
|
// Sequenced assignments of tuples is not valid, make the result a "void" type.
|
|
|
|
_assignment.annotation().type = make_shared<TupleType>();
|
2015-10-14 13:19:50 +00:00
|
|
|
expectType(_assignment.rightHandSide(), *tupleType);
|
|
|
|
}
|
|
|
|
else if (t->category() == Type::Category::Mapping)
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_assignment.location(), "Mappings cannot be assigned to.");
|
2015-09-16 14:56:30 +00:00
|
|
|
_assignment.rightHandSide().accept(*this);
|
|
|
|
}
|
|
|
|
else if (_assignment.assignmentOperator() == Token::Assign)
|
|
|
|
expectType(_assignment.rightHandSide(), *t);
|
|
|
|
else
|
|
|
|
{
|
|
|
|
// compound assignment
|
|
|
|
_assignment.rightHandSide().accept(*this);
|
|
|
|
TypePointer resultType = t->binaryOperatorResult(
|
|
|
|
Token::AssignmentToBinaryOp(_assignment.assignmentOperator()),
|
|
|
|
type(_assignment.rightHandSide())
|
|
|
|
);
|
|
|
|
if (!resultType || *resultType != *t)
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_assignment.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Operator " +
|
|
|
|
string(Token::toString(_assignment.assignmentOperator())) +
|
|
|
|
" not compatible with types " +
|
|
|
|
t->toString() +
|
|
|
|
" and " +
|
|
|
|
type(_assignment.rightHandSide())->toString()
|
|
|
|
);
|
|
|
|
}
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
2015-10-12 21:02:35 +00:00
|
|
|
bool TypeChecker::visit(TupleExpression const& _tuple)
|
|
|
|
{
|
|
|
|
vector<ASTPointer<Expression>> const& components = _tuple.components();
|
|
|
|
TypePointers types;
|
2016-01-11 20:25:59 +00:00
|
|
|
|
2015-10-12 21:02:35 +00:00
|
|
|
if (_tuple.annotation().lValueRequested)
|
|
|
|
{
|
2016-01-11 20:25:59 +00:00
|
|
|
if (_tuple.isInlineArray())
|
|
|
|
fatalTypeError(_tuple.location(), "Inline array type cannot be declared as LValue.");
|
2015-10-12 21:02:35 +00:00
|
|
|
for (auto const& component: components)
|
|
|
|
if (component)
|
|
|
|
{
|
|
|
|
requireLValue(*component);
|
|
|
|
types.push_back(type(*component));
|
|
|
|
}
|
|
|
|
else
|
|
|
|
types.push_back(TypePointer());
|
2016-01-04 08:11:04 +00:00
|
|
|
if (components.size() == 1)
|
|
|
|
_tuple.annotation().type = type(*components[0]);
|
|
|
|
else
|
|
|
|
_tuple.annotation().type = make_shared<TupleType>(types);
|
2015-10-12 21:02:35 +00:00
|
|
|
// If some of the components are not LValues, the error is reported above.
|
|
|
|
_tuple.annotation().isLValue = true;
|
|
|
|
}
|
|
|
|
else
|
|
|
|
{
|
2016-01-12 05:41:20 +00:00
|
|
|
TypePointer inlineArrayType;
|
2015-10-12 21:02:35 +00:00
|
|
|
for (size_t i = 0; i < components.size(); ++i)
|
|
|
|
{
|
|
|
|
// Outside of an lvalue-context, the only situation where a component can be empty is (x,).
|
|
|
|
if (!components[i] && !(i == 1 && components.size() == 2))
|
2015-12-16 18:55:52 +00:00
|
|
|
fatalTypeError(_tuple.location(), "Tuple component cannot be empty.");
|
2015-10-12 21:02:35 +00:00
|
|
|
else if (components[i])
|
|
|
|
{
|
|
|
|
components[i]->accept(*this);
|
|
|
|
types.push_back(type(*components[i]));
|
2016-01-11 20:25:59 +00:00
|
|
|
if (_tuple.isInlineArray())
|
|
|
|
solAssert(!!types[i], "Inline array cannot have empty components");
|
|
|
|
if (i == 0 && _tuple.isInlineArray())
|
|
|
|
inlineArrayType = types[i]->mobileType();
|
|
|
|
else if (_tuple.isInlineArray() && inlineArrayType)
|
|
|
|
inlineArrayType = Type::commonType(inlineArrayType, types[i]->mobileType());
|
2015-10-12 21:02:35 +00:00
|
|
|
}
|
|
|
|
else
|
|
|
|
types.push_back(TypePointer());
|
|
|
|
}
|
2016-01-11 20:25:59 +00:00
|
|
|
if (_tuple.isInlineArray())
|
|
|
|
{
|
|
|
|
if (!inlineArrayType)
|
|
|
|
fatalTypeError(_tuple.location(), "Unable to deduce common type for array elements.");
|
|
|
|
_tuple.annotation().type = make_shared<ArrayType>(DataLocation::Memory, inlineArrayType, types.size());
|
|
|
|
}
|
2015-10-12 21:02:35 +00:00
|
|
|
else
|
|
|
|
{
|
2016-01-11 20:25:59 +00:00
|
|
|
if (components.size() == 1)
|
|
|
|
_tuple.annotation().type = type(*components[0]);
|
|
|
|
else
|
|
|
|
{
|
|
|
|
if (components.size() == 2 && !components[1])
|
|
|
|
types.pop_back();
|
|
|
|
_tuple.annotation().type = make_shared<TupleType>(types);
|
|
|
|
}
|
2015-10-12 21:02:35 +00:00
|
|
|
}
|
2016-01-11 20:25:59 +00:00
|
|
|
|
2015-10-12 21:02:35 +00:00
|
|
|
}
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
2015-09-16 14:56:30 +00:00
|
|
|
bool TypeChecker::visit(UnaryOperation const& _operation)
|
|
|
|
{
|
|
|
|
// Inc, Dec, Add, Sub, Not, BitNot, Delete
|
|
|
|
Token::Value op = _operation.getOperator();
|
|
|
|
if (op == Token::Value::Inc || op == Token::Value::Dec || op == Token::Value::Delete)
|
|
|
|
requireLValue(_operation.subExpression());
|
|
|
|
else
|
|
|
|
_operation.subExpression().accept(*this);
|
|
|
|
TypePointer const& subExprType = type(_operation.subExpression());
|
|
|
|
TypePointer t = type(_operation.subExpression())->unaryOperatorResult(op);
|
|
|
|
if (!t)
|
|
|
|
{
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_operation.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Unary operator " +
|
|
|
|
string(Token::toString(op)) +
|
|
|
|
" cannot be applied to type " +
|
|
|
|
subExprType->toString()
|
|
|
|
);
|
|
|
|
t = subExprType;
|
|
|
|
}
|
|
|
|
_operation.annotation().type = t;
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::endVisit(BinaryOperation const& _operation)
|
|
|
|
{
|
|
|
|
TypePointer const& leftType = type(_operation.leftExpression());
|
|
|
|
TypePointer const& rightType = type(_operation.rightExpression());
|
|
|
|
TypePointer commonType = leftType->binaryOperatorResult(_operation.getOperator(), rightType);
|
|
|
|
if (!commonType)
|
|
|
|
{
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_operation.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Operator " +
|
|
|
|
string(Token::toString(_operation.getOperator())) +
|
|
|
|
" not compatible with types " +
|
|
|
|
leftType->toString() +
|
|
|
|
" and " +
|
|
|
|
rightType->toString()
|
|
|
|
);
|
|
|
|
commonType = leftType;
|
|
|
|
}
|
|
|
|
_operation.annotation().commonType = commonType;
|
|
|
|
_operation.annotation().type =
|
|
|
|
Token::isCompareOp(_operation.getOperator()) ?
|
|
|
|
make_shared<BoolType>() :
|
|
|
|
commonType;
|
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(FunctionCall const& _functionCall)
|
|
|
|
{
|
|
|
|
bool isPositionalCall = _functionCall.names().empty();
|
|
|
|
vector<ASTPointer<Expression const>> arguments = _functionCall.arguments();
|
|
|
|
vector<ASTPointer<ASTString>> const& argumentNames = _functionCall.names();
|
|
|
|
|
|
|
|
// We need to check arguments' type first as they will be needed for overload resolution.
|
|
|
|
shared_ptr<TypePointers> argumentTypes;
|
|
|
|
if (isPositionalCall)
|
|
|
|
argumentTypes = make_shared<TypePointers>();
|
|
|
|
for (ASTPointer<Expression const> const& argument: arguments)
|
|
|
|
{
|
|
|
|
argument->accept(*this);
|
|
|
|
// only store them for positional calls
|
|
|
|
if (isPositionalCall)
|
|
|
|
argumentTypes->push_back(type(*argument));
|
|
|
|
}
|
|
|
|
if (isPositionalCall)
|
|
|
|
_functionCall.expression().annotation().argumentTypes = move(argumentTypes);
|
|
|
|
|
|
|
|
_functionCall.expression().accept(*this);
|
|
|
|
TypePointer expressionType = type(_functionCall.expression());
|
|
|
|
|
|
|
|
if (auto const* typeType = dynamic_cast<TypeType const*>(expressionType.get()))
|
|
|
|
{
|
|
|
|
_functionCall.annotation().isStructConstructorCall = (typeType->actualType()->category() == Type::Category::Struct);
|
|
|
|
_functionCall.annotation().isTypeConversion = !_functionCall.annotation().isStructConstructorCall;
|
|
|
|
}
|
|
|
|
else
|
|
|
|
_functionCall.annotation().isStructConstructorCall = _functionCall.annotation().isTypeConversion = false;
|
|
|
|
|
|
|
|
if (_functionCall.annotation().isTypeConversion)
|
|
|
|
{
|
|
|
|
TypeType const& t = dynamic_cast<TypeType const&>(*expressionType);
|
|
|
|
TypePointer resultType = t.actualType();
|
|
|
|
if (arguments.size() != 1)
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_functionCall.location(), "Exactly one argument expected for explicit type conversion.");
|
2015-09-16 14:56:30 +00:00
|
|
|
else if (!isPositionalCall)
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_functionCall.location(), "Type conversion cannot allow named arguments.");
|
2015-09-16 14:56:30 +00:00
|
|
|
else
|
|
|
|
{
|
|
|
|
TypePointer const& argType = type(*arguments.front());
|
|
|
|
if (auto argRefType = dynamic_cast<ReferenceType const*>(argType.get()))
|
|
|
|
// do not change the data location when converting
|
|
|
|
// (data location cannot yet be specified for type conversions)
|
|
|
|
resultType = ReferenceType::copyForLocationIfReference(argRefType->location(), resultType);
|
|
|
|
if (!argType->isExplicitlyConvertibleTo(*resultType))
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_functionCall.location(), "Explicit type conversion not allowed.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
_functionCall.annotation().type = resultType;
|
|
|
|
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
// Actual function call or struct constructor call.
|
|
|
|
|
|
|
|
FunctionTypePointer functionType;
|
|
|
|
|
|
|
|
/// For error message: Struct members that were removed during conversion to memory.
|
|
|
|
set<string> membersRemovedForStructConstructor;
|
|
|
|
if (_functionCall.annotation().isStructConstructorCall)
|
|
|
|
{
|
|
|
|
TypeType const& t = dynamic_cast<TypeType const&>(*expressionType);
|
|
|
|
auto const& structType = dynamic_cast<StructType const&>(*t.actualType());
|
|
|
|
functionType = structType.constructorType();
|
|
|
|
membersRemovedForStructConstructor = structType.membersMissingInMemory();
|
|
|
|
}
|
|
|
|
else
|
|
|
|
functionType = dynamic_pointer_cast<FunctionType const>(expressionType);
|
|
|
|
|
|
|
|
if (!functionType)
|
|
|
|
{
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_functionCall.location(), "Type is not callable");
|
2015-10-09 17:35:41 +00:00
|
|
|
_functionCall.annotation().type = make_shared<TupleType>();
|
2015-09-16 14:56:30 +00:00
|
|
|
return false;
|
|
|
|
}
|
2015-10-09 17:35:41 +00:00
|
|
|
else if (functionType->returnParameterTypes().size() == 1)
|
|
|
|
_functionCall.annotation().type = functionType->returnParameterTypes().front();
|
2015-09-16 14:56:30 +00:00
|
|
|
else
|
2015-10-09 17:35:41 +00:00
|
|
|
_functionCall.annotation().type = make_shared<TupleType>(functionType->returnParameterTypes());
|
2015-09-16 14:56:30 +00:00
|
|
|
|
2015-12-09 16:53:15 +00:00
|
|
|
TypePointers parameterTypes = functionType->parameterTypes();
|
2015-09-16 14:56:30 +00:00
|
|
|
if (!functionType->takesArbitraryParameters() && parameterTypes.size() != arguments.size())
|
|
|
|
{
|
|
|
|
string msg =
|
|
|
|
"Wrong argument count for function call: " +
|
|
|
|
toString(arguments.size()) +
|
|
|
|
" arguments given but expected " +
|
|
|
|
toString(parameterTypes.size()) +
|
|
|
|
".";
|
|
|
|
// Extend error message in case we try to construct a struct with mapping member.
|
|
|
|
if (_functionCall.annotation().isStructConstructorCall && !membersRemovedForStructConstructor.empty())
|
|
|
|
{
|
|
|
|
msg += " Members that have to be skipped in memory:";
|
|
|
|
for (auto const& member: membersRemovedForStructConstructor)
|
|
|
|
msg += " " + member;
|
|
|
|
}
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_functionCall.location(), msg);
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
else if (isPositionalCall)
|
|
|
|
{
|
|
|
|
// call by positional arguments
|
|
|
|
for (size_t i = 0; i < arguments.size(); ++i)
|
2015-10-07 15:32:05 +00:00
|
|
|
{
|
|
|
|
auto const& argType = type(*arguments[i]);
|
|
|
|
if (functionType->takesArbitraryParameters())
|
|
|
|
{
|
2016-03-29 20:08:51 +00:00
|
|
|
if (auto t = dynamic_cast<RationalNumberType const*>(argType.get()))
|
2016-05-10 08:26:53 +00:00
|
|
|
if (!t->mobileType())
|
|
|
|
typeError(arguments[i]->location(), "Invalid rational number (too large or division by zero).");
|
2015-10-07 15:32:05 +00:00
|
|
|
}
|
|
|
|
else if (!type(*arguments[i])->isImplicitlyConvertibleTo(*parameterTypes[i]))
|
2015-09-16 14:56:30 +00:00
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
arguments[i]->location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Invalid type for argument in function call. "
|
|
|
|
"Invalid implicit conversion from " +
|
|
|
|
type(*arguments[i])->toString() +
|
|
|
|
" to " +
|
|
|
|
parameterTypes[i]->toString() +
|
|
|
|
" requested."
|
|
|
|
);
|
2015-10-07 15:32:05 +00:00
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
else
|
|
|
|
{
|
|
|
|
// call by named arguments
|
|
|
|
auto const& parameterNames = functionType->parameterNames();
|
|
|
|
if (functionType->takesArbitraryParameters())
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_functionCall.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Named arguments cannnot be used for functions that take arbitrary parameters."
|
|
|
|
);
|
|
|
|
else if (parameterNames.size() > argumentNames.size())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_functionCall.location(), "Some argument names are missing.");
|
2015-09-16 14:56:30 +00:00
|
|
|
else if (parameterNames.size() < argumentNames.size())
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_functionCall.location(), "Too many arguments.");
|
2015-09-16 14:56:30 +00:00
|
|
|
else
|
|
|
|
{
|
|
|
|
// check duplicate names
|
|
|
|
bool duplication = false;
|
|
|
|
for (size_t i = 0; i < argumentNames.size(); i++)
|
|
|
|
for (size_t j = i + 1; j < argumentNames.size(); j++)
|
|
|
|
if (*argumentNames[i] == *argumentNames[j])
|
|
|
|
{
|
|
|
|
duplication = true;
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(arguments[i]->location(), "Duplicate named argument.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
|
|
|
// check actual types
|
|
|
|
if (!duplication)
|
|
|
|
for (size_t i = 0; i < argumentNames.size(); i++)
|
|
|
|
{
|
|
|
|
bool found = false;
|
|
|
|
for (size_t j = 0; j < parameterNames.size(); j++)
|
|
|
|
if (parameterNames[j] == *argumentNames[i])
|
|
|
|
{
|
|
|
|
found = true;
|
|
|
|
// check type convertible
|
|
|
|
if (!type(*arguments[i])->isImplicitlyConvertibleTo(*parameterTypes[j]))
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
arguments[i]->location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Invalid type for argument in function call. "
|
|
|
|
"Invalid implicit conversion from " +
|
|
|
|
type(*arguments[i])->toString() +
|
|
|
|
" to " +
|
|
|
|
parameterTypes[i]->toString() +
|
|
|
|
" requested."
|
|
|
|
);
|
|
|
|
break;
|
|
|
|
}
|
|
|
|
|
|
|
|
if (!found)
|
|
|
|
typeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_functionCall.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Named argument does not match function declaration."
|
|
|
|
);
|
|
|
|
}
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::endVisit(NewExpression const& _newExpression)
|
|
|
|
{
|
2015-11-17 00:47:47 +00:00
|
|
|
TypePointer type = _newExpression.typeName().annotation().type;
|
|
|
|
solAssert(!!type, "Type name not resolved.");
|
|
|
|
|
2015-11-16 23:06:57 +00:00
|
|
|
if (auto contractName = dynamic_cast<UserDefinedTypeName const*>(&_newExpression.typeName()))
|
|
|
|
{
|
|
|
|
auto contract = dynamic_cast<ContractDefinition const*>(&dereference(*contractName));
|
|
|
|
|
|
|
|
if (!contract)
|
|
|
|
fatalTypeError(_newExpression.location(), "Identifier is not a contract.");
|
|
|
|
if (!contract->annotation().isFullyImplemented)
|
|
|
|
typeError(_newExpression.location(), "Trying to create an instance of an abstract contract.");
|
|
|
|
|
2015-11-19 17:02:04 +00:00
|
|
|
solAssert(!!m_scope, "");
|
|
|
|
m_scope->annotation().contractDependencies.insert(contract);
|
2015-11-16 23:06:57 +00:00
|
|
|
solAssert(
|
|
|
|
!contract->annotation().linearizedBaseContracts.empty(),
|
|
|
|
"Linearized base contracts not yet available."
|
2015-09-16 14:56:30 +00:00
|
|
|
);
|
2015-11-19 17:02:04 +00:00
|
|
|
if (contractDependenciesAreCyclic(*m_scope))
|
2015-11-16 23:06:57 +00:00
|
|
|
typeError(
|
|
|
|
_newExpression.location(),
|
|
|
|
"Circular reference for contract creation (cannot create instance of derived or same contract)."
|
|
|
|
);
|
2015-09-16 14:56:30 +00:00
|
|
|
|
2016-08-31 18:43:24 +00:00
|
|
|
_newExpression.annotation().type = FunctionType::newExpressionType(*contract);
|
2015-11-16 23:06:57 +00:00
|
|
|
}
|
2015-11-17 00:47:47 +00:00
|
|
|
else if (type->category() == Type::Category::Array)
|
2015-11-16 23:06:57 +00:00
|
|
|
{
|
2015-11-17 00:47:47 +00:00
|
|
|
if (!type->canLiveOutsideStorage())
|
|
|
|
fatalTypeError(
|
|
|
|
_newExpression.typeName().location(),
|
|
|
|
"Type cannot live outside storage."
|
|
|
|
);
|
|
|
|
if (!type->isDynamicallySized())
|
|
|
|
typeError(
|
|
|
|
_newExpression.typeName().location(),
|
|
|
|
"Length has to be placed in parentheses after the array type for new expression."
|
|
|
|
);
|
|
|
|
type = ReferenceType::copyForLocationIfReference(DataLocation::Memory, type);
|
|
|
|
_newExpression.annotation().type = make_shared<FunctionType>(
|
|
|
|
TypePointers{make_shared<IntegerType>(256)},
|
|
|
|
TypePointers{type},
|
|
|
|
strings(),
|
|
|
|
strings(),
|
|
|
|
FunctionType::Location::ObjectCreation
|
|
|
|
);
|
2015-11-16 23:06:57 +00:00
|
|
|
}
|
|
|
|
else
|
|
|
|
fatalTypeError(_newExpression.location(), "Contract or array type expected.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(MemberAccess const& _memberAccess)
|
|
|
|
{
|
|
|
|
_memberAccess.expression().accept(*this);
|
|
|
|
TypePointer exprType = type(_memberAccess.expression());
|
|
|
|
ASTString const& memberName = _memberAccess.memberName();
|
|
|
|
|
|
|
|
// Retrieve the types of the arguments if this is used to call a function.
|
|
|
|
auto const& argumentTypes = _memberAccess.annotation().argumentTypes;
|
2015-11-19 17:02:04 +00:00
|
|
|
MemberList::MemberMap possibleMembers = exprType->members(m_scope).membersByName(memberName);
|
2015-09-16 14:56:30 +00:00
|
|
|
if (possibleMembers.size() > 1 && argumentTypes)
|
|
|
|
{
|
|
|
|
// do overload resolution
|
|
|
|
for (auto it = possibleMembers.begin(); it != possibleMembers.end();)
|
|
|
|
if (
|
|
|
|
it->type->category() == Type::Category::Function &&
|
2015-11-27 21:24:00 +00:00
|
|
|
!dynamic_cast<FunctionType const&>(*it->type).canTakeArguments(*argumentTypes, exprType)
|
2015-09-16 14:56:30 +00:00
|
|
|
)
|
|
|
|
it = possibleMembers.erase(it);
|
|
|
|
else
|
|
|
|
++it;
|
|
|
|
}
|
|
|
|
if (possibleMembers.size() == 0)
|
|
|
|
{
|
|
|
|
auto storageType = ReferenceType::copyForLocationIfReference(
|
|
|
|
DataLocation::Storage,
|
|
|
|
exprType
|
|
|
|
);
|
2015-11-19 17:02:04 +00:00
|
|
|
if (!storageType->members(m_scope).membersByName(memberName).empty())
|
2015-09-16 14:56:30 +00:00
|
|
|
fatalTypeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_memberAccess.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Member \"" + memberName + "\" is not available in " +
|
|
|
|
exprType->toString() +
|
|
|
|
" outside of storage."
|
|
|
|
);
|
|
|
|
fatalTypeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_memberAccess.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Member \"" + memberName + "\" not found or not visible "
|
2016-08-26 18:37:10 +00:00
|
|
|
"after argument-dependent lookup in " + exprType->toString() +
|
|
|
|
(memberName == "value" ? " - did you forget the \"payable\" modifier?" : "")
|
2015-09-16 14:56:30 +00:00
|
|
|
);
|
|
|
|
}
|
|
|
|
else if (possibleMembers.size() > 1)
|
|
|
|
fatalTypeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_memberAccess.location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Member \"" + memberName + "\" not unique "
|
2016-08-26 18:37:10 +00:00
|
|
|
"after argument-dependent lookup in " + exprType->toString() +
|
|
|
|
(memberName == "value" ? " - did you forget the \"payable\" modifier?" : "")
|
2015-09-16 14:56:30 +00:00
|
|
|
);
|
|
|
|
|
|
|
|
auto& annotation = _memberAccess.annotation();
|
|
|
|
annotation.referencedDeclaration = possibleMembers.front().declaration;
|
|
|
|
annotation.type = possibleMembers.front().type;
|
2015-11-27 21:24:00 +00:00
|
|
|
|
|
|
|
if (auto funType = dynamic_cast<FunctionType const*>(annotation.type.get()))
|
|
|
|
if (funType->bound() && !exprType->isImplicitlyConvertibleTo(*funType->selfType()))
|
|
|
|
typeError(
|
|
|
|
_memberAccess.location(),
|
|
|
|
"Function \"" + memberName + "\" cannot be called on an object of type " +
|
|
|
|
exprType->toString() + " (expected " + funType->selfType()->toString() + ")"
|
|
|
|
);
|
|
|
|
|
2015-09-16 14:56:30 +00:00
|
|
|
if (exprType->category() == Type::Category::Struct)
|
|
|
|
annotation.isLValue = true;
|
|
|
|
else if (exprType->category() == Type::Category::Array)
|
|
|
|
{
|
|
|
|
auto const& arrayType(dynamic_cast<ArrayType const&>(*exprType));
|
|
|
|
annotation.isLValue = (
|
|
|
|
memberName == "length" &&
|
|
|
|
arrayType.location() == DataLocation::Storage &&
|
|
|
|
arrayType.isDynamicallySized()
|
|
|
|
);
|
|
|
|
}
|
2016-02-03 20:34:24 +00:00
|
|
|
else if (exprType->category() == Type::Category::FixedBytes)
|
|
|
|
annotation.isLValue = false;
|
2015-09-16 14:56:30 +00:00
|
|
|
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(IndexAccess const& _access)
|
|
|
|
{
|
|
|
|
_access.baseExpression().accept(*this);
|
|
|
|
TypePointer baseType = type(_access.baseExpression());
|
|
|
|
TypePointer resultType;
|
|
|
|
bool isLValue = false;
|
|
|
|
Expression const* index = _access.indexExpression();
|
|
|
|
switch (baseType->category())
|
|
|
|
{
|
|
|
|
case Type::Category::Array:
|
|
|
|
{
|
|
|
|
ArrayType const& actualType = dynamic_cast<ArrayType const&>(*baseType);
|
|
|
|
if (!index)
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_access.location(), "Index expression cannot be omitted.");
|
2015-09-16 14:56:30 +00:00
|
|
|
else if (actualType.isString())
|
|
|
|
{
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_access.location(), "Index access for string is not possible.");
|
2015-09-16 14:56:30 +00:00
|
|
|
index->accept(*this);
|
|
|
|
}
|
|
|
|
else
|
|
|
|
{
|
|
|
|
expectType(*index, IntegerType(256));
|
2016-03-29 20:08:51 +00:00
|
|
|
if (auto numberType = dynamic_cast<RationalNumberType const*>(type(*index).get()))
|
2016-02-18 22:39:11 +00:00
|
|
|
{
|
2016-05-10 12:30:24 +00:00
|
|
|
if (!numberType->isFractional()) // error is reported above
|
|
|
|
if (!actualType.isDynamicallySized() && actualType.length() <= numberType->literalValue(nullptr))
|
|
|
|
typeError(_access.location(), "Out of bounds array access.");
|
2016-05-10 08:26:53 +00:00
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
resultType = actualType.baseType();
|
|
|
|
isLValue = actualType.location() != DataLocation::CallData;
|
|
|
|
break;
|
|
|
|
}
|
|
|
|
case Type::Category::Mapping:
|
|
|
|
{
|
|
|
|
MappingType const& actualType = dynamic_cast<MappingType const&>(*baseType);
|
|
|
|
if (!index)
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_access.location(), "Index expression cannot be omitted.");
|
2015-09-16 14:56:30 +00:00
|
|
|
else
|
|
|
|
expectType(*index, *actualType.keyType());
|
|
|
|
resultType = actualType.valueType();
|
|
|
|
isLValue = true;
|
|
|
|
break;
|
|
|
|
}
|
|
|
|
case Type::Category::TypeType:
|
|
|
|
{
|
|
|
|
TypeType const& typeType = dynamic_cast<TypeType const&>(*baseType);
|
|
|
|
if (!index)
|
|
|
|
resultType = make_shared<TypeType>(make_shared<ArrayType>(DataLocation::Memory, typeType.actualType()));
|
|
|
|
else
|
|
|
|
{
|
2016-04-12 17:36:34 +00:00
|
|
|
expectType(*index, IntegerType(256));
|
2016-03-29 20:08:51 +00:00
|
|
|
if (auto length = dynamic_cast<RationalNumberType const*>(type(*index).get()))
|
2015-09-16 14:56:30 +00:00
|
|
|
resultType = make_shared<TypeType>(make_shared<ArrayType>(
|
|
|
|
DataLocation::Memory,
|
|
|
|
typeType.actualType(),
|
|
|
|
length->literalValue(nullptr)
|
|
|
|
));
|
|
|
|
else
|
2016-09-15 16:01:13 +00:00
|
|
|
fatalTypeError(index->location(), "Integer constant expected.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
break;
|
|
|
|
}
|
2016-02-03 20:34:24 +00:00
|
|
|
case Type::Category::FixedBytes:
|
|
|
|
{
|
|
|
|
FixedBytesType const& bytesType = dynamic_cast<FixedBytesType const&>(*baseType);
|
|
|
|
if (!index)
|
|
|
|
typeError(_access.location(), "Index expression cannot be omitted.");
|
|
|
|
else
|
|
|
|
{
|
|
|
|
expectType(*index, IntegerType(256));
|
2016-03-29 20:08:51 +00:00
|
|
|
if (auto integerType = dynamic_cast<RationalNumberType const*>(type(*index).get()))
|
2016-02-03 20:34:24 +00:00
|
|
|
if (bytesType.numBytes() <= integerType->literalValue(nullptr))
|
|
|
|
typeError(_access.location(), "Out of bounds array access.");
|
|
|
|
}
|
|
|
|
resultType = make_shared<FixedBytesType>(1);
|
|
|
|
isLValue = false; // @todo this heavily depends on how it is embedded
|
|
|
|
break;
|
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
default:
|
|
|
|
fatalTypeError(
|
2015-11-04 10:49:26 +00:00
|
|
|
_access.baseExpression().location(),
|
2015-09-16 14:56:30 +00:00
|
|
|
"Indexed expression has to be a type, mapping or array (is " + baseType->toString() + ")"
|
|
|
|
);
|
|
|
|
}
|
|
|
|
_access.annotation().type = move(resultType);
|
|
|
|
_access.annotation().isLValue = isLValue;
|
|
|
|
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
bool TypeChecker::visit(Identifier const& _identifier)
|
|
|
|
{
|
2015-09-21 16:55:58 +00:00
|
|
|
IdentifierAnnotation& annotation = _identifier.annotation();
|
2015-09-16 14:56:30 +00:00
|
|
|
if (!annotation.referencedDeclaration)
|
|
|
|
{
|
|
|
|
if (!annotation.argumentTypes)
|
2015-11-04 10:49:26 +00:00
|
|
|
fatalTypeError(_identifier.location(), "Unable to determine overloaded type.");
|
2015-09-16 14:56:30 +00:00
|
|
|
if (annotation.overloadedDeclarations.empty())
|
2015-11-04 10:49:26 +00:00
|
|
|
fatalTypeError(_identifier.location(), "No candidates for overload resolution found.");
|
2015-09-16 14:56:30 +00:00
|
|
|
else if (annotation.overloadedDeclarations.size() == 1)
|
|
|
|
annotation.referencedDeclaration = *annotation.overloadedDeclarations.begin();
|
|
|
|
else
|
|
|
|
{
|
|
|
|
vector<Declaration const*> candidates;
|
|
|
|
|
|
|
|
for (Declaration const* declaration: annotation.overloadedDeclarations)
|
|
|
|
{
|
2015-11-19 17:02:04 +00:00
|
|
|
TypePointer function = declaration->type();
|
2015-09-16 14:56:30 +00:00
|
|
|
solAssert(!!function, "Requested type not present.");
|
|
|
|
auto const* functionType = dynamic_cast<FunctionType const*>(function.get());
|
|
|
|
if (functionType && functionType->canTakeArguments(*annotation.argumentTypes))
|
|
|
|
candidates.push_back(declaration);
|
|
|
|
}
|
|
|
|
if (candidates.empty())
|
2015-11-04 10:49:26 +00:00
|
|
|
fatalTypeError(_identifier.location(), "No matching declaration found after argument-dependent lookup.");
|
2015-09-16 14:56:30 +00:00
|
|
|
else if (candidates.size() == 1)
|
|
|
|
annotation.referencedDeclaration = candidates.front();
|
|
|
|
else
|
2015-11-04 10:49:26 +00:00
|
|
|
fatalTypeError(_identifier.location(), "No unique declaration found after argument-dependent lookup.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
}
|
|
|
|
solAssert(
|
|
|
|
!!annotation.referencedDeclaration,
|
|
|
|
"Referenced declaration is null after overload resolution."
|
|
|
|
);
|
|
|
|
annotation.isLValue = annotation.referencedDeclaration->isLValue();
|
2015-11-19 17:02:04 +00:00
|
|
|
annotation.type = annotation.referencedDeclaration->type();
|
2015-09-16 14:56:30 +00:00
|
|
|
if (!annotation.type)
|
2015-11-04 10:49:26 +00:00
|
|
|
fatalTypeError(_identifier.location(), "Declaration referenced before type could be determined.");
|
2015-09-16 14:56:30 +00:00
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::endVisit(ElementaryTypeNameExpression const& _expr)
|
|
|
|
{
|
2016-02-08 21:43:22 +00:00
|
|
|
_expr.annotation().type = make_shared<TypeType>(Type::fromElementaryTypeName(_expr.typeName()));
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::endVisit(Literal const& _literal)
|
|
|
|
{
|
|
|
|
_literal.annotation().type = Type::forLiteral(_literal);
|
|
|
|
if (!_literal.annotation().type)
|
2015-11-04 10:49:26 +00:00
|
|
|
fatalTypeError(_literal.location(), "Invalid literal value.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
2015-10-07 13:57:17 +00:00
|
|
|
bool TypeChecker::contractDependenciesAreCyclic(
|
|
|
|
ContractDefinition const& _contract,
|
|
|
|
std::set<ContractDefinition const*> const& _seenContracts
|
|
|
|
) const
|
|
|
|
{
|
|
|
|
// Naive depth-first search that remembers nodes already seen.
|
|
|
|
if (_seenContracts.count(&_contract))
|
|
|
|
return true;
|
|
|
|
set<ContractDefinition const*> seen(_seenContracts);
|
|
|
|
seen.insert(&_contract);
|
|
|
|
for (auto const* c: _contract.annotation().contractDependencies)
|
|
|
|
if (contractDependenciesAreCyclic(*c, seen))
|
|
|
|
return true;
|
|
|
|
return false;
|
|
|
|
}
|
|
|
|
|
2015-11-24 15:34:02 +00:00
|
|
|
Declaration const& TypeChecker::dereference(Identifier const& _identifier) const
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
|
|
|
solAssert(!!_identifier.annotation().referencedDeclaration, "Declaration not stored.");
|
|
|
|
return *_identifier.annotation().referencedDeclaration;
|
|
|
|
}
|
|
|
|
|
2015-11-24 15:34:02 +00:00
|
|
|
Declaration const& TypeChecker::dereference(UserDefinedTypeName const& _typeName) const
|
2015-11-16 23:06:57 +00:00
|
|
|
{
|
|
|
|
solAssert(!!_typeName.annotation().referencedDeclaration, "Declaration not stored.");
|
|
|
|
return *_typeName.annotation().referencedDeclaration;
|
|
|
|
}
|
|
|
|
|
2015-09-16 14:56:30 +00:00
|
|
|
void TypeChecker::expectType(Expression const& _expression, Type const& _expectedType)
|
|
|
|
{
|
|
|
|
_expression.accept(*this);
|
|
|
|
if (!type(_expression)->isImplicitlyConvertibleTo(_expectedType))
|
2016-05-05 22:47:08 +00:00
|
|
|
{
|
|
|
|
if (
|
|
|
|
type(_expression)->category() == Type::Category::RationalNumber &&
|
2016-05-10 12:30:24 +00:00
|
|
|
dynamic_pointer_cast<RationalNumberType const>(type(_expression))->isFractional() &&
|
2016-05-10 08:26:53 +00:00
|
|
|
type(_expression)->mobileType()
|
2016-05-05 22:47:08 +00:00
|
|
|
)
|
|
|
|
typeError(
|
|
|
|
_expression.location(),
|
|
|
|
"Type " +
|
|
|
|
type(_expression)->toString() +
|
|
|
|
" is not implicitly convertible to expected type " +
|
|
|
|
_expectedType.toString() +
|
|
|
|
". Try converting to type " +
|
|
|
|
type(_expression)->mobileType()->toString() +
|
2016-05-10 08:26:53 +00:00
|
|
|
" or use an explicit conversion."
|
2016-05-05 22:47:08 +00:00
|
|
|
);
|
|
|
|
else
|
|
|
|
typeError(
|
|
|
|
_expression.location(),
|
|
|
|
"Type " +
|
|
|
|
type(_expression)->toString() +
|
|
|
|
" is not implicitly convertible to expected type " +
|
|
|
|
_expectedType.toString() +
|
|
|
|
"."
|
|
|
|
);
|
|
|
|
}
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
|
|
|
void TypeChecker::requireLValue(Expression const& _expression)
|
|
|
|
{
|
2015-10-12 21:02:35 +00:00
|
|
|
_expression.annotation().lValueRequested = true;
|
2015-09-16 14:56:30 +00:00
|
|
|
_expression.accept(*this);
|
|
|
|
if (!_expression.annotation().isLValue)
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_expression.location(), "Expression has to be an lvalue.");
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
2015-11-04 10:49:26 +00:00
|
|
|
void TypeChecker::typeError(SourceLocation const& _location, string const& _description)
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
2015-10-14 18:37:41 +00:00
|
|
|
auto err = make_shared<Error>(Error::Type::TypeError);
|
2015-09-16 14:56:30 +00:00
|
|
|
*err <<
|
2015-11-04 10:49:26 +00:00
|
|
|
errinfo_sourceLocation(_location) <<
|
2015-09-16 14:56:30 +00:00
|
|
|
errinfo_comment(_description);
|
|
|
|
|
2015-09-22 09:17:54 +00:00
|
|
|
m_errors.push_back(err);
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|
|
|
|
|
2016-06-21 12:36:23 +00:00
|
|
|
void TypeChecker::warning(SourceLocation const& _location, string const& _description)
|
|
|
|
{
|
|
|
|
auto err = make_shared<Error>(Error::Type::Warning);
|
|
|
|
*err <<
|
|
|
|
errinfo_sourceLocation(_location) <<
|
|
|
|
errinfo_comment(_description);
|
|
|
|
|
|
|
|
m_errors.push_back(err);
|
|
|
|
}
|
|
|
|
|
2015-11-04 10:49:26 +00:00
|
|
|
void TypeChecker::fatalTypeError(SourceLocation const& _location, string const& _description)
|
2015-09-16 14:56:30 +00:00
|
|
|
{
|
2015-11-04 10:49:26 +00:00
|
|
|
typeError(_location, _description);
|
2015-10-15 12:36:23 +00:00
|
|
|
BOOST_THROW_EXCEPTION(FatalError());
|
2015-09-16 14:56:30 +00:00
|
|
|
}
|