ETH Price: $3,300.21 (-3.49%)
Gas: 13 Gwei

Token

AnimeInBox (AIB)
 

Overview

Max Total Supply

1,500 AIB

Holders

981

Market

Volume (24H)

N/A

Min Price (24H)

N/A

Max Price (24H)

N/A

Other Info

Balance
1 AIB
0x5Ff658b5aaEAB209dF2824dc771b0798de4770e6
Loading...
Loading
Loading...
Loading
Loading...
Loading

Click here to update the token information / general information
# Exchange Pair Price  24H Volume % Volume

Contract Source Code Verified (Exact Match)

Contract Name:
AnimeInBox

Compiler Version
v0.8.7+commit.e28d00a7

Optimization Enabled:
No with 200 runs

Other Settings:
default evmVersion, None license

Contract Source Code (Solidity)

/**
 *Submitted for verification at Etherscan.io on 2023-01-02
*/

// File: @openzeppelin/contracts/utils/cryptography/MerkleProof.sol


// OpenZeppelin Contracts (last updated v4.8.0) (utils/cryptography/MerkleProof.sol)

pragma solidity ^0.8.0;

/**
 * @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 rebuild 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 totalHashes = proofFlags.length;

        // Check proof validity.
        require(leavesLen + proof.length - 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 for 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) {
            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 rebuild 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 totalHashes = proofFlags.length;

        // Check proof validity.
        require(leavesLen + proof.length - 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 for 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) {
            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)
        }
    }
}

// File: @openzeppelin/contracts/utils/Context.sol


// OpenZeppelin Contracts v4.4.1 (utils/Context.sol)

pragma solidity ^0.8.0;

/**
 * @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;
    }
}

// File: @openzeppelin/contracts/access/Ownable.sol


// OpenZeppelin Contracts (last updated v4.7.0) (access/Ownable.sol)

pragma solidity ^0.8.0;


/**
 * @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 anymore. Can only be called by the current owner.
     *
     * NOTE: Renouncing ownership will leave the contract without an owner,
     * thereby removing 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);
    }
}

// File: @openzeppelin/contracts/utils/math/Math.sol


// OpenZeppelin Contracts (last updated v4.8.0) (utils/math/Math.sol)

pragma solidity ^0.8.0;

/**
 * @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) {
                return prod0 / denominator;
            }

            // Make sure the result is less than 2^256. Also prevents denominator == 0.
            require(denominator > prod1);

            ///////////////////////////////////////////////
            // 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 10, 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 * 8) < value ? 1 : 0);
        }
    }
}

// File: @openzeppelin/contracts/utils/Strings.sol


// OpenZeppelin Contracts (last updated v4.8.0) (utils/Strings.sol)

pragma solidity ^0.8.0;


/**
 * @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 `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);
    }
}

// File: https://github.com/distractedm1nd/solmate/blob/main/src/tokens/ERC721.sol


pragma solidity >=0.8.0;

/// @notice Modern, minimalist, and gas efficient ERC-721 implementation.
/// @author Solmate (https://github.com/Rari-Capital/solmate/blob/main/src/tokens/ERC721.sol)
/// @dev Note that balanceOf does not revert if passed the zero address, in defiance of the ERC.
abstract contract ERC721 {
    /*///////////////////////////////////////////////////////////////
                                 EVENTS
    //////////////////////////////////////////////////////////////*/

    event Transfer(address indexed from, address indexed to, uint256 indexed id);

    event Approval(address indexed owner, address indexed spender, uint256 indexed id);

    event ApprovalForAll(address indexed owner, address indexed operator, bool approved);

    /*///////////////////////////////////////////////////////////////
                          METADATA STORAGE/LOGIC
    //////////////////////////////////////////////////////////////*/

    string public name;

    string public symbol;

    function tokenURI(uint256 id) public view virtual returns (string memory);

    /*///////////////////////////////////////////////////////////////
                            ERC721 STORAGE                        
    //////////////////////////////////////////////////////////////*/

    uint256 public totalSupply;

    mapping(address => uint256) public balanceOf;

    mapping(uint256 => address) public ownerOf;

    mapping(uint256 => address) public getApproved;

    mapping(address => mapping(address => bool)) public isApprovedForAll;

    /*///////////////////////////////////////////////////////////////
                              CONSTRUCTOR
    //////////////////////////////////////////////////////////////*/

    constructor(string memory _name, string memory _symbol) {
        name = _name;
        symbol = _symbol;
    }

    /*///////////////////////////////////////////////////////////////
                              ERC721 LOGIC
    //////////////////////////////////////////////////////////////*/

    function approve(address spender, uint256 id) public virtual {
        address owner = ownerOf[id];

        require(msg.sender == owner || isApprovedForAll[owner][msg.sender], "NOT_AUTHORIZED");

        getApproved[id] = spender;

        emit Approval(owner, spender, id);
    }

    function setApprovalForAll(address operator, bool approved) public virtual {
        isApprovedForAll[msg.sender][operator] = approved;

        emit ApprovalForAll(msg.sender, operator, approved);
    }

    function transferFrom(
        address from,
        address to,
        uint256 id
    ) public virtual {
        require(from == ownerOf[id], "WRONG_FROM");

        require(to != address(0), "INVALID_RECIPIENT");

        require(
            msg.sender == from || msg.sender == getApproved[id] || isApprovedForAll[from][msg.sender],
            "NOT_AUTHORIZED"
        );

        // Underflow of the sender's balance is impossible because we check for
        // ownership above and the recipient's balance can't realistically overflow.
        unchecked {
            balanceOf[from]--;

            balanceOf[to]++;
        }

        ownerOf[id] = to;

        delete getApproved[id];

        emit Transfer(from, to, id);
    }

    function safeTransferFrom(
        address from,
        address to,
        uint256 id
    ) public virtual {
        transferFrom(from, to, id);

        require(
            to.code.length == 0 ||
                ERC721TokenReceiver(to).onERC721Received(msg.sender, from, id, "") ==
                ERC721TokenReceiver.onERC721Received.selector,
            "UNSAFE_RECIPIENT"
        );
    }

    function safeTransferFrom(
        address from,
        address to,
        uint256 id,
        bytes memory data
    ) public virtual {
        transferFrom(from, to, id);

        require(
            to.code.length == 0 ||
                ERC721TokenReceiver(to).onERC721Received(msg.sender, from, id, data) ==
                ERC721TokenReceiver.onERC721Received.selector,
            "UNSAFE_RECIPIENT"
        );
    }

    /*///////////////////////////////////////////////////////////////
                              ERC165 LOGIC
    //////////////////////////////////////////////////////////////*/

    function supportsInterface(bytes4 interfaceId) public pure virtual returns (bool) {
        return
            interfaceId == 0x01ffc9a7 || // ERC165 Interface ID for ERC165
            interfaceId == 0x80ac58cd || // ERC165 Interface ID for ERC721
            interfaceId == 0x5b5e139f; // ERC165 Interface ID for ERC721Metadata
    }

    /*///////////////////////////////////////////////////////////////
                       INTERNAL MINT/BURN LOGIC
    //////////////////////////////////////////////////////////////*/

    function _mint(address to, uint256 id) internal virtual {
        require(to != address(0), "INVALID_RECIPIENT");

        require(ownerOf[id] == address(0), "ALREADY_MINTED");

        // Counter overflow is incredibly unrealistic.
        unchecked {
            totalSupply++;

            balanceOf[to]++;
        }

        ownerOf[id] = to;

        emit Transfer(address(0), to, id);
    }

    function _burn(uint256 id) internal virtual {
        address owner = ownerOf[id];

        require(ownerOf[id] != address(0), "NOT_MINTED");

        // Ownership check above ensures no underflow.
        unchecked {
            totalSupply--;

            balanceOf[owner]--;
        }

        delete ownerOf[id];

        delete getApproved[id];

        emit Transfer(owner, address(0), id);
    }

    /*///////////////////////////////////////////////////////////////
                       INTERNAL SAFE MINT LOGIC
    //////////////////////////////////////////////////////////////*/

    function _safeMint(address to, uint256 id) internal virtual {
        _mint(to, id);

        require(
            to.code.length == 0 ||
                ERC721TokenReceiver(to).onERC721Received(msg.sender, address(0), id, "") ==
                ERC721TokenReceiver.onERC721Received.selector,
            "UNSAFE_RECIPIENT"
        );
    }

    function _safeMint(
        address to,
        uint256 id,
        bytes memory data
    ) internal virtual {
        _mint(to, id);

        require(
            to.code.length == 0 ||
                ERC721TokenReceiver(to).onERC721Received(msg.sender, address(0), id, data) ==
                ERC721TokenReceiver.onERC721Received.selector,
            "UNSAFE_RECIPIENT"
        );
    }
}

/// @notice A generic interface for a contract which properly accepts ERC721 tokens.
/// @author Solmate (https://github.com/Rari-Capital/solmate/blob/main/src/tokens/ERC721.sol)
interface ERC721TokenReceiver {
    function onERC721Received(
        address operator,
        address from,
        uint256 id,
        bytes calldata data
    ) external returns (bytes4);
}

// File: AIB.sol


pragma solidity ^0.8.7;





contract AnimeInBox is ERC721, Ownable {

    address public receivingAddress = 0xE2bD4329cC72896862E78dd590202d6066eb63e6;
    using Strings for uint256;

    constructor() ERC721("AnimeInBox","AIB") {
        unchecked {
        balanceOf[receivingAddress] += 90;
        totalSupply += 90;
        for (uint256 i = 0; i < 90; i++) {
        ownerOf[i] = receivingAddress;
        emit Transfer(address(0), receivingAddress, i);
        }}
    }

    mapping(address => uint256) public amountMinted;
    uint256 public maxMintAmount = 10;
    uint256 public maxSupply = 1500;

    bytes32 public merkleRoot;

    uint256 public wlPrice = 0.02 ether;
    uint256 public publicPrice = 0.03 ether;
    
    string public baseURI;

    enum MintStatus { PAUSED, WLMINT, PUBLIC }
    MintStatus public theStatus;

    function setWLMintPrice(uint256 _price) public onlyOwner {
        wlPrice = _price;
    }

    function setPublicMintPrice(uint256 _price) public onlyOwner {
        publicPrice = _price;
    }

    function changeStatus(uint _status) public onlyOwner {
        if      (_status == 0) { theStatus = MintStatus.PAUSED; }
        else if (_status == 1) { theStatus = MintStatus.WLMINT; }
        else if (_status == 2) { theStatus = MintStatus.PUBLIC; }
    }

    function publicMint(uint256 amount) external payable {
        
        require(theStatus == MintStatus.PUBLIC, "Not the Public Phase yet");
        require(amount > 0, "Unable to mint 0 NFTs");
        require (amount <= maxMintAmount, "You are unable to mint this amount of NFTs");
        require(msg.value >= amount * publicPrice, "Not enough Ether");
        require (totalSupply + amount <= maxSupply, "Minted out supply");
        require(msg.sender == tx.origin, "Bot prevention");
        require(amountMinted[msg.sender] + amount <= maxMintAmount, "You are unable to mint this many NFTs");

        amountMinted[msg.sender] += amount;
        uint currentId = totalSupply;

        totalSupply += amount;
        balanceOf[msg.sender] += amount;
        unchecked {
            for (uint256 ii = 0; ii < amount; ii++) {
                ownerOf[currentId + ii] = msg.sender; 
                emit Transfer(address(0), msg.sender, currentId + ii);
            }
        }
    }

    function whitelistMint(bytes32[] calldata _merkleProof , uint256 amount) external payable {
        
        require(theStatus == MintStatus.WLMINT, "Not the Whitelist Phase yet");
        require(amount > 0, "Unable to mint 0 NFTs");
        require (amount <= maxMintAmount, "You are unable to mint this amount of NFTs");
        require(msg.value >= amount * wlPrice, "Not enough Ether");
        require (totalSupply + amount <= maxSupply, "Minted out supply");
        require(msg.sender == tx.origin, "Bot prevention");
        require(amountMinted[msg.sender] + amount <= maxMintAmount, "You are unable to mint this many NFTs");
        
        bytes32 leaf = keccak256(abi.encodePacked(msg.sender));
        require(MerkleProof.verify(_merkleProof, merkleRoot, leaf), "Not whitelisted");

        amountMinted[msg.sender] += amount;
        uint currentId = totalSupply;

        totalSupply += amount;
        balanceOf[msg.sender] += amount;
        unchecked { 
            for (uint256 ii = 0; ii < amount; ii++) {
                ownerOf[currentId + ii] = msg.sender; 
                emit Transfer(address(0), msg.sender, currentId + ii);
            }
        }
    }

    function tokenURI(uint256 id) public view override virtual returns (string memory) {
        return string(abi.encodePacked(baseURI, id.toString()));
    }

    function setBaseURI(string memory _baseURI) public onlyOwner {
        baseURI = _baseURI;
    }

    function changeReceivingAddress(address _receivingAddress) public onlyOwner {
        receivingAddress = _receivingAddress;
    }
    
    function airdrop(address sendTo) public onlyOwner {
        require(totalSupply < maxSupply, "Can't airdrop");
        _mint(sendTo, totalSupply);
    }
    
    function withdraw() public onlyOwner {
        (bool success, ) = payable(receivingAddress).call{value: address(this).balance}("");
        require(success, "Failed withdrawal.");
    }

    function setMerkleRoot(bytes32 _merkleRoot) public onlyOwner {
        merkleRoot = _merkleRoot;
    }
}

Contract Security Audit

Contract ABI

