mirror of
https://github.com/ethereum/solidity
synced 2023-10-03 13:03:40 +00:00
Merge pull request #11974 from ethereum/newCodeTransformIROnly
New code transform (IR codegen only).
This commit is contained in:
commit
6b029c3349
@ -1069,9 +1069,6 @@ string IRGenerator::dispatchRoutine(ContractDefinition const& _contract)
|
||||
|
||||
string IRGenerator::memoryInit(bool _useMemoryGuard)
|
||||
{
|
||||
// TODO: Remove once we have made sure it is safe, i.e. after "Yul memory objects lite".
|
||||
// Also restore the tests removed in the commit that adds this comment.
|
||||
_useMemoryGuard = false;
|
||||
// This function should be called at the beginning of the EVM call frame
|
||||
// and thus can assume all memory to be zero, including the contents of
|
||||
// the "zero memory area" (the position CompilerUtils::zeroPointer points to).
|
||||
|
@ -23,6 +23,7 @@
|
||||
|
||||
#include <libyul/backends/evm/EVMCodeTransform.h>
|
||||
#include <libyul/backends/evm/EVMDialect.h>
|
||||
#include <libyul/backends/evm/OptimizedEVMCodeTransform.h>
|
||||
|
||||
#include <libyul/Object.h>
|
||||
#include <libyul/Exceptions.h>
|
||||
@ -62,19 +63,35 @@ void EVMObjectCompiler::run(Object& _object, bool _optimize)
|
||||
|
||||
yulAssert(_object.analysisInfo, "No analysis info.");
|
||||
yulAssert(_object.code, "No code.");
|
||||
// We do not catch and re-throw the stack too deep exception here because it is a YulException,
|
||||
// which should be native to this part of the code.
|
||||
CodeTransform transform{
|
||||
m_assembly,
|
||||
*_object.analysisInfo,
|
||||
*_object.code,
|
||||
m_dialect,
|
||||
context,
|
||||
_optimize,
|
||||
{},
|
||||
CodeTransform::UseNamedLabels::ForFirstFunctionOfEachName
|
||||
};
|
||||
transform(*_object.code);
|
||||
if (!transform.stackErrors().empty())
|
||||
BOOST_THROW_EXCEPTION(transform.stackErrors().front());
|
||||
if (_optimize && m_dialect.evmVersion().canOverchargeGasForCall())
|
||||
{
|
||||
auto stackErrors = OptimizedEVMCodeTransform::run(
|
||||
m_assembly,
|
||||
*_object.analysisInfo,
|
||||
*_object.code,
|
||||
m_dialect,
|
||||
context,
|
||||
OptimizedEVMCodeTransform::UseNamedLabels::ForFirstFunctionOfEachName
|
||||
);
|
||||
if (!stackErrors.empty())
|
||||
BOOST_THROW_EXCEPTION(stackErrors.front());
|
||||
}
|
||||
else
|
||||
{
|
||||
// We do not catch and re-throw the stack too deep exception here because it is a YulException,
|
||||
// which should be native to this part of the code.
|
||||
CodeTransform transform{
|
||||
m_assembly,
|
||||
*_object.analysisInfo,
|
||||
*_object.code,
|
||||
m_dialect,
|
||||
context,
|
||||
_optimize,
|
||||
{},
|
||||
CodeTransform::UseNamedLabels::ForFirstFunctionOfEachName
|
||||
};
|
||||
transform(*_object.code);
|
||||
if (!transform.stackErrors().empty())
|
||||
BOOST_THROW_EXCEPTION(transform.stackErrors().front());
|
||||
}
|
||||
}
|
||||
|
@ -44,7 +44,7 @@ vector<StackTooDeepError> OptimizedEVMCodeTransform::run(
|
||||
Block const& _block,
|
||||
EVMDialect const& _dialect,
|
||||
BuiltinContext& _builtinContext,
|
||||
bool _useNamedLabelsForFunctions
|
||||
UseNamedLabels _useNamedLabelsForFunctions
|
||||
)
|
||||
{
|
||||
std::unique_ptr<CFG> dfg = ControlFlowGraphBuilder::build(_analysisInfo, _dialect, _block);
|
||||
@ -170,15 +170,35 @@ void OptimizedEVMCodeTransform::operator()(CFG::Assignment const& _assignment)
|
||||
OptimizedEVMCodeTransform::OptimizedEVMCodeTransform(
|
||||
AbstractAssembly& _assembly,
|
||||
BuiltinContext& _builtinContext,
|
||||
bool _useNamedLabelsForFunctions,
|
||||
UseNamedLabels _useNamedLabelsForFunctions,
|
||||
CFG const& _dfg,
|
||||
StackLayout const& _stackLayout
|
||||
):
|
||||
m_assembly(_assembly),
|
||||
m_builtinContext(_builtinContext),
|
||||
m_useNamedLabelsForFunctions(_useNamedLabelsForFunctions),
|
||||
m_dfg(_dfg),
|
||||
m_stackLayout(_stackLayout)
|
||||
m_stackLayout(_stackLayout),
|
||||
m_functionLabels([&](){
|
||||
map<CFG::FunctionInfo const*, AbstractAssembly::LabelID> functionLabels;
|
||||
set<YulString> assignedFunctionNames;
|
||||
for (Scope::Function const* function: m_dfg.functions)
|
||||
{
|
||||
CFG::FunctionInfo const& functionInfo = m_dfg.functionInfo.at(function);
|
||||
bool nameAlreadySeen = !assignedFunctionNames.insert(function->name).second;
|
||||
if (_useNamedLabelsForFunctions == UseNamedLabels::YesAndForceUnique)
|
||||
yulAssert(!nameAlreadySeen);
|
||||
bool useNamedLabel = _useNamedLabelsForFunctions != UseNamedLabels::Never && !nameAlreadySeen;
|
||||
functionLabels[&functionInfo] = useNamedLabel ?
|
||||
m_assembly.namedLabel(
|
||||
function->name.str(),
|
||||
function->arguments.size(),
|
||||
function->returns.size(),
|
||||
functionInfo.debugData ? functionInfo.debugData->astID : nullopt
|
||||
) :
|
||||
m_assembly.newLabelId();
|
||||
}
|
||||
return functionLabels;
|
||||
}())
|
||||
{
|
||||
}
|
||||
|
||||
@ -191,15 +211,7 @@ void OptimizedEVMCodeTransform::assertLayoutCompatibility(Stack const& _currentS
|
||||
|
||||
AbstractAssembly::LabelID OptimizedEVMCodeTransform::getFunctionLabel(Scope::Function const& _function)
|
||||
{
|
||||
CFG::FunctionInfo const& functionInfo = m_dfg.functionInfo.at(&_function);
|
||||
if (!m_functionLabels.count(&functionInfo))
|
||||
m_functionLabels[&functionInfo] = m_useNamedLabelsForFunctions ? m_assembly.namedLabel(
|
||||
functionInfo.function.name.str(),
|
||||
functionInfo.function.arguments.size(),
|
||||
functionInfo.function.returns.size(),
|
||||
{}
|
||||
) : m_assembly.newLabelId();
|
||||
return m_functionLabels[&functionInfo];
|
||||
return m_functionLabels.at(&m_dfg.functionInfo.at(&_function));
|
||||
}
|
||||
|
||||
void OptimizedEVMCodeTransform::validateSlot(StackSlot const& _slot, Expression const& _expression)
|
||||
|
@ -43,13 +43,17 @@ struct StackLayout;
|
||||
class OptimizedEVMCodeTransform
|
||||
{
|
||||
public:
|
||||
/// Use named labels for functions 1) Yes and check that the names are unique
|
||||
/// 2) For none of the functions 3) for the first function of each name.
|
||||
enum class UseNamedLabels { YesAndForceUnique, Never, ForFirstFunctionOfEachName };
|
||||
|
||||
[[nodiscard]] static std::vector<StackTooDeepError> run(
|
||||
AbstractAssembly& _assembly,
|
||||
AsmAnalysisInfo& _analysisInfo,
|
||||
Block const& _block,
|
||||
EVMDialect const& _dialect,
|
||||
BuiltinContext& _builtinContext,
|
||||
bool _useNamedLabelsForFunctions = false
|
||||
UseNamedLabels _useNamedLabelsForFunctions
|
||||
);
|
||||
|
||||
/// Generate code for the function call @a _call. Only public for using with std::visit.
|
||||
@ -62,7 +66,7 @@ private:
|
||||
OptimizedEVMCodeTransform(
|
||||
AbstractAssembly& _assembly,
|
||||
BuiltinContext& _builtinContext,
|
||||
bool _useNamedLabelsForFunctions,
|
||||
UseNamedLabels _useNamedLabelsForFunctions,
|
||||
CFG const& _dfg,
|
||||
StackLayout const& _stackLayout
|
||||
);
|
||||
@ -70,6 +74,7 @@ private:
|
||||
/// Assert that it is valid to transition from @a _currentStack to @a _desiredStack.
|
||||
/// That is @a _currentStack matches each slot in @a _desiredStack that is not a JunkSlot exactly.
|
||||
static void assertLayoutCompatibility(Stack const& _currentStack, Stack const& _desiredStack);
|
||||
|
||||
/// @returns The label of the entry point of the given @a _function.
|
||||
/// Creates and stores a new label, if none exists already.
|
||||
AbstractAssembly::LabelID getFunctionLabel(Scope::Function const& _function);
|
||||
@ -94,13 +99,12 @@ private:
|
||||
|
||||
AbstractAssembly& m_assembly;
|
||||
BuiltinContext& m_builtinContext;
|
||||
bool m_useNamedLabelsForFunctions = true;
|
||||
CFG const& m_dfg;
|
||||
StackLayout const& m_stackLayout;
|
||||
Stack m_stack;
|
||||
std::map<yul::FunctionCall const*, AbstractAssembly::LabelID> m_returnLabels;
|
||||
std::map<CFG::BasicBlock const*, AbstractAssembly::LabelID> m_blockLabels;
|
||||
std::map<CFG::FunctionInfo const*, AbstractAssembly::LabelID> m_functionLabels;
|
||||
std::map<CFG::FunctionInfo const*, AbstractAssembly::LabelID> const m_functionLabels;
|
||||
/// Set of blocks already generated. If any of the contained blocks is ever jumped to, m_blockLabels should
|
||||
/// contain a jump label for it.
|
||||
std::set<CFG::BasicBlock const*> m_generated;
|
||||
|
@ -27,6 +27,13 @@
|
||||
#include <libyul/optimiser/Metrics.h>
|
||||
#include <libyul/optimiser/Semantics.h>
|
||||
|
||||
#include <libyul/backends/evm/ControlFlowGraphBuilder.h>
|
||||
#include <libyul/backends/evm/StackHelpers.h>
|
||||
#include <libyul/backends/evm/StackLayoutGenerator.h>
|
||||
|
||||
#include <libyul/AsmAnalysis.h>
|
||||
#include <libyul/AsmAnalysisInfo.h>
|
||||
|
||||
#include <libyul/CompilabilityChecker.h>
|
||||
|
||||
#include <libyul/AST.h>
|
||||
@ -162,6 +169,50 @@ void eliminateVariables(
|
||||
UnusedPruner::runUntilStabilised(_dialect, _node, _allowMSizeOptimization);
|
||||
}
|
||||
|
||||
void eliminateVariables(
|
||||
Dialect const& _dialect,
|
||||
Block& _block,
|
||||
vector<StackLayoutGenerator::StackTooDeep> const& _unreachables,
|
||||
bool _allowMSizeOptimization
|
||||
)
|
||||
{
|
||||
RematCandidateSelector selector{_dialect};
|
||||
selector(_block);
|
||||
std::map<YulString, size_t> candidates;
|
||||
for (auto [cost, candidatesWithCost]: selector.candidates())
|
||||
for (auto candidate: candidatesWithCost)
|
||||
candidates[get<0>(candidate)] = cost;
|
||||
|
||||
set<YulString> varsToEliminate;
|
||||
|
||||
// TODO: this currently ignores the fact that variables may reference other variables we want to eliminate.
|
||||
for (auto const& unreachable: _unreachables)
|
||||
{
|
||||
map<size_t, vector<YulString>> suitableCandidates;
|
||||
size_t neededSlots = unreachable.deficit;
|
||||
for (auto varName: unreachable.variableChoices)
|
||||
{
|
||||
if (varsToEliminate.count(varName))
|
||||
--neededSlots;
|
||||
else if (size_t* cost = util::valueOrNullptr(candidates, varName))
|
||||
if (!util::contains(suitableCandidates[*cost], varName))
|
||||
suitableCandidates[*cost].emplace_back(varName);
|
||||
}
|
||||
for (auto candidatesByCost: suitableCandidates)
|
||||
{
|
||||
for (auto candidate: candidatesByCost.second)
|
||||
if (neededSlots--)
|
||||
varsToEliminate.emplace(candidate);
|
||||
else
|
||||
break;
|
||||
if (!neededSlots)
|
||||
break;
|
||||
}
|
||||
}
|
||||
Rematerialiser::run(_dialect, _block, std::move(varsToEliminate), true);
|
||||
UnusedPruner::runUntilStabilised(_dialect, _block, _allowMSizeOptimization);
|
||||
}
|
||||
|
||||
}
|
||||
|
||||
bool StackCompressor::run(
|
||||
@ -176,39 +227,66 @@ bool StackCompressor::run(
|
||||
_object.code->statements.size() > 0 && holds_alternative<Block>(_object.code->statements.at(0)),
|
||||
"Need to run the function grouper before the stack compressor."
|
||||
);
|
||||
bool usesOptimizedCodeGenerator = false;
|
||||
if (auto evmDialect = dynamic_cast<EVMDialect const*>(&_dialect))
|
||||
usesOptimizedCodeGenerator =
|
||||
_optimizeStackAllocation &&
|
||||
evmDialect->evmVersion().canOverchargeGasForCall() &&
|
||||
evmDialect->providesObjectAccess();
|
||||
bool allowMSizeOptimzation = !MSizeFinder::containsMSize(_dialect, *_object.code);
|
||||
for (size_t iterations = 0; iterations < _maxIterations; iterations++)
|
||||
if (usesOptimizedCodeGenerator)
|
||||
{
|
||||
map<YulString, int> stackSurplus = CompilabilityChecker(_dialect, _object, _optimizeStackAllocation).stackDeficit;
|
||||
if (stackSurplus.empty())
|
||||
return true;
|
||||
|
||||
if (stackSurplus.count(YulString{}))
|
||||
{
|
||||
yulAssert(stackSurplus.at({}) > 0, "Invalid surplus value.");
|
||||
eliminateVariables(
|
||||
_dialect,
|
||||
std::get<Block>(_object.code->statements.at(0)),
|
||||
static_cast<size_t>(stackSurplus.at({})),
|
||||
allowMSizeOptimzation
|
||||
);
|
||||
}
|
||||
|
||||
yul::AsmAnalysisInfo analysisInfo = yul::AsmAnalyzer::analyzeStrictAssertCorrect(_dialect, _object);
|
||||
unique_ptr<CFG> cfg = ControlFlowGraphBuilder::build(analysisInfo, _dialect, *_object.code);
|
||||
Block& mainBlock = std::get<Block>(_object.code->statements.at(0));
|
||||
if (
|
||||
auto stackTooDeepErrors = StackLayoutGenerator::reportStackTooDeep(*cfg, YulString{});
|
||||
!stackTooDeepErrors.empty()
|
||||
)
|
||||
eliminateVariables(_dialect, mainBlock, stackTooDeepErrors, allowMSizeOptimzation);
|
||||
for (size_t i = 1; i < _object.code->statements.size(); ++i)
|
||||
{
|
||||
auto& fun = std::get<FunctionDefinition>(_object.code->statements[i]);
|
||||
if (!stackSurplus.count(fun.name))
|
||||
continue;
|
||||
|
||||
yulAssert(stackSurplus.at(fun.name) > 0, "Invalid surplus value.");
|
||||
eliminateVariables(
|
||||
_dialect,
|
||||
fun,
|
||||
static_cast<size_t>(stackSurplus.at(fun.name)),
|
||||
allowMSizeOptimzation
|
||||
);
|
||||
if (
|
||||
auto stackTooDeepErrors = StackLayoutGenerator::reportStackTooDeep(*cfg, fun.name);
|
||||
!stackTooDeepErrors.empty()
|
||||
)
|
||||
eliminateVariables(_dialect, fun.body, stackTooDeepErrors, allowMSizeOptimzation);
|
||||
}
|
||||
}
|
||||
else
|
||||
for (size_t iterations = 0; iterations < _maxIterations; iterations++)
|
||||
{
|
||||
map<YulString, int> stackSurplus = CompilabilityChecker(_dialect, _object, _optimizeStackAllocation).stackDeficit;
|
||||
if (stackSurplus.empty())
|
||||
return true;
|
||||
|
||||
if (stackSurplus.count(YulString{}))
|
||||
{
|
||||
yulAssert(stackSurplus.at({}) > 0, "Invalid surplus value.");
|
||||
eliminateVariables(
|
||||
_dialect,
|
||||
std::get<Block>(_object.code->statements.at(0)),
|
||||
static_cast<size_t>(stackSurplus.at({})),
|
||||
allowMSizeOptimzation
|
||||
);
|
||||
}
|
||||
|
||||
for (size_t i = 1; i < _object.code->statements.size(); ++i)
|
||||
{
|
||||
auto& fun = std::get<FunctionDefinition>(_object.code->statements[i]);
|
||||
if (!stackSurplus.count(fun.name))
|
||||
continue;
|
||||
|
||||
yulAssert(stackSurplus.at(fun.name) > 0, "Invalid surplus value.");
|
||||
eliminateVariables(
|
||||
_dialect,
|
||||
fun,
|
||||
static_cast<size_t>(stackSurplus.at(fun.name)),
|
||||
allowMSizeOptimzation
|
||||
);
|
||||
}
|
||||
}
|
||||
return false;
|
||||
}
|
||||
|
||||
|
@ -21,14 +21,18 @@
|
||||
#include <libyul/optimiser/FunctionDefinitionCollector.h>
|
||||
#include <libyul/optimiser/NameDispenser.h>
|
||||
#include <libyul/optimiser/StackToMemoryMover.h>
|
||||
#include <libyul/backends/evm/ControlFlowGraphBuilder.h>
|
||||
#include <libyul/backends/evm/EVMDialect.h>
|
||||
#include <libyul/AsmAnalysis.h>
|
||||
#include <libyul/AST.h>
|
||||
#include <libyul/CompilabilityChecker.h>
|
||||
#include <libyul/Exceptions.h>
|
||||
#include <libyul/Object.h>
|
||||
#include <libyul/Utilities.h>
|
||||
#include <libsolutil/Algorithms.h>
|
||||
#include <libsolutil/CommonData.h>
|
||||
|
||||
#include <range/v3/range/conversion.hpp>
|
||||
#include <range/v3/view/concat.hpp>
|
||||
#include <range/v3/view/take.hpp>
|
||||
|
||||
@ -114,6 +118,45 @@ u256 literalArgumentValue(FunctionCall const& _call)
|
||||
}
|
||||
}
|
||||
|
||||
void StackLimitEvader::run(
|
||||
OptimiserStepContext& _context,
|
||||
Object& _object
|
||||
)
|
||||
{
|
||||
auto const* evmDialect = dynamic_cast<EVMDialect const*>(&_context.dialect);
|
||||
yulAssert(
|
||||
evmDialect && evmDialect->providesObjectAccess(),
|
||||
"StackLimitEvader can only be run on objects using the EVMDialect with object access."
|
||||
);
|
||||
if (evmDialect && evmDialect->evmVersion().canOverchargeGasForCall())
|
||||
{
|
||||
yul::AsmAnalysisInfo analysisInfo = yul::AsmAnalyzer::analyzeStrictAssertCorrect(*evmDialect, _object);
|
||||
unique_ptr<CFG> cfg = ControlFlowGraphBuilder::build(analysisInfo, *evmDialect, *_object.code);
|
||||
run(_context, _object, StackLayoutGenerator::reportStackTooDeep(*cfg));
|
||||
}
|
||||
else
|
||||
run(_context, _object, CompilabilityChecker{
|
||||
_context.dialect,
|
||||
_object,
|
||||
true
|
||||
}.unreachableVariables);
|
||||
|
||||
}
|
||||
|
||||
void StackLimitEvader::run(
|
||||
OptimiserStepContext& _context,
|
||||
Object& _object,
|
||||
map<YulString, vector<StackLayoutGenerator::StackTooDeep>> const& _stackTooDeepErrors
|
||||
)
|
||||
{
|
||||
map<YulString, set<YulString>> unreachableVariables;
|
||||
for (auto&& [function, stackTooDeepErrors]: _stackTooDeepErrors)
|
||||
// TODO: choose wisely.
|
||||
for (auto const& stackTooDeepError: stackTooDeepErrors)
|
||||
unreachableVariables[function] += stackTooDeepError.variableChoices | ranges::views::take(stackTooDeepError.deficit) | ranges::to<set<YulString>>;
|
||||
run(_context, _object, unreachableVariables);
|
||||
}
|
||||
|
||||
void StackLimitEvader::run(
|
||||
OptimiserStepContext& _context,
|
||||
Object& _object,
|
||||
|
@ -22,6 +22,7 @@
|
||||
#pragma once
|
||||
|
||||
#include <libyul/optimiser/OptimiserStep.h>
|
||||
#include <libyul/backends/evm/StackLayoutGenerator.h>
|
||||
|
||||
namespace solidity::yul
|
||||
{
|
||||
@ -61,6 +62,25 @@ public:
|
||||
Object& _object,
|
||||
std::map<YulString, std::set<YulString>> const& _unreachableVariables
|
||||
);
|
||||
/// @a _stackTooDeepErrors can be determined by the StackLayoutGenerator.
|
||||
/// Can only be run on the EVM dialect with objects.
|
||||
/// Abort and do nothing, if no ``memoryguard`` call or several ``memoryguard`` calls
|
||||
/// with non-matching arguments are found, or if any of the @a _stackTooDeepErrors
|
||||
/// are contained in a recursive function.
|
||||
static void run(
|
||||
OptimiserStepContext& _context,
|
||||
Object& _object,
|
||||
std::map<YulString, std::vector<StackLayoutGenerator::StackTooDeep>> const& _stackTooDeepErrors
|
||||
);
|
||||
/// Determines stack too deep errors using the appropriate code generation backend.
|
||||
/// Can only be run on the EVM dialect with objects.
|
||||
/// Abort and do nothing, if no ``memoryguard`` call or several ``memoryguard`` calls
|
||||
/// with non-matching arguments are found, or if any of the unreachable variables
|
||||
/// are contained in a recursive function.
|
||||
static void run(
|
||||
OptimiserStepContext& _context,
|
||||
Object& _object
|
||||
);
|
||||
};
|
||||
|
||||
}
|
||||
|
@ -95,6 +95,12 @@ void OptimiserSuite::run(
|
||||
set<YulString> const& _externallyUsedIdentifiers
|
||||
)
|
||||
{
|
||||
EVMDialect const* evmDialect = dynamic_cast<EVMDialect const*>(&_dialect);
|
||||
bool usesOptimizedCodeGenerator =
|
||||
_optimizeStackAllocation &&
|
||||
evmDialect &&
|
||||
evmDialect->evmVersion().canOverchargeGasForCall() &&
|
||||
evmDialect->providesObjectAccess();
|
||||
set<YulString> reservedIdentifiers = _externallyUsedIdentifiers;
|
||||
reservedIdentifiers += _dialect.fixedFunctionNames();
|
||||
|
||||
@ -121,24 +127,32 @@ void OptimiserSuite::run(
|
||||
|
||||
// We ignore the return value because we will get a much better error
|
||||
// message once we perform code generation.
|
||||
StackCompressor::run(
|
||||
_dialect,
|
||||
_object,
|
||||
_optimizeStackAllocation,
|
||||
stackCompressorMaxIterations
|
||||
);
|
||||
if (!usesOptimizedCodeGenerator)
|
||||
StackCompressor::run(
|
||||
_dialect,
|
||||
_object,
|
||||
_optimizeStackAllocation,
|
||||
stackCompressorMaxIterations
|
||||
);
|
||||
suite.runSequence("fDnTOc g", ast);
|
||||
|
||||
if (EVMDialect const* dialect = dynamic_cast<EVMDialect const*>(&_dialect))
|
||||
if (evmDialect)
|
||||
{
|
||||
yulAssert(_meter, "");
|
||||
ConstantOptimiser{*dialect, *_meter}(ast);
|
||||
if (dialect->providesObjectAccess() && _optimizeStackAllocation)
|
||||
StackLimitEvader::run(suite.m_context, _object, CompilabilityChecker{
|
||||
ConstantOptimiser{*evmDialect, *_meter}(ast);
|
||||
if (usesOptimizedCodeGenerator)
|
||||
{
|
||||
StackCompressor::run(
|
||||
_dialect,
|
||||
_object,
|
||||
_optimizeStackAllocation
|
||||
}.unreachableVariables);
|
||||
_optimizeStackAllocation,
|
||||
stackCompressorMaxIterations
|
||||
);
|
||||
if (evmDialect->providesObjectAccess())
|
||||
StackLimitEvader::run(suite.m_context, _object);
|
||||
}
|
||||
else if (evmDialect->providesObjectAccess() && _optimizeStackAllocation)
|
||||
StackLimitEvader::run(suite.m_context, _object);
|
||||
}
|
||||
else if (dynamic_cast<WasmDialect const*>(&_dialect))
|
||||
{
|
||||
|
@ -66,7 +66,7 @@ IR:
|
||||
object "C_6" {
|
||||
code {
|
||||
/// @src 0:60:101 "contract C {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_6()
|
||||
@ -97,7 +97,7 @@ object "C_6" {
|
||||
object "C_6_deployed" {
|
||||
code {
|
||||
/// @src 0:60:101 "contract C {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
@ -182,11 +182,12 @@ object "C_6" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:60:101 "contract C {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_6_deployed")
|
||||
codecopy(128, dataoffset("C_6_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_6_deployed")
|
||||
codecopy(_1, dataoffset("C_6_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"debug_info_in_yul_and_evm_asm_print_all/input.sol"
|
||||
@ -194,15 +195,16 @@ object "C_6" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:60:101 "contract C {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_1)))
|
||||
let _2 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_2)))
|
||||
{
|
||||
if callvalue() { revert(_1, _1) }
|
||||
if slt(add(calldatasize(), not(3)), _1) { revert(_1, _1) }
|
||||
return(128, _1)
|
||||
if callvalue() { revert(_2, _2) }
|
||||
if slt(add(calldatasize(), not(3)), _2) { revert(_2, _2) }
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
revert(0, 0)
|
||||
|
@ -66,7 +66,7 @@ IR:
|
||||
object "C_6" {
|
||||
code {
|
||||
/// @src 0:60:101
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_6()
|
||||
@ -97,7 +97,7 @@ object "C_6" {
|
||||
object "C_6_deployed" {
|
||||
code {
|
||||
/// @src 0:60:101
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
@ -181,11 +181,12 @@ object "C_6" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:60:101
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_6_deployed")
|
||||
codecopy(128, dataoffset("C_6_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_6_deployed")
|
||||
codecopy(_1, dataoffset("C_6_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"debug_info_in_yul_and_evm_asm_print_location_only/input.sol"
|
||||
@ -193,15 +194,16 @@ object "C_6" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:60:101
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_1)))
|
||||
let _2 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_2)))
|
||||
{
|
||||
if callvalue() { revert(_1, _1) }
|
||||
if slt(add(calldatasize(), not(3)), _1) { revert(_1, _1) }
|
||||
return(128, _1)
|
||||
if callvalue() { revert(_2, _2) }
|
||||
if slt(add(calldatasize(), not(3)), _2) { revert(_2, _2) }
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
revert(0, 0)
|
||||
|
@ -63,7 +63,7 @@ IR:
|
||||
object "C_6" {
|
||||
code {
|
||||
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_6()
|
||||
@ -90,7 +90,7 @@ object "C_6" {
|
||||
object "C_6_deployed" {
|
||||
code {
|
||||
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
@ -171,26 +171,28 @@ Optimized IR:
|
||||
object "C_6" {
|
||||
code {
|
||||
{
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_6_deployed")
|
||||
codecopy(128, dataoffset("C_6_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_6_deployed")
|
||||
codecopy(_1, dataoffset("C_6_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"debug_info_in_yul_and_evm_asm_print_none/input.sol"
|
||||
object "C_6_deployed" {
|
||||
code {
|
||||
{
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_1)))
|
||||
let _2 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_2)))
|
||||
{
|
||||
if callvalue() { revert(_1, _1) }
|
||||
if slt(add(calldatasize(), not(3)), _1) { revert(_1, _1) }
|
||||
return(128, _1)
|
||||
if callvalue() { revert(_2, _2) }
|
||||
if slt(add(calldatasize(), not(3)), _2) { revert(_2, _2) }
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
revert(0, 0)
|
||||
|
@ -11,7 +11,7 @@ IR:
|
||||
object "C_2" {
|
||||
code {
|
||||
/// @src 0:265:278 "contract C {}"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_2()
|
||||
@ -42,7 +42,7 @@ object "C_2" {
|
||||
object "C_2_deployed" {
|
||||
code {
|
||||
/// @src 0:265:278 "contract C {}"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
revert_error_42b3090547df1d2001c96683413b8cf91c1b902ef5e3cb8d9f6f304cf7446f74()
|
||||
|
||||
@ -82,11 +82,12 @@ object "C_2" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:265:278 "contract C {}"
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_2_deployed")
|
||||
codecopy(128, dataoffset("C_2_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_2_deployed")
|
||||
codecopy(_1, dataoffset("C_2_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"debug_info_in_yul_snippet_escaping/input.sol"
|
||||
@ -94,7 +95,7 @@ object "C_2" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:265:278 "contract C {}"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
revert(0, 0)
|
||||
}
|
||||
}
|
||||
@ -115,7 +116,7 @@ IR:
|
||||
object "D_27" {
|
||||
code {
|
||||
/// @src 0:279:599 "contract D /** @src 0:96:165 \"contract D {...\" *\/ {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_D_27()
|
||||
@ -146,7 +147,7 @@ object "D_27" {
|
||||
object "D_27_deployed" {
|
||||
code {
|
||||
/// @src 0:279:599 "contract D /** @src 0:96:165 \"contract D {...\" *\/ {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
@ -372,7 +373,7 @@ object "D_27" {
|
||||
object "C_2" {
|
||||
code {
|
||||
/// @src 0:265:278 "contract C {}"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_2()
|
||||
@ -403,7 +404,7 @@ object "D_27" {
|
||||
object "C_2_deployed" {
|
||||
code {
|
||||
/// @src 0:265:278 "contract C {}"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
revert_error_42b3090547df1d2001c96683413b8cf91c1b902ef5e3cb8d9f6f304cf7446f74()
|
||||
|
||||
@ -448,11 +449,12 @@ object "D_27" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:279:599 "contract D /** @src 0:96:165 \"contract D {...\" *\/ {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("D_27_deployed")
|
||||
codecopy(128, dataoffset("D_27_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("D_27_deployed")
|
||||
codecopy(_1, dataoffset("D_27_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"debug_info_in_yul_snippet_escaping/input.sol"
|
||||
@ -460,26 +462,25 @@ object "D_27" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:279:599 "contract D /** @src 0:96:165 \"contract D {...\" *\/ {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_1)))
|
||||
let _2 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_2)))
|
||||
{
|
||||
if callvalue() { revert(_1, _1) }
|
||||
if slt(add(calldatasize(), not(3)), _1) { revert(_1, _1) }
|
||||
if callvalue() { revert(_2, _2) }
|
||||
if slt(add(calldatasize(), not(3)), _2) { revert(_2, _2) }
|
||||
/// @src 0:446:491 "new /// @src 0:149:156 \"new C()\"..."
|
||||
let _2 := datasize("C_2")
|
||||
let _3 := add(/** @src 0:279:599 "contract D /** @src 0:96:165 \"contract D {...\" *\/ {..." */ 128, /** @src 0:446:491 "new /// @src 0:149:156 \"new C()\"..." */ _2)
|
||||
if or(gt(_3, 0xffffffffffffffff), lt(_3, /** @src 0:279:599 "contract D /** @src 0:96:165 \"contract D {...\" *\/ {..." */ 128))
|
||||
/// @src 0:446:491 "new /// @src 0:149:156 \"new C()\"..."
|
||||
{ panic_error_0x41() }
|
||||
datacopy(/** @src 0:279:599 "contract D /** @src 0:96:165 \"contract D {...\" *\/ {..." */ 128, /** @src 0:446:491 "new /// @src 0:149:156 \"new C()\"..." */ dataoffset("C_2"), _2)
|
||||
if iszero(create(/** @src 0:279:599 "contract D /** @src 0:96:165 \"contract D {...\" *\/ {..." */ _1, 128, /** @src 0:446:491 "new /// @src 0:149:156 \"new C()\"..." */ _2))
|
||||
let _3 := datasize("C_2")
|
||||
let _4 := add(_1, _3)
|
||||
if or(gt(_4, 0xffffffffffffffff), lt(_4, _1)) { panic_error_0x41() }
|
||||
datacopy(_1, dataoffset("C_2"), _3)
|
||||
if iszero(create(/** @src 0:279:599 "contract D /** @src 0:96:165 \"contract D {...\" *\/ {..." */ _2, /** @src 0:446:491 "new /// @src 0:149:156 \"new C()\"..." */ _1, sub(_4, _1)))
|
||||
{
|
||||
/// @src 0:279:599 "contract D /** @src 0:96:165 \"contract D {...\" *\/ {..."
|
||||
let pos := mload(64)
|
||||
returndatacopy(pos, _1, returndatasize())
|
||||
returndatacopy(pos, _2, returndatasize())
|
||||
revert(pos, returndatasize())
|
||||
}
|
||||
mstore(add(allocate_memory_array_string(), 32), "/*")
|
||||
@ -539,11 +540,12 @@ object "D_27" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:265:278 "contract C {}"
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_2_deployed")
|
||||
codecopy(128, dataoffset("C_2_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_2_deployed")
|
||||
codecopy(_1, dataoffset("C_2_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"debug_info_in_yul_snippet_escaping/input.sol"
|
||||
@ -551,7 +553,7 @@ object "D_27" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:265:278 "contract C {}"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
revert(0, 0)
|
||||
}
|
||||
}
|
||||
|
@ -11,7 +11,7 @@ IR:
|
||||
object "C_81" {
|
||||
code {
|
||||
/// @src 0:82:370 "contract C {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_81()
|
||||
@ -42,7 +42,7 @@ object "C_81" {
|
||||
object "C_81_deployed" {
|
||||
code {
|
||||
/// @src 0:82:370 "contract C {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
|
@ -13,7 +13,7 @@
|
||||
},
|
||||
"calldata_array_index_access_uint256_dyn_calldata":
|
||||
{
|
||||
"entryPoint": 168,
|
||||
"entryPoint": 152,
|
||||
"parameterSlots": 2,
|
||||
"returnSlots": 1
|
||||
}
|
||||
|
@ -11,11 +11,12 @@ object "C_7" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:117 "contract C {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_7_deployed")
|
||||
codecopy(128, dataoffset("C_7_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_7_deployed")
|
||||
codecopy(_1, dataoffset("C_7_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"ir_compiler_inheritance_nosubobjects/input.sol"
|
||||
@ -23,7 +24,7 @@ object "C_7" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:117 "contract C {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
revert(0, 0)
|
||||
}
|
||||
}
|
||||
@ -44,11 +45,12 @@ object "D_10" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:118:137 "contract D is C {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("D_10_deployed")
|
||||
codecopy(128, dataoffset("D_10_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("D_10_deployed")
|
||||
codecopy(_1, dataoffset("D_10_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"ir_compiler_inheritance_nosubobjects/input.sol"
|
||||
@ -56,7 +58,7 @@ object "D_10" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:118:137 "contract D is C {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
revert(0, 0)
|
||||
}
|
||||
}
|
||||
|
@ -11,11 +11,12 @@ object "C_3" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:95 "contract C {}"
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_3_deployed")
|
||||
codecopy(128, dataoffset("C_3_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_3_deployed")
|
||||
codecopy(_1, dataoffset("C_3_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"ir_compiler_subobjects/input.sol"
|
||||
@ -23,7 +24,7 @@ object "C_3" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:95 "contract C {}"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
revert(0, 0)
|
||||
}
|
||||
}
|
||||
@ -44,11 +45,12 @@ object "D_16" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:96:165 "contract D {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("D_16_deployed")
|
||||
codecopy(128, dataoffset("D_16_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("D_16_deployed")
|
||||
codecopy(_1, dataoffset("D_16_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"ir_compiler_subobjects/input.sol"
|
||||
@ -56,35 +58,35 @@ object "D_16" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:96:165 "contract D {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_1)))
|
||||
let _2 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_2)))
|
||||
{
|
||||
if callvalue() { revert(_1, _1) }
|
||||
if slt(add(calldatasize(), not(3)), _1) { revert(_1, _1) }
|
||||
/// @src 0:149:156 "new C()"
|
||||
let _2 := datasize("C_3")
|
||||
let _3 := add(/** @src 0:96:165 "contract D {..." */ 128, /** @src 0:149:156 "new C()" */ _2)
|
||||
if or(gt(_3, 0xffffffffffffffff), lt(_3, /** @src 0:96:165 "contract D {..." */ 128))
|
||||
if callvalue() { revert(_2, _2) }
|
||||
if slt(add(calldatasize(), not(3)), _2) { revert(_2, _2) }
|
||||
/// @src 0:149:156 "new C()"
|
||||
let _3 := datasize("C_3")
|
||||
let _4 := add(_1, _3)
|
||||
if or(gt(_4, 0xffffffffffffffff), lt(_4, _1))
|
||||
{
|
||||
/// @src 0:96:165 "contract D {..."
|
||||
mstore(_1, shl(224, 0x4e487b71))
|
||||
mstore(_2, shl(224, 0x4e487b71))
|
||||
mstore(4, 0x41)
|
||||
revert(_1, 0x24)
|
||||
revert(_2, 0x24)
|
||||
}
|
||||
/// @src 0:149:156 "new C()"
|
||||
datacopy(/** @src 0:96:165 "contract D {..." */ 128, /** @src 0:149:156 "new C()" */ dataoffset("C_3"), _2)
|
||||
if iszero(create(/** @src 0:96:165 "contract D {..." */ _1, 128, /** @src 0:149:156 "new C()" */ _2))
|
||||
datacopy(_1, dataoffset("C_3"), _3)
|
||||
if iszero(create(/** @src 0:96:165 "contract D {..." */ _2, /** @src 0:149:156 "new C()" */ _1, sub(_4, _1)))
|
||||
{
|
||||
/// @src 0:96:165 "contract D {..."
|
||||
let pos := mload(64)
|
||||
returndatacopy(pos, _1, returndatasize())
|
||||
returndatacopy(pos, _2, returndatasize())
|
||||
revert(pos, returndatasize())
|
||||
}
|
||||
return(mload(64), _1)
|
||||
return(mload(64), _2)
|
||||
}
|
||||
}
|
||||
revert(0, 0)
|
||||
@ -95,11 +97,12 @@ object "D_16" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:95 "contract C {}"
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_3_deployed")
|
||||
codecopy(128, dataoffset("C_3_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_3_deployed")
|
||||
codecopy(_1, dataoffset("C_3_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"ir_compiler_subobjects/input.sol"
|
||||
@ -107,7 +110,7 @@ object "D_16" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:95 "contract C {}"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
revert(0, 0)
|
||||
}
|
||||
}
|
||||
|
@ -23,15 +23,16 @@ object "D_12" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:161 "contract D {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_1)))
|
||||
let _2 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_2)))
|
||||
{
|
||||
if callvalue() { revert(_1, _1) }
|
||||
if slt(add(calldatasize(), not(3)), _1) { revert(_1, _1) }
|
||||
return(128, _1)
|
||||
if callvalue() { revert(_2, _2) }
|
||||
if slt(add(calldatasize(), not(3)), _2) { revert(_2, _2) }
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
revert(0, 0)
|
||||
|
@ -11,11 +11,12 @@ object "D_8" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:153 "contract D {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("D_8_deployed")
|
||||
codecopy(128, dataoffset("D_8_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("D_8_deployed")
|
||||
codecopy(_1, dataoffset("D_8_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"ir_with_assembly_no_memoryguard_runtime/input.sol"
|
||||
|
@ -11,11 +11,12 @@ object "C_7" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:62:285 "contract C {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_7_deployed")
|
||||
codecopy(128, dataoffset("C_7_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_7_deployed")
|
||||
codecopy(_1, dataoffset("C_7_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"keccak_optimization_low_runs/input.sol"
|
||||
|
@ -11,11 +11,12 @@ object "C_59" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:346:625 "contract C {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_59_deployed")
|
||||
codecopy(128, dataoffset("C_59_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_59_deployed")
|
||||
codecopy(_1, dataoffset("C_59_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"name_simplifier/input.sol"
|
||||
@ -23,7 +24,7 @@ object "C_59" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:346:625 "contract C {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
|
@ -23,7 +23,7 @@ object "MyContract" {
|
||||
|
||||
|
||||
Binary representation:
|
||||
33600055600b806011600039806000f3fe60005460005260206000f3
|
||||
33600055600b8060106000396000f3fe60005460005260206000f3
|
||||
|
||||
Text representation:
|
||||
/* "object_compiler/input.yul":128:136 */
|
||||
@ -34,15 +34,13 @@ Text representation:
|
||||
sstore
|
||||
/* "object_compiler/input.yul":240:259 */
|
||||
dataSize(sub_0)
|
||||
dup1
|
||||
/* "object_compiler/input.yul":217:238 */
|
||||
dup1
|
||||
dataOffset(sub_0)
|
||||
/* "object_compiler/input.yul":125:126 */
|
||||
0x00
|
||||
/* "object_compiler/input.yul":205:260 */
|
||||
codecopy
|
||||
/* "object_compiler/input.yul":275:294 */
|
||||
dup1
|
||||
/* "object_compiler/input.yul":125:126 */
|
||||
0x00
|
||||
/* "object_compiler/input.yul":265:295 */
|
||||
|
@ -11,11 +11,12 @@ object "Arraysum_34" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:80:429 "contract Arraysum {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("Arraysum_34_deployed")
|
||||
codecopy(128, dataoffset("Arraysum_34_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("Arraysum_34_deployed")
|
||||
codecopy(_1, dataoffset("Arraysum_34_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"optimizer_array_sload/input.sol"
|
||||
@ -23,7 +24,7 @@ object "Arraysum_34" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:80:429 "contract Arraysum {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
|
@ -11,7 +11,7 @@ IR:
|
||||
object "C_15" {
|
||||
code {
|
||||
/// @src 0:59:147 "contract C {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_15()
|
||||
@ -57,7 +57,7 @@ object "C_15" {
|
||||
object "C_15_deployed" {
|
||||
code {
|
||||
/// @src 0:59:147 "contract C {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
|
File diff suppressed because it is too large
Load Diff
@ -72,7 +72,7 @@ sub_0: assembly {
|
||||
object \"C_6\" {
|
||||
code {
|
||||
/// @src 0:60:101 \"contract C {...\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_6()
|
||||
@ -103,7 +103,7 @@ object \"C_6\" {
|
||||
object \"C_6_deployed\" {
|
||||
code {
|
||||
/// @src 0:60:101 \"contract C {...\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
@ -187,11 +187,12 @@ object \"C_6\" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:60:101 \"contract C {...\"
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize(\"C_6_deployed\")
|
||||
codecopy(128, dataoffset(\"C_6_deployed\"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize(\"C_6_deployed\")
|
||||
codecopy(_1, dataoffset(\"C_6_deployed\"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:\"C\"
|
||||
@ -199,15 +200,16 @@ object \"C_6\" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:60:101 \"contract C {...\"
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_1)))
|
||||
let _2 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_2)))
|
||||
{
|
||||
if callvalue() { revert(_1, _1) }
|
||||
if slt(add(calldatasize(), not(3)), _1) { revert(_1, _1) }
|
||||
return(128, _1)
|
||||
if callvalue() { revert(_2, _2) }
|
||||
if slt(add(calldatasize(), not(3)), _2) { revert(_2, _2) }
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
revert(0, 0)
|
||||
|
@ -72,7 +72,7 @@ sub_0: assembly {
|
||||
object \"C_6\" {
|
||||
code {
|
||||
/// @src 0:60:101
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_6()
|
||||
@ -103,7 +103,7 @@ object \"C_6\" {
|
||||
object \"C_6_deployed\" {
|
||||
code {
|
||||
/// @src 0:60:101
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
@ -186,11 +186,12 @@ object \"C_6\" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:60:101
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize(\"C_6_deployed\")
|
||||
codecopy(128, dataoffset(\"C_6_deployed\"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize(\"C_6_deployed\")
|
||||
codecopy(_1, dataoffset(\"C_6_deployed\"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:\"C\"
|
||||
@ -198,15 +199,16 @@ object \"C_6\" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:60:101
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_1)))
|
||||
let _2 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_2)))
|
||||
{
|
||||
if callvalue() { revert(_1, _1) }
|
||||
if slt(add(calldatasize(), not(3)), _1) { revert(_1, _1) }
|
||||
return(128, _1)
|
||||
if callvalue() { revert(_2, _2) }
|
||||
if slt(add(calldatasize(), not(3)), _2) { revert(_2, _2) }
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
revert(0, 0)
|
||||
|
@ -69,7 +69,7 @@ sub_0: assembly {
|
||||
object \"C_6\" {
|
||||
code {
|
||||
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_6()
|
||||
@ -96,7 +96,7 @@ object \"C_6\" {
|
||||
object \"C_6_deployed\" {
|
||||
code {
|
||||
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
@ -176,26 +176,28 @@ object \"C_6\" {
|
||||
object \"C_6\" {
|
||||
code {
|
||||
{
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize(\"C_6_deployed\")
|
||||
codecopy(128, dataoffset(\"C_6_deployed\"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize(\"C_6_deployed\")
|
||||
codecopy(_1, dataoffset(\"C_6_deployed\"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:\"C\"
|
||||
object \"C_6_deployed\" {
|
||||
code {
|
||||
{
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_1)))
|
||||
let _2 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_2)))
|
||||
{
|
||||
if callvalue() { revert(_1, _1) }
|
||||
if slt(add(calldatasize(), not(3)), _1) { revert(_1, _1) }
|
||||
return(128, _1)
|
||||
if callvalue() { revert(_2, _2) }
|
||||
if slt(add(calldatasize(), not(3)), _2) { revert(_2, _2) }
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
revert(0, 0)
|
||||
|
@ -10,7 +10,7 @@
|
||||
object \"C_54\" {
|
||||
code {
|
||||
/// @src 0:79:435 \"contract C...\"
|
||||
mstore(64, 160)
|
||||
mstore(64, memoryguard(160))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
let _1 := copy_arguments_for_constructor_20_object_C_54()
|
||||
@ -161,7 +161,7 @@ object \"C_54\" {
|
||||
object \"C_54_deployed\" {
|
||||
code {
|
||||
/// @src 0:79:435 \"contract C...\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
@ -592,30 +592,31 @@ object \"C_54\" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:79:435 \"contract C...\"
|
||||
mstore(64, 160)
|
||||
let _1 := memoryguard(0xa0)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let programSize := datasize(\"C_54\")
|
||||
let argSize := sub(codesize(), programSize)
|
||||
let newFreePtr := add(160, and(add(argSize, 31), not(31)))
|
||||
if or(gt(newFreePtr, sub(shl(64, 1), 1)), lt(newFreePtr, 160))
|
||||
let newFreePtr := add(_1, and(add(argSize, 31), not(31)))
|
||||
if or(gt(newFreePtr, sub(shl(64, 1), 1)), lt(newFreePtr, _1))
|
||||
{
|
||||
mstore(/** @src -1:-1:-1 */ 0, /** @src 0:79:435 \"contract C...\" */ shl(224, 0x4e487b71))
|
||||
mstore(4, 0x41)
|
||||
revert(/** @src -1:-1:-1 */ 0, /** @src 0:79:435 \"contract C...\" */ 0x24)
|
||||
}
|
||||
mstore(64, newFreePtr)
|
||||
codecopy(160, programSize, argSize)
|
||||
if slt(argSize, 32)
|
||||
codecopy(_1, programSize, argSize)
|
||||
if slt(sub(add(_1, argSize), _1), 32)
|
||||
{
|
||||
revert(/** @src -1:-1:-1 */ 0, 0)
|
||||
}
|
||||
/// @src 0:79:435 \"contract C...\"
|
||||
constructor_C(mload(160))
|
||||
let _1 := mload(64)
|
||||
let _2 := datasize(\"C_54_deployed\")
|
||||
codecopy(_1, dataoffset(\"C_54_deployed\"), _2)
|
||||
setimmutable(_1, \"8\", mload(128))
|
||||
return(_1, _2)
|
||||
constructor_C(mload(_1))
|
||||
let _2 := mload(64)
|
||||
let _3 := datasize(\"C_54_deployed\")
|
||||
codecopy(_2, dataoffset(\"C_54_deployed\"), _3)
|
||||
setimmutable(_2, \"8\", mload(128))
|
||||
return(_2, _3)
|
||||
}
|
||||
/// @ast-id 20 @src 0:182:230 \"constructor(int _init)...\"
|
||||
function constructor_C(var_init)
|
||||
@ -631,7 +632,7 @@ object \"C_54\" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:79:435 \"contract C...\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
@ -774,7 +775,7 @@ object \"C_54\" {
|
||||
object \"D_72\" {
|
||||
code {
|
||||
/// @src 1:91:166 \"contract D is C(3)...\"
|
||||
mstore(64, 160)
|
||||
mstore(64, memoryguard(160))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
let _1 := copy_arguments_for_constructor_71_object_D_72()
|
||||
@ -993,7 +994,7 @@ object \"D_72\" {
|
||||
object \"D_72_deployed\" {
|
||||
code {
|
||||
/// @src 1:91:166 \"contract D is C(3)...\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
@ -1424,30 +1425,31 @@ object \"D_72\" {
|
||||
code {
|
||||
{
|
||||
/// @src 1:91:166 \"contract D is C(3)...\"
|
||||
mstore(64, 160)
|
||||
let _1 := memoryguard(0xa0)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let programSize := datasize(\"D_72\")
|
||||
let argSize := sub(codesize(), programSize)
|
||||
let newFreePtr := add(160, and(add(argSize, 31), not(31)))
|
||||
if or(gt(newFreePtr, sub(shl(64, 1), 1)), lt(newFreePtr, 160))
|
||||
let newFreePtr := add(_1, and(add(argSize, 31), not(31)))
|
||||
if or(gt(newFreePtr, sub(shl(64, 1), 1)), lt(newFreePtr, _1))
|
||||
{
|
||||
mstore(/** @src -1:-1:-1 */ 0, /** @src 1:91:166 \"contract D is C(3)...\" */ shl(224, 0x4e487b71))
|
||||
mstore(4, 0x41)
|
||||
revert(/** @src -1:-1:-1 */ 0, /** @src 1:91:166 \"contract D is C(3)...\" */ 0x24)
|
||||
}
|
||||
mstore(64, newFreePtr)
|
||||
codecopy(160, programSize, argSize)
|
||||
if slt(argSize, 32)
|
||||
codecopy(_1, programSize, argSize)
|
||||
if slt(sub(add(_1, argSize), _1), 32)
|
||||
{
|
||||
revert(/** @src -1:-1:-1 */ 0, 0)
|
||||
}
|
||||
/// @src 1:91:166 \"contract D is C(3)...\"
|
||||
constructor_D(mload(160))
|
||||
let _1 := mload(64)
|
||||
let _2 := datasize(\"D_72_deployed\")
|
||||
codecopy(_1, dataoffset(\"D_72_deployed\"), _2)
|
||||
setimmutable(_1, \"8\", mload(128))
|
||||
return(_1, _2)
|
||||
constructor_D(mload(_1))
|
||||
let _2 := mload(64)
|
||||
let _3 := datasize(\"D_72_deployed\")
|
||||
codecopy(_2, dataoffset(\"D_72_deployed\"), _3)
|
||||
setimmutable(_2, \"8\", mload(128))
|
||||
return(_2, _3)
|
||||
}
|
||||
/// @ast-id 71 @src 1:113:164 \"constructor(int _init2)...\"
|
||||
function constructor_D(var_init2)
|
||||
@ -1471,7 +1473,7 @@ object \"D_72\" {
|
||||
code {
|
||||
{
|
||||
/// @src 1:91:166 \"contract D is C(3)...\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
|
@ -17,7 +17,7 @@
|
||||
(local $z3 i64)
|
||||
(local $_1 i64)
|
||||
(block $label_
|
||||
(local.set $p (call $u256_to_i32_726))
|
||||
(local.set $p (call $u256_to_i32_716))
|
||||
(local.set $r (i32.add (local.get $p) (i32.const 64)))
|
||||
(if (i32.lt_u (local.get $r) (local.get $p)) (then
|
||||
(unreachable)))
|
||||
@ -30,14 +30,14 @@
|
||||
(call $eth.getCallValue (i32.const 0))
|
||||
(local.set $z3 (i64.load (i32.const 8)))
|
||||
(if (i32.eqz (i64.eqz (i64.or (i64.or (i64.const 0) (i64.const 0)) (i64.or (local.get $z3) (i64.load (i32.const 0)))))) (then
|
||||
(call $eth.revert (call $to_internal_i32ptr) (call $u256_to_i32_344))))
|
||||
(call $eth.revert (call $to_internal_i32ptr_334) (call $u256_to_i32_333))))
|
||||
(local.set $_1 (datasize \"C_3_deployed\"))
|
||||
(call $eth.codeCopy (call $to_internal_i32ptr_348) (call $u256_to_i32 (dataoffset \"C_3_deployed\")) (call $u256_to_i32 (local.get $_1)))
|
||||
(call $eth.finish (call $to_internal_i32ptr_348) (call $u256_to_i32 (local.get $_1)))
|
||||
(call $eth.codeCopy (call $to_internal_i32ptr) (call $u256_to_i32 (dataoffset \"C_3_deployed\")) (call $u256_to_i32 (local.get $_1)))
|
||||
(call $eth.finish (call $to_internal_i32ptr) (call $u256_to_i32 (local.get $_1)))
|
||||
)
|
||||
)
|
||||
|
||||
(func $u256_to_i32_344
|
||||
(func $u256_to_i32_333
|
||||
(result i32)
|
||||
(local $v i32)
|
||||
(local $_1 i64)
|
||||
@ -68,7 +68,7 @@
|
||||
(local.get $v)
|
||||
)
|
||||
|
||||
(func $u256_to_i32_726
|
||||
(func $u256_to_i32_716
|
||||
(result i32)
|
||||
(local $v i32)
|
||||
(block $label__3
|
||||
@ -82,12 +82,12 @@
|
||||
(local.get $v)
|
||||
)
|
||||
|
||||
(func $to_internal_i32ptr
|
||||
(func $to_internal_i32ptr_334
|
||||
(result i32)
|
||||
(local $r i32)
|
||||
(local $p i32)
|
||||
(block $label__4
|
||||
(local.set $p (call $u256_to_i32_344))
|
||||
(local.set $p (call $u256_to_i32_333))
|
||||
(local.set $r (i32.add (local.get $p) (i32.const 64)))
|
||||
(if (i32.lt_u (local.get $r) (local.get $p)) (then
|
||||
(unreachable)))
|
||||
@ -96,7 +96,7 @@
|
||||
(local.get $r)
|
||||
)
|
||||
|
||||
(func $to_internal_i32ptr_348
|
||||
(func $to_internal_i32ptr
|
||||
(result i32)
|
||||
(local $r i32)
|
||||
(local $v i32)
|
||||
|
@ -9,7 +9,7 @@
|
||||
object \"C_7\" {
|
||||
code {
|
||||
/// @src 0:79:121 \"contract C { function f() public pure {} }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue()
|
||||
{
|
||||
revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb()
|
||||
@ -29,7 +29,7 @@ object \"C_7\" {
|
||||
object \"C_7_deployed\" {
|
||||
code {
|
||||
/// @src 0:79:121 \"contract C { function f() public pure {} }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let selector := shift_right_224_unsigned(calldataload(0))
|
||||
|
@ -10,7 +10,7 @@
|
||||
object \"C_7\" {
|
||||
code {
|
||||
/// @src 0:79:121 \"contract C { function f() public pure {} }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_7()
|
||||
@ -41,7 +41,7 @@ object \"C_7\" {
|
||||
object \"C_7_deployed\" {
|
||||
code {
|
||||
/// @src 0:79:121 \"contract C { function f() public pure {} }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
|
@ -10,7 +10,7 @@
|
||||
object \"C_3\" {
|
||||
code {
|
||||
/// @src 0:79:92 \"contract C {}\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_3()
|
||||
@ -41,7 +41,7 @@ object \"C_3\" {
|
||||
object \"C_3_deployed\" {
|
||||
code {
|
||||
/// @src 0:79:92 \"contract C {}\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
revert_error_42b3090547df1d2001c96683413b8cf91c1b902ef5e3cb8d9f6f304cf7446f74()
|
||||
|
||||
@ -79,7 +79,7 @@ object \"C_3\" {
|
||||
object \"D_16\" {
|
||||
code {
|
||||
/// @src 0:93:146 \"contract D { function f() public { C c = new C(); } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_D_16()
|
||||
@ -110,7 +110,7 @@ object \"D_16\" {
|
||||
object \"D_16_deployed\" {
|
||||
code {
|
||||
/// @src 0:93:146 \"contract D { function f() public { C c = new C(); } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
@ -212,7 +212,7 @@ object \"D_16\" {
|
||||
object \"C_3\" {
|
||||
code {
|
||||
/// @src 0:79:92 \"contract C {}\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_3()
|
||||
@ -243,7 +243,7 @@ object \"D_16\" {
|
||||
object \"C_3_deployed\" {
|
||||
code {
|
||||
/// @src 0:79:92 \"contract C {}\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
revert_error_42b3090547df1d2001c96683413b8cf91c1b902ef5e3cb8d9f6f304cf7446f74()
|
||||
|
||||
|
@ -1,10 +1,12 @@
|
||||
{"contracts":{"A":{"object":{"evm":{"assembly":" /* \"A\":17:18 */
|
||||
{"contracts":{"A":{"object":{"evm":{"assembly":" /* \"A\":38:39 */
|
||||
0x00
|
||||
/* \"A\":11:19 */
|
||||
dup1
|
||||
mload
|
||||
/* \"A\":20:40 */
|
||||
sstore
|
||||
/* \"A\":0:42 */
|
||||
stop
|
||||
","bytecode":{"functionDebugData":{},"generatedSources":[],"linkReferences":{},"object":"<BYTECODE REMOVED>","opcodes":"<OPCODES REMOVED>","sourceMap":"<SOURCEMAP REMOVED>"}},"ir":"object \"object\" {
|
||||
code {
|
||||
let x := mload(0)
|
||||
|
@ -1,10 +1,12 @@
|
||||
{"contracts":{"A":{"object":{"evm":{"assembly":" /* \"A\":17:18 */
|
||||
0x00
|
||||
dup1
|
||||
/* \"A\":11:19 */
|
||||
dup1
|
||||
mload
|
||||
/* \"A\":20:40 */
|
||||
sstore
|
||||
/* \"A\":0:42 */
|
||||
stop
|
||||
","bytecode":{"functionDebugData":{},"generatedSources":[],"linkReferences":{},"object":"<BYTECODE REMOVED>","opcodes":"<OPCODES REMOVED>","sourceMap":"<SOURCEMAP REMOVED>"}},"ir":"object \"object\" {
|
||||
code {
|
||||
let x := mload(0)
|
||||
|
@ -1,17 +1,15 @@
|
||||
{"contracts":{"A":{"object":{"evm":{"assembly":" /* \"A\":16:17 */
|
||||
0x01
|
||||
dup1
|
||||
/* \"A\":27:28 */
|
||||
0x00
|
||||
/* \"A\":20:32 */
|
||||
sstore
|
||||
pop
|
||||
/* \"A\":50:51 */
|
||||
0x02
|
||||
dup1
|
||||
/* \"A\":61:63 */
|
||||
0x20
|
||||
/* \"A\":54:67 */
|
||||
sstore
|
||||
pop
|
||||
/* \"A\":0:72 */
|
||||
stop
|
||||
"}}}},"errors":[{"component":"general","formattedMessage":"Yul is still experimental. Please use the output with care.","message":"Yul is still experimental. Please use the output with care.","severity":"warning","type":"Warning"}]}
|
||||
|
@ -25,7 +25,7 @@ object "C_6" {
|
||||
|
||||
|
||||
Binary representation:
|
||||
60806040523415600e57600080fd5b600e601c600039600e6000f3fe60806040523615600055600080fd
|
||||
608060405234601557600e601b600039600e6000f35b600080fdfe60806040523615600055600080fd
|
||||
|
||||
Text representation:
|
||||
/* "strict_asm_optimizer_steps/input.yul":45:48 */
|
||||
@ -37,17 +37,8 @@ Text representation:
|
||||
/* "strict_asm_optimizer_steps/input.yul":61:72 */
|
||||
callvalue
|
||||
/* "strict_asm_optimizer_steps/input.yul":58:89 */
|
||||
iszero
|
||||
tag_1
|
||||
jumpi
|
||||
/* "strict_asm_optimizer_steps/input.yul":85:86 */
|
||||
0x00
|
||||
/* "strict_asm_optimizer_steps/input.yul":82:83 */
|
||||
dup1
|
||||
/* "strict_asm_optimizer_steps/input.yul":75:87 */
|
||||
revert
|
||||
/* "strict_asm_optimizer_steps/input.yul":58:89 */
|
||||
tag_1:
|
||||
/* "strict_asm_optimizer_steps/input.yul":138:162 */
|
||||
dataSize(sub_0)
|
||||
/* "strict_asm_optimizer_steps/input.yul":110:136 */
|
||||
@ -62,6 +53,13 @@ tag_1:
|
||||
0x00
|
||||
/* "strict_asm_optimizer_steps/input.yul":172:207 */
|
||||
return
|
||||
/* "strict_asm_optimizer_steps/input.yul":73:89 */
|
||||
tag_1:
|
||||
/* "strict_asm_optimizer_steps/input.yul":85:86 */
|
||||
0x00
|
||||
/* "strict_asm_optimizer_steps/input.yul":75:87 */
|
||||
dup1
|
||||
revert
|
||||
stop
|
||||
|
||||
sub_0: assembly {
|
||||
@ -81,8 +79,7 @@ sub_0: assembly {
|
||||
sstore
|
||||
/* "strict_asm_optimizer_steps/input.yul":576:577 */
|
||||
0x00
|
||||
/* "strict_asm_optimizer_steps/input.yul":573:574 */
|
||||
dup1
|
||||
/* "strict_asm_optimizer_steps/input.yul":566:578 */
|
||||
dup1
|
||||
revert
|
||||
}
|
||||
|
@ -11,7 +11,7 @@ IR:
|
||||
object "test_11" {
|
||||
code {
|
||||
/// @src 0:79:169 "contract test {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_test_11()
|
||||
@ -42,7 +42,7 @@ object "test_11" {
|
||||
object "test_11_deployed" {
|
||||
code {
|
||||
/// @src 0:79:169 "contract test {..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
|
@ -17,11 +17,12 @@ object "C_3" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:95 "contract C {}"
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_3_deployed")
|
||||
codecopy(128, dataoffset("C_3_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_3_deployed")
|
||||
codecopy(_1, dataoffset("C_3_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"viair_subobjects/input.sol"
|
||||
@ -29,7 +30,7 @@ object "C_3" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:95 "contract C {}"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
revert(0, 0)
|
||||
}
|
||||
}
|
||||
@ -56,11 +57,12 @@ object "D_16" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:96:165 "contract D {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("D_16_deployed")
|
||||
codecopy(128, dataoffset("D_16_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("D_16_deployed")
|
||||
codecopy(_1, dataoffset("D_16_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"viair_subobjects/input.sol"
|
||||
@ -68,35 +70,35 @@ object "D_16" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:96:165 "contract D {..."
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let _1 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_1)))
|
||||
let _2 := 0
|
||||
if eq(0x26121ff0, shr(224, calldataload(_2)))
|
||||
{
|
||||
if callvalue() { revert(_1, _1) }
|
||||
if slt(add(calldatasize(), not(3)), _1) { revert(_1, _1) }
|
||||
/// @src 0:149:156 "new C()"
|
||||
let _2 := datasize("C_3")
|
||||
let _3 := add(/** @src 0:96:165 "contract D {..." */ 128, /** @src 0:149:156 "new C()" */ _2)
|
||||
if or(gt(_3, 0xffffffffffffffff), lt(_3, /** @src 0:96:165 "contract D {..." */ 128))
|
||||
if callvalue() { revert(_2, _2) }
|
||||
if slt(add(calldatasize(), not(3)), _2) { revert(_2, _2) }
|
||||
/// @src 0:149:156 "new C()"
|
||||
let _3 := datasize("C_3")
|
||||
let _4 := add(_1, _3)
|
||||
if or(gt(_4, 0xffffffffffffffff), lt(_4, _1))
|
||||
{
|
||||
/// @src 0:96:165 "contract D {..."
|
||||
mstore(_1, shl(224, 0x4e487b71))
|
||||
mstore(_2, shl(224, 0x4e487b71))
|
||||
mstore(4, 0x41)
|
||||
revert(_1, 0x24)
|
||||
revert(_2, 0x24)
|
||||
}
|
||||
/// @src 0:149:156 "new C()"
|
||||
datacopy(/** @src 0:96:165 "contract D {..." */ 128, /** @src 0:149:156 "new C()" */ dataoffset("C_3"), _2)
|
||||
if iszero(create(/** @src 0:96:165 "contract D {..." */ _1, 128, /** @src 0:149:156 "new C()" */ _2))
|
||||
datacopy(_1, dataoffset("C_3"), _3)
|
||||
if iszero(create(/** @src 0:96:165 "contract D {..." */ _2, /** @src 0:149:156 "new C()" */ _1, sub(_4, _1)))
|
||||
{
|
||||
/// @src 0:96:165 "contract D {..."
|
||||
let pos := mload(64)
|
||||
returndatacopy(pos, _1, returndatasize())
|
||||
returndatacopy(pos, _2, returndatasize())
|
||||
revert(pos, returndatasize())
|
||||
}
|
||||
return(mload(64), _1)
|
||||
return(mload(64), _2)
|
||||
}
|
||||
}
|
||||
revert(0, 0)
|
||||
@ -107,11 +109,12 @@ object "D_16" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:95 "contract C {}"
|
||||
mstore(64, 128)
|
||||
let _1 := memoryguard(0x80)
|
||||
mstore(64, _1)
|
||||
if callvalue() { revert(0, 0) }
|
||||
let _1 := datasize("C_3_deployed")
|
||||
codecopy(128, dataoffset("C_3_deployed"), _1)
|
||||
return(128, _1)
|
||||
let _2 := datasize("C_3_deployed")
|
||||
codecopy(_1, dataoffset("C_3_deployed"), _2)
|
||||
return(_1, _2)
|
||||
}
|
||||
}
|
||||
/// @use-src 0:"viair_subobjects/input.sol"
|
||||
@ -119,7 +122,7 @@ object "D_16" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:82:95 "contract C {}"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
revert(0, 0)
|
||||
}
|
||||
}
|
||||
|
@ -21,20 +21,18 @@ object "RunsTest1" {
|
||||
|
||||
|
||||
Binary representation:
|
||||
602480600d600039806000f3fe7fabc1234500000000000000000000000000000000000000000000000000000000600055
|
||||
602580600c6000396000f3fe7fabc123450000000000000000000000000000000000000000000000000000000060005500
|
||||
|
||||
Text representation:
|
||||
/* "yul_optimize_runs/input.yul":106:125 */
|
||||
dataSize(sub_0)
|
||||
dup1
|
||||
/* "yul_optimize_runs/input.yul":83:104 */
|
||||
dup1
|
||||
dataOffset(sub_0)
|
||||
/* "yul_optimize_runs/input.yul":80:81 */
|
||||
0x00
|
||||
/* "yul_optimize_runs/input.yul":71:126 */
|
||||
codecopy
|
||||
/* "yul_optimize_runs/input.yul":145:164 */
|
||||
dup1
|
||||
/* "yul_optimize_runs/input.yul":80:81 */
|
||||
0x00
|
||||
/* "yul_optimize_runs/input.yul":135:165 */
|
||||
@ -48,4 +46,6 @@ sub_0: assembly {
|
||||
0x00
|
||||
/* "yul_optimize_runs/input.yul":270:288 */
|
||||
sstore
|
||||
/* "yul_optimize_runs/input.yul":208:298 */
|
||||
stop
|
||||
}
|
||||
|
@ -11,7 +11,7 @@ object "C_7" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:80:112 "contract C..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
if callvalue()
|
||||
{
|
||||
revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb()
|
||||
@ -30,7 +30,7 @@ object "C_7" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:80:112 "contract C..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
revert_error_42b3090547df1d2001c96683413b8cf91c1b902ef5e3cb8d9f6f304cf7446f74()
|
||||
}
|
||||
function revert_error_42b3090547df1d2001c96683413b8cf91c1b902ef5e3cb8d9f6f304cf7446f74()
|
||||
|
@ -11,7 +11,7 @@ object "C_6" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:60:103 "contract C..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
if callvalue()
|
||||
{
|
||||
revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb()
|
||||
@ -121,7 +121,7 @@ object "C_6" {
|
||||
code {
|
||||
{
|
||||
/// @src 0:60:103 "contract C..."
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(0x80))
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
let selector := shift_right_unsigned(calldataload(0))
|
||||
|
@ -10,7 +10,7 @@
|
||||
object \"C_11\" {
|
||||
code {
|
||||
/// @src 0:78:164 \"contract C { function f() external pure returns (string memory) { return \\\"abcabc\\\"; } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_11()
|
||||
@ -41,7 +41,7 @@ object \"C_11\" {
|
||||
object \"C_11_deployed\" {
|
||||
code {
|
||||
/// @src 0:78:164 \"contract C { function f() external pure returns (string memory) { return \\\"abcabc\\\"; } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
|
@ -10,7 +10,7 @@
|
||||
object \"C_11\" {
|
||||
code {
|
||||
/// @src 0:78:158 \"contract C { function f() external pure returns (bytes32) { return \\\"abcabc\\\"; } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_11()
|
||||
@ -41,7 +41,7 @@ object \"C_11\" {
|
||||
object \"C_11_deployed\" {
|
||||
code {
|
||||
/// @src 0:78:158 \"contract C { function f() external pure returns (bytes32) { return \\\"abcabc\\\"; } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
|
@ -10,7 +10,7 @@
|
||||
object \"C_11\" {
|
||||
code {
|
||||
/// @src 0:78:159 \"contract C { function f() external pure returns (bytes4) { return 0x61626364; } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_11()
|
||||
@ -41,7 +41,7 @@ object \"C_11\" {
|
||||
object \"C_11_deployed\" {
|
||||
code {
|
||||
/// @src 0:78:159 \"contract C { function f() external pure returns (bytes4) { return 0x61626364; } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
|
@ -10,7 +10,7 @@
|
||||
object \"C_11\" {
|
||||
code {
|
||||
/// @src 0:78:243 \"contract C { function f() external pure returns (string memory) { return \\\"abcdabcdcafecafeabcdabcdcafecafeffffzzzzoooo0123456789,.<,>.?:;'[{]}|`~!@#$%^&*()-_=+\\\"; } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_11()
|
||||
@ -41,7 +41,7 @@ object \"C_11\" {
|
||||
object \"C_11_deployed\" {
|
||||
code {
|
||||
/// @src 0:78:243 \"contract C { function f() external pure returns (string memory) { return \\\"abcdabcdcafecafeabcdabcdcafecafeffffzzzzoooo0123456789,.<,>.?:;'[{]}|`~!@#$%^&*()-_=+\\\"; } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
|
@ -10,7 +10,7 @@
|
||||
object \"C_11\" {
|
||||
code {
|
||||
/// @src 0:78:159 \"contract C { function f() external pure returns (bytes4) { return 0xaabbccdd; } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
if callvalue() { revert_error_ca66f745a3ce8ff40e2ccaf1ad45db7774001b90d25810abd9040049be7bf4bb() }
|
||||
|
||||
constructor_C_11()
|
||||
@ -41,7 +41,7 @@ object \"C_11\" {
|
||||
object \"C_11_deployed\" {
|
||||
code {
|
||||
/// @src 0:78:159 \"contract C { function f() external pure returns (bytes4) { return 0xaabbccdd; } }\"
|
||||
mstore(64, 128)
|
||||
mstore(64, memoryguard(128))
|
||||
|
||||
if iszero(lt(calldatasize(), 4))
|
||||
{
|
||||
|
@ -14,7 +14,7 @@ object "object" {
|
||||
|
||||
|
||||
Binary representation:
|
||||
612000515061616002600055
|
||||
61200051506161600260005500
|
||||
|
||||
Text representation:
|
||||
/* "yul_verbatim_msize/input.yul":125:131 */
|
||||
@ -30,3 +30,5 @@ Text representation:
|
||||
0x00
|
||||
/* "yul_verbatim_msize/input.yul":162:174 */
|
||||
sstore
|
||||
/* "yul_verbatim_msize/input.yul":0:176 */
|
||||
stop
|
||||
|
@ -24,6 +24,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 0x20, 0x8, 0x40, 0x3, 0x9, 0xa, 0xb
|
||||
// gas irOptimized: 203522
|
||||
// gas irOptimized: 203312
|
||||
// gas legacy: 206084
|
||||
// gas legacyOptimized: 203068
|
||||
|
@ -60,10 +60,10 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test_bytes() ->
|
||||
// gas irOptimized: 394829
|
||||
// gas irOptimized: 377545
|
||||
// gas legacy: 423563
|
||||
// gas legacyOptimized: 331391
|
||||
// test_uint256() ->
|
||||
// gas irOptimized: 553331
|
||||
// gas irOptimized: 528726
|
||||
// gas legacy: 591392
|
||||
// gas legacyOptimized: 456137
|
||||
|
@ -26,6 +26,6 @@ contract C {
|
||||
// ----
|
||||
// library: L
|
||||
// f() -> 8, 7, 1, 2, 7, 12
|
||||
// gas irOptimized: 167615
|
||||
// gas irOptimized: 167580
|
||||
// gas legacy: 169475
|
||||
// gas legacyOptimized: 167397
|
||||
|
@ -61,10 +61,10 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test_bytes() ->
|
||||
// gas irOptimized: 394829
|
||||
// gas irOptimized: 377545
|
||||
// gas legacy: 423563
|
||||
// gas legacyOptimized: 331391
|
||||
// test_uint256() ->
|
||||
// gas irOptimized: 553331
|
||||
// gas irOptimized: 528726
|
||||
// gas legacy: 591392
|
||||
// gas legacyOptimized: 456137
|
||||
|
@ -53,6 +53,6 @@ contract C {
|
||||
// f2() -> 0x20, 0xa0, 0x1, 0x60, 0x2, 0x3, "abc"
|
||||
// f3() -> 0x20, 0xa0, 0x1, 0x60, 0x2, 0x3, "abc"
|
||||
// f4() -> 0x20, 0x160, 0x1, 0x80, 0xc0, 0x2, 0x3, "abc", 0x7, 0x40, 0x2, 0x2, 0x3
|
||||
// gas irOptimized: 113296
|
||||
// gas irOptimized: 113361
|
||||
// gas legacy: 114900
|
||||
// gas legacyOptimized: 112606
|
||||
|
@ -32,6 +32,6 @@ contract C is B {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 77
|
||||
// gas irOptimized: 121699
|
||||
// gas irOptimized: 120044
|
||||
// gas legacy: 155221
|
||||
// gas legacyOptimized: 111678
|
||||
|
@ -40,5 +40,5 @@ contract C is B {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 5, 10
|
||||
// gas irOptimized: 88225
|
||||
// gas irOptimized: 87578
|
||||
// gas legacy: 99137
|
||||
|
@ -21,6 +21,6 @@ contract C {
|
||||
// f(uint256[][1]): 32, 32, 0 -> true
|
||||
// f(uint256[][1]): 32, 32, 1, 42 -> true
|
||||
// f(uint256[][1]): 32, 32, 8, 421, 422, 423, 424, 425, 426, 427, 428 -> true
|
||||
// gas irOptimized: 177581
|
||||
// gas irOptimized: 172204
|
||||
// gas legacy: 141900
|
||||
// gas legacyOptimized: 121788
|
||||
|
@ -19,10 +19,10 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// h(uint256[2][]): 0x20, 3, 123, 124, 223, 224, 323, 324 -> 32, 256, 0x20, 3, 123, 124, 223, 224, 323, 324
|
||||
// gas irOptimized: 181123
|
||||
// gas irOptimized: 180925
|
||||
// gas legacy: 184929
|
||||
// gas legacyOptimized: 181504
|
||||
// i(uint256[2][2]): 123, 124, 223, 224 -> 32, 128, 123, 124, 223, 224
|
||||
// gas irOptimized: 112627
|
||||
// gas irOptimized: 112535
|
||||
// gas legacy: 115468
|
||||
// gas legacyOptimized: 112988
|
||||
|
@ -11,6 +11,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f(bytes): 0x20, 0x80, 0x21, 0x40, 0x7, "abcdefg" -> 0x21, 0x40, 0x7, "abcdefg"
|
||||
// gas irOptimized: 135996
|
||||
// gas irOptimized: 135918
|
||||
// gas legacy: 137190
|
||||
// gas legacyOptimized: 136082
|
||||
|
@ -14,7 +14,7 @@ contract Test {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// set(uint24[3][]): 0x20, 0x06, 0x01, 0x02, 0x03, 0x04, 0x05, 0x06, 0x07, 0x08, 0x09, 0x0a, 0x0b, 0x0c, 0x0d, 0x0e, 0x0f, 0x10, 0x11, 0x12 -> 0x06
|
||||
// gas irOptimized: 189239
|
||||
// gas irOptimized: 189910
|
||||
// gas legacy: 211149
|
||||
// gas legacyOptimized: 206054
|
||||
// data(uint256,uint256): 0x02, 0x02 -> 0x09
|
||||
|
@ -47,7 +47,7 @@ contract c {
|
||||
// gas legacyOptimized: 58606
|
||||
// storageEmpty -> 0
|
||||
// test_long() -> 67
|
||||
// gas irOptimized: 90759
|
||||
// gas irOptimized: 89148
|
||||
// gas legacy: 103590
|
||||
// gas legacyOptimized: 101044
|
||||
// storageEmpty -> 0
|
||||
|
@ -19,6 +19,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 0
|
||||
// gas irOptimized: 165224
|
||||
// gas irOptimized: 158143
|
||||
// gas legacy: 189715
|
||||
// gas legacyOptimized: 184472
|
||||
|
@ -15,7 +15,7 @@ contract c {
|
||||
// ----
|
||||
// getLength() -> 0
|
||||
// set(): 1, 2 -> true
|
||||
// gas irOptimized: 110439
|
||||
// gas irOptimized: 110433
|
||||
// gas legacy: 110726
|
||||
// gas legacyOptimized: 110567
|
||||
// getLength() -> 68
|
||||
|
@ -22,7 +22,7 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// store(uint256[9],uint8[3][]): 21, 22, 23, 24, 25, 26, 27, 28, 29, 0x140, 4, 1, 2, 3, 11, 12, 13, 21, 22, 23, 31, 32, 33 -> 32
|
||||
// gas irOptimized: 650971
|
||||
// gas irOptimized: 650669
|
||||
// gas legacy: 694515
|
||||
// gas legacyOptimized: 694013
|
||||
// retrieve() -> 9, 28, 9, 28, 4, 3, 32
|
||||
|
@ -23,6 +23,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> true
|
||||
// gas irOptimized: 92843
|
||||
// gas irOptimized: 92740
|
||||
// gas legacy: 93035
|
||||
// gas legacyOptimized: 92257
|
||||
|
@ -48,6 +48,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> true
|
||||
// gas irOptimized: 153927
|
||||
// gas irOptimized: 153260
|
||||
// gas legacy: 155961
|
||||
// gas legacyOptimized: 153588
|
||||
|
@ -15,6 +15,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 0
|
||||
// gas irOptimized: 135145
|
||||
// gas irOptimized: 135098
|
||||
// gas legacy: 135313
|
||||
// gas legacyOptimized: 134548
|
||||
|
@ -42,11 +42,11 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 0
|
||||
// gas irOptimized: 92855
|
||||
// gas irOptimized: 92800
|
||||
// gas legacy: 93006
|
||||
// gas legacyOptimized: 92261
|
||||
// g() -> 0
|
||||
// h() -> 0
|
||||
// gas irOptimized: 92922
|
||||
// gas irOptimized: 92862
|
||||
// gas legacy: 93028
|
||||
// gas legacyOptimized: 92303
|
||||
|
@ -21,6 +21,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 0x01000000000000000000000000000000000000000000000000, 0x02000000000000000000000000000000000000000000000000, 0x03000000000000000000000000000000000000000000000000, 0x04000000000000000000000000000000000000000000000000, 0x05000000000000000000000000000000000000000000000000
|
||||
// gas irOptimized: 212669
|
||||
// gas irOptimized: 212571
|
||||
// gas legacy: 221883
|
||||
// gas legacyOptimized: 220734
|
||||
|
@ -37,12 +37,12 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 0x02000202
|
||||
// gas irOptimized: 4660920
|
||||
// gas irOptimized: 4652092
|
||||
// gas legacy: 4578341
|
||||
// gas legacyOptimized: 4548354
|
||||
// storageEmpty -> 1
|
||||
// clear() -> 0, 0
|
||||
// gas irOptimized: 4491908
|
||||
// gas irOptimized: 4483169
|
||||
// gas legacy: 4410769
|
||||
// gas legacyOptimized: 4382531
|
||||
// storageEmpty -> 1
|
||||
|
@ -15,6 +15,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test(uint256[2][]): 32, 3, 7, 8, 9, 10, 11, 12 -> 10
|
||||
// gas irOptimized: 690506
|
||||
// gas irOptimized: 690205
|
||||
// gas legacy: 686268
|
||||
// gas legacyOptimized: 685688
|
||||
|
@ -19,6 +19,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 5, 4
|
||||
// gas irOptimized: 226130
|
||||
// gas irOptimized: 225956
|
||||
// gas legacy: 233801
|
||||
// gas legacyOptimized: 232816
|
||||
|
@ -24,6 +24,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 3, 4
|
||||
// gas irOptimized: 190944
|
||||
// gas irOptimized: 190480
|
||||
// gas legacy: 195353
|
||||
// gas legacyOptimized: 192441
|
||||
|
@ -17,7 +17,7 @@ contract c {
|
||||
// ----
|
||||
// setData1(uint256,uint256,uint256): 10, 5, 4 ->
|
||||
// copyStorageStorage() ->
|
||||
// gas irOptimized: 111488
|
||||
// gas irOptimized: 111426
|
||||
// gas legacy: 109278
|
||||
// gas legacyOptimized: 109268
|
||||
// getData2(uint256): 5 -> 10, 4
|
||||
|
@ -20,6 +20,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 5, 4
|
||||
// gas irOptimized: 272806
|
||||
// gas irOptimized: 272736
|
||||
// gas legacy: 270834
|
||||
// gas legacyOptimized: 269960
|
||||
|
@ -14,6 +14,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 9, 4
|
||||
// gas irOptimized: 123172
|
||||
// gas irOptimized: 123162
|
||||
// gas legacy: 123579
|
||||
// gas legacyOptimized: 123208
|
||||
|
@ -18,6 +18,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 8, 0
|
||||
// gas irOptimized: 236016
|
||||
// gas irOptimized: 236090
|
||||
// gas legacy: 234695
|
||||
// gas legacyOptimized: 234103
|
||||
|
@ -19,7 +19,7 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 4, 5
|
||||
// gas irOptimized: 239134
|
||||
// gas irOptimized: 238826
|
||||
// gas legacy: 238736
|
||||
// gas legacyOptimized: 237159
|
||||
// storageEmpty -> 1
|
||||
|
@ -17,6 +17,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 0x20, 2, 0x40, 0xa0, 2, 0, 1, 2, 2, 3
|
||||
// gas irOptimized: 161746
|
||||
// gas irOptimized: 161780
|
||||
// gas legacy: 162278
|
||||
// gas legacyOptimized: 159955
|
||||
|
@ -20,6 +20,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 0xffffffff, 0x0000000000000000000000000a00090008000700060005000400030002000100, 0x0000000000000000000000000000000000000000000000000000000000000000
|
||||
// gas irOptimized: 132180
|
||||
// gas irOptimized: 129167
|
||||
// gas legacy: 186406
|
||||
// gas legacyOptimized: 166126
|
||||
|
@ -22,6 +22,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 0x04000000000000000000000000000000000000000000000000, 0x0, 0x0
|
||||
// gas irOptimized: 93855
|
||||
// gas irOptimized: 93858
|
||||
// gas legacy: 97451
|
||||
// gas legacyOptimized: 94200
|
||||
|
@ -22,6 +22,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 0x01000000000000000000000000000000000000000000000000, 0x02000000000000000000000000000000000000000000000000, 0x03000000000000000000000000000000000000000000000000, 0x04000000000000000000000000000000000000000000000000, 0x0
|
||||
// gas irOptimized: 294958
|
||||
// gas irOptimized: 294772
|
||||
// gas legacy: 303653
|
||||
// gas legacyOptimized: 301999
|
||||
|
@ -22,6 +22,6 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 0x01000000000000000000000000000000000000000000000000, 0x02000000000000000000000000000000000000000000000000, 0x03000000000000000000000000000000000000000000000000, 0x04000000000000000000000000000000000000000000000000, 0x00
|
||||
// gas irOptimized: 274022
|
||||
// gas irOptimized: 273963
|
||||
// gas legacy: 276381
|
||||
// gas legacyOptimized: 275453
|
||||
|
@ -38,10 +38,10 @@ contract c {
|
||||
// compileViaYul: true
|
||||
// ----
|
||||
// test1(uint256[][]): 0x20, 2, 0x40, 0x40, 2, 23, 42 -> 2, 65
|
||||
// gas irOptimized: 181755
|
||||
// gas irOptimized: 181308
|
||||
// test2(uint256[][2]): 0x20, 0x40, 0x40, 2, 23, 42 -> 2, 65
|
||||
// gas irOptimized: 158111
|
||||
// gas irOptimized: 157901
|
||||
// test3(uint256[2][]): 0x20, 2, 23, 42, 23, 42 -> 2, 65
|
||||
// gas irOptimized: 135282
|
||||
// gas irOptimized: 135108
|
||||
// test4(uint256[2][2]): 23, 42, 23, 42 -> 65
|
||||
// gas irOptimized: 111460
|
||||
// gas irOptimized: 111428
|
||||
|
@ -40,12 +40,12 @@ contract Test {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 24
|
||||
// gas irOptimized: 227254
|
||||
// gas irOptimized: 227167
|
||||
// gas legacy: 227133
|
||||
// gas legacyOptimized: 226547
|
||||
// test1() -> 3
|
||||
// test2() -> 6
|
||||
// test3() -> 24
|
||||
// gas irOptimized: 133753
|
||||
// gas irOptimized: 133621
|
||||
// gas legacy: 134295
|
||||
// gas legacyOptimized: 133383
|
||||
|
@ -17,4 +17,4 @@ contract C {
|
||||
// compileViaYul: true
|
||||
// ----
|
||||
// f((uint128,uint64,uint128)[]): 0x20, 3, 0, 0, 12, 0, 11, 0, 10, 0, 0 -> 10, 11, 12
|
||||
// gas irOptimized: 121194
|
||||
// gas irOptimized: 121048
|
||||
|
@ -19,4 +19,4 @@ contract C {
|
||||
// compileViaYul: true
|
||||
// ----
|
||||
// f() -> 10, 11, 12
|
||||
// gas irOptimized: 119201
|
||||
// gas irOptimized: 119149
|
||||
|
@ -23,4 +23,4 @@ contract C {
|
||||
// compileViaYul: true
|
||||
// ----
|
||||
// f((uint256[])[]): 0x20, 3, 0x60, 0x60, 0x60, 0x20, 3, 1, 2, 3 -> 3, 1
|
||||
// gas irOptimized: 330385
|
||||
// gas irOptimized: 328592
|
||||
|
@ -26,4 +26,4 @@ contract C {
|
||||
// compileViaYul: true
|
||||
// ----
|
||||
// f() -> 3, 3, 3, 1
|
||||
// gas irOptimized: 183411
|
||||
// gas irOptimized: 183316
|
||||
|
@ -15,6 +15,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 1, 2, 3
|
||||
// gas irOptimized: 132580
|
||||
// gas irOptimized: 132298
|
||||
// gas legacy: 134619
|
||||
// gas legacyOptimized: 131940
|
||||
|
@ -12,7 +12,7 @@ contract Test {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// set(uint24[]): 0x20, 18, 1, 2, 3, 4, 5, 6, 7, 8, 9, 10, 11, 12, 13, 14, 15, 16, 17, 18 -> 18
|
||||
// gas irOptimized: 99873
|
||||
// gas irOptimized: 99616
|
||||
// gas legacy: 103563
|
||||
// gas legacyOptimized: 101397
|
||||
// data(uint256): 7 -> 8
|
||||
|
@ -7,11 +7,11 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// set(uint256): 1, 2 -> true
|
||||
// gas irOptimized: 110678
|
||||
// gas irOptimized: 110699
|
||||
// gas legacy: 111091
|
||||
// gas legacyOptimized: 110736
|
||||
// set(uint256): 2, 2, 3, 4, 5 -> true
|
||||
// gas irOptimized: 177635
|
||||
// gas irOptimized: 177659
|
||||
// gas legacy: 178021
|
||||
// gas legacyOptimized: 177666
|
||||
// storageEmpty -> 0
|
||||
|
@ -19,25 +19,25 @@ contract c {
|
||||
// ----
|
||||
// f(uint256): 0 -> 0x20, 0x00
|
||||
// f(uint256): 31 -> 0x20, 0x1f, 0x0102030405060708090a0b0c0d0e0f101112131415161718191a1b1c1d1e00
|
||||
// gas irOptimized: 125470
|
||||
// gas irOptimized: 121741
|
||||
// gas legacy: 124364
|
||||
// gas legacyOptimized: 119898
|
||||
// f(uint256): 32 -> 0x20, 0x20, 1780731860627700044960722568376592200742329637303199754547598369979440671
|
||||
// gas irOptimized: 134121
|
||||
// gas irOptimized: 130733
|
||||
// gas legacy: 135431
|
||||
// gas legacyOptimized: 130829
|
||||
// f(uint256): 33 -> 0x20, 33, 1780731860627700044960722568376592200742329637303199754547598369979440671, 0x2000000000000000000000000000000000000000000000000000000000000000
|
||||
// gas irOptimized: 141217
|
||||
// gas irOptimized: 137732
|
||||
// gas legacy: 142238
|
||||
// gas legacyOptimized: 137518
|
||||
// f(uint256): 63 -> 0x20, 0x3f, 1780731860627700044960722568376592200742329637303199754547598369979440671, 14532552714582660066924456880521368950258152170031413196862950297402215316992
|
||||
// gas irOptimized: 158957
|
||||
// gas irOptimized: 152352
|
||||
// gas legacy: 160728
|
||||
// gas legacyOptimized: 152168
|
||||
// f(uint256): 12 -> 0x20, 0x0c, 0x0102030405060708090a0b0000000000000000000000000000000000000000
|
||||
// gas legacy: 59345
|
||||
// gas legacyOptimized: 57279
|
||||
// f(uint256): 129 -> 0x20, 0x81, 1780731860627700044960722568376592200742329637303199754547598369979440671, 0x202122232425262728292a2b2c2d2e2f303132333435363738393a3b3c3d3e3f, 29063324697304692433803953038474361308315562010425523193971352996434451193439, 0x606162636465666768696a6b6c6d6e6f707172737475767778797a7b7c7d7e7f, -57896044618658097711785492504343953926634992332820282019728792003956564819968
|
||||
// gas irOptimized: 419485
|
||||
// gas irOptimized: 406089
|
||||
// gas legacy: 423017
|
||||
// gas legacyOptimized: 406021
|
||||
|
@ -11,6 +11,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f(uint256[]): 0x20, 0x03, 0x1, 0x2, 0x3 -> 0x1
|
||||
// gas irOptimized: 111204
|
||||
// gas irOptimized: 111161
|
||||
// gas legacy: 111565
|
||||
// gas legacyOptimized: 111347
|
||||
|
@ -37,11 +37,11 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 0x40, 0x80, 6, 0x6162636465660000000000000000000000000000000000000000000000000000, 0x49, 0x3132333435363738393031323334353637383930313233343536373839303120, 0x3132333435363738393031323334353637383930313233343536373839303120, 0x3132333435363738390000000000000000000000000000000000000000000000
|
||||
// gas irOptimized: 179947
|
||||
// gas irOptimized: 179952
|
||||
// gas legacy: 180694
|
||||
// gas legacyOptimized: 180088
|
||||
// g() -> 0x40, 0xc0, 0x49, 0x3132333435363738393031323334353637383930313233343536373839303120, 0x3132333435363738393031323334353637383930313233343536373839303120, 0x3132333435363738390000000000000000000000000000000000000000000000, 0x11, 0x3132333435363738393233343536373839000000000000000000000000000000
|
||||
// gas irOptimized: 107322
|
||||
// gas irOptimized: 107332
|
||||
// gas legacy: 107895
|
||||
// gas legacyOptimized: 107254
|
||||
// h() -> 0x40, 0x60, 0x00, 0x00
|
||||
|
@ -48,6 +48,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 0xff
|
||||
// gas irOptimized: 121438
|
||||
// gas irOptimized: 121145
|
||||
// gas legacy: 128035
|
||||
// gas legacyOptimized: 123476
|
||||
|
@ -18,6 +18,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// test() -> 7
|
||||
// gas irOptimized: 126212
|
||||
// gas irOptimized: 126552
|
||||
// gas legacy: 205196
|
||||
// gas legacyOptimized: 204987
|
||||
|
@ -9,7 +9,7 @@ contract c {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// set(): 1, 2, 3, 4, 5 -> true
|
||||
// gas irOptimized: 177396
|
||||
// gas irOptimized: 177417
|
||||
// gas legacy: 177656
|
||||
// gas legacyOptimized: 177496
|
||||
// storageEmpty -> 0
|
||||
|
@ -20,6 +20,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 3
|
||||
// gas irOptimized: 131095
|
||||
// gas irOptimized: 129916
|
||||
// gas legacy: 130307
|
||||
// gas legacyOptimized: 129363
|
||||
|
@ -19,6 +19,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 1, 2, 3, 4, 5, 6, 7
|
||||
// gas irOptimized: 207030
|
||||
// gas irOptimized: 207785
|
||||
// gas legacy: 212325
|
||||
// gas legacyOptimized: 211486
|
||||
|
@ -13,6 +13,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 0x20, 0x02, 0x40, 0x80, 3, 0x6162630000000000000000000000000000000000000000000000000000000000, 0x99, 44048183304486788312148433451363384677562265908331949128489393215789685032262, 32241931068525137014058842823026578386641954854143559838526554899205067598957, 49951309422467613961193228765530489307475214998374779756599339590522149884499, 0x54555658595a6162636465666768696a6b6c6d6e6f707172737475767778797a, 0x4142434445464748494a4b4c4d4e4f5051525354555658595a00000000000000
|
||||
// gas irOptimized: 202750
|
||||
// gas irOptimized: 202840
|
||||
// gas legacy: 204459
|
||||
// gas legacyOptimized: 203437
|
||||
|
@ -20,6 +20,6 @@ contract C {
|
||||
// compileViaYul: also
|
||||
// ----
|
||||
// f() -> 1, 2, 3, 4, 5, 6, 7
|
||||
// gas irOptimized: 207030
|
||||
// gas irOptimized: 207785
|
||||
// gas legacy: 212330
|
||||
// gas legacyOptimized: 211491
|
||||
|
Some files were not shown because too many files have changed in this diff Show More
Loading…
Reference in New Issue
Block a user