Source Code
Cross-Chain Transactions
Loading...
Loading
Contract Name:
ManyChainMultiSig
Compiler Version
v0.8.19+commit.7dd6d404
Contract Source Code (Solidity)
/**
*Submitted for verification at fraxscan.com on 2025-02-19
*/
// SPDX-License-Identifier: BUSL-1.1
pragma solidity =0.8.19 ^0.8.0;
// lib/openzeppelin-contracts/contracts/utils/Context.sol
// OpenZeppelin Contracts v4.4.1 (utils/Context.sol)
/**
* @dev Provides information about the current execution context, including the
* sender of the transaction and its data. While these are generally available
* via msg.sender and msg.data, they should not be accessed in such a direct
* manner, since when dealing with meta-transactions the account sending and
* paying for execution may not be the actual sender (as far as an application
* is concerned).
*
* This contract is only required for intermediate, library-like contracts.
*/
abstract contract Context {
function _msgSender() internal view virtual returns (address) {
return msg.sender;
}
function _msgData() internal view virtual returns (bytes calldata) {
return msg.data;
}
}
// lib/openzeppelin-contracts/contracts/utils/cryptography/MerkleProof.sol
// OpenZeppelin Contracts (last updated v4.9.2) (utils/cryptography/MerkleProof.sol)
/**
* @dev These functions deal with verification of Merkle Tree proofs.
*
* The tree and the proofs can be generated using our
* https://github.com/OpenZeppelin/merkle-tree[JavaScript library].
* You will find a quickstart guide in the readme.
*
* WARNING: You should avoid using leaf values that are 64 bytes long prior to
* hashing, or use a hash function other than keccak256 for hashing leaves.
* This is because the concatenation of a sorted pair of internal nodes in
* the merkle tree could be reinterpreted as a leaf value.
* OpenZeppelin's JavaScript library generates merkle trees that are safe
* against this attack out of the box.
*/
library MerkleProof {
/**
* @dev Returns true if a `leaf` can be proved to be a part of a Merkle tree
* defined by `root`. For this, a `proof` must be provided, containing
* sibling hashes on the branch from the leaf to the root of the tree. Each
* pair of leaves and each pair of pre-images are assumed to be sorted.
*/
function verify(bytes32[] memory proof, bytes32 root, bytes32 leaf) internal pure returns (bool) {
return processProof(proof, leaf) == root;
}
/**
* @dev Calldata version of {verify}
*
* _Available since v4.7._
*/
function verifyCalldata(bytes32[] calldata proof, bytes32 root, bytes32 leaf) internal pure returns (bool) {
return processProofCalldata(proof, leaf) == root;
}
/**
* @dev Returns the rebuilt hash obtained by traversing a Merkle tree up
* from `leaf` using `proof`. A `proof` is valid if and only if the rebuilt
* hash matches the root of the tree. When processing the proof, the pairs
* of leafs & pre-images are assumed to be sorted.
*
* _Available since v4.4._
*/
function processProof(bytes32[] memory proof, bytes32 leaf) internal pure returns (bytes32) {
bytes32 computedHash = leaf;
for (uint256 i = 0; i < proof.length; i++) {
computedHash = _hashPair(computedHash, proof[i]);
}
return computedHash;
}
/**
* @dev Calldata version of {processProof}
*
* _Available since v4.7._
*/
function processProofCalldata(bytes32[] calldata proof, bytes32 leaf) internal pure returns (bytes32) {
bytes32 computedHash = leaf;
for (uint256 i = 0; i < proof.length; i++) {
computedHash = _hashPair(computedHash, proof[i]);
}
return computedHash;
}
/**
* @dev Returns true if the `leaves` can be simultaneously proven to be a part of a merkle tree defined by
* `root`, according to `proof` and `proofFlags` as described in {processMultiProof}.
*
* CAUTION: Not all merkle trees admit multiproofs. See {processMultiProof} for details.
*
* _Available since v4.7._
*/
function multiProofVerify(
bytes32[] memory proof,
bool[] memory proofFlags,
bytes32 root,
bytes32[] memory leaves
) internal pure returns (bool) {
return processMultiProof(proof, proofFlags, leaves) == root;
}
/**
* @dev Calldata version of {multiProofVerify}
*
* CAUTION: Not all merkle trees admit multiproofs. See {processMultiProof} for details.
*
* _Available since v4.7._
*/
function multiProofVerifyCalldata(
bytes32[] calldata proof,
bool[] calldata proofFlags,
bytes32 root,
bytes32[] memory leaves
) internal pure returns (bool) {
return processMultiProofCalldata(proof, proofFlags, leaves) == root;
}
/**
* @dev Returns the root of a tree reconstructed from `leaves` and sibling nodes in `proof`. The reconstruction
* proceeds by incrementally reconstructing all inner nodes by combining a leaf/inner node with either another
* leaf/inner node or a proof sibling node, depending on whether each `proofFlags` item is true or false
* respectively.
*
* CAUTION: Not all merkle trees admit multiproofs. To use multiproofs, it is sufficient to ensure that: 1) the tree
* is complete (but not necessarily perfect), 2) the leaves to be proven are in the opposite order they are in the
* tree (i.e., as seen from right to left starting at the deepest layer and continuing at the next layer).
*
* _Available since v4.7._
*/
function processMultiProof(
bytes32[] memory proof,
bool[] memory proofFlags,
bytes32[] memory leaves
) internal pure returns (bytes32 merkleRoot) {
// This function rebuilds the root hash by traversing the tree up from the leaves. The root is rebuilt by
// consuming and producing values on a queue. The queue starts with the `leaves` array, then goes onto the
// `hashes` array. At the end of the process, the last hash in the `hashes` array should contain the root of
// the merkle tree.
uint256 leavesLen = leaves.length;
uint256 proofLen = proof.length;
uint256 totalHashes = proofFlags.length;
// Check proof validity.
require(leavesLen + proofLen - 1 == totalHashes, "MerkleProof: invalid multiproof");
// The xxxPos values are "pointers" to the next value to consume in each array. All accesses are done using
// `xxx[xxxPos++]`, which return the current value and increment the pointer, thus mimicking a queue's "pop".
bytes32[] memory hashes = new bytes32[](totalHashes);
uint256 leafPos = 0;
uint256 hashPos = 0;
uint256 proofPos = 0;
// At each step, we compute the next hash using two values:
// - a value from the "main queue". If not all leaves have been consumed, we get the next leaf, otherwise we
// get the next hash.
// - depending on the flag, either another value from the "main queue" (merging branches) or an element from the
// `proof` array.
for (uint256 i = 0; i < totalHashes; i++) {
bytes32 a = leafPos < leavesLen ? leaves[leafPos++] : hashes[hashPos++];
bytes32 b = proofFlags[i]
? (leafPos < leavesLen ? leaves[leafPos++] : hashes[hashPos++])
: proof[proofPos++];
hashes[i] = _hashPair(a, b);
}
if (totalHashes > 0) {
require(proofPos == proofLen, "MerkleProof: invalid multiproof");
unchecked {
return hashes[totalHashes - 1];
}
} else if (leavesLen > 0) {
return leaves[0];
} else {
return proof[0];
}
}
/**
* @dev Calldata version of {processMultiProof}.
*
* CAUTION: Not all merkle trees admit multiproofs. See {processMultiProof} for details.
*
* _Available since v4.7._
*/
function processMultiProofCalldata(
bytes32[] calldata proof,
bool[] calldata proofFlags,
bytes32[] memory leaves
) internal pure returns (bytes32 merkleRoot) {
// This function rebuilds the root hash by traversing the tree up from the leaves. The root is rebuilt by
// consuming and producing values on a queue. The queue starts with the `leaves` array, then goes onto the
// `hashes` array. At the end of the process, the last hash in the `hashes` array should contain the root of
// the merkle tree.
uint256 leavesLen = leaves.length;
uint256 proofLen = proof.length;
uint256 totalHashes = proofFlags.length;
// Check proof validity.
require(leavesLen + proofLen - 1 == totalHashes, "MerkleProof: invalid multiproof");
// The xxxPos values are "pointers" to the next value to consume in each array. All accesses are done using
// `xxx[xxxPos++]`, which return the current value and increment the pointer, thus mimicking a queue's "pop".
bytes32[] memory hashes = new bytes32[](totalHashes);
uint256 leafPos = 0;
uint256 hashPos = 0;
uint256 proofPos = 0;
// At each step, we compute the next hash using two values:
// - a value from the "main queue". If not all leaves have been consumed, we get the next leaf, otherwise we
// get the next hash.
// - depending on the flag, either another value from the "main queue" (merging branches) or an element from the
// `proof` array.
for (uint256 i = 0; i < totalHashes; i++) {
bytes32 a = leafPos < leavesLen ? leaves[leafPos++] : hashes[hashPos++];
bytes32 b = proofFlags[i]
? (leafPos < leavesLen ? leaves[leafPos++] : hashes[hashPos++])
: proof[proofPos++];
hashes[i] = _hashPair(a, b);
}
if (totalHashes > 0) {
require(proofPos == proofLen, "MerkleProof: invalid multiproof");
unchecked {
return hashes[totalHashes - 1];
}
} else if (leavesLen > 0) {
return leaves[0];
} else {
return proof[0];
}
}
function _hashPair(bytes32 a, bytes32 b) private pure returns (bytes32) {
return a < b ? _efficientHash(a, b) : _efficientHash(b, a);
}
function _efficientHash(bytes32 a, bytes32 b) private pure returns (bytes32 value) {
/// @solidity memory-safe-assembly
assembly {
mstore(0x00, a)
mstore(0x20, b)
value := keccak256(0x00, 0x40)
}
}
}
// lib/openzeppelin-contracts/contracts/utils/math/Math.sol
// OpenZeppelin Contracts (last updated v4.9.0) (utils/math/Math.sol)
/**
* @dev Standard math utilities missing in the Solidity language.
*/
library Math {
enum Rounding {
Down, // Toward negative infinity
Up, // Toward infinity
Zero // Toward zero
}
/**
* @dev Returns the largest of two numbers.
*/
function max(uint256 a, uint256 b) internal pure returns (uint256) {
return a > b ? a : b;
}
/**
* @dev Returns the smallest of two numbers.
*/
function min(uint256 a, uint256 b) internal pure returns (uint256) {
return a < b ? a : b;
}
/**
* @dev Returns the average of two numbers. The result is rounded towards
* zero.
*/
function average(uint256 a, uint256 b) internal pure returns (uint256) {
// (a + b) / 2 can overflow.
return (a & b) + (a ^ b) / 2;
}
/**
* @dev Returns the ceiling of the division of two numbers.
*
* This differs from standard division with `/` in that it rounds up instead
* of rounding down.
*/
function ceilDiv(uint256 a, uint256 b) internal pure returns (uint256) {
// (a + b - 1) / b can overflow on addition, so we distribute.
return a == 0 ? 0 : (a - 1) / b + 1;
}
/**
* @notice Calculates floor(x * y / denominator) with full precision. Throws if result overflows a uint256 or denominator == 0
* @dev Original credit to Remco Bloemen under MIT license (https://xn--2-umb.com/21/muldiv)
* with further edits by Uniswap Labs also under MIT license.
*/
function mulDiv(uint256 x, uint256 y, uint256 denominator) internal pure returns (uint256 result) {
unchecked {
// 512-bit multiply [prod1 prod0] = x * y. Compute the product mod 2^256 and mod 2^256 - 1, then use
// use the Chinese Remainder Theorem to reconstruct the 512 bit result. The result is stored in two 256
// variables such that product = prod1 * 2^256 + prod0.
uint256 prod0; // Least significant 256 bits of the product
uint256 prod1; // Most significant 256 bits of the product
assembly {
let mm := mulmod(x, y, not(0))
prod0 := mul(x, y)
prod1 := sub(sub(mm, prod0), lt(mm, prod0))
}
// Handle non-overflow cases, 256 by 256 division.
if (prod1 == 0) {
// Solidity will revert if denominator == 0, unlike the div opcode on its own.
// The surrounding unchecked block does not change this fact.
// See https://docs.soliditylang.org/en/latest/control-structures.html#checked-or-unchecked-arithmetic.
return prod0 / denominator;
}
// Make sure the result is less than 2^256. Also prevents denominator == 0.
require(denominator > prod1, "Math: mulDiv overflow");
///////////////////////////////////////////////
// 512 by 256 division.
///////////////////////////////////////////////
// Make division exact by subtracting the remainder from [prod1 prod0].
uint256 remainder;
assembly {
// Compute remainder using mulmod.
remainder := mulmod(x, y, denominator)
// Subtract 256 bit number from 512 bit number.
prod1 := sub(prod1, gt(remainder, prod0))
prod0 := sub(prod0, remainder)
}
// Factor powers of two out of denominator and compute largest power of two divisor of denominator. Always >= 1.
// See https://cs.stackexchange.com/q/138556/92363.
// Does not overflow because the denominator cannot be zero at this stage in the function.
uint256 twos = denominator & (~denominator + 1);
assembly {
// Divide denominator by twos.
denominator := div(denominator, twos)
// Divide [prod1 prod0] by twos.
prod0 := div(prod0, twos)
// Flip twos such that it is 2^256 / twos. If twos is zero, then it becomes one.
twos := add(div(sub(0, twos), twos), 1)
}
// Shift in bits from prod1 into prod0.
prod0 |= prod1 * twos;
// Invert denominator mod 2^256. Now that denominator is an odd number, it has an inverse modulo 2^256 such
// that denominator * inv = 1 mod 2^256. Compute the inverse by starting with a seed that is correct for
// four bits. That is, denominator * inv = 1 mod 2^4.
uint256 inverse = (3 * denominator) ^ 2;
// Use the Newton-Raphson iteration to improve the precision. Thanks to Hensel's lifting lemma, this also works
// in modular arithmetic, doubling the correct bits in each step.
inverse *= 2 - denominator * inverse; // inverse mod 2^8
inverse *= 2 - denominator * inverse; // inverse mod 2^16
inverse *= 2 - denominator * inverse; // inverse mod 2^32
inverse *= 2 - denominator * inverse; // inverse mod 2^64
inverse *= 2 - denominator * inverse; // inverse mod 2^128
inverse *= 2 - denominator * inverse; // inverse mod 2^256
// Because the division is now exact we can divide by multiplying with the modular inverse of denominator.
// This will give us the correct result modulo 2^256. Since the preconditions guarantee that the outcome is
// less than 2^256, this is the final result. We don't need to compute the high bits of the result and prod1
// is no longer required.
result = prod0 * inverse;
return result;
}
}
/**
* @notice Calculates x * y / denominator with full precision, following the selected rounding direction.
*/
function mulDiv(uint256 x, uint256 y, uint256 denominator, Rounding rounding) internal pure returns (uint256) {
uint256 result = mulDiv(x, y, denominator);
if (rounding == Rounding.Up && mulmod(x, y, denominator) > 0) {
result += 1;
}
return result;
}
/**
* @dev Returns the square root of a number. If the number is not a perfect square, the value is rounded down.
*
* Inspired by Henry S. Warren, Jr.'s "Hacker's Delight" (Chapter 11).
*/
function sqrt(uint256 a) internal pure returns (uint256) {
if (a == 0) {
return 0;
}
// For our first guess, we get the biggest power of 2 which is smaller than the square root of the target.
//
// We know that the "msb" (most significant bit) of our target number `a` is a power of 2 such that we have
// `msb(a) <= a < 2*msb(a)`. This value can be written `msb(a)=2**k` with `k=log2(a)`.
//
// This can be rewritten `2**log2(a) <= a < 2**(log2(a) + 1)`
// → `sqrt(2**k) <= sqrt(a) < sqrt(2**(k+1))`
// → `2**(k/2) <= sqrt(a) < 2**((k+1)/2) <= 2**(k/2 + 1)`
//
// Consequently, `2**(log2(a) / 2)` is a good first approximation of `sqrt(a)` with at least 1 correct bit.
uint256 result = 1 << (log2(a) >> 1);
// At this point `result` is an estimation with one bit of precision. We know the true value is a uint128,
// since it is the square root of a uint256. Newton's method converges quadratically (precision doubles at
// every iteration). We thus need at most 7 iteration to turn our partial result with one bit of precision
// into the expected uint128 result.
unchecked {
result = (result + a / result) >> 1;
result = (result + a / result) >> 1;
result = (result + a / result) >> 1;
result = (result + a / result) >> 1;
result = (result + a / result) >> 1;
result = (result + a / result) >> 1;
result = (result + a / result) >> 1;
return min(result, a / result);
}
}
/**
* @notice Calculates sqrt(a), following the selected rounding direction.
*/
function sqrt(uint256 a, Rounding rounding) internal pure returns (uint256) {
unchecked {
uint256 result = sqrt(a);
return result + (rounding == Rounding.Up && result * result < a ? 1 : 0);
}
}
/**
* @dev Return the log in base 2, rounded down, of a positive value.
* Returns 0 if given 0.
*/
function log2(uint256 value) internal pure returns (uint256) {
uint256 result = 0;
unchecked {
if (value >> 128 > 0) {
value >>= 128;
result += 128;
}
if (value >> 64 > 0) {
value >>= 64;
result += 64;
}
if (value >> 32 > 0) {
value >>= 32;
result += 32;
}
if (value >> 16 > 0) {
value >>= 16;
result += 16;
}
if (value >> 8 > 0) {
value >>= 8;
result += 8;
}
if (value >> 4 > 0) {
value >>= 4;
result += 4;
}
if (value >> 2 > 0) {
value >>= 2;
result += 2;
}
if (value >> 1 > 0) {
result += 1;
}
}
return result;
}
/**
* @dev Return the log in base 2, following the selected rounding direction, of a positive value.
* Returns 0 if given 0.
*/
function log2(uint256 value, Rounding rounding) internal pure returns (uint256) {
unchecked {
uint256 result = log2(value);
return result + (rounding == Rounding.Up && 1 << result < value ? 1 : 0);
}
}
/**
* @dev Return the log in base 10, rounded down, of a positive value.
* Returns 0 if given 0.
*/
function log10(uint256 value) internal pure returns (uint256) {
uint256 result = 0;
unchecked {
if (value >= 10 ** 64) {
value /= 10 ** 64;
result += 64;
}
if (value >= 10 ** 32) {
value /= 10 ** 32;
result += 32;
}
if (value >= 10 ** 16) {
value /= 10 ** 16;
result += 16;
}
if (value >= 10 ** 8) {
value /= 10 ** 8;
result += 8;
}
if (value >= 10 ** 4) {
value /= 10 ** 4;
result += 4;
}
if (value >= 10 ** 2) {
value /= 10 ** 2;
result += 2;
}
if (value >= 10 ** 1) {
result += 1;
}
}
return result;
}
/**
* @dev Return the log in base 10, following the selected rounding direction, of a positive value.
* Returns 0 if given 0.
*/
function log10(uint256 value, Rounding rounding) internal pure returns (uint256) {
unchecked {
uint256 result = log10(value);
return result + (rounding == Rounding.Up && 10 ** result < value ? 1 : 0);
}
}
/**
* @dev Return the log in base 256, rounded down, of a positive value.
* Returns 0 if given 0.
*
* Adding one to the result gives the number of pairs of hex symbols needed to represent `value` as a hex string.
*/
function log256(uint256 value) internal pure returns (uint256) {
uint256 result = 0;
unchecked {
if (value >> 128 > 0) {
value >>= 128;
result += 16;
}
if (value >> 64 > 0) {
value >>= 64;
result += 8;
}
if (value >> 32 > 0) {
value >>= 32;
result += 4;
}
if (value >> 16 > 0) {
value >>= 16;
result += 2;
}
if (value >> 8 > 0) {
result += 1;
}
}
return result;
}
/**
* @dev Return the log in base 256, following the selected rounding direction, of a positive value.
* Returns 0 if given 0.
*/
function log256(uint256 value, Rounding rounding) internal pure returns (uint256) {
unchecked {
uint256 result = log256(value);
return result + (rounding == Rounding.Up && 1 << (result << 3) < value ? 1 : 0);
}
}
}
// lib/openzeppelin-contracts/contracts/utils/math/SignedMath.sol
// OpenZeppelin Contracts (last updated v4.8.0) (utils/math/SignedMath.sol)
/**
* @dev Standard signed math utilities missing in the Solidity language.
*/
library SignedMath {
/**
* @dev Returns the largest of two signed numbers.
*/
function max(int256 a, int256 b) internal pure returns (int256) {
return a > b ? a : b;
}
/**
* @dev Returns the smallest of two signed numbers.
*/
function min(int256 a, int256 b) internal pure returns (int256) {
return a < b ? a : b;
}
/**
* @dev Returns the average of two signed numbers without overflow.
* The result is rounded towards zero.
*/
function average(int256 a, int256 b) internal pure returns (int256) {
// Formula from the book "Hacker's Delight"
int256 x = (a & b) + ((a ^ b) >> 1);
return x + (int256(uint256(x) >> 255) & (a ^ b));
}
/**
* @dev Returns the absolute unsigned value of a signed value.
*/
function abs(int256 n) internal pure returns (uint256) {
unchecked {
// must be unchecked in order to support `n = type(int256).min`
return uint256(n >= 0 ? n : -n);
}
}
}
// lib/openzeppelin-contracts/contracts/access/Ownable.sol
// OpenZeppelin Contracts (last updated v4.9.0) (access/Ownable.sol)
/**
* @dev Contract module which provides a basic access control mechanism, where
* there is an account (an owner) that can be granted exclusive access to
* specific functions.
*
* By default, the owner account will be the one that deploys the contract. This
* can later be changed with {transferOwnership}.
*
* This module is used through inheritance. It will make available the modifier
* `onlyOwner`, which can be applied to your functions to restrict their use to
* the owner.
*/
abstract contract Ownable is Context {
address private _owner;
event OwnershipTransferred(address indexed previousOwner, address indexed newOwner);
/**
* @dev Initializes the contract setting the deployer as the initial owner.
*/
constructor() {
_transferOwnership(_msgSender());
}
/**
* @dev Throws if called by any account other than the owner.
*/
modifier onlyOwner() {
_checkOwner();
_;
}
/**
* @dev Returns the address of the current owner.
*/
function owner() public view virtual returns (address) {
return _owner;
}
/**
* @dev Throws if the sender is not the owner.
*/
function _checkOwner() internal view virtual {
require(owner() == _msgSender(), "Ownable: caller is not the owner");
}
/**
* @dev Leaves the contract without owner. It will not be possible to call
* `onlyOwner` functions. Can only be called by the current owner.
*
* NOTE: Renouncing ownership will leave the contract without an owner,
* thereby disabling any functionality that is only available to the owner.
*/
function renounceOwnership() public virtual onlyOwner {
_transferOwnership(address(0));
}
/**
* @dev Transfers ownership of the contract to a new account (`newOwner`).
* Can only be called by the current owner.
*/
function transferOwnership(address newOwner) public virtual onlyOwner {
require(newOwner != address(0), "Ownable: new owner is the zero address");
_transferOwnership(newOwner);
}
/**
* @dev Transfers ownership of the contract to a new account (`newOwner`).
* Internal function without access restriction.
*/
function _transferOwnership(address newOwner) internal virtual {
address oldOwner = _owner;
_owner = newOwner;
emit OwnershipTransferred(oldOwner, newOwner);
}
}
// lib/openzeppelin-contracts/contracts/access/Ownable2Step.sol
// OpenZeppelin Contracts (last updated v4.9.0) (access/Ownable2Step.sol)
/**
* @dev Contract module which provides access control mechanism, where
* there is an account (an owner) that can be granted exclusive access to
* specific functions.
*
* By default, the owner account will be the one that deploys the contract. This
* can later be changed with {transferOwnership} and {acceptOwnership}.
*
* This module is used through inheritance. It will make available all functions
* from parent (Ownable).
*/
abstract contract Ownable2Step is Ownable {
address private _pendingOwner;
event OwnershipTransferStarted(address indexed previousOwner, address indexed newOwner);
/**
* @dev Returns the address of the pending owner.
*/
function pendingOwner() public view virtual returns (address) {
return _pendingOwner;
}
/**
* @dev Starts the ownership transfer of the contract to a new account. Replaces the pending transfer if there is one.
* Can only be called by the current owner.
*/
function transferOwnership(address newOwner) public virtual override onlyOwner {
_pendingOwner = newOwner;
emit OwnershipTransferStarted(owner(), newOwner);
}
/**
* @dev Transfers ownership of the contract to a new account (`newOwner`) and deletes any pending owner.
* Internal function without access restriction.
*/
function _transferOwnership(address newOwner) internal virtual override {
delete _pendingOwner;
super._transferOwnership(newOwner);
}
/**
* @dev The new owner accepts the ownership transfer.
*/
function acceptOwnership() public virtual {
address sender = _msgSender();
require(pendingOwner() == sender, "Ownable2Step: caller is not the new owner");
_transferOwnership(sender);
}
}
// lib/openzeppelin-contracts/contracts/utils/Strings.sol
// OpenZeppelin Contracts (last updated v4.9.0) (utils/Strings.sol)
/**
* @dev String operations.
*/
library Strings {
bytes16 private constant _SYMBOLS = "0123456789abcdef";
uint8 private constant _ADDRESS_LENGTH = 20;
/**
* @dev Converts a `uint256` to its ASCII `string` decimal representation.
*/
function toString(uint256 value) internal pure returns (string memory) {
unchecked {
uint256 length = Math.log10(value) + 1;
string memory buffer = new string(length);
uint256 ptr;
/// @solidity memory-safe-assembly
assembly {
ptr := add(buffer, add(32, length))
}
while (true) {
ptr--;
/// @solidity memory-safe-assembly
assembly {
mstore8(ptr, byte(mod(value, 10), _SYMBOLS))
}
value /= 10;
if (value == 0) break;
}
return buffer;
}
}
/**
* @dev Converts a `int256` to its ASCII `string` decimal representation.
*/
function toString(int256 value) internal pure returns (string memory) {
return string(abi.encodePacked(value < 0 ? "-" : "", toString(SignedMath.abs(value))));
}
/**
* @dev Converts a `uint256` to its ASCII `string` hexadecimal representation.
*/
function toHexString(uint256 value) internal pure returns (string memory) {
unchecked {
return toHexString(value, Math.log256(value) + 1);
}
}
/**
* @dev Converts a `uint256` to its ASCII `string` hexadecimal representation with fixed length.
*/
function toHexString(uint256 value, uint256 length) internal pure returns (string memory) {
bytes memory buffer = new bytes(2 * length + 2);
buffer[0] = "0";
buffer[1] = "x";
for (uint256 i = 2 * length + 1; i > 1; --i) {
buffer[i] = _SYMBOLS[value & 0xf];
value >>= 4;
}
require(value == 0, "Strings: hex length insufficient");
return string(buffer);
}
/**
* @dev Converts an `address` with fixed length of 20 bytes to its not checksummed ASCII `string` hexadecimal representation.
*/
function toHexString(address addr) internal pure returns (string memory) {
return toHexString(uint256(uint160(addr)), _ADDRESS_LENGTH);
}
/**
* @dev Returns true if the two strings are equal.
*/
function equal(string memory a, string memory b) internal pure returns (bool) {
return keccak256(bytes(a)) == keccak256(bytes(b));
}
}
// lib/openzeppelin-contracts/contracts/utils/cryptography/ECDSA.sol
// OpenZeppelin Contracts (last updated v4.9.0) (utils/cryptography/ECDSA.sol)
/**
* @dev Elliptic Curve Digital Signature Algorithm (ECDSA) operations.
*
* These functions can be used to verify that a message was signed by the holder
* of the private keys of a given address.
*/
library ECDSA {
enum RecoverError {
NoError,
InvalidSignature,
InvalidSignatureLength,
InvalidSignatureS,
InvalidSignatureV // Deprecated in v4.8
}
function _throwError(RecoverError error) private pure {
if (error == RecoverError.NoError) {
return; // no error: do nothing
} else if (error == RecoverError.InvalidSignature) {
revert("ECDSA: invalid signature");
} else if (error == RecoverError.InvalidSignatureLength) {
revert("ECDSA: invalid signature length");
} else if (error == RecoverError.InvalidSignatureS) {
revert("ECDSA: invalid signature 's' value");
}
}
/**
* @dev Returns the address that signed a hashed message (`hash`) with
* `signature` or error string. This address can then be used for verification purposes.
*
* The `ecrecover` EVM opcode allows for malleable (non-unique) signatures:
* this function rejects them by requiring the `s` value to be in the lower
* half order, and the `v` value to be either 27 or 28.
*
* IMPORTANT: `hash` _must_ be the result of a hash operation for the
* verification to be secure: it is possible to craft signatures that
* recover to arbitrary addresses for non-hashed data. A safe way to ensure
* this is by receiving a hash of the original message (which may otherwise
* be too long), and then calling {toEthSignedMessageHash} on it.
*
* Documentation for signature generation:
* - with https://web3js.readthedocs.io/en/v1.3.4/web3-eth-accounts.html#sign[Web3.js]
* - with https://docs.ethers.io/v5/api/signer/#Signer-signMessage[ethers]
*
* _Available since v4.3._
*/
function tryRecover(bytes32 hash, bytes memory signature) internal pure returns (address, RecoverError) {
if (signature.length == 65) {
bytes32 r;
bytes32 s;
uint8 v;
// ecrecover takes the signature parameters, and the only way to get them
// currently is to use assembly.
/// @solidity memory-safe-assembly
assembly {
r := mload(add(signature, 0x20))
s := mload(add(signature, 0x40))
v := byte(0, mload(add(signature, 0x60)))
}
return tryRecover(hash, v, r, s);
} else {
return (address(0), RecoverError.InvalidSignatureLength);
}
}
/**
* @dev Returns the address that signed a hashed message (`hash`) with
* `signature`. This address can then be used for verification purposes.
*
* The `ecrecover` EVM opcode allows for malleable (non-unique) signatures:
* this function rejects them by requiring the `s` value to be in the lower
* half order, and the `v` value to be either 27 or 28.
*
* IMPORTANT: `hash` _must_ be the result of a hash operation for the
* verification to be secure: it is possible to craft signatures that
* recover to arbitrary addresses for non-hashed data. A safe way to ensure
* this is by receiving a hash of the original message (which may otherwise
* be too long), and then calling {toEthSignedMessageHash} on it.
*/
function recover(bytes32 hash, bytes memory signature) internal pure returns (address) {
(address recovered, RecoverError error) = tryRecover(hash, signature);
_throwError(error);
return recovered;
}
/**
* @dev Overload of {ECDSA-tryRecover} that receives the `r` and `vs` short-signature fields separately.
*
* See https://eips.ethereum.org/EIPS/eip-2098[EIP-2098 short signatures]
*
* _Available since v4.3._
*/
function tryRecover(bytes32 hash, bytes32 r, bytes32 vs) internal pure returns (address, RecoverError) {
bytes32 s = vs & bytes32(0x7fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff);
uint8 v = uint8((uint256(vs) >> 255) + 27);
return tryRecover(hash, v, r, s);
}
/**
* @dev Overload of {ECDSA-recover} that receives the `r and `vs` short-signature fields separately.
*
* _Available since v4.2._
*/
function recover(bytes32 hash, bytes32 r, bytes32 vs) internal pure returns (address) {
(address recovered, RecoverError error) = tryRecover(hash, r, vs);
_throwError(error);
return recovered;
}
/**
* @dev Overload of {ECDSA-tryRecover} that receives the `v`,
* `r` and `s` signature fields separately.
*
* _Available since v4.3._
*/
function tryRecover(bytes32 hash, uint8 v, bytes32 r, bytes32 s) internal pure returns (address, RecoverError) {
// EIP-2 still allows signature malleability for ecrecover(). Remove this possibility and make the signature
// unique. Appendix F in the Ethereum Yellow paper (https://ethereum.github.io/yellowpaper/paper.pdf), defines
// the valid range for s in (301): 0 < s < secp256k1n ÷ 2 + 1, and for v in (302): v ∈ {27, 28}. Most
// signatures from current libraries generate a unique signature with an s-value in the lower half order.
//
// If your library generates malleable signatures, such as s-values in the upper range, calculate a new s-value
// with 0xFFFFFFFFFFFFFFFFFFFFFFFFFFFFFFFEBAAEDCE6AF48A03BBFD25E8CD0364141 - s1 and flip v from 27 to 28 or
// vice versa. If your library also generates signatures with 0/1 for v instead 27/28, add 27 to v to accept
// these malleable signatures as well.
if (uint256(s) > 0x7FFFFFFFFFFFFFFFFFFFFFFFFFFFFFFF5D576E7357A4501DDFE92F46681B20A0) {
return (address(0), RecoverError.InvalidSignatureS);
}
// If the signature is valid (and not malleable), return the signer address
address signer = ecrecover(hash, v, r, s);
if (signer == address(0)) {
return (address(0), RecoverError.InvalidSignature);
}
return (signer, RecoverError.NoError);
}
/**
* @dev Overload of {ECDSA-recover} that receives the `v`,
* `r` and `s` signature fields separately.
*/
function recover(bytes32 hash, uint8 v, bytes32 r, bytes32 s) internal pure returns (address) {
(address recovered, RecoverError error) = tryRecover(hash, v, r, s);
_throwError(error);
return recovered;
}
/**
* @dev Returns an Ethereum Signed Message, created from a `hash`. This
* produces hash corresponding to the one signed with the
* https://eth.wiki/json-rpc/API#eth_sign[`eth_sign`]
* JSON-RPC method as part of EIP-191.
*
* See {recover}.
*/
function toEthSignedMessageHash(bytes32 hash) internal pure returns (bytes32 message) {
// 32 is the length in bytes of hash,
// enforced by the type signature above
/// @solidity memory-safe-assembly
assembly {
mstore(0x00, "\x19Ethereum Signed Message:\n32")
mstore(0x1c, hash)
message := keccak256(0x00, 0x3c)
}
}
/**
* @dev Returns an Ethereum Signed Message, created from `s`. This
* produces hash corresponding to the one signed with the
* https://eth.wiki/json-rpc/API#eth_sign[`eth_sign`]
* JSON-RPC method as part of EIP-191.
*
* See {recover}.
*/
function toEthSignedMessageHash(bytes memory s) internal pure returns (bytes32) {
return keccak256(abi.encodePacked("\x19Ethereum Signed Message:\n", Strings.toString(s.length), s));
}
/**
* @dev Returns an Ethereum Signed Typed Data, created from a
* `domainSeparator` and a `structHash`. This produces hash corresponding
* to the one signed with the
* https://eips.ethereum.org/EIPS/eip-712[`eth_signTypedData`]
* JSON-RPC method as part of EIP-712.
*
* See {recover}.
*/
function toTypedDataHash(bytes32 domainSeparator, bytes32 structHash) internal pure returns (bytes32 data) {
/// @solidity memory-safe-assembly
assembly {
let ptr := mload(0x40)
mstore(ptr, "\x19\x01")
mstore(add(ptr, 0x02), domainSeparator)
mstore(add(ptr, 0x22), structHash)
data := keccak256(ptr, 0x42)
}
}
/**
* @dev Returns an Ethereum Signed Data with intended validator, created from a
* `validator` and `data` according to the version 0 of EIP-191.
*
* See {recover}.
*/
function toDataWithIntendedValidatorHash(address validator, bytes memory data) internal pure returns (bytes32) {
return keccak256(abi.encodePacked("\x19\x00", validator, data));
}
}
// src/ManyChainMultiSig.sol
// Should be used as the first 32 bytes of the pre-image of the leaf that holds a
// op. This value is for domain separation of the different values stored in the
// Merkle tree.
bytes32 constant MANY_CHAIN_MULTI_SIG_DOMAIN_SEPARATOR_OP =
keccak256("MANY_CHAIN_MULTI_SIG_DOMAIN_SEPARATOR_OP");
// Should be used as the first 32 bytes of the pre-image of the leaf that holds the
// root metadata. This value is for domain separation of the different values stored in the
// Merkle tree.
bytes32 constant MANY_CHAIN_MULTI_SIG_DOMAIN_SEPARATOR_METADATA =
keccak256("MANY_CHAIN_MULTI_SIG_DOMAIN_SEPARATOR_METADATA");
/// @notice This is a multi-sig contract that supports signing many transactions (called "ops" in
/// the context of this contract to prevent confusion with transactions on the underlying chain)
/// targeting many chains with a single set of signatures. Authorized ops along with some metadata
/// are stored in a Merkle tree, which is generated offchain. Each op has an associated chain id,
/// ManyChainMultiSig contract address and nonce. The nonce enables us to enforce the
/// (per-ManyChainMultiSig contract instance) ordering of ops.
///
/// At any time, this contract stores at most one Merkle root. In the typical case, all ops
/// in the Merkle tree are expected to be executed before another root is set. Since the Merkle root
/// itself reveals ~ no information about the tree's contents, we take two measures to improve
/// transparency. First, we attach an expiration time to each Merkle root after which it cannot
/// be used any more. Second, we embed metadata in the tree itself that has to be proven/revealed
/// to the contract when a new root is set; the metadata contains the range of nonces (and thus
/// number of ops) in the tree intended for the ManyChainMultiSig contract instance on which the
/// root is being set.
///
/// Once a root is registered, *anyone* is allowed to furnish proofs of op inclusion in the Merkle
/// tree and execute the corresponding op. The contract enforces that ops are executed in the
/// correct order and with the correct arguments. A notable exception to this is the gas limit of
/// the call, which can be freely determined by the executor. We expect (transitive) callees to
/// implement standard behavior of simply reverting if insufficient gas is provided. In particular,
/// this means callees should not have non-reverting gas-dependent branches.
///
/// Note: In the typical case, we expect the time from a root being set to all of the ops
/// therein having been executed to be on the order of a couple of minutes.
contract ManyChainMultiSig is Ownable2Step {
receive() external payable {}
uint8 public constant NUM_GROUPS = 32;
uint8 public constant MAX_NUM_SIGNERS = 200;
struct Signer {
address addr;
uint8 index; // index of signer in s_config.signers
uint8 group; // 0 <= group < NUM_GROUPS. Each signer can only be in one group.
}
// s_signers is used to easily validate the existence of the signer by its address. We still
// have signers stored in s_config in order to easily deactivate them when a new config is set.
mapping(address => Signer) s_signers;
// Signing groups are arranged in a tree. Each group is an interior node and has its own quorum.
// Signers are the leaves of the tree. A signer/leaf node is successful iff it furnishes a valid
// signature. A group/interior node is successful iff a quorum of its children are successful.
// setRoot succeeds only if the root group is successful.
// Here is an example:
//
// ┌──────┐
// ┌─►│2-of-3│◄───────┐
// │ └──────┘ │
// │ ▲ │
// │ │ │
// ┌──┴───┐ ┌──┴───┐ ┌───┴────┐
// ┌──►│1-of-2│ │2-of-2│ │signer A│
// │ └──────┘ └──────┘ └────────┘
// │ ▲ ▲ ▲
// │ │ │ │ ┌──────┐
// │ │ │ └─────┤1-of-2│◄─┐
// │ │ │ └──────┘ │
// ┌───────┴┐ ┌────┴───┐ ┌┴───────┐ ▲ │
// │signer B│ │signer C│ │signer D│ │ │
// └────────┘ └────────┘ └────────┘ │ │
// │ │
// ┌──────┴─┐ ┌────┴───┐
// │signer E│ │signer F│
// └────────┘ └────────┘
//
// - If signers [A, B] sign, they can set a root.
// - If signers [B, D, E] sign, they can set a root.
// - If signers [B, D, E, F] sign, they can set a root. (Either E's or F's signature was
// superfluous.)
// - If signers [B, C, D] sign, they cannot set a root, because the 2-of-2 group on the second
// level isn't successful and therefore the root group isn't successful either.
//
// To map this tree to a Config, we:
// - create an entry in signers for each signer (sorted by address in ascending order)
// - assign the root group to index 0 and have it be its own parent
// - assign an index to each non-root group, such that each group's parent has a lower index
// than the group itself
// For example, we could transform the above tree structure into:
// groupQuorums = [2, 1, 2, 1] + [0, 0, ...] (rightpad with 0s to NUM_GROUPS)
// groupParents = [0, 0, 0, 2] + [0, 0, ...] (rightpad with 0s to NUM_GROUPS)
// and assuming that address(A) < address(C) < address(E) < address(F) < address(D) < address(B)
// signers = [
// {addr: address(A), index: 0, group: 0}, {addr: address(C), index: 1, group: 1},
// {addr: address(E), index: 2, group: 3}, {addr: address(F), index: 3, group: 3},
// {addr: address(D), index: 4, group: 2}, {addr: address(B), index: 5, group: 1},
// ]
struct Config {
Signer[] signers;
// groupQuorums[i] stores the quorum for the i-th signer group. Any group with
// groupQuorums[i] = 0 is considered disabled. The i-th group is successful if
// it is enabled and at least groupQuorums[i] of its children are successful.
uint8[NUM_GROUPS] groupQuorums;
// groupParents[i] stores the parent group of the i-th signer group. We ensure that the
// groups form a tree structure (where the root/0-th signer group points to itself as
// parent) by enforcing
// - (i != 0) implies (groupParents[i] < i)
// - groupParents[0] == 0
uint8[NUM_GROUPS] groupParents;
}
Config s_config;
// Remember signedHashes that this contract has seen. Each signedHash can only be set once.
mapping(bytes32 => bool) s_seenSignedHashes;
// MerkleRoots are a bit tricky since they reveal almost no information about the contents of
// the tree they authenticate. To mitigate this, we enforce that this contract can only execute
// ops from a single root at any given point in time. We further associate an expiry
// with each root to ensure that messages are executed in a timely manner. setRoot and various
// execute calls are expected to happen in quick succession. We put the expiring root and
// opCount in same struct in order to reduce gas costs of reading and writing.
struct ExpiringRootAndOpCount {
bytes32 root;
// We prefer using block.timestamp instead of block.number, as a single
// root may target many chains. We assume that block.timestamp can
// be manipulated by block producers but only within relatively tight
// bounds (a few minutes at most).
uint32 validUntil;
// each ManyChainMultiSig instance has it own independent opCount.
uint40 opCount;
}
ExpiringRootAndOpCount s_expiringRootAndOpCount;
/// @notice Each root also authenticates metadata about itself (stored as one of the leaves)
/// which must be revealed when the root is set.
///
/// @dev We need to be careful that abi.encode(MANY_CHAIN_MULTI_SIG_DOMAIN_SEPARATOR_METADATA, RootMetadata)
/// is greater than 64 bytes to prevent collisions with internal nodes in the Merkle tree. See
/// openzeppelin-contracts/contracts/utils/cryptography/MerkleProof.sol:15 for details.
struct RootMetadata {
// chainId and multiSig uniquely identify a ManyChainMultiSig contract instance that the
// root is destined for.
// uint256 since it is unclear if we can represent chainId as uint64. There is a proposal (
// https://ethereum-magicians.org/t/eip-2294-explicit-bound-to-chain-id/11090) to
// bound chainid to 64 bits, but it is still unresolved.
uint256 chainId;
address multiSig;
// opCount before adding this root
uint40 preOpCount;
// opCount after executing all ops in this root
uint40 postOpCount;
// override whatever root was already stored in this contract even if some of its
// ops weren't executed.
// Important: it is strongly recommended that offchain code set this to false by default.
// Be careful setting this to true as it may break assumptions about what transactions from
// the previous root have already been executed.
bool overridePreviousRoot;
}
RootMetadata s_rootMetadata;
/// @notice An ECDSA signature.
struct Signature {
uint8 v;
bytes32 r;
bytes32 s;
}
/// @notice setRoot Sets a new expiring root.
///
/// @param root is the new expiring root.
/// @param validUntil is the time by which root is valid
/// @param metadata is the authenticated metadata about the root, which is stored as one of
/// the leaves.
/// @param metadataProof is the MerkleProof of inclusion of the metadata in the Merkle tree.
/// @param signatures the ECDSA signatures on (root, validUntil).
///
/// @dev the message (root, validUntil) should be signed by a sufficient set of signers.
/// This signature authenticates also the metadata.
///
/// @dev this method can be executed by anyone who has the root and valid signatures.
/// as we validate the correctness of signatures, this imposes no risk.
function setRoot(
bytes32 root,
uint32 validUntil,
RootMetadata calldata metadata,
bytes32[] calldata metadataProof,
Signature[] calldata signatures
) external {
bytes32 signedHash = ECDSA.toEthSignedMessageHash(keccak256(abi.encode(root, validUntil)));
// Each (root, validUntil) tuple can only bet set once. For example, this prevents a
// scenario where there are two signed roots with overridePreviousRoot = true and
// an adversary keeps alternatively calling setRoot(root1), setRoot(root2),
// setRoot(root1), ...
if (s_seenSignedHashes[signedHash]) {
revert SignedHashAlreadySeen();
}
// verify ECDSA signatures on (root, validUntil) and ensure that the root group is successful
{
// verify sigs and count number of signers in each group
Signer memory signer;
address prevAddress = address(0x0);
uint8[NUM_GROUPS] memory groupVoteCounts; // number of votes per group
for (uint256 i = 0; i < signatures.length; i++) {
Signature calldata sig = signatures[i];
address signerAddress = ECDSA.recover(signedHash, sig.v, sig.r, sig.s);
// the off-chain system is required to sort the signatures by the
// signer address in an increasing order
if (prevAddress >= signerAddress) {
revert SignersAddressesMustBeStrictlyIncreasing();
}
prevAddress = signerAddress;
signer = s_signers[signerAddress];
if (signer.addr != signerAddress) {
revert InvalidSigner();
}
uint8 group = signer.group;
while (true) {
groupVoteCounts[group]++;
if (groupVoteCounts[group] != s_config.groupQuorums[group]) {
// bail out unless we just hit the quorum. we only hit each quorum once,
// so we never move on to the parent of a group more than once.
break;
}
if (group == 0) {
// reached root
break;
}
group = s_config.groupParents[group];
}
}
// the group at the root of the tree (with index 0) determines whether the vote passed,
// we cannot proceed if it isn't configured with a valid (non-zero) quorum
if (s_config.groupQuorums[0] == 0) {
revert MissingConfig();
}
// did the root group reach its quorum?
if (groupVoteCounts[0] < s_config.groupQuorums[0]) {
revert InsufficientSigners();
}
}
if (validUntil < block.timestamp) {
revert ValidUntilHasAlreadyPassed();
}
{
// verify metadataProof
bytes32 hashedLeaf =
keccak256(abi.encode(MANY_CHAIN_MULTI_SIG_DOMAIN_SEPARATOR_METADATA, metadata));
if (!MerkleProof.verify(metadataProof, root, hashedLeaf)) {
revert ProofCannotBeVerified();
}
}
if (block.chainid != metadata.chainId) {
revert WrongChainId();
}
if (address(this) != metadata.multiSig) {
revert WrongMultiSig();
}
uint40 opCount = s_expiringRootAndOpCount.opCount;
// don't allow a new root to be set if there are still outstanding ops that have not been
// executed, unless overridePreviousRoot is set
if (opCount != s_rootMetadata.postOpCount && !metadata.overridePreviousRoot) {
revert PendingOps();
}
// the signers are responsible for tracking opCount offchain and ensuring that
// preOpCount equals to opCount
if (opCount != metadata.preOpCount) {
revert WrongPreOpCount();
}
if (metadata.preOpCount > metadata.postOpCount) {
revert WrongPostOpCount();
}
// done with validation, persist in in contract state
s_seenSignedHashes[signedHash] = true;
s_expiringRootAndOpCount = ExpiringRootAndOpCount({
root: root,
validUntil: validUntil,
opCount: metadata.preOpCount
});
s_rootMetadata = metadata;
emit NewRoot(root, validUntil, metadata);
}
/// @notice an op to be executed by the ManyChainMultiSig contract
///
/// @dev We need to be careful that abi.encode(LEAF_OP_DOMAIN_SEPARATOR, RootMetadata)
/// is greater than 64 bytes to prevent collisions with internal nodes in the Merkle tree. See
/// openzeppelin-contracts/contracts/utils/cryptography/MerkleProof.sol:15 for details.
struct Op {
uint256 chainId;
address multiSig;
uint40 nonce;
address to;
uint256 value;
bytes data;
}
/// @notice Execute the received op after verifying the proof of its inclusion in the
/// current Merkle tree. The op should be the next op according to the order
/// enforced by the merkle tree whose root is stored in s_expiringRootAndOpCount, i.e., the
/// nonce of the op should be equal to s_expiringRootAndOpCount.opCount.
///
/// @param op is Op to be executed
/// @param proof is the MerkleProof for the op's inclusion in the MerkleTree which its
/// root is the s_expiringRootAndOpCount.root.
///
/// @dev ANYONE can call this function! That's intentional. Callers can only execute verified,
/// ordered ops in the Merkle tree.
///
/// @dev we perform a raw call to each target. Raw calls to targets that don't have associated
/// contract code will always succeed regardless of data.
///
/// @dev the gas limit of the call can be freely determined by the caller of this function.
/// We expect callees to revert if they run out of gas.
function execute(Op calldata op, bytes32[] calldata proof) external payable {
ExpiringRootAndOpCount memory currentExpiringRootAndOpCount = s_expiringRootAndOpCount;
if (s_rootMetadata.postOpCount <= currentExpiringRootAndOpCount.opCount) {
revert PostOpCountReached();
}
if (op.chainId != block.chainid) {
revert WrongChainId();
}
if (op.multiSig != address(this)) {
revert WrongMultiSig();
}
if (block.timestamp > currentExpiringRootAndOpCount.validUntil) {
revert RootExpired();
}
if (op.nonce != currentExpiringRootAndOpCount.opCount) {
revert WrongNonce();
}
// verify that the op exists in the merkle tree
bytes32 hashedLeaf = keccak256(abi.encode(MANY_CHAIN_MULTI_SIG_DOMAIN_SEPARATOR_OP, op));
if (!MerkleProof.verify(proof, currentExpiringRootAndOpCount.root, hashedLeaf)) {
revert ProofCannotBeVerified();
}
// increase the counter *before* execution to prevent reentrancy issues
s_expiringRootAndOpCount.opCount = currentExpiringRootAndOpCount.opCount + 1;
_execute(op.to, op.value, op.data);
emit OpExecuted(op.nonce, op.to, op.data, op.value);
}
/// @notice sets a new s_config. If clearRoot is true, then it also invalidates
/// s_expiringRootAndOpCount.root.
///
/// @param signerAddresses holds the addresses of the active signers. The addresses must be in
/// ascending order.
/// @param signerGroups maps each signer to its group
/// @param groupQuorums holds the required number of valid signatures in each group.
/// A group i is called successful group if at least groupQuorum[i] distinct signers provide a
/// valid signature.
/// @param groupParents holds each group's parent. The groups must be arranged in a tree s.t.
/// group 0 is the root of the tree and the i-th group's parent has index j less than i.
/// Iff setRoot is called with a set of signatures that causes the root group to be successful,
/// setRoot allows a root to be set.
/// @param clearRoot, if set to true, invalidates the current root. This option is needed to
/// invalidate the current root, so to prevent further ops from being executed. This
/// might be used when the current root was signed under a loser group configuration or when
/// some previous signers aren't trusted any more.
function setConfig(
address[] calldata signerAddresses,
uint8[] calldata signerGroups,
uint8[NUM_GROUPS] calldata groupQuorums,
uint8[NUM_GROUPS] calldata groupParents,
bool clearRoot
) external onlyOwner {
if (signerAddresses.length == 0 || signerAddresses.length > MAX_NUM_SIGNERS) {
revert OutOfBoundsNumOfSigners();
}
if (signerAddresses.length != signerGroups.length) {
revert SignerGroupsLengthMismatch();
}
{
// validate group structure
// counts the number of children of each group
uint8[NUM_GROUPS] memory groupChildrenCounts;
// first, we count the signers as children
for (uint256 i = 0; i < signerGroups.length; i++) {
if (signerGroups[i] >= NUM_GROUPS) {
revert OutOfBoundsGroup();
}
groupChildrenCounts[signerGroups[i]]++;
}
// second, we iterate backwards so as to check each group and propagate counts from
// child group to parent groups up the tree to the root
for (uint256 j = 0; j < NUM_GROUPS; j++) {
uint256 i = NUM_GROUPS - 1 - j;
// ensure we have a well-formed group tree. the root should have itself as parent
if ((i != 0 && groupParents[i] >= i) || (i == 0 && groupParents[i] != 0)) {
revert GroupTreeNotWellFormed();
}
bool disabled = groupQuorums[i] == 0;
if (disabled) {
// a disabled group shouldn't have any children
if (0 < groupChildrenCounts[i]) {
revert SignerInDisabledGroup();
}
} else {
// ensure that the group quorum can be met
if (groupChildrenCounts[i] < groupQuorums[i]) {
revert OutOfBoundsGroupQuorum();
}
groupChildrenCounts[groupParents[i]]++;
// the above line clobbers groupChildrenCounts[0] in last iteration, don't use it after the loop ends
}
}
}
Signer[] memory oldSigners = s_config.signers;
// remove any old signer addresses
for (uint256 i = 0; i < oldSigners.length; i++) {
address oldSignerAddress = oldSigners[i].addr;
delete s_signers[oldSignerAddress];
s_config.signers.pop();
}
// we cannot just write s_config = Config({...}) because solc doesn't support that
assert(s_config.signers.length == 0);
s_config.groupQuorums = groupQuorums;
s_config.groupParents = groupParents;
// add new signers' addresses, we require that the signers' list be a strictly monotone
// increasing sequence
address prevSigner = address(0x0);
for (uint256 i = 0; i < signerAddresses.length; i++) {
if (prevSigner >= signerAddresses[i]) {
revert SignersAddressesMustBeStrictlyIncreasing();
}
Signer memory signer =
Signer({addr: signerAddresses[i], index: uint8(i), group: signerGroups[i]});
s_signers[signerAddresses[i]] = signer;
s_config.signers.push(signer);
prevSigner = signerAddresses[i];
}
if (clearRoot) {
// clearRoot is equivalent to overriding with a completely empty root
uint40 opCount = s_expiringRootAndOpCount.opCount;
s_expiringRootAndOpCount =
ExpiringRootAndOpCount({root: 0, validUntil: 0, opCount: opCount});
s_rootMetadata = RootMetadata({
chainId: block.chainid,
multiSig: address(this),
preOpCount: opCount,
postOpCount: opCount,
overridePreviousRoot: true
});
}
emit ConfigSet(s_config, clearRoot);
}
/// @notice Execute an op's call. Performs a raw call that always succeeds if the
/// target isn't a contract.
function _execute(address target, uint256 value, bytes calldata data) internal virtual {
(bool success, bytes memory ret) = target.call{value: value}(data);
if (!success) {
revert CallReverted(ret);
}
}
/*
* Getters
*/
function getConfig() public view returns (Config memory) {
return s_config;
}
function getOpCount() public view returns (uint40) {
return s_expiringRootAndOpCount.opCount;
}
function getRoot() public view returns (bytes32 root, uint32 validUntil) {
ExpiringRootAndOpCount memory currentRootAndOpCount = s_expiringRootAndOpCount;
return (currentRootAndOpCount.root, currentRootAndOpCount.validUntil);
}
function getRootMetadata() public view returns (RootMetadata memory) {
return s_rootMetadata;
}
/*
* Events and Errors
*/
/// @notice Emitted when a new root is set.
event NewRoot(bytes32 indexed root, uint32 validUntil, RootMetadata metadata);
/// @notice Emitted when a new config is set.
event ConfigSet(Config config, bool isRootCleared);
/// @notice Emitted when an op gets successfully executed.
event OpExecuted(uint40 indexed nonce, address to, bytes data, uint256 value);
/// @notice Thrown when number of signers is 0 or greater than MAX_NUM_SIGNERS.
error OutOfBoundsNumOfSigners();
/// @notice Thrown when signerAddresses and signerGroups have different lengths.
error SignerGroupsLengthMismatch();
/// @notice Thrown when number of some signer's group is greater than (NUM_GROUPS-1).
error OutOfBoundsGroup();
/// @notice Thrown when the group tree isn't well-formed.
error GroupTreeNotWellFormed();
/// @notice Thrown when the quorum of some group is larger than the number of signers in it.
error OutOfBoundsGroupQuorum();
/// @notice Thrown when a disabled group contains a signer.
error SignerInDisabledGroup();
/// @notice Thrown when the signers' addresses are not a strictly increasing monotone sequence.
/// Prevents signers from including more than one signature.
error SignersAddressesMustBeStrictlyIncreasing();
/// @notice Thrown when the signature corresponds to invalid signer.
error InvalidSigner();
/// @notice Thrown when there is no sufficient set of valid signatures provided to make the
/// root group successful.
error InsufficientSigners();
/// @notice Thrown when attempt to set metadata or execute op for another chain.
error WrongChainId();
/// @notice Thrown when the multiSig address in metadata or op is
/// incompatible with the address of this contract.
error WrongMultiSig();
/// @notice Thrown when the preOpCount <= postOpCount invariant is violated.
error WrongPostOpCount();
/// @notice Thrown when attempting to set a new root while there are still pending ops
/// from the previous root without explicitly overriding it.
error PendingOps();
/// @notice Thrown when preOpCount in metadata is incompatible with the current opCount.
error WrongPreOpCount();
/// @notice Thrown when the provided merkle proof cannot be verified.
error ProofCannotBeVerified();
/// @notice Thrown when attempt to execute an op after
/// s_expiringRootAndOpCount.validUntil has passed.
error RootExpired();
/// @notice Thrown when attempt to bypass the enforced ops' order in the merkle tree or
/// re-execute an op.
error WrongNonce();
/// @notice Thrown when attempting to execute an op even though opCount equals
/// metadata.postOpCount.
error PostOpCountReached();
/// @notice Thrown when the underlying call in _execute() reverts.
error CallReverted(bytes error);
/// @notice Thrown when attempt to set past validUntil for the root.
error ValidUntilHasAlreadyPassed();
/// @notice Thrown when setRoot() is called before setting a config.
error MissingConfig();
/// @notice Thrown when attempt to set the same (root, validUntil) in setRoot().
error SignedHashAlreadySeen();
}Contract Security Audit
- No Contract Security Audit Submitted- Submit Audit Here
Contract ABI
API[{"inputs":[{"internalType":"bytes","name":"error","type":"bytes"}],"name":"CallReverted","type":"error"},{"inputs":[],"name":"GroupTreeNotWellFormed","type":"error"},{"inputs":[],"name":"InsufficientSigners","type":"error"},{"inputs":[],"name":"InvalidSigner","type":"error"},{"inputs":[],"name":"MissingConfig","type":"error"},{"inputs":[],"name":"OutOfBoundsGroup","type":"error"},{"inputs":[],"name":"OutOfBoundsGroupQuorum","type":"error"},{"inputs":[],"name":"OutOfBoundsNumOfSigners","type":"error"},{"inputs":[],"name":"PendingOps","type":"error"},{"inputs":[],"name":"PostOpCountReached","type":"error"},{"inputs":[],"name":"ProofCannotBeVerified","type":"error"},{"inputs":[],"name":"RootExpired","type":"error"},{"inputs":[],"name":"SignedHashAlreadySeen","type":"error"},{"inputs":[],"name":"SignerGroupsLengthMismatch","type":"error"},{"inputs":[],"name":"SignerInDisabledGroup","type":"error"},{"inputs":[],"name":"SignersAddressesMustBeStrictlyIncreasing","type":"error"},{"inputs":[],"name":"ValidUntilHasAlreadyPassed","type":"error"},{"inputs":[],"name":"WrongChainId","type":"error"},{"inputs":[],"name":"WrongMultiSig","type":"error"},{"inputs":[],"name":"WrongNonce","type":"error"},{"inputs":[],"name":"WrongPostOpCount","type":"error"},{"inputs":[],"name":"WrongPreOpCount","type":"error"},{"anonymous":false,"inputs":[{"components":[{"components":[{"internalType":"address","name":"addr","type":"address"},{"internalType":"uint8","name":"index","type":"uint8"},{"internalType":"uint8","name":"group","type":"uint8"}],"internalType":"struct ManyChainMultiSig.Signer[]","name":"signers","type":"tuple[]"},{"internalType":"uint8[32]","name":"groupQuorums","type":"uint8[32]"},{"internalType":"uint8[32]","name":"groupParents","type":"uint8[32]"}],"indexed":false,"internalType":"struct ManyChainMultiSig.Config","name":"config","type":"tuple"},{"indexed":false,"internalType":"bool","name":"isRootCleared","type":"bool"}],"name":"ConfigSet","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"bytes32","name":"root","type":"bytes32"},{"indexed":false,"internalType":"uint32","name":"validUntil","type":"uint32"},{"components":[{"internalType":"uint256","name":"chainId","type":"uint256"},{"internalType":"address","name":"multiSig","type":"address"},{"internalType":"uint40","name":"preOpCount","type":"uint40"},{"internalType":"uint40","name":"postOpCount","type":"uint40"},{"internalType":"bool","name":"overridePreviousRoot","type":"bool"}],"indexed":false,"internalType":"struct ManyChainMultiSig.RootMetadata","name":"metadata","type":"tuple"}],"name":"NewRoot","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"uint40","name":"nonce","type":"uint40"},{"indexed":false,"internalType":"address","name":"to","type":"address"},{"indexed":false,"internalType":"bytes","name":"data","type":"bytes"},{"indexed":false,"internalType":"uint256","name":"value","type":"uint256"}],"name":"OpExecuted","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"previousOwner","type":"address"},{"indexed":true,"internalType":"address","name":"newOwner","type":"address"}],"name":"OwnershipTransferStarted","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"previousOwner","type":"address"},{"indexed":true,"internalType":"address","name":"newOwner","type":"address"}],"name":"OwnershipTransferred","type":"event"},{"inputs":[],"name":"MAX_NUM_SIGNERS","outputs":[{"internalType":"uint8","name":"","type":"uint8"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"NUM_GROUPS","outputs":[{"internalType":"uint8","name":"","type":"uint8"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"acceptOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"components":[{"internalType":"uint256","name":"chainId","type":"uint256"},{"internalType":"address","name":"multiSig","type":"address"},{"internalType":"uint40","name":"nonce","type":"uint40"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"value","type":"uint256"},{"internalType":"bytes","name":"data","type":"bytes"}],"internalType":"struct ManyChainMultiSig.Op","name":"op","type":"tuple"},{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"}],"name":"execute","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"getConfig","outputs":[{"components":[{"components":[{"internalType":"address","name":"addr","type":"address"},{"internalType":"uint8","name":"index","type":"uint8"},{"internalType":"uint8","name":"group","type":"uint8"}],"internalType":"struct ManyChainMultiSig.Signer[]","name":"signers","type":"tuple[]"},{"internalType":"uint8[32]","name":"groupQuorums","type":"uint8[32]"},{"internalType":"uint8[32]","name":"groupParents","type":"uint8[32]"}],"internalType":"struct ManyChainMultiSig.Config","name":"","type":"tuple"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"getOpCount","outputs":[{"internalType":"uint40","name":"","type":"uint40"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"getRoot","outputs":[{"internalType":"bytes32","name":"root","type":"bytes32"},{"internalType":"uint32","name":"validUntil","type":"uint32"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"getRootMetadata","outputs":[{"components":[{"internalType":"uint256","name":"chainId","type":"uint256"},{"internalType":"address","name":"multiSig","type":"address"},{"internalType":"uint40","name":"preOpCount","type":"uint40"},{"internalType":"uint40","name":"postOpCount","type":"uint40"},{"internalType":"bool","name":"overridePreviousRoot","type":"bool"}],"internalType":"struct ManyChainMultiSig.RootMetadata","name":"","type":"tuple"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"owner","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"pendingOwner","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address[]","name":"signerAddresses","type":"address[]"},{"internalType":"uint8[]","name":"signerGroups","type":"uint8[]"},{"internalType":"uint8[32]","name":"groupQuorums","type":"uint8[32]"},{"internalType":"uint8[32]","name":"groupParents","type":"uint8[32]"},{"internalType":"bool","name":"clearRoot","type":"bool"}],"name":"setConfig","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"root","type":"bytes32"},{"internalType":"uint32","name":"validUntil","type":"uint32"},{"components":[{"internalType":"uint256","name":"chainId","type":"uint256"},{"internalType":"address","name":"multiSig","type":"address"},{"internalType":"uint40","name":"preOpCount","type":"uint40"},{"internalType":"uint40","name":"postOpCount","type":"uint40"},{"internalType":"bool","name":"overridePreviousRoot","type":"bool"}],"internalType":"struct ManyChainMultiSig.RootMetadata","name":"metadata","type":"tuple"},{"internalType":"bytes32[]","name":"metadataProof","type":"bytes32[]"},{"components":[{"internalType":"uint8","name":"v","type":"uint8"},{"internalType":"bytes32","name":"r","type":"bytes32"},{"internalType":"bytes32","name":"s","type":"bytes32"}],"internalType":"struct ManyChainMultiSig.Signature[]","name":"signatures","type":"tuple[]"}],"name":"setRoot","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"newOwner","type":"address"}],"name":"transferOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"stateMutability":"payable","type":"receive"}]Contract Creation Code
60806040523480156200001157600080fd5b506200001d3362000023565b62000091565b600180546001600160a01b03191690556200003e8162000041565b50565b600080546001600160a01b038381166001600160a01b0319831681178455604051919092169283917f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e09190a35050565b61264380620000a16000396000f3fe6080604052600436106100e15760003560e01c8063846c67ef1161007f578063b759d68511610059578063b759d68514610345578063c3f909d414610358578063e30c39781461037a578063f2fde38b1461039857600080fd5b8063846c67ef146102de5780638da5cb5b146102fe578063a76f55981461033057600080fd5b80636b45fb3e116100bb5780636b45fb3e146101a3578063715018a61461029257806379ba5097146102a95780637cc38b28146102be57600080fd5b80635a2519ef146100ed5780635ca1e16514610119578063627e8a3b1461016f57600080fd5b366100e857005b600080fd5b3480156100f957600080fd5b50610102602081565b60405160ff90911681526020015b60405180910390f35b34801561012557600080fd5b506040805160608101825260075480825260085463ffffffff81166020808501829052600160201b90920464ffffffffff1693850193909352835191825281019190915201610110565b34801561017b57600080fd5b50600854600160201b900464ffffffffff1660405164ffffffffff9091168152602001610110565b3480156101af57600080fd5b5061023b6040805160a081018252600080825260208201819052918101829052606081018290526080810191909152506040805160a0810182526009548152600a546001600160a01b0381166020830152600160a01b810464ffffffffff90811693830193909352600160c81b81049092166060820152600160f01b90910460ff161515608082015290565b6040516101109190815181526020808301516001600160a01b03169082015260408083015164ffffffffff908116918301919091526060808401519091169082015260809182015115159181019190915260a00190565b34801561029e57600080fd5b506102a76103b8565b005b3480156102b557600080fd5b506102a76103cc565b3480156102ca57600080fd5b506102a76102d9366004611b5b565b61044b565b3480156102ea57600080fd5b506102a76102f9366004611c5f565b610a2f565b34801561030a57600080fd5b506000546001600160a01b03165b6040516001600160a01b039091168152602001610110565b34801561033c57600080fd5b5061010260c881565b6102a7610353366004611d0a565b6111a2565b34801561036457600080fd5b5061036d61144d565b6040516101109190611dab565b34801561038657600080fd5b506001546001600160a01b0316610318565b3480156103a457600080fd5b506102a76103b3366004611e5f565b61158f565b6103c0611600565b6103ca600061165a565b565b60015433906001600160a01b0316811461043f5760405162461bcd60e51b815260206004820152602960248201527f4f776e61626c6532537465703a2063616c6c6572206973206e6f7420746865206044820152683732bb9037bbb732b960b91b60648201526084015b60405180910390fd5b6104488161165a565b50565b60006104bb888860405160200161047292919091825263ffffffff16602082015260400190565b604051602081830303815290604052805190602001207f19457468657265756d205369676e6564204d6573736167653a0a3332000000006000908152601c91909152603c902090565b60008181526006602052604090205490915060ff16156104ee576040516348c2688b60e01b815260040160405180910390fd5b6040805160608101825260008082526020820181905291810182905290610513611a19565b60005b858110156106de573687878381811061053157610531611e7c565b6060029190910191506000905061055e8761054f6020850185611e92565b84602001358560400135611673565b9050806001600160a01b0316856001600160a01b03161061059257604051630946dd8160e31b815260040160405180910390fd5b6001600160a01b038082166000818152600260209081526040918290208251606081018452905494851680825260ff600160a01b8704811693830193909352600160a81b90950490911691810191909152975091955085911461060857604051632057875960e21b815260040160405180910390fd5b60408601515b848160ff166020811061062357610623611e7c565b6020020180519061063382611ecb565b60ff9081169091526004915082166020811061065157610651611e7c565b602091828204019190069054906101000a900460ff1660ff16858260ff166020811061067f5761067f611e7c565b602002015160ff16036106c85760ff8116156106c857600560ff8216602081106106ab576106ab611e7c565b602081049091015460ff601f9092166101000a900416905061060e565b50505080806106d690611eea565b915050610516565b5060045460ff1660000361070557604051635530c2e560e11b815260040160405180910390fd5b600454815160ff91821691161015610730576040516361774dcf60e11b815260040160405180910390fd5b505050428763ffffffff16101561075a5760405163582bd22960e11b815260040160405180910390fd5b60007fe6b82be989101b4eb519770114b997b97b3c8707515286748a871717f0e4ea1c8760405160200161078f929190611f82565b6040516020818303038152906040528051906020012090506107e78686808060200260200160405190810160405280939291908181526020018383602002808284376000920191909152508d925085915061169b9050565b6108035760405162948a8760e61b815260040160405180910390fd5b5046863514610824576040516217e1ef60ea1b815260040160405180910390fd5b6108346040870160208801611e5f565b6001600160a01b0316306001600160a01b03161461086557604051639a84601560e01b815260040160405180910390fd5b600854600a5464ffffffffff600160201b909204821691600160c81b9091041681148015906108a1575061089f60a0880160808901611f96565b155b156108bf57604051633230825b60e01b815260040160405180910390fd5b6108cf6060880160408901611fb3565b64ffffffffff168164ffffffffff16146108fc5760405163a255a76360e01b815260040160405180910390fd5b61090c6080880160608901611fb3565b64ffffffffff166109236060890160408a01611fb3565b64ffffffffff161115610949576040516318c26a5f60e31b815260040160405180910390fd5b600082815260066020908152604091829020805460ff191660011790558151606080820184528c825263ffffffff8c1692820192909252918281019161099491908b01908b01611fb3565b64ffffffffff9081169091528151600755602082015160088054604090940151909216600160201b0268ffffffffffffffffff1990931663ffffffff909116179190911790558660096109e78282611fd0565b905050887f7ea643ae44677f24e0d6f40168893712daaf729b0a38fe7702d21cb544c841018989604051610a1c929190612067565b60405180910390a2505050505050505050565b610a37611600565b851580610a44575060c886115b15610a6257604051633c3b072960e21b815260040160405180910390fd5b858414610a8257604051630f1f305360e41b815260040160405180910390fd5b610a8a611a19565b60005b85811015610b42576020878783818110610aa957610aa9611e7c565b9050602002016020810190610abe9190611e92565b60ff1610610adf57604051635cd7472960e11b815260040160405180910390fd5b81878783818110610af257610af2611e7c565b9050602002016020810190610b079190611e92565b60ff1660208110610b1a57610b1a611e7c565b60200201805190610b2a82611ecb565b60ff1690525080610b3a81611eea565b915050610a8d565b5060005b6020811015610d3457600081610b5e60016020612081565b60ff16610b6b919061209a565b90508015801590610ba3575080858260208110610b8a57610b8a611e7c565b602002016020810190610b9d9190611e92565b60ff1610155b80610bdd575080158015610bdd5750848160208110610bc457610bc4611e7c565b602002016020810190610bd79190611e92565b60ff1615155b15610bfe576040516001627ce2ed60e11b0319815260040160405180910390fd5b6000868260208110610c1257610c12611e7c565b602002016020810190610c259190611e92565b60ff161590508015610c6e57838260208110610c4357610c43611e7c565b602002015160ff1615610c6957604051638db4e75d60e01b815260040160405180910390fd5b610d1f565b868260208110610c8057610c80611e7c565b602002016020810190610c939190611e92565b60ff16848360208110610ca857610ca8611e7c565b602002015160ff161015610ccf57604051635d8009b760e11b815260040160405180910390fd5b83868360208110610ce257610ce2611e7c565b602002016020810190610cf59190611e92565b60ff1660208110610d0857610d08611e7c565b60200201805190610d1882611ecb565b60ff169052505b50508080610d2c90611eea565b915050610b46565b505060006003600001805480602002602001604051908101604052809291908181526020016000905b82821015610db457600084815260209081902060408051606081018252918501546001600160a01b038116835260ff600160a01b8204811684860152600160a81b9091041690820152825260019092019101610d5d565b50505050905060005b8151811015610e58576000828281518110610dda57610dda611e7c565b602090810291909101810151516001600160a01b03811660009081526002909252604090912080546001600160b01b0319169055600380549192509080610e2357610e236120ad565b600082815260209020810160001990810180546001600160b01b03191690550190555080610e5081611eea565b915050610dbd565b5060035415610e6957610e696120c3565b610e766004856020611a38565b50610e846005846020611a38565b506000805b8881101561108c57898982818110610ea357610ea3611e7c565b9050602002016020810190610eb89190611e5f565b6001600160a01b0316826001600160a01b031610610ee957604051630946dd8160e31b815260040160405180910390fd5b600060405180606001604052808c8c85818110610f0857610f08611e7c565b9050602002016020810190610f1d9190611e5f565b6001600160a01b031681526020018360ff1681526020018a8a85818110610f4657610f46611e7c565b9050602002016020810190610f5b9190611e92565b60ff169052905080600260008d8d86818110610f7957610f79611e7c565b9050602002016020810190610f8e9190611e5f565b6001600160a01b0390811682526020808301939093526040918201600090812085518154878701519786015160ff908116600160a81b90810260ff60a81b199a8316600160a01b9081026001600160a81b0319958616968a1696909617959095178b161790945560038054600181018255955289517fc2575a0e9e593c00f959f8c92f12db2869c3395a3b0502d05e2516446f71f85b9095018054988b0151978b01518216909402961690910295169190921617929092179092169190911790558a8a8381811061106157611061611e7c565b90506020020160208101906110769190611e5f565b925050808061108490611eea565b915050610e89565b50821561115d5760088054604080516060808201835260008083526020808401829052600160201b80870464ffffffffff1694860185905260079290925568ffffffffffffffffff1990951690830217909455815160a08101835246808252309482018590529281018290529384018190526001608090940193909352600955600a8054600160f01b6001600160c81b031990911664ffffffffff60a01b1990931692909217600160a01b84021765ffffffffffff60c81b1916600160c81b90930260ff60f01b1916929092171790555b7f0a4974ad206b9c736f9ab2feac1c9b1d043fe4ef377c70ae45659f2ef089f03e60038460405161118f929190612361565b60405180910390a1505050505050505050565b60408051606081018252600754815260085463ffffffff8116602083015264ffffffffff600160201b9091048116928201839052600a549192600160c81b9092041611611202576040516315b6266360e31b815260040160405180910390fd5b83354614611222576040516217e1ef60ea1b815260040160405180910390fd5b306112336040860160208701611e5f565b6001600160a01b03161461125a57604051639a84601560e01b815260040160405180910390fd5b806020015163ffffffff16421115611285576040516309ba674360e41b815260040160405180910390fd5b806040015164ffffffffff168460400160208101906112a49190611fb3565b64ffffffffff16146112c95760405163d9c6386f60e01b815260040160405180910390fd5b60007f08d275622006c4ca82d03f498e90163cafd53c663a48470c3b52ac8bfbd9f52c856040516020016112fe92919061242e565b604051602081830303815290604052805190602001209050611356848480806020026020016040519081016040528093929190818152602001838360200280828437600092019190915250508551915084905061169b565b6113725760405162948a8760e61b815260040160405180910390fd5b60408201516113829060016124f7565b6008805464ffffffffff92909216600160201b0268ffffffffff00000000199092169190911790556113d46113bd6080870160608801611e5f565b60808701356113cf60a089018961251c565b6116b3565b6113e46060860160408701611fb3565b64ffffffffff167f87d58fdd48be753fb9ef4ec8a5895086c401506da8b4d752abc90602c3e62d1d61141c6080880160608901611e5f565b61142960a089018961251c565b896080013560405161143e9493929190612563565b60405180910390a25050505050565b611455611ace565b604080516003805460806020820284018101909452606083018181529293919284929091849160009085015b828210156114d857600084815260209081902060408051606081018252918501546001600160a01b038116835260ff600160a01b8204811684860152600160a81b9091041690820152825260019092019101611481565b50505090825250604080516104008101918290526020928301929091600185019190826000855b825461010083900a900460ff168152602060019283018181049485019490930390920291018084116114ff575050509284525050604080516104008101918290526020938401939092506002850191826000855b825461010083900a900460ff16815260206001928301818104948501949093039092029101808411611553579050505050505081525050905090565b611597611600565b600180546001600160a01b0383166001600160a01b031990911681179091556115c86000546001600160a01b031690565b6001600160a01b03167f38d16b8cac22d99fc7c124b9cd0de2d3fa1faef420bfe791d8c362d765e2270060405160405180910390a350565b6000546001600160a01b031633146103ca5760405162461bcd60e51b815260206004820181905260248201527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e65726044820152606401610436565b600180546001600160a01b031916905561044881611740565b600080600061168487878787611790565b9150915061169181611854565b5095945050505050565b6000826116a8858461199e565b1490505b9392505050565b600080856001600160a01b03168585856040516116d1929190612599565b60006040518083038185875af1925050503d806000811461170e576040519150601f19603f3d011682016040523d82523d6000602084013e611713565b606091505b50915091508161173857806040516370de1b4b60e01b815260040161043691906125a9565b505050505050565b600080546001600160a01b038381166001600160a01b0319831681178455604051919092169283917f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e09190a35050565b6000807f7fffffffffffffffffffffffffffffff5d576e7357a4501ddfe92f46681b20a08311156117c7575060009050600361184b565b6040805160008082526020820180845289905260ff881692820192909252606081018690526080810185905260019060a0016020604051602081039080840390855afa15801561181b573d6000803e3d6000fd5b5050604051601f1901519150506001600160a01b0381166118445760006001925092505061184b565b9150600090505b94509492505050565b6000816004811115611868576118686125f7565b036118705750565b6001816004811115611884576118846125f7565b036118d15760405162461bcd60e51b815260206004820152601860248201527f45434453413a20696e76616c6964207369676e617475726500000000000000006044820152606401610436565b60028160048111156118e5576118e56125f7565b036119325760405162461bcd60e51b815260206004820152601f60248201527f45434453413a20696e76616c6964207369676e6174757265206c656e677468006044820152606401610436565b6003816004811115611946576119466125f7565b036104485760405162461bcd60e51b815260206004820152602260248201527f45434453413a20696e76616c6964207369676e6174757265202773272076616c604482015261756560f01b6064820152608401610436565b600081815b84518110156119e3576119cf828683815181106119c2576119c2611e7c565b60200260200101516119ed565b9150806119db81611eea565b9150506119a3565b5090505b92915050565b6000818310611a095760008281526020849052604090206116ac565b5060009182526020526040902090565b6040518061040001604052806020906020820280368337509192915050565b600183019183908215611abe5791602002820160005b83821115611a8f57833560ff1683826101000a81548160ff021916908360ff1602179055509260200192600101602081600001049283019260010302611a4e565b8015611abc5782816101000a81549060ff0219169055600101602081600001049283019260010302611a8f565b505b50611aca929150611afa565b5090565b604051806060016040528060608152602001611ae8611a19565b8152602001611af5611a19565b905290565b5b80821115611aca5760008155600101611afb565b60008083601f840112611b2157600080fd5b50813567ffffffffffffffff811115611b3957600080fd5b6020830191508360208260051b8501011115611b5457600080fd5b9250929050565b6000806000806000806000878903610120811215611b7857600080fd5b88359750602089013563ffffffff81168114611b9357600080fd5b965060a0603f1982011215611ba757600080fd5b5060408801945060e088013567ffffffffffffffff80821115611bc957600080fd5b611bd58b838c01611b0f565b90965094506101008a0135915080821115611bef57600080fd5b818a0191508a601f830112611c0357600080fd5b813581811115611c1257600080fd5b8b6020606083028501011115611c2757600080fd5b60208301945080935050505092959891949750929550565b8061040081018310156119e757600080fd5b801515811461044857600080fd5b6000806000806000806000610860888a031215611c7b57600080fd5b873567ffffffffffffffff80821115611c9357600080fd5b611c9f8b838c01611b0f565b909950975060208a0135915080821115611cb857600080fd5b50611cc58a828b01611b0f565b9096509450611cd990508960408a01611c3f565b9250611ce9896104408a01611c3f565b9150610840880135611cfa81611c51565b8091505092959891949750929550565b600080600060408486031215611d1f57600080fd5b833567ffffffffffffffff80821115611d3757600080fd5b9085019060c08288031215611d4b57600080fd5b90935060208501359080821115611d6157600080fd5b50611d6e86828701611b0f565b9497909650939450505050565b8060005b6020808210611d8e5750611da5565b825160ff1685529384019390910190600101611d7f565b50505050565b6020808252825161082083830152805161084084018190526000929182019083906108608601905b80831015611e1857835180516001600160a01b031683528581015160ff9081168785015260409182015116908301529284019260019290920191606090910190611dd3565b509286015192611e2b6040870185611d7b565b60408701519350611e40610440870185611d7b565b9695505050505050565b6001600160a01b038116811461044857600080fd5b600060208284031215611e7157600080fd5b81356116ac81611e4a565b634e487b7160e01b600052603260045260246000fd5b600060208284031215611ea457600080fd5b813560ff811681146116ac57600080fd5b634e487b7160e01b600052601160045260246000fd5b600060ff821660ff8103611ee157611ee1611eb5565b60010192915050565b600060018201611efc57611efc611eb5565b5060010190565b64ffffffffff8116811461044857600080fd5b803582526020810135611f2881611e4a565b6001600160a01b031660208301526040810135611f4481611f03565b64ffffffffff9081166040840152606082013590611f6182611f03565b1660608301526080810135611f7581611c51565b8015156080840152505050565b82815260c081016116ac6020830184611f16565b600060208284031215611fa857600080fd5b81356116ac81611c51565b600060208284031215611fc557600080fd5b81356116ac81611f03565b81358155600181016020830135611fe681611e4a565b81546040850135611ff681611f03565b606086013561200481611f03565b608087013561201281611c51565b60c89190911b64ffffffffff60c81b1660a09290921b64ffffffffff60a01b166001600160f81b0319939093166001600160a01b039490941693909317919091171790151560f01b60ff60f01b161790555050565b63ffffffff8316815260c081016116ac6020830184611f16565b60ff82811682821603908111156119e7576119e7611eb5565b818103818111156119e7576119e7611eb5565b634e487b7160e01b600052603160045260246000fd5b634e487b7160e01b600052600160045260246000fd5b8060005b602080601f8301106120ef5750611da5565b825460ff8082168752600882901c8116838801526040612118818901838560101c1660ff169052565b606061212d818a01848660181c1660ff169052565b6080612141818b018587891c1660ff169052565b60a09550612158868b01858760281c1660ff169052565b60c061216d818c01868860301c1660ff169052565b60e0612182818d01878960381c1660ff169052565b60ff87861c8716166101008d01526121a56101208d01878960481c1660ff169052565b6121ba6101408d01878960501c1660ff169052565b6121cf6101608d01878960581c1660ff169052565b60ff87851c8716166101808d01526121f26101a08d01878960681c1660ff169052565b6122076101c08d01878960701c1660ff169052565b61221c6101e08d01878960781c1660ff169052565b60ff87841c8716166102008d015261223f6102208d01878960881c1660ff169052565b6122546102408d01878960901c1660ff169052565b6122696102608d01878960981c1660ff169052565b60ff87891c8716166102808d015261228c6102a08d01878960a81c1660ff169052565b6122a16102c08d01878960b01c1660ff169052565b6122b66102e08d01878960b81c1660ff169052565b60ff87831c8716166103008d01526122d96103208d01878960c81c1660ff169052565b6122ee6103408d01878960d01c1660ff169052565b6123036103608d01878960d81c1660ff169052565b60ff87821c8716166103808d0152505050505061232b6103a08801828460e81c1660ff169052565b6123406103c08801828460f01c1660ff169052565b5060f81c6103e08601525061040090930192600191909101906020016120dd565b600060408083526108608301610820828501528086548083526108808601915087600052602092508260002060005b828110156123d05781546001600160a01b038116855260ff60a082901c81168787015260a89190911c168685015260609093019260019182019101612390565b5050506123e360608601600189016120d9565b6123f46104608601600289016120d9565b941515930192909252509092915050565b81835281816020850137506000828201602090810191909152601f909101601f19169091010190565b82815260406020820152813560408201526000602083013561244f81611e4a565b6001600160a01b03908116606084015260408401359061246e82611f03565b64ffffffffff821660808501526060850135915061248b82611e4a565b1660a083810191909152608084013560c084015283013536849003601e190181126124b557600080fd5b830160208101903567ffffffffffffffff8111156124d257600080fd5b8036038213156124e157600080fd5b60c060e0850152611e4061010085018284612405565b64ffffffffff81811683821601908082111561251557612515611eb5565b5092915050565b6000808335601e1984360301811261253357600080fd5b83018035915067ffffffffffffffff82111561254e57600080fd5b602001915036819003821315611b5457600080fd5b6001600160a01b03851681526060602082018190526000906125889083018587612405565b905082604083015295945050505050565b8183823760009101908152919050565b600060208083528351808285015260005b818110156125d6578581018301518582016040015282016125ba565b506000604082860101526040601f19601f8301168501019250505092915050565b634e487b7160e01b600052602160045260246000fdfea2646970667358221220789e10e5d6588dc4b26dba62aaa06971ed6ac6cbd43499f78a57e1d8415d671c64736f6c63430008130033
Deployed Bytecode
0x6080604052600436106100e15760003560e01c8063846c67ef1161007f578063b759d68511610059578063b759d68514610345578063c3f909d414610358578063e30c39781461037a578063f2fde38b1461039857600080fd5b8063846c67ef146102de5780638da5cb5b146102fe578063a76f55981461033057600080fd5b80636b45fb3e116100bb5780636b45fb3e146101a3578063715018a61461029257806379ba5097146102a95780637cc38b28146102be57600080fd5b80635a2519ef146100ed5780635ca1e16514610119578063627e8a3b1461016f57600080fd5b366100e857005b600080fd5b3480156100f957600080fd5b50610102602081565b60405160ff90911681526020015b60405180910390f35b34801561012557600080fd5b506040805160608101825260075480825260085463ffffffff81166020808501829052600160201b90920464ffffffffff1693850193909352835191825281019190915201610110565b34801561017b57600080fd5b50600854600160201b900464ffffffffff1660405164ffffffffff9091168152602001610110565b3480156101af57600080fd5b5061023b6040805160a081018252600080825260208201819052918101829052606081018290526080810191909152506040805160a0810182526009548152600a546001600160a01b0381166020830152600160a01b810464ffffffffff90811693830193909352600160c81b81049092166060820152600160f01b90910460ff161515608082015290565b6040516101109190815181526020808301516001600160a01b03169082015260408083015164ffffffffff908116918301919091526060808401519091169082015260809182015115159181019190915260a00190565b34801561029e57600080fd5b506102a76103b8565b005b3480156102b557600080fd5b506102a76103cc565b3480156102ca57600080fd5b506102a76102d9366004611b5b565b61044b565b3480156102ea57600080fd5b506102a76102f9366004611c5f565b610a2f565b34801561030a57600080fd5b506000546001600160a01b03165b6040516001600160a01b039091168152602001610110565b34801561033c57600080fd5b5061010260c881565b6102a7610353366004611d0a565b6111a2565b34801561036457600080fd5b5061036d61144d565b6040516101109190611dab565b34801561038657600080fd5b506001546001600160a01b0316610318565b3480156103a457600080fd5b506102a76103b3366004611e5f565b61158f565b6103c0611600565b6103ca600061165a565b565b60015433906001600160a01b0316811461043f5760405162461bcd60e51b815260206004820152602960248201527f4f776e61626c6532537465703a2063616c6c6572206973206e6f7420746865206044820152683732bb9037bbb732b960b91b60648201526084015b60405180910390fd5b6104488161165a565b50565b60006104bb888860405160200161047292919091825263ffffffff16602082015260400190565b604051602081830303815290604052805190602001207f19457468657265756d205369676e6564204d6573736167653a0a3332000000006000908152601c91909152603c902090565b60008181526006602052604090205490915060ff16156104ee576040516348c2688b60e01b815260040160405180910390fd5b6040805160608101825260008082526020820181905291810182905290610513611a19565b60005b858110156106de573687878381811061053157610531611e7c565b6060029190910191506000905061055e8761054f6020850185611e92565b84602001358560400135611673565b9050806001600160a01b0316856001600160a01b03161061059257604051630946dd8160e31b815260040160405180910390fd5b6001600160a01b038082166000818152600260209081526040918290208251606081018452905494851680825260ff600160a01b8704811693830193909352600160a81b90950490911691810191909152975091955085911461060857604051632057875960e21b815260040160405180910390fd5b60408601515b848160ff166020811061062357610623611e7c565b6020020180519061063382611ecb565b60ff9081169091526004915082166020811061065157610651611e7c565b602091828204019190069054906101000a900460ff1660ff16858260ff166020811061067f5761067f611e7c565b602002015160ff16036106c85760ff8116156106c857600560ff8216602081106106ab576106ab611e7c565b602081049091015460ff601f9092166101000a900416905061060e565b50505080806106d690611eea565b915050610516565b5060045460ff1660000361070557604051635530c2e560e11b815260040160405180910390fd5b600454815160ff91821691161015610730576040516361774dcf60e11b815260040160405180910390fd5b505050428763ffffffff16101561075a5760405163582bd22960e11b815260040160405180910390fd5b60007fe6b82be989101b4eb519770114b997b97b3c8707515286748a871717f0e4ea1c8760405160200161078f929190611f82565b6040516020818303038152906040528051906020012090506107e78686808060200260200160405190810160405280939291908181526020018383602002808284376000920191909152508d925085915061169b9050565b6108035760405162948a8760e61b815260040160405180910390fd5b5046863514610824576040516217e1ef60ea1b815260040160405180910390fd5b6108346040870160208801611e5f565b6001600160a01b0316306001600160a01b03161461086557604051639a84601560e01b815260040160405180910390fd5b600854600a5464ffffffffff600160201b909204821691600160c81b9091041681148015906108a1575061089f60a0880160808901611f96565b155b156108bf57604051633230825b60e01b815260040160405180910390fd5b6108cf6060880160408901611fb3565b64ffffffffff168164ffffffffff16146108fc5760405163a255a76360e01b815260040160405180910390fd5b61090c6080880160608901611fb3565b64ffffffffff166109236060890160408a01611fb3565b64ffffffffff161115610949576040516318c26a5f60e31b815260040160405180910390fd5b600082815260066020908152604091829020805460ff191660011790558151606080820184528c825263ffffffff8c1692820192909252918281019161099491908b01908b01611fb3565b64ffffffffff9081169091528151600755602082015160088054604090940151909216600160201b0268ffffffffffffffffff1990931663ffffffff909116179190911790558660096109e78282611fd0565b905050887f7ea643ae44677f24e0d6f40168893712daaf729b0a38fe7702d21cb544c841018989604051610a1c929190612067565b60405180910390a2505050505050505050565b610a37611600565b851580610a44575060c886115b15610a6257604051633c3b072960e21b815260040160405180910390fd5b858414610a8257604051630f1f305360e41b815260040160405180910390fd5b610a8a611a19565b60005b85811015610b42576020878783818110610aa957610aa9611e7c565b9050602002016020810190610abe9190611e92565b60ff1610610adf57604051635cd7472960e11b815260040160405180910390fd5b81878783818110610af257610af2611e7c565b9050602002016020810190610b079190611e92565b60ff1660208110610b1a57610b1a611e7c565b60200201805190610b2a82611ecb565b60ff1690525080610b3a81611eea565b915050610a8d565b5060005b6020811015610d3457600081610b5e60016020612081565b60ff16610b6b919061209a565b90508015801590610ba3575080858260208110610b8a57610b8a611e7c565b602002016020810190610b9d9190611e92565b60ff1610155b80610bdd575080158015610bdd5750848160208110610bc457610bc4611e7c565b602002016020810190610bd79190611e92565b60ff1615155b15610bfe576040516001627ce2ed60e11b0319815260040160405180910390fd5b6000868260208110610c1257610c12611e7c565b602002016020810190610c259190611e92565b60ff161590508015610c6e57838260208110610c4357610c43611e7c565b602002015160ff1615610c6957604051638db4e75d60e01b815260040160405180910390fd5b610d1f565b868260208110610c8057610c80611e7c565b602002016020810190610c939190611e92565b60ff16848360208110610ca857610ca8611e7c565b602002015160ff161015610ccf57604051635d8009b760e11b815260040160405180910390fd5b83868360208110610ce257610ce2611e7c565b602002016020810190610cf59190611e92565b60ff1660208110610d0857610d08611e7c565b60200201805190610d1882611ecb565b60ff169052505b50508080610d2c90611eea565b915050610b46565b505060006003600001805480602002602001604051908101604052809291908181526020016000905b82821015610db457600084815260209081902060408051606081018252918501546001600160a01b038116835260ff600160a01b8204811684860152600160a81b9091041690820152825260019092019101610d5d565b50505050905060005b8151811015610e58576000828281518110610dda57610dda611e7c565b602090810291909101810151516001600160a01b03811660009081526002909252604090912080546001600160b01b0319169055600380549192509080610e2357610e236120ad565b600082815260209020810160001990810180546001600160b01b03191690550190555080610e5081611eea565b915050610dbd565b5060035415610e6957610e696120c3565b610e766004856020611a38565b50610e846005846020611a38565b506000805b8881101561108c57898982818110610ea357610ea3611e7c565b9050602002016020810190610eb89190611e5f565b6001600160a01b0316826001600160a01b031610610ee957604051630946dd8160e31b815260040160405180910390fd5b600060405180606001604052808c8c85818110610f0857610f08611e7c565b9050602002016020810190610f1d9190611e5f565b6001600160a01b031681526020018360ff1681526020018a8a85818110610f4657610f46611e7c565b9050602002016020810190610f5b9190611e92565b60ff169052905080600260008d8d86818110610f7957610f79611e7c565b9050602002016020810190610f8e9190611e5f565b6001600160a01b0390811682526020808301939093526040918201600090812085518154878701519786015160ff908116600160a81b90810260ff60a81b199a8316600160a01b9081026001600160a81b0319958616968a1696909617959095178b161790945560038054600181018255955289517fc2575a0e9e593c00f959f8c92f12db2869c3395a3b0502d05e2516446f71f85b9095018054988b0151978b01518216909402961690910295169190921617929092179092169190911790558a8a8381811061106157611061611e7c565b90506020020160208101906110769190611e5f565b925050808061108490611eea565b915050610e89565b50821561115d5760088054604080516060808201835260008083526020808401829052600160201b80870464ffffffffff1694860185905260079290925568ffffffffffffffffff1990951690830217909455815160a08101835246808252309482018590529281018290529384018190526001608090940193909352600955600a8054600160f01b6001600160c81b031990911664ffffffffff60a01b1990931692909217600160a01b84021765ffffffffffff60c81b1916600160c81b90930260ff60f01b1916929092171790555b7f0a4974ad206b9c736f9ab2feac1c9b1d043fe4ef377c70ae45659f2ef089f03e60038460405161118f929190612361565b60405180910390a1505050505050505050565b60408051606081018252600754815260085463ffffffff8116602083015264ffffffffff600160201b9091048116928201839052600a549192600160c81b9092041611611202576040516315b6266360e31b815260040160405180910390fd5b83354614611222576040516217e1ef60ea1b815260040160405180910390fd5b306112336040860160208701611e5f565b6001600160a01b03161461125a57604051639a84601560e01b815260040160405180910390fd5b806020015163ffffffff16421115611285576040516309ba674360e41b815260040160405180910390fd5b806040015164ffffffffff168460400160208101906112a49190611fb3565b64ffffffffff16146112c95760405163d9c6386f60e01b815260040160405180910390fd5b60007f08d275622006c4ca82d03f498e90163cafd53c663a48470c3b52ac8bfbd9f52c856040516020016112fe92919061242e565b604051602081830303815290604052805190602001209050611356848480806020026020016040519081016040528093929190818152602001838360200280828437600092019190915250508551915084905061169b565b6113725760405162948a8760e61b815260040160405180910390fd5b60408201516113829060016124f7565b6008805464ffffffffff92909216600160201b0268ffffffffff00000000199092169190911790556113d46113bd6080870160608801611e5f565b60808701356113cf60a089018961251c565b6116b3565b6113e46060860160408701611fb3565b64ffffffffff167f87d58fdd48be753fb9ef4ec8a5895086c401506da8b4d752abc90602c3e62d1d61141c6080880160608901611e5f565b61142960a089018961251c565b896080013560405161143e9493929190612563565b60405180910390a25050505050565b611455611ace565b604080516003805460806020820284018101909452606083018181529293919284929091849160009085015b828210156114d857600084815260209081902060408051606081018252918501546001600160a01b038116835260ff600160a01b8204811684860152600160a81b9091041690820152825260019092019101611481565b50505090825250604080516104008101918290526020928301929091600185019190826000855b825461010083900a900460ff168152602060019283018181049485019490930390920291018084116114ff575050509284525050604080516104008101918290526020938401939092506002850191826000855b825461010083900a900460ff16815260206001928301818104948501949093039092029101808411611553579050505050505081525050905090565b611597611600565b600180546001600160a01b0383166001600160a01b031990911681179091556115c86000546001600160a01b031690565b6001600160a01b03167f38d16b8cac22d99fc7c124b9cd0de2d3fa1faef420bfe791d8c362d765e2270060405160405180910390a350565b6000546001600160a01b031633146103ca5760405162461bcd60e51b815260206004820181905260248201527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e65726044820152606401610436565b600180546001600160a01b031916905561044881611740565b600080600061168487878787611790565b9150915061169181611854565b5095945050505050565b6000826116a8858461199e565b1490505b9392505050565b600080856001600160a01b03168585856040516116d1929190612599565b60006040518083038185875af1925050503d806000811461170e576040519150601f19603f3d011682016040523d82523d6000602084013e611713565b606091505b50915091508161173857806040516370de1b4b60e01b815260040161043691906125a9565b505050505050565b600080546001600160a01b038381166001600160a01b0319831681178455604051919092169283917f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e09190a35050565b6000807f7fffffffffffffffffffffffffffffff5d576e7357a4501ddfe92f46681b20a08311156117c7575060009050600361184b565b6040805160008082526020820180845289905260ff881692820192909252606081018690526080810185905260019060a0016020604051602081039080840390855afa15801561181b573d6000803e3d6000fd5b5050604051601f1901519150506001600160a01b0381166118445760006001925092505061184b565b9150600090505b94509492505050565b6000816004811115611868576118686125f7565b036118705750565b6001816004811115611884576118846125f7565b036118d15760405162461bcd60e51b815260206004820152601860248201527f45434453413a20696e76616c6964207369676e617475726500000000000000006044820152606401610436565b60028160048111156118e5576118e56125f7565b036119325760405162461bcd60e51b815260206004820152601f60248201527f45434453413a20696e76616c6964207369676e6174757265206c656e677468006044820152606401610436565b6003816004811115611946576119466125f7565b036104485760405162461bcd60e51b815260206004820152602260248201527f45434453413a20696e76616c6964207369676e6174757265202773272076616c604482015261756560f01b6064820152608401610436565b600081815b84518110156119e3576119cf828683815181106119c2576119c2611e7c565b60200260200101516119ed565b9150806119db81611eea565b9150506119a3565b5090505b92915050565b6000818310611a095760008281526020849052604090206116ac565b5060009182526020526040902090565b6040518061040001604052806020906020820280368337509192915050565b600183019183908215611abe5791602002820160005b83821115611a8f57833560ff1683826101000a81548160ff021916908360ff1602179055509260200192600101602081600001049283019260010302611a4e565b8015611abc5782816101000a81549060ff0219169055600101602081600001049283019260010302611a8f565b505b50611aca929150611afa565b5090565b604051806060016040528060608152602001611ae8611a19565b8152602001611af5611a19565b905290565b5b80821115611aca5760008155600101611afb565b60008083601f840112611b2157600080fd5b50813567ffffffffffffffff811115611b3957600080fd5b6020830191508360208260051b8501011115611b5457600080fd5b9250929050565b6000806000806000806000878903610120811215611b7857600080fd5b88359750602089013563ffffffff81168114611b9357600080fd5b965060a0603f1982011215611ba757600080fd5b5060408801945060e088013567ffffffffffffffff80821115611bc957600080fd5b611bd58b838c01611b0f565b90965094506101008a0135915080821115611bef57600080fd5b818a0191508a601f830112611c0357600080fd5b813581811115611c1257600080fd5b8b6020606083028501011115611c2757600080fd5b60208301945080935050505092959891949750929550565b8061040081018310156119e757600080fd5b801515811461044857600080fd5b6000806000806000806000610860888a031215611c7b57600080fd5b873567ffffffffffffffff80821115611c9357600080fd5b611c9f8b838c01611b0f565b909950975060208a0135915080821115611cb857600080fd5b50611cc58a828b01611b0f565b9096509450611cd990508960408a01611c3f565b9250611ce9896104408a01611c3f565b9150610840880135611cfa81611c51565b8091505092959891949750929550565b600080600060408486031215611d1f57600080fd5b833567ffffffffffffffff80821115611d3757600080fd5b9085019060c08288031215611d4b57600080fd5b90935060208501359080821115611d6157600080fd5b50611d6e86828701611b0f565b9497909650939450505050565b8060005b6020808210611d8e5750611da5565b825160ff1685529384019390910190600101611d7f565b50505050565b6020808252825161082083830152805161084084018190526000929182019083906108608601905b80831015611e1857835180516001600160a01b031683528581015160ff9081168785015260409182015116908301529284019260019290920191606090910190611dd3565b509286015192611e2b6040870185611d7b565b60408701519350611e40610440870185611d7b565b9695505050505050565b6001600160a01b038116811461044857600080fd5b600060208284031215611e7157600080fd5b81356116ac81611e4a565b634e487b7160e01b600052603260045260246000fd5b600060208284031215611ea457600080fd5b813560ff811681146116ac57600080fd5b634e487b7160e01b600052601160045260246000fd5b600060ff821660ff8103611ee157611ee1611eb5565b60010192915050565b600060018201611efc57611efc611eb5565b5060010190565b64ffffffffff8116811461044857600080fd5b803582526020810135611f2881611e4a565b6001600160a01b031660208301526040810135611f4481611f03565b64ffffffffff9081166040840152606082013590611f6182611f03565b1660608301526080810135611f7581611c51565b8015156080840152505050565b82815260c081016116ac6020830184611f16565b600060208284031215611fa857600080fd5b81356116ac81611c51565b600060208284031215611fc557600080fd5b81356116ac81611f03565b81358155600181016020830135611fe681611e4a565b81546040850135611ff681611f03565b606086013561200481611f03565b608087013561201281611c51565b60c89190911b64ffffffffff60c81b1660a09290921b64ffffffffff60a01b166001600160f81b0319939093166001600160a01b039490941693909317919091171790151560f01b60ff60f01b161790555050565b63ffffffff8316815260c081016116ac6020830184611f16565b60ff82811682821603908111156119e7576119e7611eb5565b818103818111156119e7576119e7611eb5565b634e487b7160e01b600052603160045260246000fd5b634e487b7160e01b600052600160045260246000fd5b8060005b602080601f8301106120ef5750611da5565b825460ff8082168752600882901c8116838801526040612118818901838560101c1660ff169052565b606061212d818a01848660181c1660ff169052565b6080612141818b018587891c1660ff169052565b60a09550612158868b01858760281c1660ff169052565b60c061216d818c01868860301c1660ff169052565b60e0612182818d01878960381c1660ff169052565b60ff87861c8716166101008d01526121a56101208d01878960481c1660ff169052565b6121ba6101408d01878960501c1660ff169052565b6121cf6101608d01878960581c1660ff169052565b60ff87851c8716166101808d01526121f26101a08d01878960681c1660ff169052565b6122076101c08d01878960701c1660ff169052565b61221c6101e08d01878960781c1660ff169052565b60ff87841c8716166102008d015261223f6102208d01878960881c1660ff169052565b6122546102408d01878960901c1660ff169052565b6122696102608d01878960981c1660ff169052565b60ff87891c8716166102808d015261228c6102a08d01878960a81c1660ff169052565b6122a16102c08d01878960b01c1660ff169052565b6122b66102e08d01878960b81c1660ff169052565b60ff87831c8716166103008d01526122d96103208d01878960c81c1660ff169052565b6122ee6103408d01878960d01c1660ff169052565b6123036103608d01878960d81c1660ff169052565b60ff87821c8716166103808d0152505050505061232b6103a08801828460e81c1660ff169052565b6123406103c08801828460f01c1660ff169052565b5060f81c6103e08601525061040090930192600191909101906020016120dd565b600060408083526108608301610820828501528086548083526108808601915087600052602092508260002060005b828110156123d05781546001600160a01b038116855260ff60a082901c81168787015260a89190911c168685015260609093019260019182019101612390565b5050506123e360608601600189016120d9565b6123f46104608601600289016120d9565b941515930192909252509092915050565b81835281816020850137506000828201602090810191909152601f909101601f19169091010190565b82815260406020820152813560408201526000602083013561244f81611e4a565b6001600160a01b03908116606084015260408401359061246e82611f03565b64ffffffffff821660808501526060850135915061248b82611e4a565b1660a083810191909152608084013560c084015283013536849003601e190181126124b557600080fd5b830160208101903567ffffffffffffffff8111156124d257600080fd5b8036038213156124e157600080fd5b60c060e0850152611e4061010085018284612405565b64ffffffffff81811683821601908082111561251557612515611eb5565b5092915050565b6000808335601e1984360301811261253357600080fd5b83018035915067ffffffffffffffff82111561254e57600080fd5b602001915036819003821315611b5457600080fd5b6001600160a01b03851681526060602082018190526000906125889083018587612405565b905082604083015295945050505050565b8183823760009101908152919050565b600060208083528351808285015260005b818110156125d6578581018301518582016040015282016125ba565b506000604082860101526040601f19601f8301168501019250505092915050565b634e487b7160e01b600052602160045260246000fdfea2646970667358221220789e10e5d6588dc4b26dba62aaa06971ed6ac6cbd43499f78a57e1d8415d671c64736f6c63430008130033
Deployed Bytecode Sourcemap
44729:25691:0:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;44816:37;;;;;;;;;;;;44851:2;44816:37;;;;;266:4:1;254:17;;;236:36;;224:2;209:18;44816:37:0;;;;;;;;66686:250;;;;;;;;;;-1:-1:-1;66770:78:0;;;;;;;;66824:24;66770:78;;;;;;;;;;;;;;;;-1:-1:-1;;;66770:78:0;;;;;;;;;;;;66686:250;;455:25:1;;;496:18;;489:51;;;;428:18;66686:250:0;283:263:1;66569:109:0;;;;;;;;;;-1:-1:-1;66638:32:0;;-1:-1:-1;;;66638:32:0;;;;66569:109;;725:12:1;713:25;;;695:44;;683:2;668:18;66569:109:0;551:194:1;66944:109:0;;;;;;;;;;;;-1:-1:-1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;67024:21:0;;;;;;;;67031:14;67024:21;;;;;-1:-1:-1;;;;;67024:21:0;;;;;;-1:-1:-1;;;67024:21:0;;;;;;;;;;;;;-1:-1:-1;;;67024:21:0;;;;;;;;;-1:-1:-1;;;67024:21:0;;;;;;;;;;;;66944:109;;;;;;;1071:13:1;;1053:32;;1145:4;1133:17;;;1127:24;-1:-1:-1;;;;;1123:50:1;1101:20;;;1094:80;1221:4;1209:17;;;1203:24;1246:12;1296:21;;;1274:20;;;1267:51;;;;1378:4;1366:17;;;1360:24;1356:33;;;1334:20;;;1327:63;1460:4;1448:17;;;1442:24;1435:32;1428:40;1406:20;;;1399:70;;;;1040:3;1025:19;;846:629;27111:103:0;;;;;;;;;;;;;:::i;:::-;;29693:216;;;;;;;;;;;;;:::i;53111:4666::-;;;;;;;;;;-1:-1:-1;53111:4666:0;;;;;:::i;:::-;;:::i;61898:4153::-;;;;;;;;;;-1:-1:-1;61898:4153:0;;;;;:::i;:::-;;:::i;26470:87::-;;;;;;;;;;-1:-1:-1;26516:7:0;26543:6;-1:-1:-1;;;;;26543:6:0;26470:87;;;-1:-1:-1;;;;;4818:32:1;;;4800:51;;4788:2;4773:18;26470:87:0;4654:203:1;44860:43:0;;;;;;;;;;;;44900:3;44860:43;;59349:1328;;;;;;:::i;:::-;;:::i;66470:91::-;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;28781:101::-;;;;;;;;;;-1:-1:-1;28861:13:0;;-1:-1:-1;;;;;28861:13:0;28781:101;;29081:181;;;;;;;;;;-1:-1:-1;29081:181:0;;;;;:::i;:::-;;:::i;27111:103::-;26356:13;:11;:13::i;:::-;27176:30:::1;27203:1;27176:18;:30::i;:::-;27111:103::o:0;29693:216::-;28861:13;;810:10;;-1:-1:-1;;;;;28861:13:0;29794:24;;29786:78;;;;-1:-1:-1;;;29786:78:0;;7820:2:1;29786:78:0;;;7802:21:1;7859:2;7839:18;;;7832:30;7898:34;7878:18;;;7871:62;-1:-1:-1;;;7949:18:1;;;7942:39;7998:19;;29786:78:0;;;;;;;;;29875:26;29894:6;29875:18;:26::i;:::-;29735:174;29693:216::o;53111:4666::-;53332:18;53353:69;53403:4;53409:10;53392:28;;;;;;;;455:25:1;;;528:10;516:23;511:2;496:18;;489:51;443:2;428:18;;283:263;53392:28:0;;;;;;;;;;;;;53382:39;;;;;;40264:34;40059:15;40251:48;;;40320:4;40313:18;;;;40372:4;40356:21;;;39990:405;53353:69;53741:30;;;;:18;:30;;;;;;53332:90;;-1:-1:-1;53741:30:0;;53737:93;;;53795:23;;-1:-1:-1;;;53795:23:0;;;;;;;;;;;53737:93;-1:-1:-1;;;;;;;;;;;;;;;;;;;;;;;;;54114:40:0;;:::i;:::-;54203:9;54198:1376;54218:21;;;54198:1376;;;54265:22;54290:10;;54301:1;54290:13;;;;;;;:::i;:::-;;;;;;;;-1:-1:-1;54322:21:0;;-1:-1:-1;54346:46:0;54360:10;54372:5;;;;54290:13;54372:5;:::i;:::-;54379:3;:5;;;54386:3;:5;;;54346:13;:46::i;:::-;54322:70;;54571:13;-1:-1:-1;;;;;54556:28:0;:11;-1:-1:-1;;;;;54556:28:0;;54552:126;;54616:42;;-1:-1:-1;;;54616:42:0;;;;;;;;;;;54552:126;-1:-1:-1;;;;;54753:24:0;;;;;;;:9;:24;;;;;;;;;54744:33;;;;;;;;;;;;;;;;-1:-1:-1;;;54744:33:0;;;;;;;;;;;-1:-1:-1;;;54744:33:0;;;;;;;;;;;;;;-1:-1:-1;54710:13:0;;-1:-1:-1;54710:13:0;;54800:28;54796:99;;54860:15;;-1:-1:-1;;;54860:15:0;;;;;;;;;;;54796:99;54927:12;;;;54958:601;54994:15;55010:5;54994:22;;;;;;;;;:::i;:::-;;;;:24;;;;;;:::i;:::-;;;;;;;;55071:21;;-1:-1:-1;55071:28:0;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;55045:54;;:15;55061:5;55045:22;;;;;;;;;:::i;:::-;;;;;:54;;;55315:5;55041:303;55370:10;;;55366:113;55450:5;55366:113;55511:21;:28;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;-1:-1:-1;54958:601:0;;;54246:1328;;;54241:3;;;;;:::i;:::-;;;;54198:1376;;;-1:-1:-1;55781:21:0;:24;;;55803:1;55781:29;55777:92;;55838:15;;-1:-1:-1;;;55838:15:0;;;;;;;;;;;55777:92;55961:21;:24;55940:18;;55961:24;;;;55940:45;;;55936:114;;;56013:21;;-1:-1:-1;;;56013:21:0;;;;;;;;;;;55936:114;53945:2116;;;56090:15;56077:10;:28;;;56073:96;;;56129:28;;-1:-1:-1;;;56129:28:0;;;;;;;;;;;56073:96;56233:18;42659:59;56340:8;56281:68;;;;;;;;;:::i;:::-;;;;;;;;;;;;;56271:79;;;;;;56233:117;;56370:51;56389:13;;56370:51;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;56404:4:0;;-1:-1:-1;56410:10:0;;-1:-1:-1;56370:18:0;;-1:-1:-1;56370:51:0:i;:::-;56365:123;;56449:23;;-1:-1:-1;;;56449:23:0;;;;;;;;;;;56365:123;-1:-1:-1;56515:13:0;56532:16;;56515:33;56511:87;;56572:14;;-1:-1:-1;;;56572:14:0;;;;;;;;;;;56511:87;56631:17;;;;;;;;:::i;:::-;-1:-1:-1;;;;;56614:34:0;56622:4;-1:-1:-1;;;;;56614:34:0;;56610:89;;56672:15;;-1:-1:-1;;;56672:15:0;;;;;;;;;;;56610:89;56728:32;;56944:26;;56728:32;-1:-1:-1;;;56728:32:0;;;;;;-1:-1:-1;;;56944:26:0;;;;56933:37;;;;;:71;;-1:-1:-1;56975:29:0;;;;;;;;:::i;:::-;56974:30;56933:71;56929:123;;;57028:12;;-1:-1:-1;;;57028:12:0;;;;;;;;;;;56929:123;57208:19;;;;;;;;:::i;:::-;57197:30;;:7;:30;;;57193:87;;57251:17;;-1:-1:-1;;;57251:17:0;;;;;;;;;;;57193:87;57318:20;;;;;;;;:::i;:::-;57296:42;;:19;;;;;;;;:::i;:::-;:42;;;57292:100;;;57362:18;;-1:-1:-1;;;57362:18:0;;;;;;;;;;;57292:100;57467:30;;;;:18;:30;;;;;;;;;:37;;-1:-1:-1;;57467:37:0;57500:4;57467:37;;;57542:140;;;;;;;;;;;;;;;;;;;;;;;;;;57651:19;;;;;;;;;:::i;:::-;57542:140;;;;;;;57515:167;;:24;:167;;;;;;;;;;;;;;;;-1:-1:-1;;;57515:167:0;-1:-1:-1;;57515:167:0;;;;;;;;;;;;;;57710:8;57693:14;:25;57710:8;57693:14;:25;:::i;:::-;;;;57742:4;57734:35;57748:10;57760:8;57734:35;;;;;;;:::i;:::-;;;;;;;;53321:4456;;53111:4666;;;;;;;:::o;61898:4153::-;26356:13;:11;:13::i;:::-;62168:27;;;:71:::1;;-1:-1:-1::0;44900:3:0::1;62199:40:::0;::::1;62168:71;62164:136;;;62263:25;;-1:-1:-1::0;;;62263:25:0::1;;;;;;;;;;;62164:136;62316:45:::0;;::::1;62312:113;;62385:28;;-1:-1:-1::0;;;62385:28:0::1;;;;;;;;;;;62312:113;62553:44;;:::i;:::-;62673:9;62668:244;62688:23:::0;;::::1;62668:244;;;44851:2;62741:12:::0;;62754:1;62741:15;;::::1;;;;;:::i;:::-;;;;;;;;;;;;;;:::i;:::-;:29;;;62737:103;;62802:18;;-1:-1:-1::0;;;62802:18:0::1;;;;;;;;;;;62737:103;62858:19;62878:12;;62891:1;62878:15;;;;;;;:::i;:::-;;;;;;;;;;;;;;:::i;:::-;62858:36;;;;;;;;;:::i;:::-;;;;:38:::0;;;::::1;::::0;::::1;:::i;:::-;;;::::0;;-1:-1:-1;62713:3:0;::::1;::::0;::::1;:::i;:::-;;;;62668:244;;;;63097:9;63092:1106;44851:2;63112:14:::0;::::1;63092:1106;;;63152:9;63181:1:::0;63164:14:::1;63177:1;44851:2;63164:14;:::i;:::-;:18;;;;;;:::i;:::-;63152:30:::0;-1:-1:-1;63305:6:0;;;::::1;::::0;:30:::1;;;63334:1;63315:12;63328:1;63315:15;;;;;;;:::i;:::-;;;;;;;;;;;;:::i;:::-;:20;;;;63305:30;63304:68;;;-1:-1:-1::0;63341:6:0;;:30;::::1;;;;63351:12;63364:1;63351:15;;;;;;;:::i;:::-;;;;;;;;;;;;:::i;:::-;:20;;::::0;::::1;63341:30;63300:148;;;63404:24;;-1:-1:-1::0;;;;;;63404:24:0::1;;;;;;;;;;;63300:148;63466:13;63482:12;63495:1;63482:15;;;;;;;:::i;:::-;;;;;;;;;;;;:::i;:::-;:20;;::::0;;-1:-1:-1;63521:662:0;::::1;;;63635:19;63655:1;63635:22;;;;;;;:::i;:::-;;;;::::0;63631:26:::1;;::::0;63627:113:::1;;63693:23;;-1:-1:-1::0;;;63693:23:0::1;;;;;;;;;;;63627:113;63521:662;;;63881:12;63894:1;63881:15;;;;;;;:::i;:::-;;;;;;;;;;;;:::i;:::-;63856:40;;:19;63876:1;63856:22;;;;;;;:::i;:::-;;;;;:40;;;63852:128;;;63932:24;;-1:-1:-1::0;;;63932:24:0::1;;;;;;;;;;;63852:128;64002:19;64022:12;64035:1;64022:15;;;;;;;:::i;:::-;;;;;;;;;;;;:::i;:::-;64002:36;;;;;;;;;:::i;:::-;;;;:38:::0;;;::::1;::::0;::::1;:::i;:::-;;;::::0;;-1:-1:-1;63521:662:0::1;63133:1065;;63128:3;;;;;:::i;:::-;;;;63092:1106;;;;62437:1772;64221:26;64250:8;:16;;64221:45;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;::::0;;;::::1;::::0;;;;::::1;::::0;;::::1;::::0;::::1;::::0;;;;::::1;::::0;-1:-1:-1;;;;;64221:45:0;::::1;::::0;;::::1;-1:-1:-1::0;;;64221:45:0;::::1;::::0;::::1;::::0;;::::1;::::0;-1:-1:-1;;;64221:45:0;;::::1;;::::0;;;;;;;;;::::1;::::0;::::1;;;;;;;;;;64326:9;64321:206;64345:10;:17;64341:1;:21;64321:206;;;64384:24;64411:10;64422:1;64411:13;;;;;;;;:::i;:::-;;::::0;;::::1;::::0;;;;;;;:18;-1:-1:-1;;;;;64451:27:0;::::1;64411:18;64451:27:::0;;;:9:::1;:27:::0;;;;;;;64444:34;;-1:-1:-1;;;;;;64444:34:0;;;64493:8:::1;:22:::0;;64411:18;;-1:-1:-1;64493:8:0;:22;::::1;;;;:::i;:::-;;::::0;;;::::1;::::0;;;;-1:-1:-1;;64493:22:0;;;;;-1:-1:-1;;;;;;64493:22:0;;;;;;-1:-1:-1;64364:3:0;::::1;::::0;::::1;:::i;:::-;;;;64321:206;;;-1:-1:-1::0;64638:8:0::1;:23:::0;:28;64631:36:::1;;;;:::i;:::-;64678;:21:::0;64702:12;64678:36:::1;;:::i;:::-;-1:-1:-1::0;64725:36:0::1;:21:::0;64749:12;64725:36:::1;;:::i;:::-;;64903:18;64952:9:::0;64947:474:::1;64967:26:::0;;::::1;64947:474;;;65033:15;;65049:1;65033:18;;;;;;;:::i;:::-;;;;;;;;;;;;;;:::i;:::-;-1:-1:-1::0;;;;;65019:32:0::1;:10;-1:-1:-1::0;;;;;65019:32:0::1;;65015:122;;65079:42;;-1:-1:-1::0;;;65079:42:0::1;;;;;;;;;;;65015:122;65151:20;65191:75;;;;;;;;65205:15;;65221:1;65205:18;;;;;;;:::i;:::-;;;;;;;;;;;;;;:::i;:::-;-1:-1:-1::0;;;;;65191:75:0::1;;;;;65238:1;65191:75;;;;;;65249:12;;65262:1;65249:15;;;;;;;:::i;:::-;;;;;;;;;;;;;;:::i;:::-;65191:75;;::::0;;65151:115;-1:-1:-1;65151:115:0;65281:9:::1;:29;65291:15:::0;;65307:1;65291:18;;::::1;;;;;:::i;:::-;;;;;;;;;;;;;;:::i;:::-;-1:-1:-1::0;;;;;65281:29:0;;::::1;::::0;;::::1;::::0;;::::1;::::0;;;;;;;;-1:-1:-1;65281:29:0;;;:38;;;;;;::::1;::::0;;;::::1;::::0;::::1;::::0;;::::1;-1:-1:-1::0;;;65281:38:0;;::::1;-1:-1:-1::0;;;;65281:38:0;;::::1;-1:-1:-1::0;;;65281:38:0;;::::1;-1:-1:-1::0;;;;;;65281:38:0;;;;;::::1;::::0;;;;;;;::::1;::::0;::::1;;::::0;;;65334:8:::1;:29:::0;;65281:38;65334:29;::::1;::::0;;;;;;;;;::::1;::::0;;;;::::1;::::0;;;::::1;::::0;;::::1;::::0;;::::1;::::0;::::1;::::0;;::::1;::::0;;;;;::::1;::::0;;;;::::1;::::0;;::::1;::::0;;;::::1;::::0;;65391:15;;65407:1;65391:18;;::::1;;;;;:::i;:::-;;;;;;;;;;;;;;:::i;:::-;65378:31;;65000:421;64995:3;;;;;:::i;:::-;;;;64947:474;;;;65437:9;65433:565;;;65563:32:::0;;;65654:66:::1;::::0;;::::1;::::0;;::::1;::::0;;-1:-1:-1;65654:66:0;;;::::1;::::0;;::::1;::::0;;;-1:-1:-1;;;65563:32:0;;::::1;;;65654:66:::0;;;;;;65563:24:::1;65610:110:::0;;;;-1:-1:-1;;65610:110:0;;;;;::::1;;::::0;;;65752:234;;::::1;::::0;::::1;::::0;;65793:13:::1;65752:234:::0;;;65843:4:::1;65752:234:::0;;::::1;::::0;;;;;;;;;;;;;;;-1:-1:-1;65752:234:0;;;;;;;;65735:14:::1;:251:::0;;;;-1:-1:-1;;;;;;;;;65735:251:0;;;-1:-1:-1;;;;65735:251:0;;;;;;;-1:-1:-1;;;65735:251:0;::::1;;-1:-1:-1::0;;;;65735:251:0;-1:-1:-1;;;65735:251:0;;::::1;-1:-1:-1::0;;;;65735:251:0;;;;;::::1;::::0;;65433:565:::1;66013:30;66023:8;66033:9;66013:30;;;;;;;:::i;:::-;;;;;;;;62153:3898;;61898:4153:::0;;;;;;;:::o;59349:1328::-;59436:86;;;;;;;;59498:24;59436:86;;;;;;;;;;;;;-1:-1:-1;;;59436:86:0;;;;;;;;;;;59539:26;;59436:86;;-1:-1:-1;;;59539:26:0;;;;:67;59535:127;;59630:20;;-1:-1:-1;;;59630:20:0;;;;;;;;;;;59535:127;59678:10;;59692:13;59678:27;59674:81;;59729:14;;-1:-1:-1;;;59729:14:0;;;;;;;;;;;59674:81;59794:4;59771:11;;;;;;;;:::i;:::-;-1:-1:-1;;;;;59771:28:0;;59767:83;;59823:15;;-1:-1:-1;;;59823:15:0;;;;;;;;;;;59767:83;59884:29;:40;;;59866:58;;:15;:58;59862:111;;;59948:13;;-1:-1:-1;;;59948:13:0;;;;;;;;;;;59862:111;60001:29;:37;;;59989:49;;:2;:8;;;;;;;;;;:::i;:::-;:49;;;59985:101;;60062:12;;-1:-1:-1;;;60062:12:0;;;;;;;;;;;59985:101;60155:18;42335:53;60239:2;60186:56;;;;;;;;;:::i;:::-;;;;;;;;;;;;;60176:67;;;;;;60155:88;;60259:73;60278:5;;60259:73;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;60285:34:0;;;-1:-1:-1;60321:10:0;;-1:-1:-1;60259:18:0;:73::i;:::-;60254:137;;60356:23;;-1:-1:-1;;;60356:23:0;;;;;;;;;;;60254:137;60519:37;;;;:41;;60559:1;60519:41;:::i;:::-;60484:32;:76;;;;;;;-1:-1:-1;;;60484:76:0;-1:-1:-1;;60484:76:0;;;;;;;;;60573:34;60582:5;;;;;;;;:::i;:::-;60589:8;;;;60599:7;;;;60589:2;60599:7;:::i;:::-;60573:8;:34::i;:::-;60634:8;;;;;;;;:::i;:::-;60623:46;;;60644:5;;;;;;;;:::i;:::-;60651:7;;;;:2;:7;:::i;:::-;60660:2;:8;;;60623:46;;;;;;;;;:::i;:::-;;;;;;;;59425:1252;;59349:1328;;;:::o;66470:91::-;66512:13;;:::i;:::-;66538:15;;;66545:8;66538:15;;;;;;;;;;;;;;;;;;;;;66545:8;;66538:15;;;;66545:8;;-1:-1:-1;;66538:15:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;;;;66538:15:0;;;;;-1:-1:-1;;;66538:15:0;;;;;;;;-1:-1:-1;;;66538:15:0;;;;;;;;;;;;;;;;;;;-1:-1:-1;;;66538:15:0;;;-1:-1:-1;66538:15:0;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;66538:15:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;;66538:15:0;;;-1:-1:-1;;66538:15:0;;;;;;;;;;;;;;;;;-1:-1:-1;66538:15:0;;;;;-1:-1:-1;66538:15:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;66470:91;:::o;29081:181::-;26356:13;:11;:13::i;:::-;29171::::1;:24:::0;;-1:-1:-1;;;;;29171:24:0;::::1;-1:-1:-1::0;;;;;;29171:24:0;;::::1;::::0;::::1;::::0;;;29236:7:::1;26516::::0;26543:6;-1:-1:-1;;;;;26543:6:0;;26470:87;29236:7:::1;-1:-1:-1::0;;;;;29211:43:0::1;;;;;;;;;;;29081:181:::0;:::o;26635:132::-;26516:7;26543:6;-1:-1:-1;;;;;26543:6:0;810:10;26699:23;26691:68;;;;-1:-1:-1;;;26691:68:0;;19413:2:1;26691:68:0;;;19395:21:1;;;19432:18;;;19425:30;19491:34;19471:18;;;19464:62;19543:18;;26691:68:0;19211:356:1;29452:156:0;29542:13;29535:20;;-1:-1:-1;;;;;;29535:20:0;;;29566:34;29591:8;29566:24;:34::i;39454:236::-;39539:7;39560:17;39579:18;39601:25;39612:4;39618:1;39621;39624;39601:10;:25::i;:::-;39559:67;;;;39637:18;39649:5;39637:11;:18::i;:::-;-1:-1:-1;39673:9:0;39454:236;-1:-1:-1;;;;;39454:236:0:o;2144:156::-;2235:4;2288;2259:25;2272:5;2279:4;2259:12;:25::i;:::-;:33;2252:40;;2144:156;;;;;;:::o;66180:247::-;66279:12;66293:16;66313:6;-1:-1:-1;;;;;66313:11:0;66332:5;66339:4;;66313:31;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;66278:66;;;;66360:7;66355:65;;66404:3;66391:17;;-1:-1:-1;;;66391:17:0;;;;;;;;:::i;66355:65::-;66267:160;;66180:247;;;;:::o;27730:191::-;27804:16;27823:6;;-1:-1:-1;;;;;27840:17:0;;;-1:-1:-1;;;;;;27840:17:0;;;;;;27873:40;;27823:6;;;;;;;27873:40;;27804:16;27873:40;27793:128;27730:191;:::o;37838:1477::-;37926:7;;38860:66;38847:79;;38843:163;;;-1:-1:-1;38959:1:0;;-1:-1:-1;38963:30:0;38943:51;;38843:163;39120:24;;;39103:14;39120:24;;;;;;;;;20626:25:1;;;20699:4;20687:17;;20667:18;;;20660:45;;;;20721:18;;;20714:34;;;20764:18;;;20757:34;;;39120:24:0;;20598:19:1;;39120:24:0;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;39120:24:0;;-1:-1:-1;;39120:24:0;;;-1:-1:-1;;;;;;;39159:20:0;;39155:103;;39212:1;39216:29;39196:50;;;;;;;39155:103;39278:6;-1:-1:-1;39286:20:0;;-1:-1:-1;37838:1477:0;;;;;;;;:::o;33298:521::-;33376:20;33367:5;:29;;;;;;;;:::i;:::-;;33363:449;;33298:521;:::o;33363:449::-;33474:29;33465:5;:38;;;;;;;;:::i;:::-;;33461:351;;33520:34;;-1:-1:-1;;;33520:34:0;;21136:2:1;33520:34:0;;;21118:21:1;21175:2;21155:18;;;21148:30;21214:26;21194:18;;;21187:54;21258:18;;33520:34:0;20934:348:1;33461:351:0;33585:35;33576:5;:44;;;;;;;;:::i;:::-;;33572:240;;33637:41;;-1:-1:-1;;;33637:41:0;;21489:2:1;33637:41:0;;;21471:21:1;21528:2;21508:18;;;21501:30;21567:33;21547:18;;;21540:61;21618:18;;33637:41:0;21287:355:1;33572:240:0;33709:30;33700:5;:39;;;;;;;;:::i;:::-;;33696:116;;33756:44;;-1:-1:-1;;;33756:44:0;;21849:2:1;33756:44:0;;;21831:21:1;21888:2;21868:18;;;21861:30;21927:34;21907:18;;;21900:62;-1:-1:-1;;;21978:18:1;;;21971:32;22020:19;;33756:44:0;21647:398:1;2943:296:0;3026:7;3069:4;3026:7;3084:118;3108:5;:12;3104:1;:16;3084:118;;;3157:33;3167:12;3181:5;3187:1;3181:8;;;;;;;;:::i;:::-;;;;;;;3157:9;:33::i;:::-;3142:48;-1:-1:-1;3122:3:0;;;;:::i;:::-;;;;3084:118;;;-1:-1:-1;3219:12:0;-1:-1:-1;2943:296:0;;;;;:::o;10381:149::-;10444:7;10475:1;10471;:5;:51;;10606:13;10700:15;;;10736:4;10729:15;;;10783:4;10767:21;;10471:51;;;-1:-1:-1;10606:13:0;10700:15;;;10736:4;10729:15;10783:4;10767:21;;;10381:149::o;-1:-1:-1:-;;;;;;;;;;;;;;;;;;;;;;;;:::o;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;:::o;:::-;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;:::o;:::-;;;;;;;;;;;;;;;1480:367:1;1543:8;1553:6;1607:3;1600:4;1592:6;1588:17;1584:27;1574:55;;1625:1;1622;1615:12;1574:55;-1:-1:-1;1648:20:1;;1691:18;1680:30;;1677:50;;;1723:1;1720;1713:12;1677:50;1760:4;1752:6;1748:17;1736:29;;1820:3;1813:4;1803:6;1800:1;1796:14;1788:6;1784:27;1780:38;1777:47;1774:67;;;1837:1;1834;1827:12;1774:67;1480:367;;;;;:::o;1852:1359::-;2061:6;2069;2077;2085;2093;2101;2109;2153:9;2144:7;2140:23;2183:3;2179:2;2175:12;2172:32;;;2200:1;2197;2190:12;2172:32;2236:9;2223:23;2213:33;;2296:2;2285:9;2281:18;2268:32;2340:10;2333:5;2329:22;2322:5;2319:33;2309:61;;2366:1;2363;2356:12;2309:61;2389:5;-1:-1:-1;2428:3:1;-1:-1:-1;;2410:16:1;;2406:26;2403:46;;;2445:1;2442;2435:12;2403:46;;2483:2;2472:9;2468:18;2458:28;;2537:3;2526:9;2522:19;2509:33;2561:18;2602:2;2594:6;2591:14;2588:34;;;2618:1;2615;2608:12;2588:34;2657:70;2719:7;2710:6;2699:9;2695:22;2657:70;:::i;:::-;2746:8;;-1:-1:-1;2631:96:1;-1:-1:-1;2834:3:1;2819:19;;2806:33;;-1:-1:-1;2851:16:1;;;2848:36;;;2880:1;2877;2870:12;2848:36;2918:8;2907:9;2903:24;2893:34;;2965:7;2958:4;2954:2;2950:13;2946:27;2936:55;;2987:1;2984;2977:12;2936:55;3027:2;3014:16;3053:2;3045:6;3042:14;3039:34;;;3069:1;3066;3059:12;3039:34;3125:7;3120:2;3112:4;3104:6;3100:17;3096:2;3092:26;3088:35;3085:48;3082:68;;;3146:1;3143;3136:12;3082:68;3177:2;3173;3169:11;3159:21;;3199:6;3189:16;;;;;1852:1359;;;;;;;;;;:::o;3216:159::-;3308:6;3341:4;3329:17;;3326:26;-1:-1:-1;3323:46:1;;;3365:1;3362;3355:12;3380:118;3466:5;3459:13;3452:21;3445:5;3442:32;3432:60;;3488:1;3485;3478:12;3503:1146;3695:6;3703;3711;3719;3727;3735;3743;3796:4;3784:9;3775:7;3771:23;3767:34;3764:54;;;3814:1;3811;3804:12;3764:54;3854:9;3841:23;3883:18;3924:2;3916:6;3913:14;3910:34;;;3940:1;3937;3930:12;3910:34;3979:70;4041:7;4032:6;4021:9;4017:22;3979:70;:::i;:::-;4068:8;;-1:-1:-1;3953:96:1;-1:-1:-1;4156:2:1;4141:18;;4128:32;;-1:-1:-1;4172:16:1;;;4169:36;;;4201:1;4198;4191:12;4169:36;;4240:72;4304:7;4293:8;4282:9;4278:24;4240:72;:::i;:::-;4331:8;;-1:-1:-1;4214:98:1;-1:-1:-1;4385:60:1;;-1:-1:-1;4437:7:1;4432:2;4417:18;;4385:60;:::i;:::-;4375:70;;4464:62;4518:7;4511:4;4500:9;4496:20;4464:62;:::i;:::-;4454:72;;4576:4;4565:9;4561:20;4548:34;4591:28;4613:5;4591:28;:::i;:::-;4638:5;4628:15;;;3503:1146;;;;;;;;;;:::o;4862:718::-;4979:6;4987;4995;5048:2;5036:9;5027:7;5023:23;5019:32;5016:52;;;5064:1;5061;5054:12;5016:52;5104:9;5091:23;5133:18;5174:2;5166:6;5163:14;5160:34;;;5190:1;5187;5180:12;5160:34;5213:22;;;;5269:3;5251:16;;;5247:26;5244:46;;;5286:1;5283;5276:12;5244:46;5309:2;;-1:-1:-1;5364:2:1;5349:18;;5336:32;;5380:16;;;5377:36;;;5409:1;5406;5399:12;5377:36;;5448:72;5512:7;5501:8;5490:9;5486:24;5448:72;:::i;:::-;4862:718;;5539:8;;-1:-1:-1;5422:98:1;;-1:-1:-1;;;;4862:718:1:o;5585:371::-;5676:5;5699:1;5709:241;5773:4;5806:2;5803:1;5800:9;5790:30;;5813:5;;;5790:30;5849:13;;5864:4;5845:24;5833:37;;5890:12;;;;5925:15;;;;5736:1;5729:9;5709:241;;;5713:3;;5585:371;;:::o;5961:1264::-;6130:2;6141:21;;;6234:13;;6283:6;6263:18;;;6256:34;6339:19;;6200:4;6185:20;;6367:22;;;6101:4;;6130:2;6448:21;;;6101:4;;6420;6405:20;;;6497:456;6511:6;6508:1;6505:13;6497:456;;;6570:13;;6612:9;;-1:-1:-1;;;;;6608:35:1;6596:48;;6685:11;;;6679:18;6720:4;6758:23;;;6744:12;;;6737:45;6805:4;6853:11;;;6847:18;6843:27;6829:12;;;6822:49;6928:15;;;;6640:1;6526:9;;;;;6900:4;6891:14;;;;6497:456;;;-1:-1:-1;6990:15:1;;;6984:22;;7015:60;7069:4;7054:20;;6984:22;7015:60;:::i;:::-;7124:4;7116:6;7112:17;7106:24;7084:46;;7139:60;7193:4;7182:9;7178:20;7162:14;7139:60;:::i;:::-;7216:3;5961:1264;-1:-1:-1;;;;;;5961:1264:1:o;7230:131::-;-1:-1:-1;;;;;7305:31:1;;7295:42;;7285:70;;7351:1;7348;7341:12;7366:247;7425:6;7478:2;7466:9;7457:7;7453:23;7449:32;7446:52;;;7494:1;7491;7484:12;7446:52;7533:9;7520:23;7552:31;7577:5;7552:31;:::i;8028:127::-;8089:10;8084:3;8080:20;8077:1;8070:31;8120:4;8117:1;8110:15;8144:4;8141:1;8134:15;8160:269;8217:6;8270:2;8258:9;8249:7;8245:23;8241:32;8238:52;;;8286:1;8283;8276:12;8238:52;8325:9;8312:23;8375:4;8368:5;8364:16;8357:5;8354:27;8344:55;;8395:1;8392;8385:12;8434:127;8495:10;8490:3;8486:20;8483:1;8476:31;8526:4;8523:1;8516:15;8550:4;8547:1;8540:15;8566:175;8603:3;8647:4;8640:5;8636:16;8676:4;8667:7;8664:17;8661:43;;8684:18;;:::i;:::-;8733:1;8720:15;;8566:175;-1:-1:-1;;8566:175:1:o;8746:135::-;8785:3;8806:17;;;8803:43;;8826:18;;:::i;:::-;-1:-1:-1;8873:1:1;8862:13;;8746:135::o;8886:123::-;8971:12;8964:5;8960:24;8953:5;8950:35;8940:63;;8999:1;8996;8989:12;9014:743;9114:5;9101:19;9096:3;9089:32;9169:4;9162:5;9158:16;9145:30;9184:33;9209:7;9184:33;:::i;:::-;-1:-1:-1;;;;;9249:33:1;9242:4;9233:14;;9226:57;9331:4;9320:16;;9307:30;9346:32;9307:30;9346:32;:::i;:::-;9397:12;9441:16;;;9434:4;9425:14;;9418:40;9506:4;9495:16;;9482:30;;9521:32;9482:30;9521:32;:::i;:::-;9585:16;9578:4;9569:14;;9562:40;9650:4;9639:16;;9626:30;9665;9626;9665;:::i;:::-;9741:7;9734:15;9727:23;9720:4;9715:3;9711:14;9704:47;;9014:743;;:::o;9762:344::-;9999:25;;;9986:3;9971:19;;10033:67;10096:2;10081:18;;10073:6;10033:67;:::i;10111:241::-;10167:6;10220:2;10208:9;10199:7;10195:23;10191:32;10188:52;;;10236:1;10233;10226:12;10188:52;10275:9;10262:23;10294:28;10316:5;10294:28;:::i;10357:245::-;10415:6;10468:2;10456:9;10447:7;10443:23;10439:32;10436:52;;;10484:1;10481;10474:12;10436:52;10523:9;10510:23;10542:30;10566:5;10542:30;:::i;10607:886::-;10780:5;10767:19;10761:4;10754:33;10824:1;10818:4;10814:12;10874:2;10867:5;10863:14;10850:28;10887:33;10912:7;10887:33;:::i;:::-;10945:10;10939:17;11004:2;10997:5;10993:14;10980:28;11017:32;11041:7;11017:32;:::i;:::-;11097:2;11090:5;11086:14;11073:28;11110:32;11134:7;11110:32;:::i;:::-;11190:3;11183:5;11179:15;11166:29;11204:30;11226:7;11204:30;:::i;:::-;11295:3;11272:17;;;;-1:-1:-1;;;11268:46:1;11415:3;11323:17;;;;-1:-1:-1;;;11319:46:1;-1:-1:-1;;;;;;11370:22:1;;;;-1:-1:-1;;;;;11394:33:1;;;;11367:61;;;;11316:113;;;;11265:165;11452:15;;11445:23;11475:3;11436:33;-1:-1:-1;;;11432:53:1;11262:224;11243:244;;-1:-1:-1;;10607:886:1:o;11498:359::-;11763:10;11751:23;;11733:42;;11720:3;11705:19;;11784:67;11847:2;11832:18;;11824:6;11784:67;:::i;11862:151::-;11952:4;11945:12;;;11931;;;11927:31;;11970:14;;11967:40;;;11987:18;;:::i;12018:128::-;12085:9;;;12106:11;;;12103:37;;;12120:18;;:::i;12151:127::-;12212:10;12207:3;12203:20;12200:1;12193:31;12243:4;12240:1;12233:15;12267:4;12264:1;12257:15;12283:127;12344:10;12339:3;12335:20;12332:1;12325:31;12375:4;12372:1;12365:15;12399:4;12396:1;12389:15;12415:2792;12514:5;12547:1;12557:2644;12680:4;12732:2;12727;12714:11;12710:20;12707:28;12697:49;;12739:5;;;12697:49;12771:13;;12807:4;12841:13;;;58:29;;12898:1;12894:12;;;12890:21;;12913:12;;;58:29;12949:2;12964:54;13014:2;13009:3;13005:12;13000:2;12993:4;12989:2;12985:13;12981:22;81:4;70:16;58:29;;14:75;12964:54;13041:2;13056:54;13106:2;13101:3;13097:12;13092:2;13085:4;13081:2;13077:13;13073:22;81:4;70:16;58:29;;14:75;13056:54;13133:3;13149:54;13199:2;13194:3;13190:12;13185:2;13178:4;13174:2;13170:13;13166:22;81:4;70:16;58:29;;14:75;13149:54;13226:3;13216:13;;13242:54;13292:2;13287:3;13283:12;13278:2;13271:4;13267:2;13263:13;13259:22;81:4;70:16;58:29;;14:75;13242:54;13319:3;13335:54;13385:2;13380:3;13376:12;13371:2;13364:4;13360:2;13356:13;13352:22;81:4;70:16;58:29;;14:75;13335:54;13412:3;13428:54;13478:2;13473:3;13469:12;13464:2;13457:4;13453:2;13449:13;13445:22;81:4;70:16;58:29;;14:75;13428:54;81:4;13516:13;;;13512:22;;70:16;13545:3;13536:13;;58:29;13563:55;13613:3;13608;13604:13;13599:2;13592:4;13588:2;13584:13;13580:22;81:4;70:16;58:29;;14:75;13563:55;13631;13681:3;13676;13672:13;13667:2;13660:4;13656:2;13652:13;13648:22;81:4;70:16;58:29;;14:75;13631:55;13699;13749:3;13744;13740:13;13735:2;13728:4;13724:2;13720:13;13716:22;81:4;70:16;58:29;;14:75;13699:55;81:4;13788:13;;;13784:22;;70:16;13817:3;13808:13;;58:29;13835:56;13886:3;13881;13877:13;13872:2;13865:4;13860:3;13856:14;13852:23;81:4;70:16;58:29;;14:75;13835:56;13904;13955:3;13950;13946:13;13941:2;13934:4;13929:3;13925:14;13921:23;81:4;70:16;58:29;;14:75;13904:56;13973;14024:3;14019;14015:13;14010:2;14003:4;13998:3;13994:14;13990:23;81:4;70:16;58:29;;14:75;13973:56;81:4;14063:13;;;14059:22;;70:16;14092:3;14083:13;;58:29;14110:56;14161:3;14156;14152:13;14147:2;14140:4;14135:3;14131:14;14127:23;81:4;70:16;58:29;;14:75;14110:56;14179;14230:3;14225;14221:13;14216:2;14209:4;14204:3;14200:14;14196:23;81:4;70:16;58:29;;14:75;14179:56;14248;14299:3;14294;14290:13;14285:2;14278:4;14273:3;14269:14;14265:23;81:4;70:16;58:29;;14:75;14248:56;81:4;14338:13;;;14334:22;;70:16;14367:3;14358:13;;58:29;14385:56;14436:3;14431;14427:13;14422:2;14415:4;14410:3;14406:14;14402:23;81:4;70:16;58:29;;14:75;14385:56;14454;14505:3;14500;14496:13;14491:2;14484:4;14479:3;14475:14;14471:23;81:4;70:16;58:29;;14:75;14454:56;14523;14574:3;14569;14565:13;14560:2;14553:4;14548:3;14544:14;14540:23;81:4;70:16;58:29;;14:75;14523:56;81:4;14613:13;;;14609:22;;70:16;14642:3;14633:13;;58:29;14660:56;14711:3;14706;14702:13;14697:2;14690:4;14685:3;14681:14;14677:23;81:4;70:16;58:29;;14:75;14660:56;14729;14780:3;14775;14771:13;14766:2;14759:4;14754:3;14750:14;14746:23;81:4;70:16;58:29;;14:75;14729:56;14798;14849:3;14844;14840:13;14835:2;14828:4;14823:3;14819:14;14815:23;81:4;70:16;58:29;;14:75;14798:56;81:4;14888:13;;;14884:22;;70:16;14917:3;14908:13;;58:29;14867:55;;;;;14935:56;14986:3;14981;14977:13;14972:2;14965:4;14960:3;14956:14;14952:23;81:4;70:16;58:29;;14:75;14935:56;15004;15055:3;15050;15046:13;15041:2;15034:4;15029:3;15025:14;15021:23;81:4;70:16;58:29;;14:75;15004:56;-1:-1:-1;15094:3:1;15090:14;15115:3;15106:13;;58:29;-1:-1:-1;15149:4:1;15140:14;;;;15189:1;15177:14;;;;;12632:4;12615:22;12557:2644;;15212:1174;15371:4;15400:2;15429;15418:9;15411:21;15470:4;15459:9;15455:20;15511:6;15506:2;15495:9;15491:18;15484:34;15538:6;15573;15567:13;15604:6;15596;15589:22;15642:4;15631:9;15627:20;15620:27;;15666:6;15663:1;15656:17;15692:4;15682:14;;15732:2;15729:1;15719:16;15753:1;15763:388;15777:6;15774:1;15771:13;15763:388;;;15843:13;;-1:-1:-1;;;;;15881:35:1;;15869:48;;15940:4;15904:3;15982:19;;;15978:28;;15964:12;;;15957:50;16049:3;16045:19;;;;16041:28;16027:12;;;16020:50;16099:4;16090:14;;;;15913:1;16127:14;;;;15792:9;15763:388;;;15767:3;;;16160:68;16222:4;16211:9;16207:20;16203:1;16195:6;16191:14;16160:68;:::i;:::-;16237:71;16302:4;16291:9;16287:20;16280:4;16272:6;16268:17;16237:71;:::i;:::-;820:13;;813:21;16361:18;;801:34;;;;-1:-1:-1;16325:3:1;;15212:1174;-1:-1:-1;;15212:1174:1:o;16391:266::-;16479:6;16474:3;16467:19;16531:6;16524:5;16517:4;16512:3;16508:14;16495:43;-1:-1:-1;16583:1:1;16558:16;;;16576:4;16554:27;;;16547:38;;;;16639:2;16618:15;;;-1:-1:-1;;16614:29:1;16605:39;;;16601:50;;16391:266::o;16662:1422::-;16861:6;16850:9;16843:25;16904:2;16899;16888:9;16884:18;16877:30;16956:6;16943:20;16938:2;16927:9;16923:18;16916:48;16824:4;17011:2;17003:6;16999:15;16986:29;17024:31;17049:5;17024:31;:::i;:::-;-1:-1:-1;;;;;17129:14:1;;;17124:2;17109:18;;17102:42;17193:2;17181:15;;17168:29;;17206:32;17168:29;17206:32;:::i;:::-;17288:12;17279:7;17275:26;17269:3;17258:9;17254:19;17247:55;17351:2;17343:6;17339:15;17326:29;17311:44;;17364:33;17389:7;17364:33;:::i;:::-;17434:16;17428:3;17413:19;;;17406:45;;;;17514:3;17502:16;;17489:30;17482:4;17467:20;;17460:60;17568:16;;17555:30;17636:14;17632:27;;;-1:-1:-1;;17628:41:1;17604:66;;17594:94;;17684:1;17681;17674:12;17594:94;17712:31;;17824:2;17811:16;;;17766:21;17850:18;17839:30;;17836:50;;;17882:1;17879;17872:12;17836:50;17931:6;17915:14;17911:27;17902:7;17898:41;17895:61;;;17952:1;17949;17942:12;17895:61;17993:4;17987:3;17976:9;17972:19;17965:33;18015:63;18073:3;18062:9;18058:19;18050:6;18041:7;18015:63;:::i;18089:174::-;18156:12;18188:10;;;18200;;;18184:27;;18223:11;;;18220:37;;;18237:18;;:::i;:::-;18220:37;18089:174;;;;:::o;18268:521::-;18345:4;18351:6;18411:11;18398:25;18505:2;18501:7;18490:8;18474:14;18470:29;18466:43;18446:18;18442:68;18432:96;;18524:1;18521;18514:12;18432:96;18551:33;;18603:20;;;-1:-1:-1;18646:18:1;18635:30;;18632:50;;;18678:1;18675;18668:12;18632:50;18711:4;18699:17;;-1:-1:-1;18742:14:1;18738:27;;;18728:38;;18725:58;;;18779:1;18776;18769:12;18794:412;-1:-1:-1;;;;;19007:32:1;;18989:51;;19076:2;19071;19056:18;;19049:30;;;-1:-1:-1;;19096:61:1;;19138:18;;19130:6;19122;19096:61;:::i;:::-;19088:69;;19193:6;19188:2;19177:9;19173:18;19166:34;18794:412;;;;;;;:::o;19572:271::-;19755:6;19747;19742:3;19729:33;19711:3;19781:16;;19806:13;;;19781:16;19572:271;-1:-1:-1;19572:271:1:o;19848:546::-;19958:4;19987:2;20016;20005:9;19998:21;20048:6;20042:13;20091:6;20086:2;20075:9;20071:18;20064:34;20116:1;20126:140;20140:6;20137:1;20134:13;20126:140;;;20235:14;;;20231:23;;20225:30;20201:17;;;20220:2;20197:26;20190:66;20155:10;;20126:140;;;20130:3;20315:1;20310:2;20301:6;20290:9;20286:22;20282:31;20275:42;20385:2;20378;20374:7;20369:2;20361:6;20357:15;20353:29;20342:9;20338:45;20334:54;20326:62;;;;19848:546;;;;:::o;20802:127::-;20863:10;20858:3;20854:20;20851:1;20844:31;20894:4;20891:1;20884:15;20918:4;20915:1;20908:15
Swarm Source
ipfs://789e10e5d6588dc4b26dba62aaa06971ed6ac6cbd43499f78a57e1d8415d671c
Loading...
Loading
Loading...
Loading
Loading...
Loading
Net Worth in USD
$0.00
Net Worth in FRAX
0
Token Allocations
FRAX
100.00%
Multichain Portfolio | 35 Chains
| Chain | Token | Portfolio % | Price | Amount | Value |
|---|---|---|---|---|---|
| FRAXTAL | 100.00% | $1 | 0.000000002514 | <$0.000001 |
Loading...
Loading
Loading...
Loading
Loading...
Loading
[ Download: CSV Export ]
[ Download: CSV Export ]
A contract address hosts a smart contract, which is a set of code stored on the blockchain that runs when predetermined conditions are met. Learn more about addresses in our Knowledge Base.