[{"inputs":[],"stateMutability":"nonpayable","type":"constructor"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"spender","type":"address"},{"indexed":true,"internalType":"uint256","name":"id","type":"uint256"}],"name":"Approval","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"operator","type":"address"},{"indexed":false,"internalType":"bool","name":"approved","type":"bool"}],"name":"ApprovalForAll","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"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"},{"indexed":true,"internalType":"uint256","name":"id","type":"uint256"}],"name":"Transfer","type":"event"},{"inputs":[{"internalType":"address","name":"sendTo","type":"address"}],"name":"airdrop","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"amountMinted","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"spender","type":"address"},{"internalType":"uint256","name":"id","type":"uint256"}],"name":"approve","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"balanceOf","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"baseURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"_receivingAddress","type":"address"}],"name":"changeReceivingAddress","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_status","type":"uint256"}],"name":"changeStatus","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"","type":"uint256"}],"name":"getApproved","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"},{"internalType":"address","name":"","type":"address"}],"name":"isApprovedForAll","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxMintAmount","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxSupply","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"merkleRoot","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"name","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"owner","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"","type":"uint256"}],"name":"ownerOf","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"amount","type":"uint256"}],"name":"publicMint","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"publicPrice","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"receivingAddress","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"id","type":"uint256"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"id","type":"uint256"},{"internalType":"bytes","name":"data","type":"bytes"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"operator","type":"address"},{"internalType":"bool","name":"approved","type":"bool"}],"name":"setApprovalForAll","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"_baseURI","type":"string"}],"name":"setBaseURI","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"_merkleRoot","type":"bytes32"}],"name":"setMerkleRoot","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_price","type":"uint256"}],"name":"setPublicMintPrice","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_price","type":"uint256"}],"name":"setWLMintPrice","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes4","name":"interfaceId","type":"bytes4"}],"name":"supportsInterface","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"pure","type":"function"},{"inputs":[],"name":"symbol","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"theStatus","outputs":[{"internalType":"enum AnimeInBox.MintStatus","name":"","type":"uint8"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"id","type":"uint256"}],"name":"tokenURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"totalSupply","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"id","type":"uint256"}],"name":"transferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"newOwner","type":"address"}],"name":"transferOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32[]","name":"_merkleProof","type":"bytes32[]"},{"internalType":"uint256","name":"amount","type":"uint256"}],"name":"whitelistMint","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"withdraw","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"wlPrice","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"}]

608060405273e2bd4329cc72896862e78dd590202d6066eb63e6600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550600a80556105dc600b5566470de4df820000600d55666a94d74f430000600e553480156200008657600080fd5b506040518060400160405280600a81526020017f416e696d65496e426f78000000000000000000000000000000000000000000008152506040518060400160405280600381526020017f414942000000000000000000000000000000000000000000000000000000000081525081600090805190602001906200010b929190620003aa565b50806001908051906020019062000124929190620003aa565b505050620001476200013b620002dc60201b60201c565b620002e460201b60201c565b605a60036000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282540192505081905550605a60026000828254019250508190555060005b605a811015620002d557600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff166004600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555080600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a48080600101915050620001cb565b50620004bf565b600033905090565b6000600760009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600760006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b828054620003b8906200045a565b90600052602060002090601f016020900481019282620003dc576000855562000428565b82601f10620003f757805160ff191683800117855562000428565b8280016001018555821562000428579182015b82811115620004275782518255916020019190600101906200040a565b5b5090506200043791906200043b565b5090565b5b80821115620004565760008160009055506001016200043c565b5090565b600060028204905060018216806200047357607f821691505b602082108114156200048a576200048962000490565b5b50919050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b613e4f80620004cf6000396000f3fe60806040526004361061020f5760003560e01c80636352211e11610118578063b88d4fde116100a0578063e1e62b021161006f578063e1e62b021461075d578063e8025d7714610786578063e985e9c5146107af578063f2fde38b146107ec578063fd7c074f146108155761020f565b8063b88d4fde146106a1578063c7f8d01a146106ca578063c87b56dd146106f5578063d5abeb01146107325761020f565b80637cb64759116100e75780637cb64759146105ce5780638da5cb5b146105f757806395d89b4114610622578063a22cb4651461064d578063a945bf80146106765761020f565b80636352211e146105125780636c0360eb1461054f57806370a082311461057a578063715018a6146105b75761020f565b80632904e6d91161019b57806342842e0e1161016a57806342842e0e1461042f578063438a67e71461045857806355f804b3146104955780635d82cf6e146104be5780636102ca36146104e75761020f565b80632904e6d9146103b55780632db11544146103d15780632eb4a7ab146103ed5780633ccfd60b146104185761020f565b806318160ddd116101e257806318160ddd146102e25780631db87be81461030d57806321860a0514610338578063239c70ae1461036157806323b872dd1461038c5761020f565b806301ffc9a71461021457806306fdde0314610251578063081812fc1461027c578063095ea7b3146102b9575b600080fd5b34801561022057600080fd5b5061023b60048036038101906102369190612cb3565b61083e565b60405161024891906132c8565b60405180910390f35b34801561025d57600080fd5b506102666108d0565b6040516102739190613319565b60405180910390f35b34801561028857600080fd5b506102a3600480360381019061029e9190612d56565b61095e565b6040516102b09190613217565b60405180910390f35b3480156102c557600080fd5b506102e060048036038101906102db9190612be6565b610991565b005b3480156102ee57600080fd5b506102f7610b7a565b604051610304919061357b565b60405180910390f35b34801561031957600080fd5b50610322610b80565b60405161032f9190613217565b60405180910390f35b34801561034457600080fd5b5061035f600480360381019061035a9190612a63565b610ba6565b005b34801561036d57600080fd5b50610376610c03565b604051610383919061357b565b60405180910390f35b34801561039857600080fd5b506103b360048036038101906103ae9190612ad0565b610c09565b005b6103cf60048036038101906103ca9190612c26565b611009565b005b6103eb60048036038101906103e69190612d56565b6114fc565b005b3480156103f957600080fd5b50610402611933565b60405161040f91906132e3565b60405180910390f35b34801561042457600080fd5b5061042d611939565b005b34801561043b57600080fd5b5061045660048036038101906104519190612ad0565b611a12565b005b34801561046457600080fd5b5061047f600480360381019061047a9190612a63565b611b59565b60405161048c919061357b565b60405180910390f35b3480156104a157600080fd5b506104bc60048036038101906104b79190612d0d565b611b71565b005b3480156104ca57600080fd5b506104e560048036038101906104e09190612d56565b611b93565b005b3480156104f357600080fd5b506104fc611ba5565b60405161050991906132fe565b60405180910390f35b34801561051e57600080fd5b5061053960048036038101906105349190612d56565b611bb8565b6040516105469190613217565b60405180910390f35b34801561055b57600080fd5b50610564611beb565b6040516105719190613319565b60405180910390f35b34801561058657600080fd5b506105a1600480360381019061059c9190612a63565b611c79565b6040516105ae919061357b565b60405180910390f35b3480156105c357600080fd5b506105cc611c91565b005b3480156105da57600080fd5b506105f560048036038101906105f09190612c86565b611ca5565b005b34801561060357600080fd5b5061060c611cb7565b6040516106199190613217565b60405180910390f35b34801561062e57600080fd5b50610637611ce1565b6040516106449190613319565b60405180910390f35b34801561065957600080fd5b50610674600480360381019061066f9190612ba6565b611d6f565b005b34801561068257600080fd5b5061068b611e6c565b604051610698919061357b565b60405180910390f35b3480156106ad57600080fd5b506106c860048036038101906106c39190612b23565b611e72565b005b3480156106d657600080fd5b506106df611fbc565b6040516106ec919061357b565b60405180910390f35b34801561070157600080fd5b5061071c60048036038101906107179190612d56565b611fc2565b6040516107299190613319565b60405180910390f35b34801561073e57600080fd5b50610747611ff6565b604051610754919061357b565b60405180910390f35b34801561076957600080fd5b50610784600480360381019061077f9190612d56565b611ffc565b005b34801561079257600080fd5b506107ad60048036038101906107a89190612d56565b61200e565b005b3480156107bb57600080fd5b506107d660048036038101906107d19190612a90565b6120c2565b6040516107e391906132c8565b60405180910390f35b3480156107f857600080fd5b50610813600480360381019061080e9190612a63565b6120f1565b005b34801561082157600080fd5b5061083c60048036038101906108379190612a63565b612175565b005b60006301ffc9a760e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916148061089957506380ac58cd60e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b806108c95750635b5e139f60e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b9050919050565b600080546108dd90613815565b80601f016020809104026020016040519081016040528092919081815260200182805461090990613815565b80156109565780601f1061092b57610100808354040283529160200191610956565b820191906000526020600020905b81548152906001019060200180831161093957829003601f168201915b505050505081565b60056020528060005260406000206000915054906101000a900473ffffffffffffffffffffffffffffffffffffffff1681565b60006004600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1690508073ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff161480610a895750600660008273ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff165b610ac8576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610abf906134fb565b60405180910390fd5b826005600084815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550818373ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff167f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92560405160405180910390a4505050565b60025481565b600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1681565b610bae6121c1565b600b5460025410610bf4576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610beb9061339b565b60405180910390fd5b610c008160025461223f565b50565b600a5481565b6004600082815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff1614610caa576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610ca19061355b565b60405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415610d1a576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610d11906133bb565b60405180910390fd5b8273ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff161480610db257506005600082815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff16145b80610e435750600660008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff165b610e82576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610e79906134fb565b60405180910390fd5b600360008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000815480929190600190039190505550600360008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008154809291906001019190505550816004600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055506005600082815260200190815260200160002060006101000a81549073ffffffffffffffffffffffffffffffffffffffff0219169055808273ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4505050565b6001600281111561101d5761101c613943565b5b601060009054906101000a900460ff16600281111561103f5761103e613943565b5b1461107f576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016110769061351b565b60405180910390fd5b600081116110c2576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016110b9906133fb565b60405180910390fd5b600a54811115611107576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016110fe9061343b565b60405180910390fd5b600d548161111591906136d6565b341015611157576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161114e9061349b565b60405180910390fd5b600b54816002546111689190613680565b11156111a9576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016111a09061333b565b60405180910390fd5b3273ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff1614611217576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161120e906133db565b60405180910390fd5b600a5481600960003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020546112659190613680565b11156112a6576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161129d9061353b565b60405180910390fd5b6000336040516020016112b991906131c3565b60405160208183030381529060405280519060200120905061131f848480806020026020016040519081016040528093929190818152602001838360200280828437600081840152601f19601f82011690508083019250505050505050600c5483612464565b61135e576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016113559061341b565b60405180910390fd5b81600960003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282546113ad9190613680565b925050819055506000600254905082600260008282546113cd9190613680565b9250508190555082600360003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282546114239190613680565b9250508190555060005b838110156114f4573360046000838501815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508082013373ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4808060010191505061142d565b505050505050565b60028081111561150f5761150e613943565b5b601060009054906101000a900460ff16600281111561153157611530613943565b5b14611571576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611568906134bb565b60405180910390fd5b600081116115b4576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016115ab906133fb565b60405180910390fd5b600a548111156115f9576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016115f09061343b565b60405180910390fd5b600e548161160791906136d6565b341015611649576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016116409061349b565b60405180910390fd5b600b548160025461165a9190613680565b111561169b576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016116929061333b565b60405180910390fd5b3273ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff1614611709576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611700906133db565b60405180910390fd5b600a5481600960003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020546117579190613680565b1115611798576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161178f9061353b565b60405180910390fd5b80600960003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282546117e79190613680565b925050819055506000600254905081600260008282546118079190613680565b9250508190555081600360003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600082825461185d9190613680565b9250508190555060005b8281101561192e573360046000838501815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508082013373ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a48080600101915050611867565b505050565b600c5481565b6119416121c1565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff164760405161198990613202565b60006040518083038185875af1925050503d80600081146119c6576040519150601f19603f3d011682016040523d82523d6000602084013e6119cb565b606091505b5050905080611a0f576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611a069061337b565b60405180910390fd5b50565b611a1d838383610c09565b60008273ffffffffffffffffffffffffffffffffffffffff163b1480611b15575063150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff19168273ffffffffffffffffffffffffffffffffffffffff1663150b7a023386856040518463ffffffff1660e01b8152600401611aa29392919061327e565b602060405180830381600087803b158015611abc57600080fd5b505af1158015611ad0573d6000803e3d6000fd5b505050506040513d601f19601f82011682018060405250810190611af49190612ce0565b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b611b54576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611b4b9061345b565b60405180910390fd5b505050565b60096020528060005260406000206000915090505481565b611b796121c1565b80600f9080519060200190611b8f92919061280c565b5050565b611b9b6121c1565b80600e8190555050565b601060009054906101000a900460ff1681565b60046020528060005260406000206000915054906101000a900473ffffffffffffffffffffffffffffffffffffffff1681565b600f8054611bf890613815565b80601f0160208091040260200160405190810160405280929190818152602001828054611c2490613815565b8015611c715780601f10611c4657610100808354040283529160200191611c71565b820191906000526020600020905b815481529060010190602001808311611c5457829003601f168201915b505050505081565b60036020528060005260406000206000915090505481565b611c996121c1565b611ca3600061247b565b565b611cad6121c1565b80600c8190555050565b6000600760009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b60018054611cee90613815565b80601f0160208091040260200160405190810160405280929190818152602001828054611d1a90613815565b8015611d675780601f10611d3c57610100808354040283529160200191611d67565b820191906000526020600020905b815481529060010190602001808311611d4a57829003601f168201915b505050505081565b80600660003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060006101000a81548160ff0219169083151502179055508173ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff167f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c3183604051611e6091906132c8565b60405180910390a35050565b600e5481565b611e7d848484610c09565b60008373ffffffffffffffffffffffffffffffffffffffff163b1480611f77575063150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff19168373ffffffffffffffffffffffffffffffffffffffff1663150b7a02338786866040518563ffffffff1660e01b8152600401611f049493929190613232565b602060405180830381600087803b158015611f1e57600080fd5b505af1158015611f32573d6000803e3d6000fd5b505050506040513d601f19601f82011682018060405250810190611f569190612ce0565b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b611fb6576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611fad9061345b565b60405180910390fd5b50505050565b600d5481565b6060600f611fcf83612541565b604051602001611fe09291906131de565b6040516020818303038152906040529050919050565b600b5481565b6120046121c1565b80600d8190555050565b6120166121c1565b600081141561204f576000601060006101000a81548160ff0219169083600281111561204557612044613943565b5b02179055506120bf565b6001811415612088576001601060006101000a81548160ff0219169083600281111561207e5761207d613943565b5b02179055506120be565b60028114156120bd576002601060006101000a81548160ff021916908360028111156120b7576120b6613943565b5b02179055505b5b5b50565b60066020528160005260406000206020528060005260406000206000915091509054906101000a900460ff1681565b6120f96121c1565b600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff161415612169576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016121609061335b565b60405180910390fd5b6121728161247b565b50565b61217d6121c1565b80600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555050565b6121c9612619565b73ffffffffffffffffffffffffffffffffffffffff166121e7611cb7565b73ffffffffffffffffffffffffffffffffffffffff161461223d576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016122349061347b565b60405180910390fd5b565b600073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff1614156122af576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016122a6906133bb565b60405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff166004600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1614612351576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612348906134db565b60405180910390fd5b600260008154809291906001019190505550600360008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008154809291906001019190505550816004600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550808273ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a45050565b6000826124718584612621565b1490509392505050565b6000600760009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600760006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b60606000600161255084612677565b01905060008167ffffffffffffffff81111561256f5761256e6139d0565b5b6040519080825280601f01601f1916602001820160405280156125a15781602001600182028036833780820191505090505b509050600082602001820190505b60011561260e578080600190039150507f3031323334353637383961626364656600000000000000000000000000000000600a86061a8153600a85816125f8576125f7613914565b5b04945060008514156126095761260e565b6125af565b819350505050919050565b600033905090565b60008082905060005b845181101561266c576126578286838151811061264a576126496139a1565b5b60200260200101516127ca565b9150808061266490613878565b91505061262a565b508091505092915050565b600080600090507a184f03e93ff9f4daa797ed6e38ed64bf6a1f01000000000000000083106126d5577a184f03e93ff9f4daa797ed6e38ed64bf6a1f01000000000000000083816126cb576126ca613914565b5b0492506040810190505b6d04ee2d6d415b85acef81000000008310612712576d04ee2d6d415b85acef8100000000838161270857612707613914565b5b0492506020810190505b662386f26fc10000831061274157662386f26fc10000838161273757612736613914565b5b0492506010810190505b6305f5e100831061276a576305f5e10083816127605761275f613914565b5b0492506008810190505b612710831061278f57612710838161278557612784613914565b5b0492506004810190505b606483106127b257606483816127a8576127a7613914565b5b0492506002810190505b600a83106127c1576001810190505b80915050919050565b60008183106127e2576127dd82846127f5565b6127ed565b6127ec83836127f5565b5b905092915050565b600082600052816020526040600020905092915050565b82805461281890613815565b90600052602060002090601f01602090048101928261283a5760008555612881565b82601f1061285357805160ff1916838001178555612881565b82800160010185558215612881579182015b82811115612880578251825591602001919060010190612865565b5b50905061288e9190612892565b5090565b5b808211156128ab576000816000905550600101612893565b5090565b60006128c26128bd846135bb565b613596565b9050828152602081018484840111156128de576128dd613a0e565b5b6128e98482856137d3565b509392505050565b60006129046128ff846135ec565b613596565b9050828152602081018484840111156129205761291f613a0e565b5b61292b8482856137d3565b509392505050565b60008135905061294281613da6565b92915050565b60008083601f84011261295e5761295d613a04565b5b8235905067ffffffffffffffff81111561297b5761297a6139ff565b5b60208301915083602082028301111561299757612996613a09565b5b9250929050565b6000813590506129ad81613dbd565b92915050565b6000813590506129c281613dd4565b92915050565b6000813590506129d781613deb565b92915050565b6000815190506129ec81613deb565b92915050565b600082601f830112612a0757612a06613a04565b5b8135612a178482602086016128af565b91505092915050565b600082601f830112612a3557612a34613a04565b5b8135612a458482602086016128f1565b91505092915050565b600081359050612a5d81613e02565b92915050565b600060208284031215612a7957612a78613a18565b5b6000612a8784828501612933565b91505092915050565b60008060408385031215612aa757612aa6613a18565b5b6000612ab585828601612933565b9250506020612ac685828601612933565b9150509250929050565b600080600060608486031215612ae957612ae8613a18565b5b6000612af786828701612933565b9350506020612b0886828701612933565b9250506040612b1986828701612a4e565b9150509250925092565b60008060008060808587031215612b3d57612b3c613a18565b5b6000612b4b87828801612933565b9450506020612b5c87828801612933565b9350506040612b6d87828801612a4e565b925050606085013567ffffffffffffffff811115612b8e57612b8d613a13565b5b612b9a878288016129f2565b91505092959194509250565b60008060408385031215612bbd57612bbc613a18565b5b6000612bcb85828601612933565b9250506020612bdc8582860161299e565b9150509250929050565b60008060408385031215612bfd57612bfc613a18565b5b6000612c0b85828601612933565b9250506020612c1c85828601612a4e565b9150509250929050565b600080600060408486031215612c3f57612c3e613a18565b5b600084013567ffffffffffffffff811115612c5d57612c5c613a13565b5b612c6986828701612948565b93509350506020612c7c86828701612a4e565b9150509250925092565b600060208284031215612c9c57612c9b613a18565b5b6000612caa848285016129b3565b91505092915050565b600060208284031215612cc957612cc8613a18565b5b6000612cd7848285016129c8565b91505092915050565b600060208284031215612cf657612cf5613a18565b5b6000612d04848285016129dd565b91505092915050565b600060208284031215612d2357612d22613a18565b5b600082013567ffffffffffffffff811115612d4157612d40613a13565b5b612d4d84828501612a20565b91505092915050565b600060208284031215612d6c57612d6b613a18565b5b6000612d7a84828501612a4e565b91505092915050565b612d8c81613730565b82525050565b612da3612d9e82613730565b6138c1565b82525050565b612db281613742565b82525050565b612dc18161374e565b82525050565b6000612dd282613632565b612ddc8185613648565b9350612dec8185602086016137e2565b612df581613a1d565b840191505092915050565b612e09816137c1565b82525050565b6000612e1a8261363d565b612e248185613664565b9350612e348185602086016137e2565b612e3d81613a1d565b840191505092915050565b6000612e538261363d565b612e5d8185613675565b9350612e6d8185602086016137e2565b80840191505092915050565b60008154612e8681613815565b612e908186613675565b94506001821660008114612eab5760018114612ebc57612eef565b60ff19831686528186019350612eef565b612ec58561361d565b60005b83811015612ee757815481890152600182019150602081019050612ec8565b838801955050505b50505092915050565b6000612f05601183613664565b9150612f1082613a3b565b602082019050919050565b6000612f28602683613664565b9150612f3382613a64565b604082019050919050565b6000612f4b601283613664565b9150612f5682613ab3565b602082019050919050565b6000612f6e600d83613664565b9150612f7982613adc565b602082019050919050565b6000612f91601183613664565b9150612f9c82613b05565b602082019050919050565b6000612fb4600e83613664565b9150612fbf82613b2e565b602082019050919050565b6000612fd7601583613664565b9150612fe282613b57565b602082019050919050565b6000612ffa600f83613664565b915061300582613b80565b602082019050919050565b600061301d602a83613664565b915061302882613ba9565b604082019050919050565b6000613040601083613664565b915061304b82613bf8565b602082019050919050565b6000613063602083613664565b915061306e82613c21565b602082019050919050565b6000613086600083613648565b915061309182613c4a565b600082019050919050565b60006130a9600083613659565b91506130b482613c4a565b600082019050919050565b60006130cc601083613664565b91506130d782613c4d565b602082019050919050565b60006130ef601883613664565b91506130fa82613c76565b602082019050919050565b6000613112600e83613664565b915061311d82613c9f565b602082019050919050565b6000613135600e83613664565b915061314082613cc8565b602082019050919050565b6000613158601b83613664565b915061316382613cf1565b602082019050919050565b600061317b602583613664565b915061318682613d1a565b604082019050919050565b600061319e600a83613664565b91506131a982613d69565b602082019050919050565b6131bd816137b7565b82525050565b60006131cf8284612d92565b60148201915081905092915050565b60006131ea8285612e79565b91506131f68284612e48565b91508190509392505050565b600061320d8261309c565b9150819050919050565b600060208201905061322c6000830184612d83565b92915050565b60006080820190506132476000830187612d83565b6132546020830186612d83565b61326160408301856131b4565b81810360608301526132738184612dc7565b905095945050505050565b60006080820190506132936000830186612d83565b6132a06020830185612d83565b6132ad60408301846131b4565b81810360608301526132be81613079565b9050949350505050565b60006020820190506132dd6000830184612da9565b92915050565b60006020820190506132f86000830184612db8565b92915050565b60006020820190506133136000830184612e00565b92915050565b600060208201905081810360008301526133338184612e0f565b905092915050565b6000602082019050818103600083015261335481612ef8565b9050919050565b6000602082019050818103600083015261337481612f1b565b9050919050565b6000602082019050818103600083015261339481612f3e565b9050919050565b600060208201905081810360008301526133b481612f61565b9050919050565b600060208201905081810360008301526133d481612f84565b9050919050565b600060208201905081810360008301526133f481612fa7565b9050919050565b6000602082019050818103600083015261341481612fca565b9050919050565b6000602082019050818103600083015261343481612fed565b9050919050565b6000602082019050818103600083015261345481613010565b9050919050565b6000602082019050818103600083015261347481613033565b9050919050565b6000602082019050818103600083015261349481613056565b9050919050565b600060208201905081810360008301526134b4816130bf565b9050919050565b600060208201905081810360008301526134d4816130e2565b9050919050565b600060208201905081810360008301526134f481613105565b9050919050565b6000602082019050818103600083015261351481613128565b9050919050565b600060208201905081810360008301526135348161314b565b9050919050565b600060208201905081810360008301526135548161316e565b9050919050565b6000602082019050818103600083015261357481613191565b9050919050565b600060208201905061359060008301846131b4565b92915050565b60006135a06135b1565b90506135ac8282613847565b919050565b6000604051905090565b600067ffffffffffffffff8211156135d6576135d56139d0565b5b6135df82613a1d565b9050602081019050919050565b600067ffffffffffffffff821115613607576136066139d0565b5b61361082613a1d565b9050602081019050919050565b60008190508160005260206000209050919050565b600081519050919050565b600081519050919050565b600082825260208201905092915050565b600081905092915050565b600082825260208201905092915050565b600081905092915050565b600061368b826137b7565b9150613696836137b7565b9250827fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff038211156136cb576136ca6138e5565b5b828201905092915050565b60006136e1826137b7565b91506136ec836137b7565b9250817fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff0483118215151615613725576137246138e5565b5b828202905092915050565b600061373b82613797565b9050919050565b60008115159050919050565b6000819050919050565b60007fffffffff0000000000000000000000000000000000000000000000000000000082169050919050565b600081905061379282613d92565b919050565b600073ffffffffffffffffffffffffffffffffffffffff82169050919050565b6000819050919050565b60006137cc82613784565b9050919050565b82818337600083830152505050565b60005b838110156138005780820151818401526020810190506137e5565b8381111561380f576000848401525b50505050565b6000600282049050600182168061382d57607f821691505b6020821081141561384157613840613972565b5b50919050565b61385082613a1d565b810181811067ffffffffffffffff8211171561386f5761386e6139d0565b5b80604052505050565b6000613883826137b7565b91507fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff8214156138b6576138b56138e5565b5b600182019050919050565b60006138cc826138d3565b9050919050565b60006138de82613a2e565b9050919050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602160045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b600080fd5b600080fd5b600080fd5b600080fd5b600080fd5b600080fd5b6000601f19601f8301169050919050565b60008160601b9050919050565b7f4d696e746564206f757420737570706c79000000000000000000000000000000600082015250565b7f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160008201527f6464726573730000000000000000000000000000000000000000000000000000602082015250565b7f4661696c6564207769746864726177616c2e0000000000000000000000000000600082015250565b7f43616e27742061697264726f7000000000000000000000000000000000000000600082015250565b7f494e56414c49445f524543495049454e54000000000000000000000000000000600082015250565b7f426f742070726576656e74696f6e000000000000000000000000000000000000600082015250565b7f556e61626c6520746f206d696e742030204e4654730000000000000000000000600082015250565b7f4e6f742077686974656c69737465640000000000000000000000000000000000600082015250565b7f596f752061726520756e61626c6520746f206d696e74207468697320616d6f7560008201527f6e74206f66204e46547300000000000000000000000000000000000000000000602082015250565b7f554e534146455f524543495049454e5400000000000000000000000000000000600082015250565b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b50565b7f4e6f7420656e6f75676820457468657200000000000000000000000000000000600082015250565b7f4e6f7420746865205075626c6963205068617365207965740000000000000000600082015250565b7f414c52454144595f4d494e544544000000000000000000000000000000000000600082015250565b7f4e4f545f415554484f52495a4544000000000000000000000000000000000000600082015250565b7f4e6f74207468652057686974656c697374205068617365207965740000000000600082015250565b7f596f752061726520756e61626c6520746f206d696e742074686973206d616e7960008201527f204e465473000000000000000000000000000000000000000000000000000000602082015250565b7f57524f4e475f46524f4d00000000000000000000000000000000000000000000600082015250565b60038110613da357613da2613943565b5b50565b613daf81613730565b8114613dba57600080fd5b50565b613dc681613742565b8114613dd157600080fd5b50565b613ddd8161374e565b8114613de857600080fd5b50565b613df481613758565b8114613dff57600080fd5b50565b613e0b816137b7565b8114613e1657600080fd5b5056fea26469706673582212206db58f9eb5afd7d9ba1323832d1f50afd7528007dc0b8799366788efc8014e9e64736f6c63430008070033

Deployed Bytecode

0x60806040526004361061020f5760003560e01c80636352211e11610118578063b88d4fde116100a0578063e1e62b021161006f578063e1e62b021461075d578063e8025d7714610786578063e985e9c5146107af578063f2fde38b146107ec578063fd7c074f146108155761020f565b8063b88d4fde146106a1578063c7f8d01a146106ca578063c87b56dd146106f5578063d5abeb01146107325761020f565b80637cb64759116100e75780637cb64759146105ce5780638da5cb5b146105f757806395d89b4114610622578063a22cb4651461064d578063a945bf80146106765761020f565b80636352211e146105125780636c0360eb1461054f57806370a082311461057a578063715018a6146105b75761020f565b80632904e6d91161019b57806342842e0e1161016a57806342842e0e1461042f578063438a67e71461045857806355f804b3146104955780635d82cf6e146104be5780636102ca36146104e75761020f565b80632904e6d9146103b55780632db11544146103d15780632eb4a7ab146103ed5780633ccfd60b146104185761020f565b806318160ddd116101e257806318160ddd146102e25780631db87be81461030d57806321860a0514610338578063239c70ae1461036157806323b872dd1461038c5761020f565b806301ffc9a71461021457806306fdde0314610251578063081812fc1461027c578063095ea7b3146102b9575b600080fd5b34801561022057600080fd5b5061023b60048036038101906102369190612cb3565b61083e565b60405161024891906132c8565b60405180910390f35b34801561025d57600080fd5b506102666108d0565b6040516102739190613319565b60405180910390f35b34801561028857600080fd5b506102a3600480360381019061029e9190612d56565b61095e565b6040516102b09190613217565b60405180910390f35b3480156102c557600080fd5b506102e060048036038101906102db9190612be6565b610991565b005b3480156102ee57600080fd5b506102f7610b7a565b604051610304919061357b565b60405180910390f35b34801561031957600080fd5b50610322610b80565b60405161032f9190613217565b60405180910390f35b34801561034457600080fd5b5061035f600480360381019061035a9190612a63565b610ba6565b005b34801561036d57600080fd5b50610376610c03565b604051610383919061357b565b60405180910390f35b34801561039857600080fd5b506103b360048036038101906103ae9190612ad0565b610c09565b005b6103cf60048036038101906103ca9190612c26565b611009565b005b6103eb60048036038101906103e69190612d56565b6114fc565b005b3480156103f957600080fd5b50610402611933565b60405161040f91906132e3565b60405180910390f35b34801561042457600080fd5b5061042d611939565b005b34801561043b57600080fd5b5061045660048036038101906104519190612ad0565b611a12565b005b34801561046457600080fd5b5061047f600480360381019061047a9190612a63565b611b59565b60405161048c919061357b565b60405180910390f35b3480156104a157600080fd5b506104bc60048036038101906104b79190612d0d565b611b71565b005b3480156104ca57600080fd5b506104e560048036038101906104e09190612d56565b611b93565b005b3480156104f357600080fd5b506104fc611ba5565b60405161050991906132fe565b60405180910390f35b34801561051e57600080fd5b5061053960048036038101906105349190612d56565b611bb8565b6040516105469190613217565b60405180910390f35b34801561055b57600080fd5b50610564611beb565b6040516105719190613319565b60405180910390f35b34801561058657600080fd5b506105a1600480360381019061059c9190612a63565b611c79565b6040516105ae919061357b565b60405180910390f35b3480156105c357600080fd5b506105cc611c91565b005b3480156105da57600080fd5b506105f560048036038101906105f09190612c86565b611ca5565b005b34801561060357600080fd5b5061060c611cb7565b6040516106199190613217565b60405180910390f35b34801561062e57600080fd5b50610637611ce1565b6040516106449190613319565b60405180910390f35b34801561065957600080fd5b50610674600480360381019061066f9190612ba6565b611d6f565b005b34801561068257600080fd5b5061068b611e6c565b604051610698919061357b565b60405180910390f35b3480156106ad57600080fd5b506106c860048036038101906106c39190612b23565b611e72565b005b3480156106d657600080fd5b506106df611fbc565b6040516106ec919061357b565b60405180910390f35b34801561070157600080fd5b5061071c60048036038101906107179190612d56565b611fc2565b6040516107299190613319565b60405180910390f35b34801561073e57600080fd5b50610747611ff6565b604051610754919061357b565b60405180910390f35b34801561076957600080fd5b50610784600480360381019061077f9190612d56565b611ffc565b005b34801561079257600080fd5b506107ad60048036038101906107a89190612d56565b61200e565b005b3480156107bb57600080fd5b506107d660048036038101906107d19190612a90565b6120c2565b6040516107e391906132c8565b60405180910390f35b3480156107f857600080fd5b50610813600480360381019061080e9190612a63565b6120f1565b005b34801561082157600080fd5b5061083c60048036038101906108379190612a63565b612175565b005b60006301ffc9a760e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916148061089957506380ac58cd60e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b806108c95750635b5e139f60e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b9050919050565b600080546108dd90613815565b80601f016020809104026020016040519081016040528092919081815260200182805461090990613815565b80156109565780601f1061092b57610100808354040283529160200191610956565b820191906000526020600020905b81548152906001019060200180831161093957829003601f168201915b505050505081565b60056020528060005260406000206000915054906101000a900473ffffffffffffffffffffffffffffffffffffffff1681565b60006004600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1690508073ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff161480610a895750600660008273ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff165b610ac8576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610abf906134fb565b60405180910390fd5b826005600084815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550818373ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff167f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92560405160405180910390a4505050565b60025481565b600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1681565b610bae6121c1565b600b5460025410610bf4576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610beb9061339b565b60405180910390fd5b610c008160025461223f565b50565b600a5481565b6004600082815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff1614610caa576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610ca19061355b565b60405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415610d1a576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610d11906133bb565b60405180910390fd5b8273ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff161480610db257506005600082815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff16145b80610e435750600660008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff165b610e82576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610e79906134fb565b60405180910390fd5b600360008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000815480929190600190039190505550600360008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008154809291906001019190505550816004600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055506005600082815260200190815260200160002060006101000a81549073ffffffffffffffffffffffffffffffffffffffff0219169055808273ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4505050565b6001600281111561101d5761101c613943565b5b601060009054906101000a900460ff16600281111561103f5761103e613943565b5b1461107f576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016110769061351b565b60405180910390fd5b600081116110c2576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016110b9906133fb565b60405180910390fd5b600a54811115611107576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016110fe9061343b565b60405180910390fd5b600d548161111591906136d6565b341015611157576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161114e9061349b565b60405180910390fd5b600b54816002546111689190613680565b11156111a9576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016111a09061333b565b60405180910390fd5b3273ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff1614611217576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161120e906133db565b60405180910390fd5b600a5481600960003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020546112659190613680565b11156112a6576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161129d9061353b565b60405180910390fd5b6000336040516020016112b991906131c3565b60405160208183030381529060405280519060200120905061131f848480806020026020016040519081016040528093929190818152602001838360200280828437600081840152601f19601f82011690508083019250505050505050600c5483612464565b61135e576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016113559061341b565b60405180910390fd5b81600960003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282546113ad9190613680565b925050819055506000600254905082600260008282546113cd9190613680565b9250508190555082600360003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282546114239190613680565b9250508190555060005b838110156114f4573360046000838501815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508082013373ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4808060010191505061142d565b505050505050565b60028081111561150f5761150e613943565b5b601060009054906101000a900460ff16600281111561153157611530613943565b5b14611571576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611568906134bb565b60405180910390fd5b600081116115b4576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016115ab906133fb565b60405180910390fd5b600a548111156115f9576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016115f09061343b565b60405180910390fd5b600e548161160791906136d6565b341015611649576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016116409061349b565b60405180910390fd5b600b548160025461165a9190613680565b111561169b576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016116929061333b565b60405180910390fd5b3273ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff1614611709576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611700906133db565b60405180910390fd5b600a5481600960003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020546117579190613680565b1115611798576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161178f9061353b565b60405180910390fd5b80600960003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282546117e79190613680565b925050819055506000600254905081600260008282546118079190613680565b9250508190555081600360003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600082825461185d9190613680565b9250508190555060005b8281101561192e573360046000838501815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508082013373ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a48080600101915050611867565b505050565b600c5481565b6119416121c1565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff164760405161198990613202565b60006040518083038185875af1925050503d80600081146119c6576040519150601f19603f3d011682016040523d82523d6000602084013e6119cb565b606091505b5050905080611a0f576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611a069061337b565b60405180910390fd5b50565b611a1d838383610c09565b60008273ffffffffffffffffffffffffffffffffffffffff163b1480611b15575063150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff19168273ffffffffffffffffffffffffffffffffffffffff1663150b7a023386856040518463ffffffff1660e01b8152600401611aa29392919061327e565b602060405180830381600087803b158015611abc57600080fd5b505af1158015611ad0573d6000803e3d6000fd5b505050506040513d601f19601f82011682018060405250810190611af49190612ce0565b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b611b54576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611b4b9061345b565b60405180910390fd5b505050565b60096020528060005260406000206000915090505481565b611b796121c1565b80600f9080519060200190611b8f92919061280c565b5050565b611b9b6121c1565b80600e8190555050565b601060009054906101000a900460ff1681565b60046020528060005260406000206000915054906101000a900473ffffffffffffffffffffffffffffffffffffffff1681565b600f8054611bf890613815565b80601f0160208091040260200160405190810160405280929190818152602001828054611c2490613815565b8015611c715780601f10611c4657610100808354040283529160200191611c71565b820191906000526020600020905b815481529060010190602001808311611c5457829003601f168201915b505050505081565b60036020528060005260406000206000915090505481565b611c996121c1565b611ca3600061247b565b565b611cad6121c1565b80600c8190555050565b6000600760009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b60018054611cee90613815565b80601f0160208091040260200160405190810160405280929190818152602001828054611d1a90613815565b8015611d675780601f10611d3c57610100808354040283529160200191611d67565b820191906000526020600020905b815481529060010190602001808311611d4a57829003601f168201915b505050505081565b80600660003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060006101000a81548160ff0219169083151502179055508173ffffffffffffffffffffffffffffffffffffffff163373ffffffffffffffffffffffffffffffffffffffff167f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c3183604051611e6091906132c8565b60405180910390a35050565b600e5481565b611e7d848484610c09565b60008373ffffffffffffffffffffffffffffffffffffffff163b1480611f77575063150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff19168373ffffffffffffffffffffffffffffffffffffffff1663150b7a02338786866040518563ffffffff1660e01b8152600401611f049493929190613232565b602060405180830381600087803b158015611f1e57600080fd5b505af1158015611f32573d6000803e3d6000fd5b505050506040513d601f19601f82011682018060405250810190611f569190612ce0565b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b611fb6576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611fad9061345b565b60405180910390fd5b50505050565b600d5481565b6060600f611fcf83612541565b604051602001611fe09291906131de565b6040516020818303038152906040529050919050565b600b5481565b6120046121c1565b80600d8190555050565b6120166121c1565b600081141561204f576000601060006101000a81548160ff0219169083600281111561204557612044613943565b5b02179055506120bf565b6001811415612088576001601060006101000a81548160ff0219169083600281111561207e5761207d613943565b5b02179055506120be565b60028114156120bd576002601060006101000a81548160ff021916908360028111156120b7576120b6613943565b5b02179055505b5b5b50565b60066020528160005260406000206020528060005260406000206000915091509054906101000a900460ff1681565b6120f96121c1565b600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff161415612169576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016121609061335b565b60405180910390fd5b6121728161247b565b50565b61217d6121c1565b80600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555050565b6121c9612619565b73ffffffffffffffffffffffffffffffffffffffff166121e7611cb7565b73ffffffffffffffffffffffffffffffffffffffff161461223d576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016122349061347b565b60405180910390fd5b565b600073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff1614156122af576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016122a6906133bb565b60405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff166004600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1614612351576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612348906134db565b60405180910390fd5b600260008154809291906001019190505550600360008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008154809291906001019190505550816004600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550808273ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a45050565b6000826124718584612621565b1490509392505050565b6000600760009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600760006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b60606000600161255084612677565b01905060008167ffffffffffffffff81111561256f5761256e6139d0565b5b6040519080825280601f01601f1916602001820160405280156125a15781602001600182028036833780820191505090505b509050600082602001820190505b60011561260e578080600190039150507f3031323334353637383961626364656600000000000000000000000000000000600a86061a8153600a85816125f8576125f7613914565b5b04945060008514156126095761260e565b6125af565b819350505050919050565b600033905090565b60008082905060005b845181101561266c576126578286838151811061264a576126496139a1565b5b60200260200101516127ca565b9150808061266490613878565b91505061262a565b508091505092915050565b600080600090507a184f03e93ff9f4daa797ed6e38ed64bf6a1f01000000000000000083106126d5577a184f03e93ff9f4daa797ed6e38ed64bf6a1f01000000000000000083816126cb576126ca613914565b5b0492506040810190505b6d04ee2d6d415b85acef81000000008310612712576d04ee2d6d415b85acef8100000000838161270857612707613914565b5b0492506020810190505b662386f26fc10000831061274157662386f26fc10000838161273757612736613914565b5b0492506010810190505b6305f5e100831061276a576305f5e10083816127605761275f613914565b5b0492506008810190505b612710831061278f57612710838161278557612784613914565b5b0492506004810190505b606483106127b257606483816127a8576127a7613914565b5b0492506002810190505b600a83106127c1576001810190505b80915050919050565b60008183106127e2576127dd82846127f5565b6127ed565b6127ec83836127f5565b5b905092915050565b600082600052816020526040600020905092915050565b82805461281890613815565b90600052602060002090601f01602090048101928261283a5760008555612881565b82601f1061285357805160ff1916838001178555612881565b82800160010185558215612881579182015b82811115612880578251825591602001919060010190612865565b5b50905061288e9190612892565b5090565b5b808211156128ab576000816000905550600101612893565b5090565b60006128c26128bd846135bb565b613596565b9050828152602081018484840111156128de576128dd613a0e565b5b6128e98482856137d3565b509392505050565b60006129046128ff846135ec565b613596565b9050828152602081018484840111156129205761291f613a0e565b5b61292b8482856137d3565b509392505050565b60008135905061294281613da6565b92915050565b60008083601f84011261295e5761295d613a04565b5b8235905067ffffffffffffffff81111561297b5761297a6139ff565b5b60208301915083602082028301111561299757612996613a09565b5b9250929050565b6000813590506129ad81613dbd565b92915050565b6000813590506129c281613dd4565b92915050565b6000813590506129d781613deb565b92915050565b6000815190506129ec81613deb565b92915050565b600082601f830112612a0757612a06613a04565b5b8135612a178482602086016128af565b91505092915050565b600082601f830112612a3557612a34613a04565b5b8135612a458482602086016128f1565b91505092915050565b600081359050612a5d81613e02565b92915050565b600060208284031215612a7957612a78613a18565b5b6000612a8784828501612933565b91505092915050565b60008060408385031215612aa757612aa6613a18565b5b6000612ab585828601612933565b9250506020612ac685828601612933565b9150509250929050565b600080600060608486031215612ae957612ae8613a18565b5b6000612af786828701612933565b9350506020612b0886828701612933565b9250506040612b1986828701612a4e565b9150509250925092565b60008060008060808587031215612b3d57612b3c613a18565b5b6000612b4b87828801612933565b9450506020612b5c87828801612933565b9350506040612b6d87828801612a4e565b925050606085013567ffffffffffffffff811115612b8e57612b8d613a13565b5b612b9a878288016129f2565b91505092959194509250565b60008060408385031215612bbd57612bbc613a18565b5b6000612bcb85828601612933565b9250506020612bdc8582860161299e565b9150509250929050565b60008060408385031215612bfd57612bfc613a18565b5b6000612c0b85828601612933565b9250506020612c1c85828601612a4e565b9150509250929050565b600080600060408486031215612c3f57612c3e613a18565b5b600084013567ffffffffffffffff811115612c5d57612c5c613a13565b5b612c6986828701612948565b93509350506020612c7c86828701612a4e565b9150509250925092565b600060208284031215612c9c57612c9b613a18565b5b6000612caa848285016129b3565b91505092915050565b600060208284031215612cc957612cc8613a18565b5b6000612cd7848285016129c8565b91505092915050565b600060208284031215612cf657612cf5613a18565b5b6000612d04848285016129dd565b91505092915050565b600060208284031215612d2357612d22613a18565b5b600082013567ffffffffffffffff811115612d4157612d40613a13565b5b612d4d84828501612a20565b91505092915050565b600060208284031215612d6c57612d6b613a18565b5b6000612d7a84828501612a4e565b91505092915050565b612d8c81613730565b82525050565b612da3612d9e82613730565b6138c1565b82525050565b612db281613742565b82525050565b612dc18161374e565b82525050565b6000612dd282613632565b612ddc8185613648565b9350612dec8185602086016137e2565b612df581613a1d565b840191505092915050565b612e09816137c1565b82525050565b6000612e1a8261363d565b612e248185613664565b9350612e348185602086016137e2565b612e3d81613a1d565b840191505092915050565b6000612e538261363d565b612e5d8185613675565b9350612e6d8185602086016137e2565b80840191505092915050565b60008154612e8681613815565b612e908186613675565b94506001821660008114612eab5760018114612ebc57612eef565b60ff19831686528186019350612eef565b612ec58561361d565b60005b83811015612ee757815481890152600182019150602081019050612ec8565b838801955050505b50505092915050565b6000612f05601183613664565b9150612f1082613a3b565b602082019050919050565b6000612f28602683613664565b9150612f3382613a64565b604082019050919050565b6000612f4b601283613664565b9150612f5682613ab3565b602082019050919050565b6000612f6e600d83613664565b9150612f7982613adc565b602082019050919050565b6000612f91601183613664565b9150612f9c82613b05565b602082019050919050565b6000612fb4600e83613664565b9150612fbf82613b2e565b602082019050919050565b6000612fd7601583613664565b9150612fe282613b57565b602082019050919050565b6000612ffa600f83613664565b915061300582613b80565b602082019050919050565b600061301d602a83613664565b915061302882613ba9565b604082019050919050565b6000613040601083613664565b915061304b82613bf8565b602082019050919050565b6000613063602083613664565b915061306e82613c21565b602082019050919050565b6000613086600083613648565b915061309182613c4a565b600082019050919050565b60006130a9600083613659565b91506130b482613c4a565b600082019050919050565b60006130cc601083613664565b91506130d782613c4d565b602082019050919050565b60006130ef601883613664565b91506130fa82613c76565b602082019050919050565b6000613112600e83613664565b915061311d82613c9f565b602082019050919050565b6000613135600e83613664565b915061314082613cc8565b602082019050919050565b6000613158601b83613664565b915061316382613cf1565b602082019050919050565b600061317b602583613664565b915061318682613d1a565b604082019050919050565b600061319e600a83613664565b91506131a982613d69565b602082019050919050565b6131bd816137b7565b82525050565b60006131cf8284612d92565b60148201915081905092915050565b60006131ea8285612e79565b91506131f68284612e48565b91508190509392505050565b600061320d8261309c565b9150819050919050565b600060208201905061322c6000830184612d83565b92915050565b60006080820190506132476000830187612d83565b6132546020830186612d83565b61326160408301856131b4565b81810360608301526132738184612dc7565b905095945050505050565b60006080820190506132936000830186612d83565b6132a06020830185612d83565b6132ad60408301846131b4565b81810360608301526132be81613079565b9050949350505050565b60006020820190506132dd6000830184612da9565b92915050565b60006020820190506132f86000830184612db8565b92915050565b60006020820190506133136000830184612e00565b92915050565b600060208201905081810360008301526133338184612e0f565b905092915050565b6000602082019050818103600083015261335481612ef8565b9050919050565b6000602082019050818103600083015261337481612f1b565b9050919050565b6000602082019050818103600083015261339481612f3e565b9050919050565b600060208201905081810360008301526133b481612f61565b9050919050565b600060208201905081810360008301526133d481612f84565b9050919050565b600060208201905081810360008301526133f481612fa7565b9050919050565b6000602082019050818103600083015261341481612fca565b9050919050565b6000602082019050818103600083015261343481612fed565b9050919050565b6000602082019050818103600083015261345481613010565b9050919050565b6000602082019050818103600083015261347481613033565b9050919050565b6000602082019050818103600083015261349481613056565b9050919050565b600060208201905081810360008301526134b4816130bf565b9050919050565b600060208201905081810360008301526134d4816130e2565b9050919050565b600060208201905081810360008301526134f481613105565b9050919050565b6000602082019050818103600083015261351481613128565b9050919050565b600060208201905081810360008301526135348161314b565b9050919050565b600060208201905081810360008301526135548161316e565b9050919050565b6000602082019050818103600083015261357481613191565b9050919050565b600060208201905061359060008301846131b4565b92915050565b60006135a06135b1565b90506135ac8282613847565b919050565b6000604051905090565b600067ffffffffffffffff8211156135d6576135d56139d0565b5b6135df82613a1d565b9050602081019050919050565b600067ffffffffffffffff821115613607576136066139d0565b5b61361082613a1d565b9050602081019050919050565b60008190508160005260206000209050919050565b600081519050919050565b600081519050919050565b600082825260208201905092915050565b600081905092915050565b600082825260208201905092915050565b600081905092915050565b600061368b826137b7565b9150613696836137b7565b9250827fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff038211156136cb576136ca6138e5565b5b828201905092915050565b60006136e1826137b7565b91506136ec836137b7565b9250817fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff0483118215151615613725576137246138e5565b5b828202905092915050565b600061373b82613797565b9050919050565b60008115159050919050565b6000819050919050565b60007fffffffff0000000000000000000000000000000000000000000000000000000082169050919050565b600081905061379282613d92565b919050565b600073ffffffffffffffffffffffffffffffffffffffff82169050919050565b6000819050919050565b60006137cc82613784565b9050919050565b82818337600083830152505050565b60005b838110156138005780820151818401526020810190506137e5565b8381111561380f576000848401525b50505050565b6000600282049050600182168061382d57607f821691505b6020821081141561384157613840613972565b5b50919050565b61385082613a1d565b810181811067ffffffffffffffff8211171561386f5761386e6139d0565b5b80604052505050565b6000613883826137b7565b91507fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff8214156138b6576138b56138e5565b5b600182019050919050565b60006138cc826138d3565b9050919050565b60006138de82613a2e565b9050919050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602160045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b600080fd5b600080fd5b600080fd5b600080fd5b600080fd5b600080fd5b6000601f19601f8301169050919050565b60008160601b9050919050565b7f4d696e746564206f757420737570706c79000000000000000000000000000000600082015250565b7f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160008201527f6464726573730000000000000000000000000000000000000000000000000000602082015250565b7f4661696c6564207769746864726177616c2e0000000000000000000000000000600082015250565b7f43616e27742061697264726f7000000000000000000000000000000000000000600082015250565b7f494e56414c49445f524543495049454e54000000000000000000000000000000600082015250565b7f426f742070726576656e74696f6e000000000000000000000000000000000000600082015250565b7f556e61626c6520746f206d696e742030204e4654730000000000000000000000600082015250565b7f4e6f742077686974656c69737465640000000000000000000000000000000000600082015250565b7f596f752061726520756e61626c6520746f206d696e74207468697320616d6f7560008201527f6e74206f66204e46547300000000000000000000000000000000000000000000602082015250565b7f554e534146455f524543495049454e5400000000000000000000000000000000600082015250565b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b50565b7f4e6f7420656e6f75676820457468657200000000000000000000000000000000600082015250565b7f4e6f7420746865205075626c6963205068617365207965740000000000000000600082015250565b7f414c52454144595f4d494e544544000000000000000000000000000000000000600082015250565b7f4e4f545f415554484f52495a4544000000000000000000000000000000000000600082015250565b7f4e6f74207468652057686974656c697374205068617365207965740000000000600082015250565b7f596f752061726520756e61626c6520746f206d696e742074686973206d616e7960008201527f204e465473000000000000000000000000000000000000000000000000000000602082015250565b7f57524f4e475f46524f4d00000000000000000000000000000000000000000000600082015250565b60038110613da357613da2613943565b5b50565b613daf81613730565b8114613dba57600080fd5b50565b613dc681613742565b8114613dd157600080fd5b50565b613ddd8161374e565b8114613de857600080fd5b50565b613df481613758565b8114613dff57600080fd5b50565b613e0b816137b7565b8114613e1657600080fd5b5056fea26469706673582212206db58f9eb5afd7d9ba1323832d1f50afd7528007dc0b8799366788efc8014e9e64736f6c63430008070033

Deployed Bytecode Sourcemap

35653:4435:0:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;32865:340;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;29415:18;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;29903:46;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;30530:289;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;29764:26;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;35701:76;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;39618:155;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;36175:33;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;31042:764;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;37989:1207;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;36975:1006;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;36255:25;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;39785:188;;;;;;;;;;;;;:::i;:::-;;31814:409;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;36121:47;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;39369:98;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;36597:100;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;36461:27;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;29852:42;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;36383:21;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;29799:44;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;12337:103;;;;;;;;;;;;;:::i;:::-;;39981:104;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;11689:87;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;29442:20;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;30827:207;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;36331:39;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;32231:439;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;36289:35;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;39204:157;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;36215:31;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;36497:92;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;36705:262;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;29958:68;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;12595:201;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;39475:131;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;32865:340;32941:4;32993:10;32978:25;;:11;:25;;;;:101;;;;33069:10;33054:25;;:11;:25;;;;32978:101;:177;;;;33145:10;33130:25;;:11;:25;;;;32978:177;32958:197;;32865:340;;;:::o;29415:18::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;29903:46::-;;;;;;;;;;;;;;;;;;;;;;:::o;30530:289::-;30602:13;30618:7;:11;30626:2;30618:11;;;;;;;;;;;;;;;;;;;;;30602:27;;30664:5;30650:19;;:10;:19;;;:58;;;;30673:16;:23;30690:5;30673:23;;;;;;;;;;;;;;;:35;30697:10;30673:35;;;;;;;;;;;;;;;;;;;;;;;;;30650:58;30642:85;;;;;;;;;;;;:::i;:::-;;;;;;;;;30758:7;30740:11;:15;30752:2;30740:15;;;;;;;;;;;;:25;;;;;;;;;;;;;;;;;;30808:2;30799:7;30783:28;;30792:5;30783:28;;;;;;;;;;;;30591:228;30530:289;;:::o;29764:26::-;;;;:::o;35701:76::-;;;;;;;;;;;;;:::o;39618:155::-;11575:13;:11;:13::i;:::-;39701:9:::1;;39687:11;;:23;39679:49;;;;;;;;;;;;:::i;:::-;;;;;;;;;39739:26;39745:6;39753:11;;39739:5;:26::i;:::-;39618:155:::0;:::o;36175:33::-;;;;:::o;31042:764::-;31178:7;:11;31186:2;31178:11;;;;;;;;;;;;;;;;;;;;;31170:19;;:4;:19;;;31162:42;;;;;;;;;;;;:::i;:::-;;;;;;;;;31239:1;31225:16;;:2;:16;;;;31217:46;;;;;;;;;;;;:::i;:::-;;;;;;;;;31312:4;31298:18;;:10;:18;;;:51;;;;31334:11;:15;31346:2;31334:15;;;;;;;;;;;;;;;;;;;;;31320:29;;:10;:29;;;31298:51;:89;;;;31353:16;:22;31370:4;31353:22;;;;;;;;;;;;;;;:34;31376:10;31353:34;;;;;;;;;;;;;;;;;;;;;;;;;31298:89;31276:153;;;;;;;;;;;;:::i;:::-;;;;;;;;;31634:9;:15;31644:4;31634:15;;;;;;;;;;;;;;;;:17;;;;;;;;;;;;;;31668:9;:13;31678:2;31668:13;;;;;;;;;;;;;;;;:15;;;;;;;;;;;;;31721:2;31707:7;:11;31715:2;31707:11;;;;;;;;;;;;:16;;;;;;;;;;;;;;;;;;31743:11;:15;31755:2;31743:15;;;;;;;;;;;;31736:22;;;;;;;;;;;31795:2;31791;31776:22;;31785:4;31776:22;;;;;;;;;;;;31042:764;;;:::o;37989:1207::-;38121:17;38108:30;;;;;;;;:::i;:::-;;:9;;;;;;;;;;;:30;;;;;;;;:::i;:::-;;;38100:70;;;;;;;;;;;;:::i;:::-;;;;;;;;;38198:1;38189:6;:10;38181:44;;;;;;;;;;;;:::i;:::-;;;;;;;;;38255:13;;38245:6;:23;;38236:79;;;;;;;;;;;;:::i;:::-;;;;;;;;;38356:7;;38347:6;:16;;;;:::i;:::-;38334:9;:29;;38326:58;;;;;;;;;;;;:::i;:::-;;;;;;;;;38428:9;;38418:6;38404:11;;:20;;;;:::i;:::-;:33;;38395:64;;;;;;;;;;;;:::i;:::-;;;;;;;;;38492:9;38478:23;;:10;:23;;;38470:50;;;;;;;;;;;;:::i;:::-;;;;;;;;;38576:13;;38566:6;38539:12;:24;38552:10;38539:24;;;;;;;;;;;;;;;;:33;;;;:::i;:::-;:50;;38531:100;;;;;;;;;;;;:::i;:::-;;;;;;;;;38652:12;38694:10;38677:28;;;;;;;;:::i;:::-;;;;;;;;;;;;;38667:39;;;;;;38652:54;;38725:50;38744:12;;38725:50;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;38758:10;;38770:4;38725:18;:50::i;:::-;38717:78;;;;;;;;;;;;:::i;:::-;;;;;;;;;38836:6;38808:12;:24;38821:10;38808:24;;;;;;;;;;;;;;;;:34;;;;;;;:::i;:::-;;;;;;;;38853:14;38870:11;;38853:28;;38909:6;38894:11;;:21;;;;;;;:::i;:::-;;;;;;;;38951:6;38926:9;:21;38936:10;38926:21;;;;;;;;;;;;;;;;:31;;;;;;;:::i;:::-;;;;;;;;38999:10;38994:184;39020:6;39015:2;:11;38994:184;;;39079:10;39053:7;:23;39073:2;39061:9;:14;39053:23;;;;;;;;;;;;:36;;;;;;;;;;;;;;;;;;39159:2;39147:9;:14;39135:10;39114:48;;39131:1;39114:48;;;;;;;;;;;;39028:4;;;;;;;38994:184;;;;38079:1117;;37989:1207;;;:::o;36975:1006::-;37070:17;37057:30;;;;;;;;:::i;:::-;;:9;;;;;;;;;;;:30;;;;;;;;:::i;:::-;;;37049:67;;;;;;;;;;;;:::i;:::-;;;;;;;;;37144:1;37135:6;:10;37127:44;;;;;;;;;;;;:::i;:::-;;;;;;;;;37201:13;;37191:6;:23;;37182:79;;;;;;;;;;;;:::i;:::-;;;;;;;;;37302:11;;37293:6;:20;;;;:::i;:::-;37280:9;:33;;37272:62;;;;;;;;;;;;:::i;:::-;;;;;;;;;37378:9;;37368:6;37354:11;;:20;;;;:::i;:::-;:33;;37345:64;;;;;;;;;;;;:::i;:::-;;;;;;;;;37442:9;37428:23;;:10;:23;;;37420:50;;;;;;;;;;;;:::i;:::-;;;;;;;;;37526:13;;37516:6;37489:12;:24;37502:10;37489:24;;;;;;;;;;;;;;;;:33;;;;:::i;:::-;:50;;37481:100;;;;;;;;;;;;:::i;:::-;;;;;;;;;37622:6;37594:12;:24;37607:10;37594:24;;;;;;;;;;;;;;;;:34;;;;;;;:::i;:::-;;;;;;;;37639:14;37656:11;;37639:28;;37695:6;37680:11;;:21;;;;;;;:::i;:::-;;;;;;;;37737:6;37712:9;:21;37722:10;37712:21;;;;;;;;;;;;;;;;:31;;;;;;;:::i;:::-;;;;;;;;37784:10;37779:184;37805:6;37800:2;:11;37779:184;;;37864:10;37838:7;:23;37858:2;37846:9;:14;37838:23;;;;;;;;;;;;:36;;;;;;;;;;;;;;;;;;37944:2;37932:9;:14;37920:10;37899:48;;37916:1;37899:48;;;;;;;;;;;;37813:4;;;;;;;37779:184;;;;37028:953;36975:1006;:::o;36255:25::-;;;;:::o;39785:188::-;11575:13;:11;:13::i;:::-;39834:12:::1;39860:16;;;;;;;;;;;39852:30;;39890:21;39852:64;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;39833:83;;;39935:7;39927:38;;;;;;;;;;;;:::i;:::-;;;;;;;;;39822:151;39785:188::o:0;31814:409::-;31938:26;31951:4;31957:2;31961;31938:12;:26::i;:::-;32017:1;31999:2;:14;;;:19;:172;;;;32126:45;;;32039:132;;;32059:2;32039:40;;;32080:10;32092:4;32098:2;32039:66;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;:132;;;;31999:172;31977:238;;;;;;;;;;;;:::i;:::-;;;;;;;;;31814:409;;;:::o;36121:47::-;;;;;;;;;;;;;;;;;:::o;39369:98::-;11575:13;:11;:13::i;:::-;39451:8:::1;39441:7;:18;;;;;;;;;;;;:::i;:::-;;39369:98:::0;:::o;36597:100::-;11575:13;:11;:13::i;:::-;36683:6:::1;36669:11;:20;;;;36597:100:::0;:::o;36461:27::-;;;;;;;;;;;;;:::o;29852:42::-;;;;;;;;;;;;;;;;;;;;;;:::o;36383:21::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;29799:44::-;;;;;;;;;;;;;;;;;:::o;12337:103::-;11575:13;:11;:13::i;:::-;12402:30:::1;12429:1;12402:18;:30::i;:::-;12337:103::o:0;39981:104::-;11575:13;:11;:13::i;:::-;40066:11:::1;40053:10;:24;;;;39981:104:::0;:::o;11689:87::-;11735:7;11762:6;;;;;;;;;;;11755:13;;11689:87;:::o;29442:20::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;30827:207::-;30954:8;30913:16;:28;30930:10;30913:28;;;;;;;;;;;;;;;:38;30942:8;30913:38;;;;;;;;;;;;;;;;:49;;;;;;;;;;;;;;;;;;31007:8;30980:46;;30995:10;30980:46;;;31017:8;30980:46;;;;;;:::i;:::-;;;;;;;;30827:207;;:::o;36331:39::-;;;;:::o;32231:439::-;32383:26;32396:4;32402:2;32406;32383:12;:26::i;:::-;32462:1;32444:2;:14;;;:19;:174;;;;32573:45;;;32484:134;;;32504:2;32484:40;;;32525:10;32537:4;32543:2;32547:4;32484:68;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;:134;;;;32444:174;32422:240;;;;;;;;;;;;:::i;:::-;;;;;;;;;32231:439;;;;:::o;36289:35::-;;;;:::o;39204:157::-;39272:13;39329:7;39338:13;:2;:11;:13::i;:::-;39312:40;;;;;;;;;:::i;:::-;;;;;;;;;;;;;39298:55;;39204:157;;;:::o;36215:31::-;;;;:::o;36497:92::-;11575:13;:11;:13::i;:::-;36575:6:::1;36565:7;:16;;;;36497:92:::0;:::o;36705:262::-;11575:13;:11;:13::i;:::-;36789:1:::1;36778:7;:12;36769:191;;;36806:17;36794:9;;:29;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;36769:191;;;36856:1;36845:7;:12;36841:119;;;36873:17;36861:9;;:29;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;36841:119;;;36923:1;36912:7;:12;36908:52;;;36940:17;36928:9;;:29;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;36908:52;36841:119;36769:191;36705:262:::0;:::o;29958:68::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;12595:201::-;11575:13;:11;:13::i;:::-;12704:1:::1;12684:22;;:8;:22;;;;12676:73;;;;;;;;;;;;:::i;:::-;;;;;;;;;12760:28;12779:8;12760:18;:28::i;:::-;12595:201:::0;:::o;39475:131::-;11575:13;:11;:13::i;:::-;39581:17:::1;39562:16;;:36;;;;;;;;;;;;;;;;;;39475:131:::0;:::o;11854:132::-;11929:12;:10;:12::i;:::-;11918:23;;:7;:5;:7::i;:::-;:23;;;11910:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;11854:132::o;33405:411::-;33494:1;33480:16;;:2;:16;;;;33472:46;;;;;;;;;;;;:::i;:::-;;;;;;;;;33562:1;33539:25;;:7;:11;33547:2;33539:11;;;;;;;;;;;;;;;;;;;;;:25;;;33531:52;;;;;;;;;;;;:::i;:::-;;;;;;;;;33677:11;;:13;;;;;;;;;;;;;33707:9;:13;33717:2;33707:13;;;;;;;;;;;;;;;;:15;;;;;;;;;;;;;33760:2;33746:7;:11;33754:2;33746:11;;;;;;;;;;;;:16;;;;;;;;;;;;;;;;;;33805:2;33801;33780:28;;33797:1;33780:28;;;;;;;;;;;;33405:411;;:::o;1222:190::-;1347:4;1400;1371:25;1384:5;1391:4;1371:12;:25::i;:::-;:33;1364:40;;1222:190;;;;;:::o;12956:191::-;13030:16;13049:6;;;;;;;;;;;13030:25;;13075:8;13066:6;;:17;;;;;;;;;;;;;;;;;;13130:8;13099:40;;13120:8;13099:40;;;;;;;;;;;;13019:128;12956:191;:::o;26459:716::-;26515:13;26566:14;26603:1;26583:17;26594:5;26583:10;:17::i;:::-;:21;26566:38;;26619:20;26653:6;26642:18;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;26619:41;;26675:11;26804:6;26800:2;26796:15;26788:6;26784:28;26777:35;;26841:288;26848:4;26841:288;;;26873:5;;;;;;;;27015:8;27010:2;27003:5;26999:14;26994:30;26989:3;26981:44;27071:2;27062:11;;;;;;:::i;:::-;;;;;27105:1;27096:5;:10;27092:21;;;27108:5;;27092:21;26841:288;;;27150:6;27143:13;;;;;26459:716;;;:::o;10240:98::-;10293:7;10320:10;10313:17;;10240:98;:::o;2089:296::-;2172:7;2192:20;2215:4;2192:27;;2235:9;2230:118;2254:5;:12;2250:1;:16;2230:118;;;2303:33;2313:12;2327:5;2333:1;2327:8;;;;;;;;:::i;:::-;;;;;;;;2303:9;:33::i;:::-;2288:48;;2268:3;;;;;:::i;:::-;;;;2230:118;;;;2365:12;2358:19;;;2089:296;;;;:::o;23325:922::-;23378:7;23398:14;23415:1;23398:18;;23465:6;23456:5;:15;23452:102;;23501:6;23492:15;;;;;;:::i;:::-;;;;;23536:2;23526:12;;;;23452:102;23581:6;23572:5;:15;23568:102;;23617:6;23608:15;;;;;;:::i;:::-;;;;;23652:2;23642:12;;;;23568:102;23697:6;23688:5;:15;23684:102;;23733:6;23724:15;;;;;;:::i;:::-;;;;;23768:2;23758:12;;;;23684:102;23813:5;23804;:14;23800:99;;23848:5;23839:14;;;;;;:::i;:::-;;;;;23882:1;23872:11;;;;23800:99;23926:5;23917;:14;23913:99;;23961:5;23952:14;;;;;;:::i;:::-;;;;;23995:1;23985:11;;;;23913:99;24039:5;24030;:14;24026:99;;24074:5;24065:14;;;;;;:::i;:::-;;;;;24108:1;24098:11;;;;24026:99;24152:5;24143;:14;24139:66;;24188:1;24178:11;;;;24139:66;24233:6;24226:13;;;23325:922;;;:::o;9129:149::-;9192:7;9223:1;9219;:5;:51;;9250:20;9265:1;9268;9250:14;:20::i;:::-;9219:51;;;9227:20;9242:1;9245;9227:14;:20::i;:::-;9219:51;9212:58;;9129:149;;;;:::o;9286:268::-;9354:13;9461:1;9455:4;9448:15;9490:1;9484:4;9477:15;9531:4;9525;9515:21;9506:30;;9286:268;;;;:::o;-1:-1:-1:-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;:::o;:::-;;;;;;;;;;;;;;;;;;;;;:::o;7:410:1:-;84:5;109:65;125:48;166:6;125:48;:::i;:::-;109:65;:::i;:::-;100:74;;197:6;190:5;183:21;235:4;228:5;224:16;273:3;264:6;259:3;255:16;252:25;249:112;;;280:79;;:::i;:::-;249:112;370:41;404:6;399:3;394;370:41;:::i;:::-;90:327;7:410;;;;;:::o;423:412::-;501:5;526:66;542:49;584:6;542:49;:::i;:::-;526:66;:::i;:::-;517:75;;615:6;608:5;601:21;653:4;646:5;642:16;691:3;682:6;677:3;673:16;670:25;667:112;;;698:79;;:::i;:::-;667:112;788:41;822:6;817:3;812;788:41;:::i;:::-;507:328;423:412;;;;;:::o;841:139::-;887:5;925:6;912:20;903:29;;941:33;968:5;941:33;:::i;:::-;841:139;;;;:::o;1003:568::-;1076:8;1086:6;1136:3;1129:4;1121:6;1117:17;1113:27;1103:122;;1144:79;;:::i;:::-;1103:122;1257:6;1244:20;1234:30;;1287:18;1279:6;1276:30;1273:117;;;1309:79;;:::i;:::-;1273:117;1423:4;1415:6;1411:17;1399:29;;1477:3;1469:4;1461:6;1457:17;1447:8;1443:32;1440:41;1437:128;;;1484:79;;:::i;:::-;1437:128;1003:568;;;;;:::o;1577:133::-;1620:5;1658:6;1645:20;1636:29;;1674:30;1698:5;1674:30;:::i;:::-;1577:133;;;;:::o;1716:139::-;1762:5;1800:6;1787:20;1778:29;;1816:33;1843:5;1816:33;:::i;:::-;1716:139;;;;:::o;1861:137::-;1906:5;1944:6;1931:20;1922:29;;1960:32;1986:5;1960:32;:::i;:::-;1861:137;;;;:::o;2004:141::-;2060:5;2091:6;2085:13;2076:22;;2107:32;2133:5;2107:32;:::i;:::-;2004:141;;;;:::o;2164:338::-;2219:5;2268:3;2261:4;2253:6;2249:17;2245:27;2235:122;;2276:79;;:::i;:::-;2235:122;2393:6;2380:20;2418:78;2492:3;2484:6;2477:4;2469:6;2465:17;2418:78;:::i;:::-;2409:87;;2225:277;2164:338;;;;:::o;2522:340::-;2578:5;2627:3;2620:4;2612:6;2608:17;2604:27;2594:122;;2635:79;;:::i;:::-;2594:122;2752:6;2739:20;2777:79;2852:3;2844:6;2837:4;2829:6;2825:17;2777:79;:::i;:::-;2768:88;;2584:278;2522:340;;;;:::o;2868:139::-;2914:5;2952:6;2939:20;2930:29;;2968:33;2995:5;2968:33;:::i;:::-;2868:139;;;;:::o;3013:329::-;3072:6;3121:2;3109:9;3100:7;3096:23;3092:32;3089:119;;;3127:79;;:::i;:::-;3089:119;3247:1;3272:53;3317:7;3308:6;3297:9;3293:22;3272:53;:::i;:::-;3262:63;;3218:117;3013:329;;;;:::o;3348:474::-;3416:6;3424;3473:2;3461:9;3452:7;3448:23;3444:32;3441:119;;;3479:79;;:::i;:::-;3441:119;3599:1;3624:53;3669:7;3660:6;3649:9;3645:22;3624:53;:::i;:::-;3614:63;;3570:117;3726:2;3752:53;3797:7;3788:6;3777:9;3773:22;3752:53;:::i;:::-;3742:63;;3697:118;3348:474;;;;;:::o;3828:619::-;3905:6;3913;3921;3970:2;3958:9;3949:7;3945:23;3941:32;3938:119;;;3976:79;;:::i;:::-;3938:119;4096:1;4121:53;4166:7;4157:6;4146:9;4142:22;4121:53;:::i;:::-;4111:63;;4067:117;4223:2;4249:53;4294:7;4285:6;4274:9;4270:22;4249:53;:::i;:::-;4239:63;;4194:118;4351:2;4377:53;4422:7;4413:6;4402:9;4398:22;4377:53;:::i;:::-;4367:63;;4322:118;3828:619;;;;;:::o;4453:943::-;4548:6;4556;4564;4572;4621:3;4609:9;4600:7;4596:23;4592:33;4589:120;;;4628:79;;:::i;:::-;4589:120;4748:1;4773:53;4818:7;4809:6;4798:9;4794:22;4773:53;:::i;:::-;4763:63;;4719:117;4875:2;4901:53;4946:7;4937:6;4926:9;4922:22;4901:53;:::i;:::-;4891:63;;4846:118;5003:2;5029:53;5074:7;5065:6;5054:9;5050:22;5029:53;:::i;:::-;5019:63;;4974:118;5159:2;5148:9;5144:18;5131:32;5190:18;5182:6;5179:30;5176:117;;;5212:79;;:::i;:::-;5176:117;5317:62;5371:7;5362:6;5351:9;5347:22;5317:62;:::i;:::-;5307:72;;5102:287;4453:943;;;;;;;:::o;5402:468::-;5467:6;5475;5524:2;5512:9;5503:7;5499:23;5495:32;5492:119;;;5530:79;;:::i;:::-;5492:119;5650:1;5675:53;5720:7;5711:6;5700:9;5696:22;5675:53;:::i;:::-;5665:63;;5621:117;5777:2;5803:50;5845:7;5836:6;5825:9;5821:22;5803:50;:::i;:::-;5793:60;;5748:115;5402:468;;;;;:::o;5876:474::-;5944:6;5952;6001:2;5989:9;5980:7;5976:23;5972:32;5969:119;;;6007:79;;:::i;:::-;5969:119;6127:1;6152:53;6197:7;6188:6;6177:9;6173:22;6152:53;:::i;:::-;6142:63;;6098:117;6254:2;6280:53;6325:7;6316:6;6305:9;6301:22;6280:53;:::i;:::-;6270:63;;6225:118;5876:474;;;;;:::o;6356:704::-;6451:6;6459;6467;6516:2;6504:9;6495:7;6491:23;6487:32;6484:119;;;6522:79;;:::i;:::-;6484:119;6670:1;6659:9;6655:17;6642:31;6700:18;6692:6;6689:30;6686:117;;;6722:79;;:::i;:::-;6686:117;6835:80;6907:7;6898:6;6887:9;6883:22;6835:80;:::i;:::-;6817:98;;;;6613:312;6964:2;6990:53;7035:7;7026:6;7015:9;7011:22;6990:53;:::i;:::-;6980:63;;6935:118;6356:704;;;;;:::o;7066:329::-;7125:6;7174:2;7162:9;7153:7;7149:23;7145:32;7142:119;;;7180:79;;:::i;:::-;7142:119;7300:1;7325:53;7370:7;7361:6;7350:9;7346:22;7325:53;:::i;:::-;7315:63;;7271:117;7066:329;;;;:::o;7401:327::-;7459:6;7508:2;7496:9;7487:7;7483:23;7479:32;7476:119;;;7514:79;;:::i;:::-;7476:119;7634:1;7659:52;7703:7;7694:6;7683:9;7679:22;7659:52;:::i;:::-;7649:62;;7605:116;7401:327;;;;:::o;7734:349::-;7803:6;7852:2;7840:9;7831:7;7827:23;7823:32;7820:119;;;7858:79;;:::i;:::-;7820:119;7978:1;8003:63;8058:7;8049:6;8038:9;8034:22;8003:63;:::i;:::-;7993:73;;7949:127;7734:349;;;;:::o;8089:509::-;8158:6;8207:2;8195:9;8186:7;8182:23;8178:32;8175:119;;;8213:79;;:::i;:::-;8175:119;8361:1;8350:9;8346:17;8333:31;8391:18;8383:6;8380:30;8377:117;;;8413:79;;:::i;:::-;8377:117;8518:63;8573:7;8564:6;8553:9;8549:22;8518:63;:::i;:::-;8508:73;;8304:287;8089:509;;;;:::o;8604:329::-;8663:6;8712:2;8700:9;8691:7;8687:23;8683:32;8680:119;;;8718:79;;:::i;:::-;8680:119;8838:1;8863:53;8908:7;8899:6;8888:9;8884:22;8863:53;:::i;:::-;8853:63;;8809:117;8604:329;;;;:::o;8939:118::-;9026:24;9044:5;9026:24;:::i;:::-;9021:3;9014:37;8939:118;;:::o;9063:157::-;9168:45;9188:24;9206:5;9188:24;:::i;:::-;9168:45;:::i;:::-;9163:3;9156:58;9063:157;;:::o;9226:109::-;9307:21;9322:5;9307:21;:::i;:::-;9302:3;9295:34;9226:109;;:::o;9341:118::-;9428:24;9446:5;9428:24;:::i;:::-;9423:3;9416:37;9341:118;;:::o;9465:360::-;9551:3;9579:38;9611:5;9579:38;:::i;:::-;9633:70;9696:6;9691:3;9633:70;:::i;:::-;9626:77;;9712:52;9757:6;9752:3;9745:4;9738:5;9734:16;9712:52;:::i;:::-;9789:29;9811:6;9789:29;:::i;:::-;9784:3;9780:39;9773:46;;9555:270;9465:360;;;;:::o;9831:157::-;9931:50;9975:5;9931:50;:::i;:::-;9926:3;9919:63;9831:157;;:::o;9994:364::-;10082:3;10110:39;10143:5;10110:39;:::i;:::-;10165:71;10229:6;10224:3;10165:71;:::i;:::-;10158:78;;10245:52;10290:6;10285:3;10278:4;10271:5;10267:16;10245:52;:::i;:::-;10322:29;10344:6;10322:29;:::i;:::-;10317:3;10313:39;10306:46;;10086:272;9994:364;;;;:::o;10364:377::-;10470:3;10498:39;10531:5;10498:39;:::i;:::-;10553:89;10635:6;10630:3;10553:89;:::i;:::-;10546:96;;10651:52;10696:6;10691:3;10684:4;10677:5;10673:16;10651:52;:::i;:::-;10728:6;10723:3;10719:16;10712:23;;10474:267;10364:377;;;;:::o;10771:845::-;10874:3;10911:5;10905:12;10940:36;10966:9;10940:36;:::i;:::-;10992:89;11074:6;11069:3;10992:89;:::i;:::-;10985:96;;11112:1;11101:9;11097:17;11128:1;11123:137;;;;11274:1;11269:341;;;;11090:520;;11123:137;11207:4;11203:9;11192;11188:25;11183:3;11176:38;11243:6;11238:3;11234:16;11227:23;;11123:137;;11269:341;11336:38;11368:5;11336:38;:::i;:::-;11396:1;11410:154;11424:6;11421:1;11418:13;11410:154;;;11498:7;11492:14;11488:1;11483:3;11479:11;11472:35;11548:1;11539:7;11535:15;11524:26;;11446:4;11443:1;11439:12;11434:17;;11410:154;;;11593:6;11588:3;11584:16;11577:23;;11276:334;;11090:520;;10878:738;;10771:845;;;;:::o;11622:366::-;11764:3;11785:67;11849:2;11844:3;11785:67;:::i;:::-;11778:74;;11861:93;11950:3;11861:93;:::i;:::-;11979:2;11974:3;11970:12;11963:19;;11622:366;;;:::o;11994:::-;12136:3;12157:67;12221:2;12216:3;12157:67;:::i;:::-;12150:74;;12233:93;12322:3;12233:93;:::i;:::-;12351:2;12346:3;12342:12;12335:19;;11994:366;;;:::o;12366:::-;12508:3;12529:67;12593:2;12588:3;12529:67;:::i;:::-;12522:74;;12605:93;12694:3;12605:93;:::i;:::-;12723:2;12718:3;12714:12;12707:19;;12366:366;;;:::o;12738:::-;12880:3;12901:67;12965:2;12960:3;12901:67;:::i;:::-;12894:74;;12977:93;13066:3;12977:93;:::i;:::-;13095:2;13090:3;13086:12;13079:19;;12738:366;;;:::o;13110:::-;13252:3;13273:67;13337:2;13332:3;13273:67;:::i;:::-;13266:74;;13349:93;13438:3;13349:93;:::i;:::-;13467:2;13462:3;13458:12;13451:19;;13110:366;;;:::o;13482:::-;13624:3;13645:67;13709:2;13704:3;13645:67;:::i;:::-;13638:74;;13721:93;13810:3;13721:93;:::i;:::-;13839:2;13834:3;13830:12;13823:19;;13482:366;;;:::o;13854:::-;13996:3;14017:67;14081:2;14076:3;14017:67;:::i;:::-;14010:74;;14093:93;14182:3;14093:93;:::i;:::-;14211:2;14206:3;14202:12;14195:19;;13854:366;;;:::o;14226:::-;14368:3;14389:67;14453:2;14448:3;14389:67;:::i;:::-;14382:74;;14465:93;14554:3;14465:93;:::i;:::-;14583:2;14578:3;14574:12;14567:19;;14226:366;;;:::o;14598:::-;14740:3;14761:67;14825:2;14820:3;14761:67;:::i;:::-;14754:74;;14837:93;14926:3;14837:93;:::i;:::-;14955:2;14950:3;14946:12;14939:19;;14598:366;;;:::o;14970:::-;15112:3;15133:67;15197:2;15192:3;15133:67;:::i;:::-;15126:74;;15209:93;15298:3;15209:93;:::i;:::-;15327:2;15322:3;15318:12;15311:19;;14970:366;;;:::o;15342:::-;15484:3;15505:67;15569:2;15564:3;15505:67;:::i;:::-;15498:74;;15581:93;15670:3;15581:93;:::i;:::-;15699:2;15694:3;15690:12;15683:19;;15342:366;;;:::o;15714:362::-;15855:3;15876:65;15939:1;15934:3;15876:65;:::i;:::-;15869:72;;15950:93;16039:3;15950:93;:::i;:::-;16068:1;16063:3;16059:11;16052:18;;15714:362;;;:::o;16082:398::-;16241:3;16262:83;16343:1;16338:3;16262:83;:::i;:::-;16255:90;;16354:93;16443:3;16354:93;:::i;:::-;16472:1;16467:3;16463:11;16456:18;;16082:398;;;:::o;16486:366::-;16628:3;16649:67;16713:2;16708:3;16649:67;:::i;:::-;16642:74;;16725:93;16814:3;16725:93;:::i;:::-;16843:2;16838:3;16834:12;16827:19;;16486:366;;;:::o;16858:::-;17000:3;17021:67;17085:2;17080:3;17021:67;:::i;:::-;17014:74;;17097:93;17186:3;17097:93;:::i;:::-;17215:2;17210:3;17206:12;17199:19;;16858:366;;;:::o;17230:::-;17372:3;17393:67;17457:2;17452:3;17393:67;:::i;:::-;17386:74;;17469:93;17558:3;17469:93;:::i;:::-;17587:2;17582:3;17578:12;17571:19;;17230:366;;;:::o;17602:::-;17744:3;17765:67;17829:2;17824:3;17765:67;:::i;:::-;17758:74;;17841:93;17930:3;17841:93;:::i;:::-;17959:2;17954:3;17950:12;17943:19;;17602:366;;;:::o;17974:::-;18116:3;18137:67;18201:2;18196:3;18137:67;:::i;:::-;18130:74;;18213:93;18302:3;18213:93;:::i;:::-;18331:2;18326:3;18322:12;18315:19;;17974:366;;;:::o;18346:::-;18488:3;18509:67;18573:2;18568:3;18509:67;:::i;:::-;18502:74;;18585:93;18674:3;18585:93;:::i;:::-;18703:2;18698:3;18694:12;18687:19;;18346:366;;;:::o;18718:::-;18860:3;18881:67;18945:2;18940:3;18881:67;:::i;:::-;18874:74;;18957:93;19046:3;18957:93;:::i;:::-;19075:2;19070:3;19066:12;19059:19;;18718:366;;;:::o;19090:118::-;19177:24;19195:5;19177:24;:::i;:::-;19172:3;19165:37;19090:118;;:::o;19214:256::-;19326:3;19341:75;19412:3;19403:6;19341:75;:::i;:::-;19441:2;19436:3;19432:12;19425:19;;19461:3;19454:10;;19214:256;;;;:::o;19476:429::-;19653:3;19675:92;19763:3;19754:6;19675:92;:::i;:::-;19668:99;;19784:95;19875:3;19866:6;19784:95;:::i;:::-;19777:102;;19896:3;19889:10;;19476:429;;;;;:::o;19911:379::-;20095:3;20117:147;20260:3;20117:147;:::i;:::-;20110:154;;20281:3;20274:10;;19911:379;;;:::o;20296:222::-;20389:4;20427:2;20416:9;20412:18;20404:26;;20440:71;20508:1;20497:9;20493:17;20484:6;20440:71;:::i;:::-;20296:222;;;;:::o;20524:640::-;20719:4;20757:3;20746:9;20742:19;20734:27;;20771:71;20839:1;20828:9;20824:17;20815:6;20771:71;:::i;:::-;20852:72;20920:2;20909:9;20905:18;20896:6;20852:72;:::i;:::-;20934;21002:2;20991:9;20987:18;20978:6;20934:72;:::i;:::-;21053:9;21047:4;21043:20;21038:2;21027:9;21023:18;21016:48;21081:76;21152:4;21143:6;21081:76;:::i;:::-;21073:84;;20524:640;;;;;;;:::o;21170:748::-;21419:4;21457:3;21446:9;21442:19;21434:27;;21471:71;21539:1;21528:9;21524:17;21515:6;21471:71;:::i;:::-;21552:72;21620:2;21609:9;21605:18;21596:6;21552:72;:::i;:::-;21634;21702:2;21691:9;21687:18;21678:6;21634:72;:::i;:::-;21753:9;21747:4;21743:20;21738:2;21727:9;21723:18;21716:48;21781:130;21906:4;21781:130;:::i;:::-;21773:138;;21170:748;;;;;;:::o;21924:210::-;22011:4;22049:2;22038:9;22034:18;22026:26;;22062:65;22124:1;22113:9;22109:17;22100:6;22062:65;:::i;:::-;21924:210;;;;:::o;22140:222::-;22233:4;22271:2;22260:9;22256:18;22248:26;;22284:71;22352:1;22341:9;22337:17;22328:6;22284:71;:::i;:::-;22140:222;;;;:::o;22368:248::-;22474:4;22512:2;22501:9;22497:18;22489:26;;22525:84;22606:1;22595:9;22591:17;22582:6;22525:84;:::i;:::-;22368:248;;;;:::o;22622:313::-;22735:4;22773:2;22762:9;22758:18;22750:26;;22822:9;22816:4;22812:20;22808:1;22797:9;22793:17;22786:47;22850:78;22923:4;22914:6;22850:78;:::i;:::-;22842:86;;22622:313;;;;:::o;22941:419::-;23107:4;23145:2;23134:9;23130:18;23122:26;;23194:9;23188:4;23184:20;23180:1;23169:9;23165:17;23158:47;23222:131;23348:4;23222:131;:::i;:::-;23214:139;;22941:419;;;:::o;23366:::-;23532:4;23570:2;23559:9;23555:18;23547:26;;23619:9;23613:4;23609:20;23605:1;23594:9;23590:17;23583:47;23647:131;23773:4;23647:131;:::i;:::-;23639:139;;23366:419;;;:::o;23791:::-;23957:4;23995:2;23984:9;23980:18;23972:26;;24044:9;24038:4;24034:20;24030:1;24019:9;24015:17;24008:47;24072:131;24198:4;24072:131;:::i;:::-;24064:139;;23791:419;;;:::o;24216:::-;24382:4;24420:2;24409:9;24405:18;24397:26;;24469:9;24463:4;24459:20;24455:1;24444:9;24440:17;24433:47;24497:131;24623:4;24497:131;:::i;:::-;24489:139;;24216:419;;;:::o;24641:::-;24807:4;24845:2;24834:9;24830:18;24822:26;;24894:9;24888:4;24884:20;24880:1;24869:9;24865:17;24858:47;24922:131;25048:4;24922:131;:::i;:::-;24914:139;;24641:419;;;:::o;25066:::-;25232:4;25270:2;25259:9;25255:18;25247:26;;25319:9;25313:4;25309:20;25305:1;25294:9;25290:17;25283:47;25347:131;25473:4;25347:131;:::i;:::-;25339:139;;25066:419;;;:::o;25491:::-;25657:4;25695:2;25684:9;25680:18;25672:26;;25744:9;25738:4;25734:20;25730:1;25719:9;25715:17;25708:47;25772:131;25898:4;25772:131;:::i;:::-;25764:139;;25491:419;;;:::o;25916:::-;26082:4;26120:2;26109:9;26105:18;26097:26;;26169:9;26163:4;26159:20;26155:1;26144:9;26140:17;26133:47;26197:131;26323:4;26197:131;:::i;:::-;26189:139;;25916:419;;;:::o;26341:::-;26507:4;26545:2;26534:9;26530:18;26522:26;;26594:9;26588:4;26584:20;26580:1;26569:9;26565:17;26558:47;26622:131;26748:4;26622:131;:::i;:::-;26614:139;;26341:419;;;:::o;26766:::-;26932:4;26970:2;26959:9;26955:18;26947:26;;27019:9;27013:4;27009:20;27005:1;26994:9;26990:17;26983:47;27047:131;27173:4;27047:131;:::i;:::-;27039:139;;26766:419;;;:::o;27191:::-;27357:4;27395:2;27384:9;27380:18;27372:26;;27444:9;27438:4;27434:20;27430:1;27419:9;27415:17;27408:47;27472:131;27598:4;27472:131;:::i;:::-;27464:139;;27191:419;;;:::o;27616:::-;27782:4;27820:2;27809:9;27805:18;27797:26;;27869:9;27863:4;27859:20;27855:1;27844:9;27840:17;27833:47;27897:131;28023:4;27897:131;:::i;:::-;27889:139;;27616:419;;;:::o;28041:::-;28207:4;28245:2;28234:9;28230:18;28222:26;;28294:9;28288:4;28284:20;28280:1;28269:9;28265:17;28258:47;28322:131;28448:4;28322:131;:::i;:::-;28314:139;;28041:419;;;:::o;28466:::-;28632:4;28670:2;28659:9;28655:18;28647:26;;28719:9;28713:4;28709:20;28705:1;28694:9;28690:17;28683:47;28747:131;28873:4;28747:131;:::i;:::-;28739:139;;28466:419;;;:::o;28891:::-;29057:4;29095:2;29084:9;29080:18;29072:26;;29144:9;29138:4;29134:20;29130:1;29119:9;29115:17;29108:47;29172:131;29298:4;29172:131;:::i;:::-;29164:139;;28891:419;;;:::o;29316:::-;29482:4;29520:2;29509:9;29505:18;29497:26;;29569:9;29563:4;29559:20;29555:1;29544:9;29540:17;29533:47;29597:131;29723:4;29597:131;:::i;:::-;29589:139;;29316:419;;;:::o;29741:::-;29907:4;29945:2;29934:9;29930:18;29922:26;;29994:9;29988:4;29984:20;29980:1;29969:9;29965:17;29958:47;30022:131;30148:4;30022:131;:::i;:::-;30014:139;;29741:419;;;:::o;30166:::-;30332:4;30370:2;30359:9;30355:18;30347:26;;30419:9;30413:4;30409:20;30405:1;30394:9;30390:17;30383:47;30447:131;30573:4;30447:131;:::i;:::-;30439:139;;30166:419;;;:::o;30591:222::-;30684:4;30722:2;30711:9;30707:18;30699:26;;30735:71;30803:1;30792:9;30788:17;30779:6;30735:71;:::i;:::-;30591:222;;;;:::o;30819:129::-;30853:6;30880:20;;:::i;:::-;30870:30;;30909:33;30937:4;30929:6;30909:33;:::i;:::-;30819:129;;;:::o;30954:75::-;30987:6;31020:2;31014:9;31004:19;;30954:75;:::o;31035:307::-;31096:4;31186:18;31178:6;31175:30;31172:56;;;31208:18;;:::i;:::-;31172:56;31246:29;31268:6;31246:29;:::i;:::-;31238:37;;31330:4;31324;31320:15;31312:23;;31035:307;;;:::o;31348:308::-;31410:4;31500:18;31492:6;31489:30;31486:56;;;31522:18;;:::i;:::-;31486:56;31560:29;31582:6;31560:29;:::i;:::-;31552:37;;31644:4;31638;31634:15;31626:23;;31348:308;;;:::o;31662:141::-;31711:4;31734:3;31726:11;;31757:3;31754:1;31747:14;31791:4;31788:1;31778:18;31770:26;;31662:141;;;:::o;31809:98::-;31860:6;31894:5;31888:12;31878:22;;31809:98;;;:::o;31913:99::-;31965:6;31999:5;31993:12;31983:22;;31913:99;;;:::o;32018:168::-;32101:11;32135:6;32130:3;32123:19;32175:4;32170:3;32166:14;32151:29;;32018:168;;;;:::o;32192:147::-;32293:11;32330:3;32315:18;;32192:147;;;;:::o;32345:169::-;32429:11;32463:6;32458:3;32451:19;32503:4;32498:3;32494:14;32479:29;;32345:169;;;;:::o;32520:148::-;32622:11;32659:3;32644:18;;32520:148;;;;:::o;32674:305::-;32714:3;32733:20;32751:1;32733:20;:::i;:::-;32728:25;;32767:20;32785:1;32767:20;:::i;:::-;32762:25;;32921:1;32853:66;32849:74;32846:1;32843:81;32840:107;;;32927:18;;:::i;:::-;32840:107;32971:1;32968;32964:9;32957:16;;32674:305;;;;:::o;32985:348::-;33025:7;33048:20;33066:1;33048:20;:::i;:::-;33043:25;;33082:20;33100:1;33082:20;:::i;:::-;33077:25;;33270:1;33202:66;33198:74;33195:1;33192:81;33187:1;33180:9;33173:17;33169:105;33166:131;;;33277:18;;:::i;:::-;33166:131;33325:1;33322;33318:9;33307:20;;32985:348;;;;:::o;33339:96::-;33376:7;33405:24;33423:5;33405:24;:::i;:::-;33394:35;;33339:96;;;:::o;33441:90::-;33475:7;33518:5;33511:13;33504:21;33493:32;;33441:90;;;:::o;33537:77::-;33574:7;33603:5;33592:16;;33537:77;;;:::o;33620:149::-;33656:7;33696:66;33689:5;33685:78;33674:89;;33620:149;;;:::o;33775:141::-;33827:7;33856:5;33845:16;;33862:48;33904:5;33862:48;:::i;:::-;33775:141;;;:::o;33922:126::-;33959:7;33999:42;33992:5;33988:54;33977:65;;33922:126;;;:::o;34054:77::-;34091:7;34120:5;34109:16;;34054:77;;;:::o;34137:141::-;34200:9;34233:39;34266:5;34233:39;:::i;:::-;34220:52;;34137:141;;;:::o;34284:154::-;34368:6;34363:3;34358;34345:30;34430:1;34421:6;34416:3;34412:16;34405:27;34284:154;;;:::o;34444:307::-;34512:1;34522:113;34536:6;34533:1;34530:13;34522:113;;;34621:1;34616:3;34612:11;34606:18;34602:1;34597:3;34593:11;34586:39;34558:2;34555:1;34551:10;34546:15;;34522:113;;;34653:6;34650:1;34647:13;34644:101;;;34733:1;34724:6;34719:3;34715:16;34708:27;34644:101;34493:258;34444:307;;;:::o;34757:320::-;34801:6;34838:1;34832:4;34828:12;34818:22;;34885:1;34879:4;34875:12;34906:18;34896:81;;34962:4;34954:6;34950:17;34940:27;;34896:81;35024:2;35016:6;35013:14;34993:18;34990:38;34987:84;;;35043:18;;:::i;:::-;34987:84;34808:269;34757:320;;;:::o;35083:281::-;35166:27;35188:4;35166:27;:::i;:::-;35158:6;35154:40;35296:6;35284:10;35281:22;35260:18;35248:10;35245:34;35242:62;35239:88;;;35307:18;;:::i;:::-;35239:88;35347:10;35343:2;35336:22;35126:238;35083:281;;:::o;35370:233::-;35409:3;35432:24;35450:5;35432:24;:::i;:::-;35423:33;;35478:66;35471:5;35468:77;35465:103;;;35548:18;;:::i;:::-;35465:103;35595:1;35588:5;35584:13;35577:20;;35370:233;;;:::o;35609:100::-;35648:7;35677:26;35697:5;35677:26;:::i;:::-;35666:37;;35609:100;;;:::o;35715:94::-;35754:7;35783:20;35797:5;35783:20;:::i;:::-;35772:31;;35715:94;;;:::o;35815:180::-;35863:77;35860:1;35853:88;35960:4;35957:1;35950:15;35984:4;35981:1;35974:15;36001:180;36049:77;36046:1;36039:88;36146:4;36143:1;36136:15;36170:4;36167:1;36160:15;36187:180;36235:77;36232:1;36225:88;36332:4;36329:1;36322:15;36356:4;36353:1;36346:15;36373:180;36421:77;36418:1;36411:88;36518:4;36515:1;36508:15;36542:4;36539:1;36532:15;36559:180;36607:77;36604:1;36597:88;36704:4;36701:1;36694:15;36728:4;36725:1;36718:15;36745:180;36793:77;36790:1;36783:88;36890:4;36887:1;36880:15;36914:4;36911:1;36904:15;36931:117;37040:1;37037;37030:12;37054:117;37163:1;37160;37153:12;37177:117;37286:1;37283;37276:12;37300:117;37409:1;37406;37399:12;37423:117;37532:1;37529;37522:12;37546:117;37655:1;37652;37645:12;37669:102;37710:6;37761:2;37757:7;37752:2;37745:5;37741:14;37737:28;37727:38;;37669:102;;;:::o;37777:94::-;37810:8;37858:5;37854:2;37850:14;37829:35;;37777:94;;;:::o;37877:167::-;38017:19;38013:1;38005:6;38001:14;37994:43;37877:167;:::o;38050:225::-;38190:34;38186:1;38178:6;38174:14;38167:58;38259:8;38254:2;38246:6;38242:15;38235:33;38050:225;:::o;38281:168::-;38421:20;38417:1;38409:6;38405:14;38398:44;38281:168;:::o;38455:163::-;38595:15;38591:1;38583:6;38579:14;38572:39;38455:163;:::o;38624:167::-;38764:19;38760:1;38752:6;38748:14;38741:43;38624:167;:::o;38797:164::-;38937:16;38933:1;38925:6;38921:14;38914:40;38797:164;:::o;38967:171::-;39107:23;39103:1;39095:6;39091:14;39084:47;38967:171;:::o;39144:165::-;39284:17;39280:1;39272:6;39268:14;39261:41;39144:165;:::o;39315:229::-;39455:34;39451:1;39443:6;39439:14;39432:58;39524:12;39519:2;39511:6;39507:15;39500:37;39315:229;:::o;39550:166::-;39690:18;39686:1;39678:6;39674:14;39667:42;39550:166;:::o;39722:182::-;39862:34;39858:1;39850:6;39846:14;39839:58;39722:182;:::o;39910:114::-;;:::o;40030:166::-;40170:18;40166:1;40158:6;40154:14;40147:42;40030:166;:::o;40202:174::-;40342:26;40338:1;40330:6;40326:14;40319:50;40202:174;:::o;40382:164::-;40522:16;40518:1;40510:6;40506:14;40499:40;40382:164;:::o;40552:::-;40692:16;40688:1;40680:6;40676:14;40669:40;40552:164;:::o;40722:177::-;40862:29;40858:1;40850:6;40846:14;40839:53;40722:177;:::o;40905:224::-;41045:34;41041:1;41033:6;41029:14;41022:58;41114:7;41109:2;41101:6;41097:15;41090:32;40905:224;:::o;41135:160::-;41275:12;41271:1;41263:6;41259:14;41252:36;41135:160;:::o;41301:120::-;41389:1;41382:5;41379:12;41369:46;;41395:18;;:::i;:::-;41369:46;41301:120;:::o;41427:122::-;41500:24;41518:5;41500:24;:::i;:::-;41493:5;41490:35;41480:63;;41539:1;41536;41529:12;41480:63;41427:122;:::o;41555:116::-;41625:21;41640:5;41625:21;:::i;:::-;41618:5;41615:32;41605:60;;41661:1;41658;41651:12;41605:60;41555:116;:::o;41677:122::-;41750:24;41768:5;41750:24;:::i;:::-;41743:5;41740:35;41730:63;;41789:1;41786;41779:12;41730:63;41677:122;:::o;41805:120::-;41877:23;41894:5;41877:23;:::i;:::-;41870:5;41867:34;41857:62;;41915:1;41912;41905:12;41857:62;41805:120;:::o;41931:122::-;42004:24;42022:5;42004:24;:::i;:::-;41997:5;41994:35;41984:63;;42043:1;42040;42033:12;41984:63;41931:122;:::o

Swarm Source

ipfs://6db58f9eb5afd7d9ba1323832d1f50afd7528007dc0b8799366788efc8014e9e
Loading...
Loading
Loading...
Loading
[ Download: CSV Export  ]
[ Download: CSV Export  ]

A token is a representation of an on-chain or off-chain asset. The token page shows information such as price, total supply, holders, transfers and social links. Learn more about this page in our Knowledge Base.