ETH Price: $3,293.55 (+1.35%)
Gas: 2 Gwei

Token

Meta-DIOs (Meta-DIOs)
 

Overview

Max Total Supply

8,888 Meta-DIOs

Holders

254

Market

Volume (24H)

N/A

Min Price (24H)

N/A

Max Price (24H)

N/A
Balance
0 Meta-DIOs
0xe1799e4bfb2890721169e07933c28144323a9223
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:
DIOsNFT

Compiler Version
v0.8.7+commit.e28d00a7

Optimization Enabled:
Yes with 1000 runs

Other Settings:
default evmVersion, None license

Contract Source Code (Solidity)

/**
 *Submitted for verification at Etherscan.io on 2022-11-15
*/

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


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

pragma solidity ^0.8.0;

/**
 * @dev These functions deal with verification of Merkle Tree proofs.
 *
 * The tree and the proofs can be generated using our
 * https://github.com/OpenZeppelin/merkle-tree[JavaScript library].
 * You will find a quickstart guide in the readme.
 *
 * WARNING: You should avoid using leaf values that are 64 bytes long prior to
 * hashing, or use a hash function other than keccak256 for hashing leaves.
 * This is because the concatenation of a sorted pair of internal nodes in
 * the merkle tree could be reinterpreted as a leaf value.
 * OpenZeppelin's JavaScript library generates merkle trees that are safe
 * against this attack out of the box.
 */
library MerkleProof {
    /**
     * @dev Returns true if a `leaf` can be proved to be a part of a Merkle tree
     * defined by `root`. For this, a `proof` must be provided, containing
     * sibling hashes on the branch from the leaf to the root of the tree. Each
     * pair of leaves and each pair of pre-images are assumed to be sorted.
     */
    function verify(
        bytes32[] memory proof,
        bytes32 root,
        bytes32 leaf
    ) internal pure returns (bool) {
        return processProof(proof, leaf) == root;
    }

    /**
     * @dev Calldata version of {verify}
     *
     * _Available since v4.7._
     */
    function verifyCalldata(
        bytes32[] calldata proof,
        bytes32 root,
        bytes32 leaf
    ) internal pure returns (bool) {
        return processProofCalldata(proof, leaf) == root;
    }

    /**
     * @dev Returns the rebuilt hash obtained by traversing a Merkle tree up
     * from `leaf` using `proof`. A `proof` is valid if and only if the rebuilt
     * hash matches the root of the tree. When processing the proof, the pairs
     * of leafs & pre-images are assumed to be sorted.
     *
     * _Available since v4.4._
     */
    function processProof(bytes32[] memory proof, bytes32 leaf) internal pure returns (bytes32) {
        bytes32 computedHash = leaf;
        for (uint256 i = 0; i < proof.length; i++) {
            computedHash = _hashPair(computedHash, proof[i]);
        }
        return computedHash;
    }

    /**
     * @dev Calldata version of {processProof}
     *
     * _Available since v4.7._
     */
    function processProofCalldata(bytes32[] calldata proof, bytes32 leaf) internal pure returns (bytes32) {
        bytes32 computedHash = leaf;
        for (uint256 i = 0; i < proof.length; i++) {
            computedHash = _hashPair(computedHash, proof[i]);
        }
        return computedHash;
    }

    /**
     * @dev Returns true if the `leaves` can be simultaneously proven to be a part of a merkle tree defined by
     * `root`, according to `proof` and `proofFlags` as described in {processMultiProof}.
     *
     * CAUTION: Not all merkle trees admit multiproofs. See {processMultiProof} for details.
     *
     * _Available since v4.7._
     */
    function multiProofVerify(
        bytes32[] memory proof,
        bool[] memory proofFlags,
        bytes32 root,
        bytes32[] memory leaves
    ) internal pure returns (bool) {
        return processMultiProof(proof, proofFlags, leaves) == root;
    }

    /**
     * @dev Calldata version of {multiProofVerify}
     *
     * CAUTION: Not all merkle trees admit multiproofs. See {processMultiProof} for details.
     *
     * _Available since v4.7._
     */
    function multiProofVerifyCalldata(
        bytes32[] calldata proof,
        bool[] calldata proofFlags,
        bytes32 root,
        bytes32[] memory leaves
    ) internal pure returns (bool) {
        return processMultiProofCalldata(proof, proofFlags, leaves) == root;
    }

    /**
     * @dev Returns the root of a tree reconstructed from `leaves` and sibling nodes in `proof`. The reconstruction
     * proceeds by incrementally reconstructing all inner nodes by combining a leaf/inner node with either another
     * leaf/inner node or a proof sibling node, depending on whether each `proofFlags` item is true or false
     * respectively.
     *
     * CAUTION: Not all merkle trees admit multiproofs. To use multiproofs, it is sufficient to ensure that: 1) the tree
     * is complete (but not necessarily perfect), 2) the leaves to be proven are in the opposite order they are in the
     * tree (i.e., as seen from right to left starting at the deepest layer and continuing at the next layer).
     *
     * _Available since v4.7._
     */
    function processMultiProof(
        bytes32[] memory proof,
        bool[] memory proofFlags,
        bytes32[] memory leaves
    ) internal pure returns (bytes32 merkleRoot) {
        // This function rebuild the root hash by traversing the tree up from the leaves. The root is rebuilt by
        // consuming and producing values on a queue. The queue starts with the `leaves` array, then goes onto the
        // `hashes` array. At the end of the process, the last hash in the `hashes` array should contain the root of
        // the merkle tree.
        uint256 leavesLen = leaves.length;
        uint256 totalHashes = proofFlags.length;

        // Check proof validity.
        require(leavesLen + proof.length - 1 == totalHashes, "MerkleProof: invalid multiproof");

        // The xxxPos values are "pointers" to the next value to consume in each array. All accesses are done using
        // `xxx[xxxPos++]`, which return the current value and increment the pointer, thus mimicking a queue's "pop".
        bytes32[] memory hashes = new bytes32[](totalHashes);
        uint256 leafPos = 0;
        uint256 hashPos = 0;
        uint256 proofPos = 0;
        // At each step, we compute the next hash using two values:
        // - a value from the "main queue". If not all leaves have been consumed, we get the next leaf, otherwise we
        //   get the next hash.
        // - depending on the flag, either another value for the "main queue" (merging branches) or an element from the
        //   `proof` array.
        for (uint256 i = 0; i < totalHashes; i++) {
            bytes32 a = leafPos < leavesLen ? leaves[leafPos++] : hashes[hashPos++];
            bytes32 b = proofFlags[i] ? leafPos < leavesLen ? leaves[leafPos++] : hashes[hashPos++] : proof[proofPos++];
            hashes[i] = _hashPair(a, b);
        }

        if (totalHashes > 0) {
            return hashes[totalHashes - 1];
        } else if (leavesLen > 0) {
            return leaves[0];
        } else {
            return proof[0];
        }
    }

    /**
     * @dev Calldata version of {processMultiProof}.
     *
     * CAUTION: Not all merkle trees admit multiproofs. See {processMultiProof} for details.
     *
     * _Available since v4.7._
     */
    function processMultiProofCalldata(
        bytes32[] calldata proof,
        bool[] calldata proofFlags,
        bytes32[] memory leaves
    ) internal pure returns (bytes32 merkleRoot) {
        // This function rebuild the root hash by traversing the tree up from the leaves. The root is rebuilt by
        // consuming and producing values on a queue. The queue starts with the `leaves` array, then goes onto the
        // `hashes` array. At the end of the process, the last hash in the `hashes` array should contain the root of
        // the merkle tree.
        uint256 leavesLen = leaves.length;
        uint256 totalHashes = proofFlags.length;

        // Check proof validity.
        require(leavesLen + proof.length - 1 == totalHashes, "MerkleProof: invalid multiproof");

        // The xxxPos values are "pointers" to the next value to consume in each array. All accesses are done using
        // `xxx[xxxPos++]`, which return the current value and increment the pointer, thus mimicking a queue's "pop".
        bytes32[] memory hashes = new bytes32[](totalHashes);
        uint256 leafPos = 0;
        uint256 hashPos = 0;
        uint256 proofPos = 0;
        // At each step, we compute the next hash using two values:
        // - a value from the "main queue". If not all leaves have been consumed, we get the next leaf, otherwise we
        //   get the next hash.
        // - depending on the flag, either another value for the "main queue" (merging branches) or an element from the
        //   `proof` array.
        for (uint256 i = 0; i < totalHashes; i++) {
            bytes32 a = leafPos < leavesLen ? leaves[leafPos++] : hashes[hashPos++];
            bytes32 b = proofFlags[i] ? leafPos < leavesLen ? leaves[leafPos++] : hashes[hashPos++] : proof[proofPos++];
            hashes[i] = _hashPair(a, b);
        }

        if (totalHashes > 0) {
            return hashes[totalHashes - 1];
        } else if (leavesLen > 0) {
            return leaves[0];
        } else {
            return proof[0];
        }
    }

    function _hashPair(bytes32 a, bytes32 b) private pure returns (bytes32) {
        return a < b ? _efficientHash(a, b) : _efficientHash(b, a);
    }

    function _efficientHash(bytes32 a, bytes32 b) private pure returns (bytes32 value) {
        /// @solidity memory-safe-assembly
        assembly {
            mstore(0x00, a)
            mstore(0x20, b)
            value := keccak256(0x00, 0x40)
        }
    }
}

// File: @openzeppelin/contracts/security/ReentrancyGuard.sol


// OpenZeppelin Contracts (last updated v4.8.0) (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() {
        _nonReentrantBefore();
        _;
        _nonReentrantAfter();
    }

    function _nonReentrantBefore() private {
        // On the first call to nonReentrant, _status will be _NOT_ENTERED
        require(_status != _ENTERED, "ReentrancyGuard: reentrant call");

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

    function _nonReentrantAfter() private {
        // 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/Context.sol


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

pragma solidity ^0.8.0;

/**
 * @dev Provides information about the current execution context, including the
 * sender of the transaction and its data. While these are generally available
 * via msg.sender and msg.data, they should not be accessed in such a direct
 * manner, since when dealing with meta-transactions the account sending and
 * paying for execution may not be the actual sender (as far as an application
 * is concerned).
 *
 * This contract is only required for intermediate, library-like contracts.
 */
abstract contract Context {
    function _msgSender() internal view virtual returns (address) {
        return msg.sender;
    }

    function _msgData() internal view virtual returns (bytes calldata) {
        return msg.data;
    }
}

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


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

pragma solidity ^0.8.0;


/**
 * @dev Contract module which provides a basic access control mechanism, where
 * there is an account (an owner) that can be granted exclusive access to
 * specific functions.
 *
 * By default, the owner account will be the one that deploys the contract. This
 * can later be changed with {transferOwnership}.
 *
 * This module is used through inheritance. It will make available the modifier
 * `onlyOwner`, which can be applied to your functions to restrict their use to
 * the owner.
 */
abstract contract Ownable is Context {
    address private _owner;

    event OwnershipTransferred(address indexed previousOwner, address indexed newOwner);

    /**
     * @dev Initializes the contract setting the deployer as the initial owner.
     */
    constructor() {
        _transferOwnership(_msgSender());
    }

    /**
     * @dev Throws if called by any account other than the owner.
     */
    modifier onlyOwner() {
        _checkOwner();
        _;
    }

    /**
     * @dev Returns the address of the current owner.
     */
    function owner() public view virtual returns (address) {
        return _owner;
    }

    /**
     * @dev Throws if the sender is not the owner.
     */
    function _checkOwner() internal view virtual {
        require(owner() == _msgSender(), "Ownable: caller is not the owner");
    }

    /**
     * @dev Leaves the contract without owner. It will not be possible to call
     * `onlyOwner` functions anymore. Can only be called by the current owner.
     *
     * NOTE: Renouncing ownership will leave the contract without an owner,
     * thereby removing any functionality that is only available to the owner.
     */
    function renounceOwnership() public virtual onlyOwner {
        _transferOwnership(address(0));
    }

    /**
     * @dev Transfers ownership of the contract to a new account (`newOwner`).
     * Can only be called by the current owner.
     */
    function transferOwnership(address newOwner) public virtual onlyOwner {
        require(newOwner != address(0), "Ownable: new owner is the zero address");
        _transferOwnership(newOwner);
    }

    /**
     * @dev Transfers ownership of the contract to a new account (`newOwner`).
     * Internal function without access restriction.
     */
    function _transferOwnership(address newOwner) internal virtual {
        address oldOwner = _owner;
        _owner = newOwner;
        emit OwnershipTransferred(oldOwner, newOwner);
    }
}

// File: IERC721A.sol


// ERC721A Contracts v4.2.3
// Creator: Chiru Labs

pragma solidity ^0.8.4;

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

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

    /**
     * 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();

    /**
     * The `quantity` minted with ERC2309 exceeds the safety limit.
     */
    error MintERC2309QuantityExceedsLimit();

    /**
     * The `extraData` cannot be set on an unintialized ownership slot.
     */
    error OwnershipNotInitializedForExtraData();

    // =============================================================
    //                            STRUCTS
    // =============================================================

    struct TokenOwnership {
        // The address of the owner.
        address addr;
        // Stores the start time of ownership with minimal overhead for tokenomics.
        uint64 startTimestamp;
        // Whether the token has been burned.
        bool burned;
        // Arbitrary data similar to `startTimestamp` that can be set via {_extraData}.
        uint24 extraData;
    }

    // =============================================================
    //                         TOKEN COUNTERS
    // =============================================================

    /**
     * @dev Returns the total number of tokens in existence.
     * Burned tokens will reduce the count.
     * To get the total number of tokens minted, please see {_totalMinted}.
     */
    function totalSupply() external view returns (uint256);

    // =============================================================
    //                            IERC165
    // =============================================================

    /**
     * @dev Returns true if this contract implements the interface defined by
     * `interfaceId`. See the corresponding
     * [EIP section](https://eips.ethereum.org/EIPS/eip-165#how-interfaces-are-identified)
     * to learn more about how these ids are created.
     *
     * This function call must use less than 30000 gas.
     */
    function supportsInterface(bytes4 interfaceId) external view returns (bool);

    // =============================================================
    //                            IERC721
    // =============================================================

    /**
     * @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`,
     * 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,
        bytes calldata data
    ) external payable;

    /**
     * @dev Equivalent to `safeTransferFrom(from, to, tokenId, '')`.
     */
    function safeTransferFrom(
        address from,
        address to,
        uint256 tokenId
    ) external payable;

    /**
     * @dev Transfers `tokenId` 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 payable;

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

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

    // =============================================================
    //                        IERC721Metadata
    // =============================================================

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

    // =============================================================
    //                           IERC2309
    // =============================================================

    /**
     * @dev Emitted when tokens in `fromTokenId` to `toTokenId`
     * (inclusive) is transferred from `from` to `to`, as defined in the
     * [ERC2309](https://eips.ethereum.org/EIPS/eip-2309) standard.
     *
     * See {_mintERC2309} for more details.
     */
    event ConsecutiveTransfer(uint256 indexed fromTokenId, uint256 toTokenId, address indexed from, address indexed to);
}
// File: ERC721A.sol


// ERC721A Contracts v4.2.3
// Creator: Chiru Labs

pragma solidity ^0.8.4;


/**
 * @dev Interface of ERC721 token receiver.
 */
interface ERC721A__IERC721Receiver {
    function onERC721Received(
        address operator,
        address from,
        uint256 tokenId,
        bytes calldata data
    ) external returns (bytes4);
}

/**
 * @title ERC721A
 *
 * @dev Implementation of the [ERC721](https://eips.ethereum.org/EIPS/eip-721)
 * Non-Fungible Token Standard, including the Metadata extension.
 * Optimized for lower gas during batch mints.
 *
 * Token IDs are minted in sequential order (e.g. 0, 1, 2, 3, ...)
 * starting from `_startTokenId()`.
 *
 * Assumptions:
 *
 * - An owner cannot have more than 2**64 - 1 (max value of uint64) of supply.
 * - The maximum token ID cannot exceed 2**256 - 1 (max value of uint256).
 */
contract ERC721A is IERC721A {
    // Bypass for a `--via-ir` bug (https://github.com/chiru-labs/ERC721A/pull/364).
    struct TokenApprovalRef {
        address value;
    }

    // =============================================================
    //                           CONSTANTS
    // =============================================================

    // Mask of an entry in packed address data.
    uint256 private constant _BITMASK_ADDRESS_DATA_ENTRY = (1 << 64) - 1;

    // The bit position of `numberMinted` in packed address data.
    uint256 private constant _BITPOS_NUMBER_MINTED = 64;

    // The bit position of `numberBurned` in packed address data.
    uint256 private constant _BITPOS_NUMBER_BURNED = 128;

    // The bit position of `aux` in packed address data.
    uint256 private constant _BITPOS_AUX = 192;

    // Mask of all 256 bits in packed address data except the 64 bits for `aux`.
    uint256 private constant _BITMASK_AUX_COMPLEMENT = (1 << 192) - 1;

    // The bit position of `startTimestamp` in packed ownership.
    uint256 private constant _BITPOS_START_TIMESTAMP = 160;

    // The bit mask of the `burned` bit in packed ownership.
    uint256 private constant _BITMASK_BURNED = 1 << 224;

    // The bit position of the `nextInitialized` bit in packed ownership.
    uint256 private constant _BITPOS_NEXT_INITIALIZED = 225;

    // The bit mask of the `nextInitialized` bit in packed ownership.
    uint256 private constant _BITMASK_NEXT_INITIALIZED = 1 << 225;

    // The bit position of `extraData` in packed ownership.
    uint256 private constant _BITPOS_EXTRA_DATA = 232;

    // Mask of all 256 bits in a packed ownership except the 24 bits for `extraData`.
    uint256 private constant _BITMASK_EXTRA_DATA_COMPLEMENT = (1 << 232) - 1;

    // The mask of the lower 160 bits for addresses.
    uint256 private constant _BITMASK_ADDRESS = (1 << 160) - 1;

    // The maximum `quantity` that can be minted with {_mintERC2309}.
    // This limit is to prevent overflows on the address data entries.
    // For a limit of 5000, a total of 3.689e15 calls to {_mintERC2309}
    // is required to cause an overflow, which is unrealistic.
    uint256 private constant _MAX_MINT_ERC2309_QUANTITY_LIMIT = 5000;

    // The `Transfer` event signature is given by:
    // `keccak256(bytes("Transfer(address,address,uint256)"))`.
    bytes32 private constant _TRANSFER_EVENT_SIGNATURE =
        0xddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef;

    // =============================================================
    //                            STORAGE
    // =============================================================

    // The next token ID to be minted.
    uint256 private _currentIndex;

    // The number of tokens burned.
    uint256 private _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 {_packedOwnershipOf} implementation for details.
    //
    // Bits Layout:
    // - [0..159]   `addr`
    // - [160..223] `startTimestamp`
    // - [224]      `burned`
    // - [225]      `nextInitialized`
    // - [232..255] `extraData`
    mapping(uint256 => uint256) private _packedOwnerships;

    // Mapping owner address to address data.
    //
    // Bits Layout:
    // - [0..63]    `balance`
    // - [64..127]  `numberMinted`
    // - [128..191] `numberBurned`
    // - [192..255] `aux`
    mapping(address => uint256) private _packedAddressData;

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

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

    // =============================================================
    //                          CONSTRUCTOR
    // =============================================================

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

    // =============================================================
    //                   TOKEN COUNTING OPERATIONS
    // =============================================================

    /**
     * @dev Returns the starting token ID.
     * To change the starting token ID, please override this function.
     */
    function _startTokenId() internal view virtual returns (uint256) {
        return 0;
    }

    /**
     * @dev Returns the next token ID to be minted.
     */
    function _nextTokenId() internal view virtual returns (uint256) {
        return _currentIndex;
    }

    /**
     * @dev Returns the total number of tokens in existence.
     * Burned tokens will reduce the count.
     * To get the total number of tokens minted, please see {_totalMinted}.
     */
    function totalSupply() public view virtual override returns (uint256) {
        // Counter underflow is impossible as _burnCounter cannot be incremented
        // more than `_currentIndex - _startTokenId()` times.
        unchecked {
            return _currentIndex - _burnCounter - _startTokenId();
        }
    }

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

    /**
     * @dev Returns the total number of tokens burned.
     */
    function _totalBurned() internal view virtual returns (uint256) {
        return _burnCounter;
    }

    // =============================================================
    //                    ADDRESS DATA OPERATIONS
    // =============================================================

    /**
     * @dev Returns the number of tokens in `owner`'s account.
     */
    function balanceOf(address owner) public view virtual override returns (uint256) {
        if (owner == address(0)) revert BalanceQueryForZeroAddress();
        return _packedAddressData[owner] & _BITMASK_ADDRESS_DATA_ENTRY;
    }

    /**
     * Returns the number of tokens minted by `owner`.
     */
    function _numberMinted(address owner) internal view returns (uint256) {
        return (_packedAddressData[owner] >> _BITPOS_NUMBER_MINTED) & _BITMASK_ADDRESS_DATA_ENTRY;
    }

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

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

    /**
     * Sets the auxiliary 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 virtual {
        uint256 packed = _packedAddressData[owner];
        uint256 auxCasted;
        // Cast `aux` with assembly to avoid redundant masking.
        assembly {
            auxCasted := aux
        }
        packed = (packed & _BITMASK_AUX_COMPLEMENT) | (auxCasted << _BITPOS_AUX);
        _packedAddressData[owner] = packed;
    }

    // =============================================================
    //                            IERC165
    // =============================================================

    /**
     * @dev Returns true if this contract implements the interface defined by
     * `interfaceId`. See the corresponding
     * [EIP section](https://eips.ethereum.org/EIPS/eip-165#how-interfaces-are-identified)
     * to learn more about how these ids are created.
     *
     * This function call must use less than 30000 gas.
     */
    function supportsInterface(bytes4 interfaceId) public view virtual override returns (bool) {
        // The interface IDs are constants representing the first 4 bytes
        // of the XOR of all function selectors in the interface.
        // See: [ERC165](https://eips.ethereum.org/EIPS/eip-165)
        // (e.g. `bytes4(i.functionA.selector ^ i.functionB.selector ^ ...)`)
        return
            interfaceId == 0x01ffc9a7 || // ERC165 interface ID for ERC165.
            interfaceId == 0x80ac58cd || // ERC165 interface ID for ERC721.
            interfaceId == 0x5b5e139f; // ERC165 interface ID for ERC721Metadata.
    }

    // =============================================================
    //                        IERC721Metadata
    // =============================================================

    /**
     * @dev Returns the token collection name.
     */
    function name() public view virtual override returns (string memory) {
        return _name;
    }

    /**
     * @dev Returns the token collection symbol.
     */
    function symbol() public view virtual override returns (string memory) {
        return _symbol;
    }

    /**
     * @dev Returns the Uniform Resource Identifier (URI) for `tokenId` token.
     */
    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, _toString(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, it can be overridden in child contracts.
     */
    function _baseURI() internal view virtual returns (string memory) {
        return '';
    }

    // =============================================================
    //                     OWNERSHIPS OPERATIONS
    // =============================================================

    /**
     * @dev Returns the owner of the `tokenId` token.
     *
     * Requirements:
     *
     * - `tokenId` must exist.
     */
    function ownerOf(uint256 tokenId) public view virtual override returns (address) {
        return address(uint160(_packedOwnershipOf(tokenId)));
    }

    /**
     * @dev Gas spent here starts off proportional to the maximum mint batch size.
     * It gradually moves to O(1) as tokens get transferred around over time.
     */
    function _ownershipOf(uint256 tokenId) internal view virtual returns (TokenOwnership memory) {
        return _unpackedOwnership(_packedOwnershipOf(tokenId));
    }

    /**
     * @dev Returns the unpacked `TokenOwnership` struct at `index`.
     */
    function _ownershipAt(uint256 index) internal view virtual returns (TokenOwnership memory) {
        return _unpackedOwnership(_packedOwnerships[index]);
    }

    /**
     * @dev Initializes the ownership slot minted at `index` for efficiency purposes.
     */
    function _initializeOwnershipAt(uint256 index) internal virtual {
        if (_packedOwnerships[index] == 0) {
            _packedOwnerships[index] = _packedOwnershipOf(index);
        }
    }

    /**
     * Returns the packed ownership data of `tokenId`.
     */
    function _packedOwnershipOf(uint256 tokenId) private view returns (uint256) {
        uint256 curr = tokenId;

        unchecked {
            if (_startTokenId() <= curr)
                if (curr < _currentIndex) {
                    uint256 packed = _packedOwnerships[curr];
                    // If not burned.
                    if (packed & _BITMASK_BURNED == 0) {
                        // Invariant:
                        // There will always be an initialized ownership slot
                        // (i.e. `ownership.addr != address(0) && ownership.burned == false`)
                        // before an unintialized ownership slot
                        // (i.e. `ownership.addr == address(0) && ownership.burned == false`)
                        // Hence, `curr` will not underflow.
                        //
                        // We can directly compare the packed value.
                        // If the address is zero, packed will be zero.
                        while (packed == 0) {
                            packed = _packedOwnerships[--curr];
                        }
                        return packed;
                    }
                }
        }
        revert OwnerQueryForNonexistentToken();
    }

    /**
     * @dev Returns the unpacked `TokenOwnership` struct from `packed`.
     */
    function _unpackedOwnership(uint256 packed) private pure returns (TokenOwnership memory ownership) {
        ownership.addr = address(uint160(packed));
        ownership.startTimestamp = uint64(packed >> _BITPOS_START_TIMESTAMP);
        ownership.burned = packed & _BITMASK_BURNED != 0;
        ownership.extraData = uint24(packed >> _BITPOS_EXTRA_DATA);
    }

    /**
     * @dev Packs ownership data into a single uint256.
     */
    function _packOwnershipData(address owner, uint256 flags) private view returns (uint256 result) {
        assembly {
            // Mask `owner` to the lower 160 bits, in case the upper bits somehow aren't clean.
            owner := and(owner, _BITMASK_ADDRESS)
            // `owner | (block.timestamp << _BITPOS_START_TIMESTAMP) | flags`.
            result := or(owner, or(shl(_BITPOS_START_TIMESTAMP, timestamp()), flags))
        }
    }

    /**
     * @dev Returns the `nextInitialized` flag set if `quantity` equals 1.
     */
    function _nextInitializedFlag(uint256 quantity) private pure returns (uint256 result) {
        // For branchless setting of the `nextInitialized` flag.
        assembly {
            // `(quantity == 1) << _BITPOS_NEXT_INITIALIZED`.
            result := shl(_BITPOS_NEXT_INITIALIZED, eq(quantity, 1))
        }
    }

    // =============================================================
    //                      APPROVAL OPERATIONS
    // =============================================================

    /**
     * @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) public payable virtual override {
        address owner = ownerOf(tokenId);

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

        _tokenApprovals[tokenId].value = to;
        emit Approval(owner, to, tokenId);
    }

    /**
     * @dev Returns the account approved for `tokenId` token.
     *
     * Requirements:
     *
     * - `tokenId` must exist.
     */
    function getApproved(uint256 tokenId) public view virtual override returns (address) {
        if (!_exists(tokenId)) revert ApprovalQueryForNonexistentToken();

        return _tokenApprovals[tokenId].value;
    }

    /**
     * @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) public virtual override {
        _operatorApprovals[_msgSenderERC721A()][operator] = approved;
        emit ApprovalForAll(_msgSenderERC721A(), operator, approved);
    }

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

    /**
     * @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. See {_mint}.
     */
    function _exists(uint256 tokenId) internal view virtual returns (bool) {
        return
            _startTokenId() <= tokenId &&
            tokenId < _currentIndex && // If within bounds,
            _packedOwnerships[tokenId] & _BITMASK_BURNED == 0; // and not burned.
    }

    /**
     * @dev Returns whether `msgSender` is equal to `approvedAddress` or `owner`.
     */
    function _isSenderApprovedOrOwner(
        address approvedAddress,
        address owner,
        address msgSender
    ) private pure returns (bool result) {
        assembly {
            // Mask `owner` to the lower 160 bits, in case the upper bits somehow aren't clean.
            owner := and(owner, _BITMASK_ADDRESS)
            // Mask `msgSender` to the lower 160 bits, in case the upper bits somehow aren't clean.
            msgSender := and(msgSender, _BITMASK_ADDRESS)
            // `msgSender == owner || msgSender == approvedAddress`.
            result := or(eq(msgSender, owner), eq(msgSender, approvedAddress))
        }
    }

    /**
     * @dev Returns the storage slot and value for the approved address of `tokenId`.
     */
    function _getApprovedSlotAndAddress(uint256 tokenId)
        private
        view
        returns (uint256 approvedAddressSlot, address approvedAddress)
    {
        TokenApprovalRef storage tokenApproval = _tokenApprovals[tokenId];
        // The following is equivalent to `approvedAddress = _tokenApprovals[tokenId].value`.
        assembly {
            approvedAddressSlot := tokenApproval.slot
            approvedAddress := sload(approvedAddressSlot)
        }
    }

    // =============================================================
    //                      TRANSFER OPERATIONS
    // =============================================================

    /**
     * @dev Transfers `tokenId` from `from` to `to`.
     *
     * 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
    ) public payable virtual override {
        uint256 prevOwnershipPacked = _packedOwnershipOf(tokenId);

        if (address(uint160(prevOwnershipPacked)) != from) revert TransferFromIncorrectOwner();

        (uint256 approvedAddressSlot, address approvedAddress) = _getApprovedSlotAndAddress(tokenId);

        // The nested ifs save around 20+ gas over a compound boolean condition.
        if (!_isSenderApprovedOrOwner(approvedAddress, from, _msgSenderERC721A()))
            if (!isApprovedForAll(from, _msgSenderERC721A())) revert TransferCallerNotOwnerNorApproved();

        if (to == address(0)) revert TransferToZeroAddress();

        _beforeTokenTransfers(from, to, tokenId, 1);

        // Clear approvals from the previous owner.
        assembly {
            if approvedAddress {
                // This is equivalent to `delete _tokenApprovals[tokenId]`.
                sstore(approvedAddressSlot, 0)
            }
        }

        // 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 {
            // We can directly increment and decrement the balances.
            --_packedAddressData[from]; // Updates: `balance -= 1`.
            ++_packedAddressData[to]; // Updates: `balance += 1`.

            // Updates:
            // - `address` to the next owner.
            // - `startTimestamp` to the timestamp of transfering.
            // - `burned` to `false`.
            // - `nextInitialized` to `true`.
            _packedOwnerships[tokenId] = _packOwnershipData(
                to,
                _BITMASK_NEXT_INITIALIZED | _nextExtraData(from, to, prevOwnershipPacked)
            );

            // If the next slot may not have been initialized (i.e. `nextInitialized == false`) .
            if (prevOwnershipPacked & _BITMASK_NEXT_INITIALIZED == 0) {
                uint256 nextTokenId = tokenId + 1;
                // If the next slot's address is zero and not burned (i.e. packed value is zero).
                if (_packedOwnerships[nextTokenId] == 0) {
                    // If the next slot is within bounds.
                    if (nextTokenId != _currentIndex) {
                        // Initialize the next slot to maintain correctness for `ownerOf(tokenId + 1)`.
                        _packedOwnerships[nextTokenId] = prevOwnershipPacked;
                    }
                }
            }
        }

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

    /**
     * @dev Equivalent to `safeTransferFrom(from, to, tokenId, '')`.
     */
    function safeTransferFrom(
        address from,
        address to,
        uint256 tokenId
    ) public payable virtual override {
        safeTransferFrom(from, to, tokenId, '');
    }

    /**
     * @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 memory _data
    ) public payable virtual override {
        transferFrom(from, to, tokenId);
        if (to.code.length != 0)
            if (!_checkContractOnERC721Received(from, to, tokenId, _data)) {
                revert TransferToNonERC721ReceiverImplementer();
            }
    }

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

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

    // =============================================================
    //                        MINT OPERATIONS
    // =============================================================

    /**
     * @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 for each mint.
     */
    function _mint(address to, uint256 quantity) internal virtual {
        uint256 startTokenId = _currentIndex;
        if (quantity == 0) revert MintZeroQuantity();

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

        // Overflows are incredibly unrealistic.
        // `balance` and `numberMinted` have a maximum limit of 2**64.
        // `tokenId` has a maximum limit of 2**256.
        unchecked {
            // Updates:
            // - `balance += quantity`.
            // - `numberMinted += quantity`.
            //
            // We can directly add to the `balance` and `numberMinted`.
            _packedAddressData[to] += quantity * ((1 << _BITPOS_NUMBER_MINTED) | 1);

            // Updates:
            // - `address` to the owner.
            // - `startTimestamp` to the timestamp of minting.
            // - `burned` to `false`.
            // - `nextInitialized` to `quantity == 1`.
            _packedOwnerships[startTokenId] = _packOwnershipData(
                to,
                _nextInitializedFlag(quantity) | _nextExtraData(address(0), to, 0)
            );

            uint256 toMasked;
            uint256 end = startTokenId + quantity;

            // Use assembly to loop and emit the `Transfer` event for gas savings.
            // The duplicated `log4` removes an extra check and reduces stack juggling.
            // The assembly, together with the surrounding Solidity code, have been
            // delicately arranged to nudge the compiler into producing optimized opcodes.
            assembly {
                // Mask `to` to the lower 160 bits, in case the upper bits somehow aren't clean.
                toMasked := and(to, _BITMASK_ADDRESS)
                // Emit the `Transfer` event.
                log4(
                    0, // Start of data (0, since no data).
                    0, // End of data (0, since no data).
                    _TRANSFER_EVENT_SIGNATURE, // Signature.
                    0, // `address(0)`.
                    toMasked, // `to`.
                    startTokenId // `tokenId`.
                )

                // The `iszero(eq(,))` check ensures that large values of `quantity`
                // that overflows uint256 will make the loop run out of gas.
                // The compiler will optimize the `iszero` away for performance.
                for {
                    let tokenId := add(startTokenId, 1)
                } iszero(eq(tokenId, end)) {
                    tokenId := add(tokenId, 1)
                } {
                    // Emit the `Transfer` event. Similar to above.
                    log4(0, 0, _TRANSFER_EVENT_SIGNATURE, 0, toMasked, tokenId)
                }
            }
            if (toMasked == 0) revert MintToZeroAddress();

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

    /**
     * @dev Mints `quantity` tokens and transfers them to `to`.
     *
     * This function is intended for efficient minting only during contract creation.
     *
     * It emits only one {ConsecutiveTransfer} as defined in
     * [ERC2309](https://eips.ethereum.org/EIPS/eip-2309),
     * instead of a sequence of {Transfer} event(s).
     *
     * Calling this function outside of contract creation WILL make your contract
     * non-compliant with the ERC721 standard.
     * For full ERC721 compliance, substituting ERC721 {Transfer} event(s) with the ERC2309
     * {ConsecutiveTransfer} event is only permissible during contract creation.
     *
     * Requirements:
     *
     * - `to` cannot be the zero address.
     * - `quantity` must be greater than 0.
     *
     * Emits a {ConsecutiveTransfer} event.
     */
    function _mintERC2309(address to, uint256 quantity) internal virtual {
        uint256 startTokenId = _currentIndex;
        if (to == address(0)) revert MintToZeroAddress();
        if (quantity == 0) revert MintZeroQuantity();
        if (quantity > _MAX_MINT_ERC2309_QUANTITY_LIMIT) revert MintERC2309QuantityExceedsLimit();

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

        // Overflows are unrealistic due to the above check for `quantity` to be below the limit.
        unchecked {
            // Updates:
            // - `balance += quantity`.
            // - `numberMinted += quantity`.
            //
            // We can directly add to the `balance` and `numberMinted`.
            _packedAddressData[to] += quantity * ((1 << _BITPOS_NUMBER_MINTED) | 1);

            // Updates:
            // - `address` to the owner.
            // - `startTimestamp` to the timestamp of minting.
            // - `burned` to `false`.
            // - `nextInitialized` to `quantity == 1`.
            _packedOwnerships[startTokenId] = _packOwnershipData(
                to,
                _nextInitializedFlag(quantity) | _nextExtraData(address(0), to, 0)
            );

            emit ConsecutiveTransfer(startTokenId, startTokenId + quantity - 1, address(0), to);

            _currentIndex = startTokenId + quantity;
        }
        _afterTokenTransfers(address(0), to, startTokenId, 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.
     *
     * See {_mint}.
     *
     * Emits a {Transfer} event for each mint.
     */
    function _safeMint(
        address to,
        uint256 quantity,
        bytes memory _data
    ) internal virtual {
        _mint(to, quantity);

        unchecked {
            if (to.code.length != 0) {
                uint256 end = _currentIndex;
                uint256 index = end - quantity;
                do {
                    if (!_checkContractOnERC721Received(address(0), to, index++, _data)) {
                        revert TransferToNonERC721ReceiverImplementer();
                    }
                } while (index < end);
                // Reentrancy protection.
                if (_currentIndex != end) revert();
            }
        }
    }

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

    // =============================================================
    //                        BURN OPERATIONS
    // =============================================================

    /**
     * @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 {
        uint256 prevOwnershipPacked = _packedOwnershipOf(tokenId);

        address from = address(uint160(prevOwnershipPacked));

        (uint256 approvedAddressSlot, address approvedAddress) = _getApprovedSlotAndAddress(tokenId);

        if (approvalCheck) {
            // The nested ifs save around 20+ gas over a compound boolean condition.
            if (!_isSenderApprovedOrOwner(approvedAddress, from, _msgSenderERC721A()))
                if (!isApprovedForAll(from, _msgSenderERC721A())) revert TransferCallerNotOwnerNorApproved();
        }

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

        // Clear approvals from the previous owner.
        assembly {
            if approvedAddress {
                // This is equivalent to `delete _tokenApprovals[tokenId]`.
                sstore(approvedAddressSlot, 0)
            }
        }

        // 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 {
            // Updates:
            // - `balance -= 1`.
            // - `numberBurned += 1`.
            //
            // We can directly decrement the balance, and increment the number burned.
            // This is equivalent to `packed -= 1; packed += 1 << _BITPOS_NUMBER_BURNED;`.
            _packedAddressData[from] += (1 << _BITPOS_NUMBER_BURNED) - 1;

            // Updates:
            // - `address` to the last owner.
            // - `startTimestamp` to the timestamp of burning.
            // - `burned` to `true`.
            // - `nextInitialized` to `true`.
            _packedOwnerships[tokenId] = _packOwnershipData(
                from,
                (_BITMASK_BURNED | _BITMASK_NEXT_INITIALIZED) | _nextExtraData(from, address(0), prevOwnershipPacked)
            );

            // If the next slot may not have been initialized (i.e. `nextInitialized == false`) .
            if (prevOwnershipPacked & _BITMASK_NEXT_INITIALIZED == 0) {
                uint256 nextTokenId = tokenId + 1;
                // If the next slot's address is zero and not burned (i.e. packed value is zero).
                if (_packedOwnerships[nextTokenId] == 0) {
                    // If the next slot is within bounds.
                    if (nextTokenId != _currentIndex) {
                        // Initialize the next slot to maintain correctness for `ownerOf(tokenId + 1)`.
                        _packedOwnerships[nextTokenId] = prevOwnershipPacked;
                    }
                }
            }
        }

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

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

    // =============================================================
    //                     EXTRA DATA OPERATIONS
    // =============================================================

    /**
     * @dev Directly sets the extra data for the ownership data `index`.
     */
    function _setExtraDataAt(uint256 index, uint24 extraData) internal virtual {
        uint256 packed = _packedOwnerships[index];
        if (packed == 0) revert OwnershipNotInitializedForExtraData();
        uint256 extraDataCasted;
        // Cast `extraData` with assembly to avoid redundant masking.
        assembly {
            extraDataCasted := extraData
        }
        packed = (packed & _BITMASK_EXTRA_DATA_COMPLEMENT) | (extraDataCasted << _BITPOS_EXTRA_DATA);
        _packedOwnerships[index] = packed;
    }

    /**
     * @dev Called during each token transfer to set the 24bit `extraData` field.
     * Intended to be overridden by the cosumer contract.
     *
     * `previousExtraData` - the value of `extraData` before transfer.
     *
     * 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 _extraData(
        address from,
        address to,
        uint24 previousExtraData
    ) internal view virtual returns (uint24) {}

    /**
     * @dev Returns the next extra data for the packed ownership data.
     * The returned result is shifted into position.
     */
    function _nextExtraData(
        address from,
        address to,
        uint256 prevOwnershipPacked
    ) private view returns (uint256) {
        uint24 extraData = uint24(prevOwnershipPacked >> _BITPOS_EXTRA_DATA);
        return uint256(_extraData(from, to, extraData)) << _BITPOS_EXTRA_DATA;
    }

    // =============================================================
    //                       OTHER OPERATIONS
    // =============================================================

    /**
     * @dev Returns the message sender (defaults to `msg.sender`).
     *
     * If you are writing GSN compatible contracts, you need to override this function.
     */
    function _msgSenderERC721A() internal view virtual returns (address) {
        return msg.sender;
    }

    /**
     * @dev Converts a uint256 to its ASCII string decimal representation.
     */
    function _toString(uint256 value) internal pure virtual returns (string memory str) {
        assembly {
            // The maximum value of a uint256 contains 78 digits (1 byte per digit), but
            // we allocate 0xa0 bytes to keep the free memory pointer 32-byte word aligned.
            // We will need 1 word for the trailing zeros padding, 1 word for the length,
            // and 3 words for a maximum of 78 digits. Total: 5 * 0x20 = 0xa0.
            let m := add(mload(0x40), 0xa0)
            // Update the free memory pointer to allocate.
            mstore(0x40, m)
            // Assign the `str` to the end.
            str := sub(m, 0x20)
            // Zeroize the slot after the string.
            mstore(str, 0)

            // Cache the end of the memory to calculate the length later.
            let end := str

            // We write the string from rightmost digit to leftmost digit.
            // The following is essentially a do-while loop that also handles the zero case.
            // prettier-ignore
            for { let temp := value } 1 {} {
                str := sub(str, 1)
                // Write the character to the pointer.
                // The ASCII index of the '0' character is 48.
                mstore8(str, add(48, mod(temp, 10)))
                // Keep dividing `temp` until zero.
                temp := div(temp, 10)
                // prettier-ignore
                if iszero(temp) { break }
            }

            let length := sub(end, str)
            // Move the pointer 32 bytes leftwards to make room for the length.
            str := sub(str, 0x20)
            // Store the length.
            mstore(str, length)
        }
    }
}
// File: DIOSNFT.sol

pragma solidity ^0.8.7;
/*
 .----------------.  .----------------.  .----------------.  .----------------. 
| .--------------. || .--------------. || .--------------. || .--------------. |
| |  ________    | || |     _____    | || |     ____     | || |    _______   | |
| | |_   ___ `.  | || |    |_   _|   | || |   .'    `.   | || |   /  ___  |  | |
| |   | |   `. \ | || |      | |     | || |  /  .--.  \  | || |  |  (__ \_|  | |
| |   | |    | | | || |      | |     | || |  | |    | |  | || |   '.___`-.   | |
| |  _| |___.' / | || |     _| |_    | || |  \  `--'  /  | || |  |`\____) |  | |
| | |________.'  | || |    |_____|   | || |   `.____.'   | || |  |_______.'  | |
| |              | || |              | || |              | || |              | |
| '--------------' || '--------------' || '--------------' || '--------------' |
 '----------------'  '----------------'  '----------------'  '----------------'                                                                       
*/





contract DIOsNFT is  ERC721A, Ownable, ReentrancyGuard {
    uint256 public constant MAX_SUPPLY = 8888;
    uint256 public constant WL1NORMAL_PRICE = 0.05 ether;
    uint256 public constant WL2DISCOUNT_PRICE = 0.03 ether;
    uint256 public constant PUB_PRICE = 0.07 ether;
    uint256 public constant WL1NORMAL_LIMIT = 2;
    uint256 public constant WL2DISCOUNT_LIMIT = 1;
    uint256 public constant WL3FM_LIMIT = 1;
    uint256 public constant PUB_LIMIT = 3;

    uint256 public constant WL1NORMAL_MAX_SUPPLY = 7910;
    uint256 public constant WL2DISCOUNT_MAX_SUPPLY = 30;
    uint256 public constant WL3FM_MAX_SUPPLY = 60;

    // mainNet
    uint256 public constant WL_SaleTime = 1668513600;
    uint256 public constant PUB_SaleTime = 1668600000;


    uint256 public minteds1 = 0;
    uint256 public minteds2 = 0;
    uint256 public minteds3 = 0;
    uint256 public minteds4 = 0;

    string public baseTokenURI;
    address public metaDataAddress ;

    mapping(address => uint256) public minteds1Map;
    mapping(address => uint256) public minteds2Map;
    mapping(address => uint256) public minteds3Map;
    mapping(address => uint256) public minteds4Map;

    mapping(address => bool) public disapprovedMarketplaces;

    bytes32 public root1 =
        0x6413a4cc6c8a43b348766863f59ba07981866a81b0f67f05b94476edb2a34f2b;
    bytes32 public root2 =
        0x656f5ac3b657fbaa450872f4ae6c2a5025d63fce686e42def340838eb672c9a2;
    bytes32 public root3 =
        0xc88bcf616c4d1031a250c488b6bdf2b343559b2610c4386343ff08f826fc2277;

    constructor(string memory _baseTokenUri)
        ERC721A("Meta-DIOs", "Meta-DIOs")
    {
        baseTokenURI = _baseTokenUri;
    }


    function WL1NORMAL_MINT(uint256 amount, bytes32[] memory proof) external payable{
        require(isWhiteLists1(proof, keccak256(abi.encodePacked(msg.sender))),"not WL1");
        require(msg.value >= amount* WL1NORMAL_PRICE,"value low");
        require(minteds1Map[msg.sender] + amount <= WL1NORMAL_LIMIT, "Limit exceeded");
        require(minteds1 + amount <= WL1NORMAL_MAX_SUPPLY, "Sold out!");
        require(block.timestamp >= WL_SaleTime , "Not on WL sale");
        require(PUB_SaleTime >= block.timestamp , "Not on WL sale");
        unchecked {
            minteds1Map[msg.sender] += amount;
            minteds1 += amount;
        }

        _mint(msg.sender, amount);
    }

    function WL2DISCOUNT_MINT(uint256 amount, bytes32[] memory proof) external payable{
        require(isWhiteLists2(proof, keccak256(abi.encodePacked(msg.sender))),"not WL2");
        require(msg.value >= amount* WL2DISCOUNT_PRICE,"value low");
        require(minteds2Map[msg.sender] + amount <= WL2DISCOUNT_LIMIT, "Limit exceeded");
        require(minteds2 + amount <= WL2DISCOUNT_MAX_SUPPLY, "Sold out!");
        require(block.timestamp >= WL_SaleTime, "Not on WL sale");
        require(PUB_SaleTime >= block.timestamp , "Not on WL sale");
        unchecked {
            minteds2Map[msg.sender] += amount;
            minteds2 += amount;
        }

        _mint(msg.sender, amount);
    }


    function WL3FM_MINT(uint256 amount, bytes32[] memory proof) external {
        require(isWhiteLists3(proof, keccak256(abi.encodePacked(msg.sender))),"not WL3");
        require(minteds3 + amount <= WL3FM_MAX_SUPPLY, "Sold out!");
        require(minteds3Map[msg.sender] + amount <= WL3FM_LIMIT, "Limit exceeded");
        require(block.timestamp >= WL_SaleTime, "Not on WL sale");
        require(PUB_SaleTime >= block.timestamp , "Not on WL sale");
        unchecked {
            minteds3Map[msg.sender] += amount;
            minteds3 += amount;
        }

        _mint(msg.sender, amount);
    }

    function PUB_MINT(uint256 amount) external payable {
        require(totalSupply() + amount <= MAX_SUPPLY, "Sold out!");
        require(minteds4Map[msg.sender] + amount <= PUB_LIMIT, "Limit exceeded");
        require(msg.value >= amount* PUB_PRICE,"value low");
        require(block.timestamp >= PUB_SaleTime, "Not on PUB sale");
        unchecked {
            minteds4Map[msg.sender] += amount;
            minteds4 += amount;
        }
        _mint(msg.sender, amount);
    }

    function isWhiteLists1(bytes32[] memory proof, bytes32 leaf)
        public
        view
        returns (bool)
    {
        return MerkleProof.verify(proof, root1, leaf);
    }

    function isWhiteLists2(bytes32[] memory proof, bytes32 leaf)
        public
        view
        returns (bool)
    {
        return MerkleProof.verify(proof, root2, leaf);
    }

    function isWhiteLists3(bytes32[] memory proof, bytes32 leaf)
        public
        view
        returns (bool)
    {
        return MerkleProof.verify(proof, root3, leaf);
    }

    receive() external payable {}

    function ownerMint(address to, uint256 amount) external onlyOwner {
        require(totalSupply() + amount <= MAX_SUPPLY, "Sold out!");
        _mint(to, amount);
    }

    function setBaseTokenURI(string calldata _uri) external onlyOwner {
        baseTokenURI = _uri;
    }

    function setMetadata(address _address) external onlyOwner {
        metaDataAddress = _address;
    }

    function setDisapprovedMarketplace(address market, bool isDisapprove)
        external
        onlyOwner
    {
        disapprovedMarketplaces[market] = isDisapprove;
    }

    function approve(address to, uint256 tokenId)
        public
        payable
        virtual
        override
    {
        require(!disapprovedMarketplaces[to], "The address is not approved");
        super.approve(to, tokenId);
    }

    function setApprovalForAll(address operator, bool approved)
        public
        virtual
        override
    {
        require(
            !disapprovedMarketplaces[operator],
            "The address is not approved"
        );
        super.setApprovalForAll(operator, approved);
    }

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

    function tokenURI(uint256 tokenId)
        public
        view
        override
        returns (string memory)
    {
        require(
            _exists(tokenId),
            "ERC721Metadata: URI query for nonexistent token"
        );
        string memory baseURI = _baseURI();
        string memory _tokenUri = IDIOSMetadata(metaDataAddress).getMetadata(tokenId);
        return
            bytes(baseURI).length != 0
                ? _tokenUri
                : "";
    }

    function _startTokenId() internal pure override returns (uint256) {
        return 1;
    }

    function withdraw() public payable onlyOwner {
        (bool success, ) = payable(msg.sender).call{
            value: address(this).balance
        }("");
        require(success);
    }
}

interface IDIOSMetadata {
    function getMetadata(uint256 tokenId) external view returns (string memory);    
}

Contract Security Audit

Contract ABI

[{"inputs":[{"internalType":"string","name":"_baseTokenUri","type":"string"}],"stateMutability":"nonpayable","type":"constructor"},{"inputs":[],"name":"ApprovalCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"ApprovalQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"BalanceQueryForZeroAddress","type":"error"},{"inputs":[],"name":"MintERC2309QuantityExceedsLimit","type":"error"},{"inputs":[],"name":"MintToZeroAddress","type":"error"},{"inputs":[],"name":"MintZeroQuantity","type":"error"},{"inputs":[],"name":"OwnerQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"OwnershipNotInitializedForExtraData","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":"uint256","name":"fromTokenId","type":"uint256"},{"indexed":false,"internalType":"uint256","name":"toTokenId","type":"uint256"},{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"}],"name":"ConsecutiveTransfer","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"},{"inputs":[],"name":"MAX_SUPPLY","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"PUB_LIMIT","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"amount","type":"uint256"}],"name":"PUB_MINT","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"PUB_PRICE","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"PUB_SaleTime","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"WL1NORMAL_LIMIT","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"WL1NORMAL_MAX_SUPPLY","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"amount","type":"uint256"},{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"}],"name":"WL1NORMAL_MINT","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"WL1NORMAL_PRICE","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"WL2DISCOUNT_LIMIT","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"WL2DISCOUNT_MAX_SUPPLY","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"amount","type":"uint256"},{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"}],"name":"WL2DISCOUNT_MINT","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"WL2DISCOUNT_PRICE","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"WL3FM_LIMIT","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"WL3FM_MAX_SUPPLY","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"amount","type":"uint256"},{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"}],"name":"WL3FM_MINT","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"WL_SaleTime","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"approve","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"}],"name":"balanceOf","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"baseTokenURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"disapprovedMarketplaces","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":[{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"},{"internalType":"bytes32","name":"leaf","type":"bytes32"}],"name":"isWhiteLists1","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"},{"internalType":"bytes32","name":"leaf","type":"bytes32"}],"name":"isWhiteLists2","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"},{"internalType":"bytes32","name":"leaf","type":"bytes32"}],"name":"isWhiteLists3","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"metaDataAddress","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"minteds1","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"minteds1Map","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"minteds2","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"minteds2Map","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"minteds3","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"minteds3Map","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"minteds4","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"minteds4Map","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":"address","name":"to","type":"address"},{"internalType":"uint256","name":"amount","type":"uint256"}],"name":"ownerMint","outputs":[],"stateMutability":"nonpayable","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":[],"name":"root1","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"root2","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"root3","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"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":"payable","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":"payable","type":"function"},{"inputs":[{"internalType":"address","name":"operator","type":"address"},{"internalType":"bool","name":"approved","type":"bool"}],"name":"setApprovalForAll","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"_uri","type":"string"}],"name":"setBaseTokenURI","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"market","type":"address"},{"internalType":"bool","name":"isDisapprove","type":"bool"}],"name":"setDisapprovedMarketplace","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"_address","type":"address"}],"name":"setMetadata","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":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"tokenURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"totalSupply","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"transferFrom","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"address","name":"newOwner","type":"address"}],"name":"transferOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"withdraw","outputs":[],"stateMutability":"payable","type":"function"},{"stateMutability":"payable","type":"receive"}]

60806040526000600a819055600b819055600c819055600d557f6413a4cc6c8a43b348766863f59ba07981866a81b0f67f05b94476edb2a34f2b6015557f656f5ac3b657fbaa450872f4ae6c2a5025d63fce686e42def340838eb672c9a26016557fc88bcf616c4d1031a250c488b6bdf2b343559b2610c4386343ff08f826fc22776017553480156200009157600080fd5b5060405162002a4d38038062002a4d833981016040819052620000b4916200023b565b6040805180820182526009808252684d6574612d44494f7360b81b602080840182815285518087019096529285528401528151919291620000f89160029162000195565b5080516200010e90600390602084019062000195565b5050600160005550620001213362000143565b600160095580516200013b90600e90602084019062000195565b50506200036a565b600880546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b828054620001a39062000317565b90600052602060002090601f016020900481019282620001c7576000855562000212565b82601f10620001e257805160ff191683800117855562000212565b8280016001018555821562000212579182015b8281111562000212578251825591602001919060010190620001f5565b506200022092915062000224565b5090565b5b8082111562000220576000815560010162000225565b600060208083850312156200024f57600080fd5b82516001600160401b03808211156200026757600080fd5b818501915085601f8301126200027c57600080fd5b81518181111562000291576200029162000354565b604051601f8201601f19908116603f01168101908382118183101715620002bc57620002bc62000354565b816040528281528886848701011115620002d557600080fd5b600093505b82841015620002f95784840186015181850187015292850192620002da565b828411156200030b5760008684830101525b98975050505050505050565b600181811c908216806200032c57607f821691505b602082108114156200034e57634e487b7160e01b600052602260045260246000fd5b50919050565b634e487b7160e01b600052604160045260246000fd5b6126d3806200037a6000396000f3fe60806040526004361061036f5760003560e01c80637b2484b6116101c6578063b88d4fde116100f7578063dbcb4c4311610095578063ef6815eb1161006f578063ef6815eb14610931578063f2fde38b14610951578063f3cb838514610971578063f5e543e01461099157600080fd5b8063dbcb4c43146108bd578063e53c6f12146108d2578063e985e9c5146108e857600080fd5b8063c87b56dd116100d1578063c87b56dd14610845578063d547cfb714610865578063d6ffe24d1461087a578063da0d2bf0146108a757600080fd5b8063b88d4fde146107ef578063bb55697614610802578063c4e987f81461081857600080fd5b80639a26895511610164578063a99e7c651161013e578063a99e7c6514610789578063aa3a8b011461079e578063b472070f146107be578063b7662133146107d957600080fd5b80639a268955146107265780639fb90e7c14610739578063a22cb4651461076957600080fd5b80638b6ed4e6116101a05780638b6ed4e6146106c05780638da5cb5b146106d35780638e887db9146106f157806395d89b411461071157600080fd5b80637b2484b61461067457806380ceba1e1461068a5780638b4feb6a146106aa57600080fd5b806332cb6b0c116102a0578063566ee2391161023e57806368546a871161021857806368546a871461060e5780636d920eb31461062457806370a082311461063f578063715018a61461065f57600080fd5b8063566ee239146105ae5780636352211e146105db57806365ae15bc146105fb57600080fd5b80633e5123b41161027a5780633e5123b4146104d75780633e582fb11461056557806342842e0e1461057b578063484b973c1461058e57600080fd5b806332cb6b0c146105275780633c6c72591461053d5780633ccfd60b1461055d57600080fd5b806318160ddd1161030d57806324fc685c116102e757806324fc685c146104bf5780632e537b1c146104d757806330176e13146104ec578063304c15b51461050c57600080fd5b806318160ddd1461047a57806323b872dd1461049757806324c6f1bd146104aa57600080fd5b8063081812fc11610349578063081812fc146103f2578063095ea7b31461042a5780630f8b08821461043f578063102357a61461046557600080fd5b806301351ac21461037b57806301ffc9a7146103b057806306fdde03146103d057600080fd5b3661037657005b600080fd5b34801561038757600080fd5b5061039b6103963660046122f0565b6109be565b60405190151581526020015b60405180910390f35b3480156103bc57600080fd5b5061039b6103cb366004612335565b6109d4565b3480156103dc57600080fd5b506103e5610a71565b6040516103a79190612520565b3480156103fe57600080fd5b5061041261040d366004612458565b610b03565b6040516001600160a01b0390911681526020016103a7565b61043d6104383660046122c6565b610b60565b005b34801561044b57600080fd5b506104576363737f4081565b6040519081526020016103a7565b34801561047157600080fd5b50610457600381565b34801561048657600080fd5b506001546000540360001901610457565b61043d6104a53660046121a3565b610bdc565b3480156104b657600080fd5b50610457603c81565b3480156104cb57600080fd5b50610457636374d0c081565b3480156104e357600080fd5b50610457600181565b3480156104f857600080fd5b5061043d61050736600461236f565b610db9565b34801561051857600080fd5b5061045766b1a2bc2ec5000081565b34801561053357600080fd5b506104576122b881565b34801561054957600080fd5b5061039b6105583660046122f0565b610dd2565b61043d610de1565b34801561057157600080fd5b50610457600b5481565b61043d6105893660046121a3565b610e41565b34801561059a57600080fd5b5061043d6105a93660046122c6565b610e5c565b3480156105ba57600080fd5b506104576105c9366004612155565b60116020526000908152604090205481565b3480156105e757600080fd5b506104126105f6366004612458565b610ec3565b61043d610609366004612458565b610ece565b34801561061a57600080fd5b5061045760165481565b34801561063057600080fd5b50610457666a94d74f43000081565b34801561064b57600080fd5b5061045761065a366004612155565b611047565b34801561066b57600080fd5b5061043d6110af565b34801561068057600080fd5b50610457611ee681565b34801561069657600080fd5b5061043d6106a536600461228a565b6110c3565b3480156106b657600080fd5b5061045760155481565b61043d6106ce366004612471565b6110f6565b3480156106df57600080fd5b506008546001600160a01b0316610412565b3480156106fd57600080fd5b5061043d61070c366004612471565b611325565b34801561071d57600080fd5b506103e5611508565b61043d610734366004612471565b611517565b34801561074557600080fd5b5061039b610754366004612155565b60146020526000908152604090205460ff1681565b34801561077557600080fd5b5061043d61078436600461228a565b611747565b34801561079557600080fd5b50610457600281565b3480156107aa57600080fd5b50600f54610412906001600160a01b031681565b3480156107ca57600080fd5b5061045766f8b0a10e47000081565b3480156107e557600080fd5b50610457600a5481565b61043d6107fd3660046121df565b6117ba565b34801561080e57600080fd5b50610457600d5481565b34801561082457600080fd5b50610457610833366004612155565b60126020526000908152604090205481565b34801561085157600080fd5b506103e5610860366004612458565b611804565b34801561087157600080fd5b506103e5611955565b34801561088657600080fd5b50610457610895366004612155565b60106020526000908152604090205481565b3480156108b357600080fd5b5061045760175481565b3480156108c957600080fd5b50610457601e81565b3480156108de57600080fd5b50610457600c5481565b3480156108f457600080fd5b5061039b610903366004612170565b6001600160a01b03918216600090815260076020908152604080832093909416825291909152205460ff1690565b34801561093d57600080fd5b5061039b61094c3660046122f0565b6119e3565b34801561095d57600080fd5b5061043d61096c366004612155565b6119f2565b34801561097d57600080fd5b5061043d61098c366004612155565b611a7f565b34801561099d57600080fd5b506104576109ac366004612155565b60136020526000908152604090205481565b60006109cd8360165484611ab6565b9392505050565b60007f01ffc9a7000000000000000000000000000000000000000000000000000000006001600160e01b031983161480610a3757507f80ac58cd000000000000000000000000000000000000000000000000000000006001600160e01b03198316145b80610a6b57507f5b5e139f000000000000000000000000000000000000000000000000000000006001600160e01b03198316145b92915050565b606060028054610a80906125ef565b80601f0160208091040260200160405190810160405280929190818152602001828054610aac906125ef565b8015610af95780601f10610ace57610100808354040283529160200191610af9565b820191906000526020600020905b815481529060010190602001808311610adc57829003601f168201915b5050505050905090565b6000610b0e82611acc565b610b44576040517fcf4700e400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b506000908152600660205260409020546001600160a01b031690565b6001600160a01b03821660009081526014602052604090205460ff1615610bce5760405162461bcd60e51b815260206004820152601b60248201527f5468652061646472657373206973206e6f7420617070726f766564000000000060448201526064015b60405180910390fd5b610bd88282611b01565b5050565b6000610be782611bc7565b9050836001600160a01b0316816001600160a01b031614610c34576040517fa114810000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b60008281526006602052604090208054338082146001600160a01b03881690911417610c9a57610c648633610903565b610c9a576040517f59c896be00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6001600160a01b038516610cda576040517fea553b3400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8015610ce557600082555b6001600160a01b038681166000908152600560205260408082208054600019019055918716808252919020805460010190554260a01b17600160e11b17600085815260046020526040902055600160e11b8316610d705760018401600081815260046020526040902054610d6e576000548114610d6e5760008181526004602052604090208490555b505b83856001600160a01b0316876001600160a01b03167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4505050505050565b610dc1611c49565b610dcd600e838361201a565b505050565b60006109cd8360175484611ab6565b610de9611c49565b604051600090339047908381818185875af1925050503d8060008114610e2b576040519150601f19603f3d011682016040523d82523d6000602084013e610e30565b606091505b5050905080610e3e57600080fd5b50565b610dcd838383604051806020016040528060008152506117ba565b610e64611c49565b6001546000546122b89183910360001901610e7f919061258c565b1115610eb95760405162461bcd60e51b8152602060048201526009602482015268536f6c64206f75742160b81b6044820152606401610bc5565b610bd88282611ca3565b6000610a6b82611bc7565b6001546000546122b89183910360001901610ee9919061258c565b1115610f235760405162461bcd60e51b8152602060048201526009602482015268536f6c64206f75742160b81b6044820152606401610bc5565b33600090815260136020526040902054600390610f4190839061258c565b1115610f805760405162461bcd60e51b815260206004820152600e60248201526d131a5b5a5d08195e18d95959195960921b6044820152606401610bc5565b610f9166f8b0a10e470000826125a4565b341015610fcc5760405162461bcd60e51b815260206004820152600960248201526876616c7565206c6f7760b81b6044820152606401610bc5565b636374d0c04210156110205760405162461bcd60e51b815260206004820152600f60248201527f4e6f74206f6e205055422073616c6500000000000000000000000000000000006044820152606401610bc5565b336000818152601360205260409020805483019055600d805483019055610e3e9082611ca3565b60006001600160a01b038216611089576040517f8f4eb60400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b506001600160a01b031660009081526005602052604090205467ffffffffffffffff1690565b6110b7611c49565b6110c16000611dcd565b565b6110cb611c49565b6001600160a01b03919091166000908152601460205260409020805460ff1916911515919091179055565b6040516bffffffffffffffffffffffff193360601b166020820152611135908290603401604051602081830303815290604052805190602001206109be565b6111815760405162461bcd60e51b815260206004820152600760248201527f6e6f7420574c32000000000000000000000000000000000000000000000000006044820152606401610bc5565b611192666a94d74f430000836125a4565b3410156111cd5760405162461bcd60e51b815260206004820152600960248201526876616c7565206c6f7760b81b6044820152606401610bc5565b336000908152601160205260409020546001906111eb90849061258c565b111561122a5760405162461bcd60e51b815260206004820152600e60248201526d131a5b5a5d08195e18d95959195960921b6044820152606401610bc5565b601e82600b5461123a919061258c565b11156112745760405162461bcd60e51b8152602060048201526009602482015268536f6c64206f75742160b81b6044820152606401610bc5565b6363737f404210156112b95760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b42636374d0c010156112fe5760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b336000818152601160205260409020805484019055600b805484019055610bd89083611ca3565b6040516bffffffffffffffffffffffff193360601b16602082015261136490829060340160405160208183030381529060405280519060200120610dd2565b6113b05760405162461bcd60e51b815260206004820152600760248201527f6e6f7420574c33000000000000000000000000000000000000000000000000006044820152606401610bc5565b603c82600c546113c0919061258c565b11156113fa5760405162461bcd60e51b8152602060048201526009602482015268536f6c64206f75742160b81b6044820152606401610bc5565b3360009081526012602052604090205460019061141890849061258c565b11156114575760405162461bcd60e51b815260206004820152600e60248201526d131a5b5a5d08195e18d95959195960921b6044820152606401610bc5565b6363737f4042101561149c5760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b42636374d0c010156114e15760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b336000818152601260205260409020805484019055600c805484019055610bd89083611ca3565b606060038054610a80906125ef565b6040516bffffffffffffffffffffffff193360601b166020820152611556908290603401604051602081830303815290604052805190602001206119e3565b6115a25760405162461bcd60e51b815260206004820152600760248201527f6e6f7420574c31000000000000000000000000000000000000000000000000006044820152606401610bc5565b6115b366b1a2bc2ec50000836125a4565b3410156115ee5760405162461bcd60e51b815260206004820152600960248201526876616c7565206c6f7760b81b6044820152606401610bc5565b3360009081526010602052604090205460029061160c90849061258c565b111561164b5760405162461bcd60e51b815260206004820152600e60248201526d131a5b5a5d08195e18d95959195960921b6044820152606401610bc5565b611ee682600a5461165c919061258c565b11156116965760405162461bcd60e51b8152602060048201526009602482015268536f6c64206f75742160b81b6044820152606401610bc5565b6363737f404210156116db5760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b42636374d0c010156117205760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b336000818152601060205260409020805484019055600a805484019055610bd89083611ca3565b6001600160a01b03821660009081526014602052604090205460ff16156117b05760405162461bcd60e51b815260206004820152601b60248201527f5468652061646472657373206973206e6f7420617070726f76656400000000006044820152606401610bc5565b610bd88282611e2c565b6117c5848484610bdc565b6001600160a01b0383163b156117fe576117e184848484611e98565b6117fe576040516368d2bf6b60e11b815260040160405180910390fd5b50505050565b606061180f82611acc565b6118815760405162461bcd60e51b815260206004820152602f60248201527f4552433732314d657461646174613a2055524920717565727920666f72206e6f60448201527f6e6578697374656e7420746f6b656e00000000000000000000000000000000006064820152608401610bc5565b600061188b611f8f565b600f546040517fa574cea4000000000000000000000000000000000000000000000000000000008152600481018690529192506000916001600160a01b039091169063a574cea49060240160006040518083038186803b1580156118ee57600080fd5b505afa158015611902573d6000803e3d6000fd5b505050506040513d6000823e601f3d908101601f1916820160405261192a91908101906123e1565b905081516000141561194b576040518060200160405280600081525061194d565b805b949350505050565b600e8054611962906125ef565b80601f016020809104026020016040519081016040528092919081815260200182805461198e906125ef565b80156119db5780601f106119b0576101008083540402835291602001916119db565b820191906000526020600020905b8154815290600101906020018083116119be57829003601f168201915b505050505081565b60006109cd8360155484611ab6565b6119fa611c49565b6001600160a01b038116611a765760405162461bcd60e51b815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201527f64647265737300000000000000000000000000000000000000000000000000006064820152608401610bc5565b610e3e81611dcd565b611a87611c49565b600f805473ffffffffffffffffffffffffffffffffffffffff19166001600160a01b0392909216919091179055565b600082611ac38584611f9e565b14949350505050565b600081600111158015611ae0575060005482105b8015610a6b575050600090815260046020526040902054600160e01b161590565b6000611b0c82610ec3565b9050336001600160a01b03821614611b5e57611b288133610903565b611b5e576040517fcfb3b94200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600082815260066020526040808220805473ffffffffffffffffffffffffffffffffffffffff19166001600160a01b0387811691821790925591518593918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a4505050565b60008180600111611c1757600054811015611c1757600081815260046020526040902054600160e01b8116611c15575b8061194b575060001901600081815260046020526040902054611bf7565b505b6040517fdf2d9b4200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6008546001600160a01b031633146110c15760405162461bcd60e51b815260206004820181905260248201527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e65726044820152606401610bc5565b60005481611cdd576040517fb562e8dd00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6001600160a01b03831660008181526005602090815260408083208054680100000000000000018802019055848352600490915281206001851460e11b4260a01b178317905582840190839083907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef8180a4600183015b818114611d8c57808360007fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a4600101611d54565b5081611dc4576040517f2e07630000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b60005550505050565b600880546001600160a01b0383811673ffffffffffffffffffffffffffffffffffffffff19831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b3360008181526007602090815260408083206001600160a01b03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b604051630a85bd0160e11b81526000906001600160a01b0385169063150b7a0290611ecd9033908990889088906004016124e4565b602060405180830381600087803b158015611ee757600080fd5b505af1925050508015611f17575060408051601f3d908101601f19168201909252611f1491810190612352565b60015b611f72573d808015611f45576040519150601f19603f3d011682016040523d82523d6000602084013e611f4a565b606091505b508051611f6a576040516368d2bf6b60e11b815260040160405180910390fd5b805181602001fd5b6001600160e01b031916630a85bd0160e11b149050949350505050565b6060600e8054610a80906125ef565b600081815b8451811015611fe357611fcf82868381518110611fc257611fc261265b565b6020026020010151611feb565b915080611fdb8161262a565b915050611fa3565b509392505050565b60008183106120075760008281526020849052604090206109cd565b60008381526020839052604090206109cd565b828054612026906125ef565b90600052602060002090601f016020900481019282612048576000855561208e565b82601f106120615782800160ff1982351617855561208e565b8280016001018555821561208e579182015b8281111561208e578235825591602001919060010190612073565b5061209a92915061209e565b5090565b5b8082111561209a576000815560010161209f565b80356001600160a01b03811681146120ca57600080fd5b919050565b600082601f8301126120e057600080fd5b8135602067ffffffffffffffff8211156120fc576120fc612671565b8160051b61210b828201612533565b83815282810190868401838801850189101561212657600080fd5b600093505b8584101561214957803583526001939093019291840191840161212b565b50979650505050505050565b60006020828403121561216757600080fd5b6109cd826120b3565b6000806040838503121561218357600080fd5b61218c836120b3565b915061219a602084016120b3565b90509250929050565b6000806000606084860312156121b857600080fd5b6121c1846120b3565b92506121cf602085016120b3565b9150604084013590509250925092565b600080600080608085870312156121f557600080fd5b6121fe856120b3565b935061220c602086016120b3565b925060408501359150606085013567ffffffffffffffff81111561222f57600080fd5b8501601f8101871361224057600080fd5b803561225361224e82612564565b612533565b81815288602083850101111561226857600080fd5b8160208401602083013760006020838301015280935050505092959194509250565b6000806040838503121561229d57600080fd5b6122a6836120b3565b9150602083013580151581146122bb57600080fd5b809150509250929050565b600080604083850312156122d957600080fd5b6122e2836120b3565b946020939093013593505050565b6000806040838503121561230357600080fd5b823567ffffffffffffffff81111561231a57600080fd5b612326858286016120cf565b95602094909401359450505050565b60006020828403121561234757600080fd5b81356109cd81612687565b60006020828403121561236457600080fd5b81516109cd81612687565b6000806020838503121561238257600080fd5b823567ffffffffffffffff8082111561239a57600080fd5b818501915085601f8301126123ae57600080fd5b8135818111156123bd57600080fd5b8660208285010111156123cf57600080fd5b60209290920196919550909350505050565b6000602082840312156123f357600080fd5b815167ffffffffffffffff81111561240a57600080fd5b8201601f8101841361241b57600080fd5b805161242961224e82612564565b81815285602083850101111561243e57600080fd5b61244f8260208301602086016125c3565b95945050505050565b60006020828403121561246a57600080fd5b5035919050565b6000806040838503121561248457600080fd5b82359150602083013567ffffffffffffffff8111156124a257600080fd5b6124ae858286016120cf565b9150509250929050565b600081518084526124d08160208601602086016125c3565b601f01601f19169290920160200192915050565b60006001600160a01b0380871683528086166020840152508360408301526080606083015261251660808301846124b8565b9695505050505050565b6020815260006109cd60208301846124b8565b604051601f8201601f1916810167ffffffffffffffff8111828210171561255c5761255c612671565b604052919050565b600067ffffffffffffffff82111561257e5761257e612671565b50601f01601f191660200190565b6000821982111561259f5761259f612645565b500190565b60008160001904831182151516156125be576125be612645565b500290565b60005b838110156125de5781810151838201526020016125c6565b838111156117fe5750506000910152565b600181811c9082168061260357607f821691505b6020821081141561262457634e487b7160e01b600052602260045260246000fd5b50919050565b600060001982141561263e5761263e612645565b5060010190565b634e487b7160e01b600052601160045260246000fd5b634e487b7160e01b600052603260045260246000fd5b634e487b7160e01b600052604160045260246000fd5b6001600160e01b031981168114610e3e57600080fdfea2646970667358221220cc6bfbbdb2da0fee5d750955ee7def5de066ffed927e9e3fc97df3a29cf8458c64736f6c63430008070033000000000000000000000000000000000000000000000000000000000000002000000000000000000000000000000000000000000000000000000000000000094d4554412d44494f730000000000000000000000000000000000000000000000

Deployed Bytecode

0x60806040526004361061036f5760003560e01c80637b2484b6116101c6578063b88d4fde116100f7578063dbcb4c4311610095578063ef6815eb1161006f578063ef6815eb14610931578063f2fde38b14610951578063f3cb838514610971578063f5e543e01461099157600080fd5b8063dbcb4c43146108bd578063e53c6f12146108d2578063e985e9c5146108e857600080fd5b8063c87b56dd116100d1578063c87b56dd14610845578063d547cfb714610865578063d6ffe24d1461087a578063da0d2bf0146108a757600080fd5b8063b88d4fde146107ef578063bb55697614610802578063c4e987f81461081857600080fd5b80639a26895511610164578063a99e7c651161013e578063a99e7c6514610789578063aa3a8b011461079e578063b472070f146107be578063b7662133146107d957600080fd5b80639a268955146107265780639fb90e7c14610739578063a22cb4651461076957600080fd5b80638b6ed4e6116101a05780638b6ed4e6146106c05780638da5cb5b146106d35780638e887db9146106f157806395d89b411461071157600080fd5b80637b2484b61461067457806380ceba1e1461068a5780638b4feb6a146106aa57600080fd5b806332cb6b0c116102a0578063566ee2391161023e57806368546a871161021857806368546a871461060e5780636d920eb31461062457806370a082311461063f578063715018a61461065f57600080fd5b8063566ee239146105ae5780636352211e146105db57806365ae15bc146105fb57600080fd5b80633e5123b41161027a5780633e5123b4146104d75780633e582fb11461056557806342842e0e1461057b578063484b973c1461058e57600080fd5b806332cb6b0c146105275780633c6c72591461053d5780633ccfd60b1461055d57600080fd5b806318160ddd1161030d57806324fc685c116102e757806324fc685c146104bf5780632e537b1c146104d757806330176e13146104ec578063304c15b51461050c57600080fd5b806318160ddd1461047a57806323b872dd1461049757806324c6f1bd146104aa57600080fd5b8063081812fc11610349578063081812fc146103f2578063095ea7b31461042a5780630f8b08821461043f578063102357a61461046557600080fd5b806301351ac21461037b57806301ffc9a7146103b057806306fdde03146103d057600080fd5b3661037657005b600080fd5b34801561038757600080fd5b5061039b6103963660046122f0565b6109be565b60405190151581526020015b60405180910390f35b3480156103bc57600080fd5b5061039b6103cb366004612335565b6109d4565b3480156103dc57600080fd5b506103e5610a71565b6040516103a79190612520565b3480156103fe57600080fd5b5061041261040d366004612458565b610b03565b6040516001600160a01b0390911681526020016103a7565b61043d6104383660046122c6565b610b60565b005b34801561044b57600080fd5b506104576363737f4081565b6040519081526020016103a7565b34801561047157600080fd5b50610457600381565b34801561048657600080fd5b506001546000540360001901610457565b61043d6104a53660046121a3565b610bdc565b3480156104b657600080fd5b50610457603c81565b3480156104cb57600080fd5b50610457636374d0c081565b3480156104e357600080fd5b50610457600181565b3480156104f857600080fd5b5061043d61050736600461236f565b610db9565b34801561051857600080fd5b5061045766b1a2bc2ec5000081565b34801561053357600080fd5b506104576122b881565b34801561054957600080fd5b5061039b6105583660046122f0565b610dd2565b61043d610de1565b34801561057157600080fd5b50610457600b5481565b61043d6105893660046121a3565b610e41565b34801561059a57600080fd5b5061043d6105a93660046122c6565b610e5c565b3480156105ba57600080fd5b506104576105c9366004612155565b60116020526000908152604090205481565b3480156105e757600080fd5b506104126105f6366004612458565b610ec3565b61043d610609366004612458565b610ece565b34801561061a57600080fd5b5061045760165481565b34801561063057600080fd5b50610457666a94d74f43000081565b34801561064b57600080fd5b5061045761065a366004612155565b611047565b34801561066b57600080fd5b5061043d6110af565b34801561068057600080fd5b50610457611ee681565b34801561069657600080fd5b5061043d6106a536600461228a565b6110c3565b3480156106b657600080fd5b5061045760155481565b61043d6106ce366004612471565b6110f6565b3480156106df57600080fd5b506008546001600160a01b0316610412565b3480156106fd57600080fd5b5061043d61070c366004612471565b611325565b34801561071d57600080fd5b506103e5611508565b61043d610734366004612471565b611517565b34801561074557600080fd5b5061039b610754366004612155565b60146020526000908152604090205460ff1681565b34801561077557600080fd5b5061043d61078436600461228a565b611747565b34801561079557600080fd5b50610457600281565b3480156107aa57600080fd5b50600f54610412906001600160a01b031681565b3480156107ca57600080fd5b5061045766f8b0a10e47000081565b3480156107e557600080fd5b50610457600a5481565b61043d6107fd3660046121df565b6117ba565b34801561080e57600080fd5b50610457600d5481565b34801561082457600080fd5b50610457610833366004612155565b60126020526000908152604090205481565b34801561085157600080fd5b506103e5610860366004612458565b611804565b34801561087157600080fd5b506103e5611955565b34801561088657600080fd5b50610457610895366004612155565b60106020526000908152604090205481565b3480156108b357600080fd5b5061045760175481565b3480156108c957600080fd5b50610457601e81565b3480156108de57600080fd5b50610457600c5481565b3480156108f457600080fd5b5061039b610903366004612170565b6001600160a01b03918216600090815260076020908152604080832093909416825291909152205460ff1690565b34801561093d57600080fd5b5061039b61094c3660046122f0565b6119e3565b34801561095d57600080fd5b5061043d61096c366004612155565b6119f2565b34801561097d57600080fd5b5061043d61098c366004612155565b611a7f565b34801561099d57600080fd5b506104576109ac366004612155565b60136020526000908152604090205481565b60006109cd8360165484611ab6565b9392505050565b60007f01ffc9a7000000000000000000000000000000000000000000000000000000006001600160e01b031983161480610a3757507f80ac58cd000000000000000000000000000000000000000000000000000000006001600160e01b03198316145b80610a6b57507f5b5e139f000000000000000000000000000000000000000000000000000000006001600160e01b03198316145b92915050565b606060028054610a80906125ef565b80601f0160208091040260200160405190810160405280929190818152602001828054610aac906125ef565b8015610af95780601f10610ace57610100808354040283529160200191610af9565b820191906000526020600020905b815481529060010190602001808311610adc57829003601f168201915b5050505050905090565b6000610b0e82611acc565b610b44576040517fcf4700e400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b506000908152600660205260409020546001600160a01b031690565b6001600160a01b03821660009081526014602052604090205460ff1615610bce5760405162461bcd60e51b815260206004820152601b60248201527f5468652061646472657373206973206e6f7420617070726f766564000000000060448201526064015b60405180910390fd5b610bd88282611b01565b5050565b6000610be782611bc7565b9050836001600160a01b0316816001600160a01b031614610c34576040517fa114810000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b60008281526006602052604090208054338082146001600160a01b03881690911417610c9a57610c648633610903565b610c9a576040517f59c896be00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6001600160a01b038516610cda576040517fea553b3400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8015610ce557600082555b6001600160a01b038681166000908152600560205260408082208054600019019055918716808252919020805460010190554260a01b17600160e11b17600085815260046020526040902055600160e11b8316610d705760018401600081815260046020526040902054610d6e576000548114610d6e5760008181526004602052604090208490555b505b83856001600160a01b0316876001600160a01b03167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4505050505050565b610dc1611c49565b610dcd600e838361201a565b505050565b60006109cd8360175484611ab6565b610de9611c49565b604051600090339047908381818185875af1925050503d8060008114610e2b576040519150601f19603f3d011682016040523d82523d6000602084013e610e30565b606091505b5050905080610e3e57600080fd5b50565b610dcd838383604051806020016040528060008152506117ba565b610e64611c49565b6001546000546122b89183910360001901610e7f919061258c565b1115610eb95760405162461bcd60e51b8152602060048201526009602482015268536f6c64206f75742160b81b6044820152606401610bc5565b610bd88282611ca3565b6000610a6b82611bc7565b6001546000546122b89183910360001901610ee9919061258c565b1115610f235760405162461bcd60e51b8152602060048201526009602482015268536f6c64206f75742160b81b6044820152606401610bc5565b33600090815260136020526040902054600390610f4190839061258c565b1115610f805760405162461bcd60e51b815260206004820152600e60248201526d131a5b5a5d08195e18d95959195960921b6044820152606401610bc5565b610f9166f8b0a10e470000826125a4565b341015610fcc5760405162461bcd60e51b815260206004820152600960248201526876616c7565206c6f7760b81b6044820152606401610bc5565b636374d0c04210156110205760405162461bcd60e51b815260206004820152600f60248201527f4e6f74206f6e205055422073616c6500000000000000000000000000000000006044820152606401610bc5565b336000818152601360205260409020805483019055600d805483019055610e3e9082611ca3565b60006001600160a01b038216611089576040517f8f4eb60400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b506001600160a01b031660009081526005602052604090205467ffffffffffffffff1690565b6110b7611c49565b6110c16000611dcd565b565b6110cb611c49565b6001600160a01b03919091166000908152601460205260409020805460ff1916911515919091179055565b6040516bffffffffffffffffffffffff193360601b166020820152611135908290603401604051602081830303815290604052805190602001206109be565b6111815760405162461bcd60e51b815260206004820152600760248201527f6e6f7420574c32000000000000000000000000000000000000000000000000006044820152606401610bc5565b611192666a94d74f430000836125a4565b3410156111cd5760405162461bcd60e51b815260206004820152600960248201526876616c7565206c6f7760b81b6044820152606401610bc5565b336000908152601160205260409020546001906111eb90849061258c565b111561122a5760405162461bcd60e51b815260206004820152600e60248201526d131a5b5a5d08195e18d95959195960921b6044820152606401610bc5565b601e82600b5461123a919061258c565b11156112745760405162461bcd60e51b8152602060048201526009602482015268536f6c64206f75742160b81b6044820152606401610bc5565b6363737f404210156112b95760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b42636374d0c010156112fe5760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b336000818152601160205260409020805484019055600b805484019055610bd89083611ca3565b6040516bffffffffffffffffffffffff193360601b16602082015261136490829060340160405160208183030381529060405280519060200120610dd2565b6113b05760405162461bcd60e51b815260206004820152600760248201527f6e6f7420574c33000000000000000000000000000000000000000000000000006044820152606401610bc5565b603c82600c546113c0919061258c565b11156113fa5760405162461bcd60e51b8152602060048201526009602482015268536f6c64206f75742160b81b6044820152606401610bc5565b3360009081526012602052604090205460019061141890849061258c565b11156114575760405162461bcd60e51b815260206004820152600e60248201526d131a5b5a5d08195e18d95959195960921b6044820152606401610bc5565b6363737f4042101561149c5760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b42636374d0c010156114e15760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b336000818152601260205260409020805484019055600c805484019055610bd89083611ca3565b606060038054610a80906125ef565b6040516bffffffffffffffffffffffff193360601b166020820152611556908290603401604051602081830303815290604052805190602001206119e3565b6115a25760405162461bcd60e51b815260206004820152600760248201527f6e6f7420574c31000000000000000000000000000000000000000000000000006044820152606401610bc5565b6115b366b1a2bc2ec50000836125a4565b3410156115ee5760405162461bcd60e51b815260206004820152600960248201526876616c7565206c6f7760b81b6044820152606401610bc5565b3360009081526010602052604090205460029061160c90849061258c565b111561164b5760405162461bcd60e51b815260206004820152600e60248201526d131a5b5a5d08195e18d95959195960921b6044820152606401610bc5565b611ee682600a5461165c919061258c565b11156116965760405162461bcd60e51b8152602060048201526009602482015268536f6c64206f75742160b81b6044820152606401610bc5565b6363737f404210156116db5760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b42636374d0c010156117205760405162461bcd60e51b815260206004820152600e60248201526d4e6f74206f6e20574c2073616c6560901b6044820152606401610bc5565b336000818152601060205260409020805484019055600a805484019055610bd89083611ca3565b6001600160a01b03821660009081526014602052604090205460ff16156117b05760405162461bcd60e51b815260206004820152601b60248201527f5468652061646472657373206973206e6f7420617070726f76656400000000006044820152606401610bc5565b610bd88282611e2c565b6117c5848484610bdc565b6001600160a01b0383163b156117fe576117e184848484611e98565b6117fe576040516368d2bf6b60e11b815260040160405180910390fd5b50505050565b606061180f82611acc565b6118815760405162461bcd60e51b815260206004820152602f60248201527f4552433732314d657461646174613a2055524920717565727920666f72206e6f60448201527f6e6578697374656e7420746f6b656e00000000000000000000000000000000006064820152608401610bc5565b600061188b611f8f565b600f546040517fa574cea4000000000000000000000000000000000000000000000000000000008152600481018690529192506000916001600160a01b039091169063a574cea49060240160006040518083038186803b1580156118ee57600080fd5b505afa158015611902573d6000803e3d6000fd5b505050506040513d6000823e601f3d908101601f1916820160405261192a91908101906123e1565b905081516000141561194b576040518060200160405280600081525061194d565b805b949350505050565b600e8054611962906125ef565b80601f016020809104026020016040519081016040528092919081815260200182805461198e906125ef565b80156119db5780601f106119b0576101008083540402835291602001916119db565b820191906000526020600020905b8154815290600101906020018083116119be57829003601f168201915b505050505081565b60006109cd8360155484611ab6565b6119fa611c49565b6001600160a01b038116611a765760405162461bcd60e51b815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201527f64647265737300000000000000000000000000000000000000000000000000006064820152608401610bc5565b610e3e81611dcd565b611a87611c49565b600f805473ffffffffffffffffffffffffffffffffffffffff19166001600160a01b0392909216919091179055565b600082611ac38584611f9e565b14949350505050565b600081600111158015611ae0575060005482105b8015610a6b575050600090815260046020526040902054600160e01b161590565b6000611b0c82610ec3565b9050336001600160a01b03821614611b5e57611b288133610903565b611b5e576040517fcfb3b94200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600082815260066020526040808220805473ffffffffffffffffffffffffffffffffffffffff19166001600160a01b0387811691821790925591518593918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a4505050565b60008180600111611c1757600054811015611c1757600081815260046020526040902054600160e01b8116611c15575b8061194b575060001901600081815260046020526040902054611bf7565b505b6040517fdf2d9b4200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6008546001600160a01b031633146110c15760405162461bcd60e51b815260206004820181905260248201527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e65726044820152606401610bc5565b60005481611cdd576040517fb562e8dd00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6001600160a01b03831660008181526005602090815260408083208054680100000000000000018802019055848352600490915281206001851460e11b4260a01b178317905582840190839083907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef8180a4600183015b818114611d8c57808360007fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a4600101611d54565b5081611dc4576040517f2e07630000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b60005550505050565b600880546001600160a01b0383811673ffffffffffffffffffffffffffffffffffffffff19831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b3360008181526007602090815260408083206001600160a01b03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b604051630a85bd0160e11b81526000906001600160a01b0385169063150b7a0290611ecd9033908990889088906004016124e4565b602060405180830381600087803b158015611ee757600080fd5b505af1925050508015611f17575060408051601f3d908101601f19168201909252611f1491810190612352565b60015b611f72573d808015611f45576040519150601f19603f3d011682016040523d82523d6000602084013e611f4a565b606091505b508051611f6a576040516368d2bf6b60e11b815260040160405180910390fd5b805181602001fd5b6001600160e01b031916630a85bd0160e11b149050949350505050565b6060600e8054610a80906125ef565b600081815b8451811015611fe357611fcf82868381518110611fc257611fc261265b565b6020026020010151611feb565b915080611fdb8161262a565b915050611fa3565b509392505050565b60008183106120075760008281526020849052604090206109cd565b60008381526020839052604090206109cd565b828054612026906125ef565b90600052602060002090601f016020900481019282612048576000855561208e565b82601f106120615782800160ff1982351617855561208e565b8280016001018555821561208e579182015b8281111561208e578235825591602001919060010190612073565b5061209a92915061209e565b5090565b5b8082111561209a576000815560010161209f565b80356001600160a01b03811681146120ca57600080fd5b919050565b600082601f8301126120e057600080fd5b8135602067ffffffffffffffff8211156120fc576120fc612671565b8160051b61210b828201612533565b83815282810190868401838801850189101561212657600080fd5b600093505b8584101561214957803583526001939093019291840191840161212b565b50979650505050505050565b60006020828403121561216757600080fd5b6109cd826120b3565b6000806040838503121561218357600080fd5b61218c836120b3565b915061219a602084016120b3565b90509250929050565b6000806000606084860312156121b857600080fd5b6121c1846120b3565b92506121cf602085016120b3565b9150604084013590509250925092565b600080600080608085870312156121f557600080fd5b6121fe856120b3565b935061220c602086016120b3565b925060408501359150606085013567ffffffffffffffff81111561222f57600080fd5b8501601f8101871361224057600080fd5b803561225361224e82612564565b612533565b81815288602083850101111561226857600080fd5b8160208401602083013760006020838301015280935050505092959194509250565b6000806040838503121561229d57600080fd5b6122a6836120b3565b9150602083013580151581146122bb57600080fd5b809150509250929050565b600080604083850312156122d957600080fd5b6122e2836120b3565b946020939093013593505050565b6000806040838503121561230357600080fd5b823567ffffffffffffffff81111561231a57600080fd5b612326858286016120cf565b95602094909401359450505050565b60006020828403121561234757600080fd5b81356109cd81612687565b60006020828403121561236457600080fd5b81516109cd81612687565b6000806020838503121561238257600080fd5b823567ffffffffffffffff8082111561239a57600080fd5b818501915085601f8301126123ae57600080fd5b8135818111156123bd57600080fd5b8660208285010111156123cf57600080fd5b60209290920196919550909350505050565b6000602082840312156123f357600080fd5b815167ffffffffffffffff81111561240a57600080fd5b8201601f8101841361241b57600080fd5b805161242961224e82612564565b81815285602083850101111561243e57600080fd5b61244f8260208301602086016125c3565b95945050505050565b60006020828403121561246a57600080fd5b5035919050565b6000806040838503121561248457600080fd5b82359150602083013567ffffffffffffffff8111156124a257600080fd5b6124ae858286016120cf565b9150509250929050565b600081518084526124d08160208601602086016125c3565b601f01601f19169290920160200192915050565b60006001600160a01b0380871683528086166020840152508360408301526080606083015261251660808301846124b8565b9695505050505050565b6020815260006109cd60208301846124b8565b604051601f8201601f1916810167ffffffffffffffff8111828210171561255c5761255c612671565b604052919050565b600067ffffffffffffffff82111561257e5761257e612671565b50601f01601f191660200190565b6000821982111561259f5761259f612645565b500190565b60008160001904831182151516156125be576125be612645565b500290565b60005b838110156125de5781810151838201526020016125c6565b838111156117fe5750506000910152565b600181811c9082168061260357607f821691505b6020821081141561262457634e487b7160e01b600052602260045260246000fd5b50919050565b600060001982141561263e5761263e612645565b5060010190565b634e487b7160e01b600052601160045260246000fd5b634e487b7160e01b600052603260045260246000fd5b634e487b7160e01b600052604160045260246000fd5b6001600160e01b031981168114610e3e57600080fdfea2646970667358221220cc6bfbbdb2da0fee5d750955ee7def5de066ffed927e9e3fc97df3a29cf8458c64736f6c63430008070033

Constructor Arguments (ABI-Encoded and is the last bytes of the Contract Creation Code above)

000000000000000000000000000000000000000000000000000000000000002000000000000000000000000000000000000000000000000000000000000000094d4554412d44494f730000000000000000000000000000000000000000000000

-----Decoded View---------------
Arg [0] : _baseTokenUri (string): META-DIOs

-----Encoded View---------------
3 Constructor Arguments found :
Arg [0] : 0000000000000000000000000000000000000000000000000000000000000020
Arg [1] : 0000000000000000000000000000000000000000000000000000000000000009
Arg [2] : 4d4554412d44494f730000000000000000000000000000000000000000000000


Deployed Bytecode Sourcemap

68534:6945:0:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;73001:184;;;;;;;;;;-1:-1:-1;73001:184:0;;;;;:::i;:::-;;:::i;:::-;;;7622:14:1;;7615:22;7597:41;;7585:2;7570:18;73001:184:0;;;;;;;;34466:639;;;;;;;;;;-1:-1:-1;34466:639:0;;;;;:::i;:::-;;:::i;35368:100::-;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;41859:218::-;;;;;;;;;;-1:-1:-1;41859:218:0;;;;;:::i;:::-;;:::i;:::-;;;-1:-1:-1;;;;;6874:55:1;;;6856:74;;6844:2;6829:18;41859:218:0;6710:226:1;74009:243:0;;;;;;:::i;:::-;;:::i;:::-;;69197:48;;;;;;;;;;;;69235:10;69197:48;;;;;7795:25:1;;;7783:2;7768:18;69197:48:0;7649:177:1;68965:37:0;;;;;;;;;;;;69001:1;68965:37;;31119:323;;;;;;;;;;-1:-1:-1;75267:1:0;31393:12;31180:7;31377:13;:28;-1:-1:-1;;31377:46:0;31119:323;;45498:2825;;;;;;:::i;:::-;;:::i;69127:45::-;;;;;;;;;;;;69170:2;69127:45;;69252:49;;;;;;;;;;;;69291:10;69252:49;;68919:39;;;;;;;;;;;;68957:1;68919:39;;73601:104;;;;;;;;;;-1:-1:-1;73601:104:0;;;;;:::i;:::-;;:::i;68644:52::-;;;;;;;;;;;;68686:10;68644:52;;68596:41;;;;;;;;;;;;68633:4;68596:41;;73193:184;;;;;;;;;;-1:-1:-1;73193:184:0;;;;;:::i;:::-;;:::i;75284:192::-;;;:::i;69346:27::-;;;;;;;;;;;;;;;;48419:193;;;;;;:::i;:::-;;:::i;73422:171::-;;;;;;;;;;-1:-1:-1;73422:171:0;;;;;:::i;:::-;;:::i;69576:46::-;;;;;;;;;;-1:-1:-1;69576:46:0;;;;;:::i;:::-;;;;;;;;;;;;;;36761:152;;;;;;;;;;-1:-1:-1;36761:152:0;;;;;:::i;:::-;;:::i;72309:492::-;;;;;;:::i;:::-;;:::i;69906:98::-;;;;;;;;;;;;;;;;68703:54;;;;;;;;;;;;68747:10;68703:54;;32303:233;;;;;;;;;;-1:-1:-1;32303:233:0;;;;;:::i;:::-;;:::i;15283:103::-;;;;;;;;;;;;;:::i;69011:51::-;;;;;;;;;;;;69058:4;69011:51;;73824:177;;;;;;;;;;-1:-1:-1;73824:177:0;;;;;:::i;:::-;;:::i;69801:98::-;;;;;;;;;;;;;;;;70972:707;;;;;;:::i;:::-;;:::i;14635:87::-;;;;;;;;;;-1:-1:-1;14708:6:0;;-1:-1:-1;;;;;14708:6:0;14635:87;;71689:612;;;;;;;;;;-1:-1:-1;71689:612:0;;;;;:::i;:::-;;:::i;35544:104::-;;;;;;;;;;;;;:::i;70264:700::-;;;;;;:::i;:::-;;:::i;69737:55::-;;;;;;;;;;-1:-1:-1;69737:55:0;;;;;:::i;:::-;;;;;;;;;;;;;;;;74260:300;;;;;;;;;;-1:-1:-1;74260:300:0;;;;;:::i;:::-;;:::i;68817:43::-;;;;;;;;;;;;68859:1;68817:43;;69483:30;;;;;;;;;;-1:-1:-1;69483:30:0;;;;-1:-1:-1;;;;;69483:30:0;;;68764:46;;;;;;;;;;;;68800:10;68764:46;;69312:27;;;;;;;;;;;;;;;;49210:407;;;;;;:::i;:::-;;:::i;69414:27::-;;;;;;;;;;;;;;;;69629:46;;;;;;;;;;-1:-1:-1;69629:46:0;;;;;:::i;:::-;;;;;;;;;;;;;;74681:494;;;;;;;;;;-1:-1:-1;74681:494:0;;;;;:::i;:::-;;:::i;69450:26::-;;;;;;;;;;;;;:::i;69523:46::-;;;;;;;;;;-1:-1:-1;69523:46:0;;;;;:::i;:::-;;;;;;;;;;;;;;70011:98;;;;;;;;;;;;;;;;69069:51;;;;;;;;;;;;69118:2;69069:51;;69380:27;;;;;;;;;;;;;;;;42808:164;;;;;;;;;;-1:-1:-1;42808:164:0;;;;;:::i;:::-;-1:-1:-1;;;;;42929:25:0;;;42905:4;42929:25;;;:18;:25;;;;;;;;:35;;;;;;;;;;;;;;;42808:164;72809:184;;;;;;;;;;-1:-1:-1;72809:184:0;;;;;:::i;:::-;;:::i;15541:201::-;;;;;;;;;;-1:-1:-1;15541:201:0;;;;;:::i;:::-;;:::i;73713:103::-;;;;;;;;;;-1:-1:-1;73713:103:0;;;;;:::i;:::-;;:::i;69682:46::-;;;;;;;;;;-1:-1:-1;69682:46:0;;;;;:::i;:::-;;;;;;;;;;;;;;73001:184;73110:4;73139:38;73158:5;73165;;73172:4;73139:18;:38::i;:::-;73132:45;73001:184;-1:-1:-1;;;73001:184:0:o;34466:639::-;34551:4;34875:25;-1:-1:-1;;;;;;34875:25:0;;;;:102;;-1:-1:-1;34952:25:0;-1:-1:-1;;;;;;34952:25:0;;;34875:102;:179;;;-1:-1:-1;35029:25:0;-1:-1:-1;;;;;;35029:25:0;;;34875:179;34855:199;34466:639;-1:-1:-1;;34466:639:0:o;35368:100::-;35422:13;35455:5;35448:12;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;35368:100;:::o;41859:218::-;41935:7;41960:16;41968:7;41960;:16::i;:::-;41955:64;;41985:34;;;;;;;;;;;;;;41955:64;-1:-1:-1;42039:24:0;;;;:15;:24;;;;;:30;-1:-1:-1;;;;;42039:30:0;;41859:218::o;74009:243::-;-1:-1:-1;;;;;74148:27:0;;;;;;:23;:27;;;;;;;;74147:28;74139:68;;;;-1:-1:-1;;;74139:68:0;;11143:2:1;74139:68:0;;;11125:21:1;11182:2;11162:18;;;11155:30;11221:29;11201:18;;;11194:57;11268:18;;74139:68:0;;;;;;;;;74218:26;74232:2;74236:7;74218:13;:26::i;:::-;74009:243;;:::o;45498:2825::-;45640:27;45670;45689:7;45670:18;:27::i;:::-;45640:57;;45755:4;-1:-1:-1;;;;;45714:45:0;45730:19;-1:-1:-1;;;;;45714:45:0;;45710:86;;45768:28;;;;;;;;;;;;;;45710:86;45810:27;44606:24;;;:15;:24;;;;;44834:26;;65625:10;44231:30;;;-1:-1:-1;;;;;43924:28:0;;44209:20;;;44206:56;45996:180;;46089:43;46106:4;65625:10;42808:164;:::i;46089:43::-;46084:92;;46141:35;;;;;;;;;;;;;;46084:92;-1:-1:-1;;;;;46193:16:0;;46189:52;;46218:23;;;;;;;;;;;;;;46189:52;46390:15;46387:160;;;46530:1;46509:19;46502:30;46387:160;-1:-1:-1;;;;;46927:24:0;;;;;;;:18;:24;;;;;;46925:26;;-1:-1:-1;;46925:26:0;;;46996:22;;;;;;;;;46994:24;;-1:-1:-1;46994:24:0;;;40150:11;40125:23;40121:41;40108:63;-1:-1:-1;;;40108:63:0;47289:26;;;;:17;:26;;;;;:175;-1:-1:-1;;;47584:47:0;;47580:627;;47689:1;47679:11;;47657:19;47812:30;;;:17;:30;;;;;;47808:384;;47950:13;;47935:11;:28;47931:242;;48097:30;;;;:17;:30;;;;;:52;;;47931:242;47638:569;47580:627;48254:7;48250:2;-1:-1:-1;;;;;48235:27:0;48244:4;-1:-1:-1;;;;;48235:27:0;;;;;;;;;;;45629:2694;;;45498:2825;;;:::o;73601:104::-;14521:13;:11;:13::i;:::-;73678:19:::1;:12;73693:4:::0;;73678:19:::1;:::i;:::-;;73601:104:::0;;:::o;73193:184::-;73302:4;73331:38;73350:5;73357;;73364:4;73331:18;:38::i;75284:192::-;14521:13;:11;:13::i;:::-;75359:82:::1;::::0;75341:12:::1;::::0;75367:10:::1;::::0;75405:21:::1;::::0;75341:12;75359:82;75341:12;75359:82;75405:21;75367:10;75359:82:::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;75340:101;;;75460:7;75452:16;;;::::0;::::1;;75329:147;75284:192::o:0;48419:193::-;48565:39;48582:4;48588:2;48592:7;48565:39;;;;;;;;;;;;:16;:39::i;73422:171::-;14521:13;:11;:13::i;:::-;75267:1;31393:12;31180:7;31377:13;68633:4:::1;::::0;73523:6;;31377:28;-1:-1:-1;;31377:46:0;73507:22:::1;;;;:::i;:::-;:36;;73499:58;;;::::0;-1:-1:-1;;;73499:58:0;;11834:2:1;73499:58:0::1;::::0;::::1;11816:21:1::0;11873:1;11853:18;;;11846:29;-1:-1:-1;;;11891:18:1;;;11884:39;11940:18;;73499:58:0::1;11632:332:1::0;73499:58:0::1;73568:17;73574:2;73578:6;73568:5;:17::i;36761:152::-:0;36833:7;36876:27;36895:7;36876:18;:27::i;72309:492::-;75267:1;31393:12;31180:7;31377:13;68633:4;;72395:6;;31377:28;-1:-1:-1;;31377:46:0;72379:22;;;;:::i;:::-;:36;;72371:58;;;;-1:-1:-1;;;72371:58:0;;11834:2:1;72371:58:0;;;11816:21:1;11873:1;11853:18;;;11846:29;-1:-1:-1;;;11891:18:1;;;11884:39;11940:18;;72371:58:0;11632:332:1;72371:58:0;72460:10;72448:23;;;;:11;:23;;;;;;69001:1;;72448:32;;72474:6;;72448:32;:::i;:::-;:45;;72440:72;;;;-1:-1:-1;;;72440:72:0;;9342:2:1;72440:72:0;;;9324:21:1;9381:2;9361:18;;;9354:30;-1:-1:-1;;;9400:18:1;;;9393:44;9454:18;;72440:72:0;9140:338:1;72440:72:0;72544:17;68800:10;72544:6;:17;:::i;:::-;72531:9;:30;;72523:51;;;;-1:-1:-1;;;72523:51:0;;10462:2:1;72523:51:0;;;10444:21:1;10501:1;10481:18;;;10474:29;-1:-1:-1;;;10519:18:1;;;10512:39;10568:18;;72523:51:0;10260:332:1;72523:51:0;69291:10;72593:15;:31;;72585:59;;;;-1:-1:-1;;;72585:59:0;;10799:2:1;72585:59:0;;;10781:21:1;10838:2;10818:18;;;10811:30;10877:17;10857:18;;;10850:45;10912:18;;72585:59:0;10597:339:1;72585:59:0;72692:10;72680:23;;;;:11;:23;;;;;:33;;;;;;72728:8;:18;;;;;;72768:25;;72707:6;72768:5;:25::i;32303:233::-;32375:7;-1:-1:-1;;;;;32399:19:0;;32395:60;;32427:28;;;;;;;;;;;;;;32395:60;-1:-1:-1;;;;;;32473:25:0;;;;;:18;:25;;;;;;26462:13;32473:55;;32303:233::o;15283:103::-;14521:13;:11;:13::i;:::-;15348:30:::1;15375:1;15348:18;:30::i;:::-;15283:103::o:0;73824:177::-;14521:13;:11;:13::i;:::-;-1:-1:-1;;;;;73947:31:0;;;::::1;;::::0;;;:23:::1;:31;::::0;;;;:46;;-1:-1:-1;;73947:46:0::1;::::0;::::1;;::::0;;;::::1;::::0;;73824:177::o;70972:707::-;71104:28;;-1:-1:-1;;71121:10:0;6415:2:1;6411:15;6407:53;71104:28:0;;;6395:66:1;71073:61:0;;71087:5;;6477:12:1;;71104:28:0;;;;;;;;;;;;71094:39;;;;;;71073:13;:61::i;:::-;71065:80;;;;-1:-1:-1;;;71065:80:0;;8257:2:1;71065:80:0;;;8239:21:1;8296:1;8276:18;;;8269:29;8334:9;8314:18;;;8307:37;8361:18;;71065:80:0;8055:330:1;71065:80:0;71177:25;68747:10;71177:6;:25;:::i;:::-;71164:9;:38;;71156:59;;;;-1:-1:-1;;;71156:59:0;;10462:2:1;71156:59:0;;;10444:21:1;10501:1;10481:18;;;10474:29;-1:-1:-1;;;10519:18:1;;;10512:39;10568:18;;71156:59:0;10260:332:1;71156:59:0;71246:10;71234:23;;;;:11;:23;;;;;;68911:1;;71234:32;;71260:6;;71234:32;:::i;:::-;:53;;71226:80;;;;-1:-1:-1;;;71226:80:0;;9342:2:1;71226:80:0;;;9324:21:1;9381:2;9361:18;;;9354:30;-1:-1:-1;;;9400:18:1;;;9393:44;9454:18;;71226:80:0;9140:338:1;71226:80:0;69118:2;71336:6;71325:8;;:17;;;;:::i;:::-;:43;;71317:65;;;;-1:-1:-1;;;71317:65:0;;11834:2:1;71317:65:0;;;11816:21:1;11873:1;11853:18;;;11846:29;-1:-1:-1;;;11891:18:1;;;11884:39;11940:18;;71317:65:0;11632:332:1;71317:65:0;69235:10;71401:15;:30;;71393:57;;;;-1:-1:-1;;;71393:57:0;;8592:2:1;71393:57:0;;;8574:21:1;8631:2;8611:18;;;8604:30;-1:-1:-1;;;8650:18:1;;;8643:44;8704:18;;71393:57:0;8390:338:1;71393:57:0;71485:15;69291:10;71469:31;;71461:59;;;;-1:-1:-1;;;71461:59:0;;8592:2:1;71461:59:0;;;8574:21:1;8631:2;8611:18;;;8604:30;-1:-1:-1;;;8650:18:1;;;8643:44;8704:18;;71461:59:0;8390:338:1;71461:59:0;71568:10;71556:23;;;;:11;:23;;;;;:33;;;;;;71604:8;:18;;;;;;71646:25;;71583:6;71646:5;:25::i;71689:612::-;71808:28;;-1:-1:-1;;71825:10:0;6415:2:1;6411:15;6407:53;71808:28:0;;;6395:66:1;71777:61:0;;71791:5;;6477:12:1;;71808:28:0;;;;;;;;;;;;71798:39;;;;;;71777:13;:61::i;:::-;71769:80;;;;-1:-1:-1;;;71769:80:0;;12171:2:1;71769:80:0;;;12153:21:1;12210:1;12190:18;;;12183:29;12248:9;12228:18;;;12221:37;12275:18;;71769:80:0;11969:330:1;71769:80:0;69170:2;71879:6;71868:8;;:17;;;;:::i;:::-;:37;;71860:59;;;;-1:-1:-1;;;71860:59:0;;11834:2:1;71860:59:0;;;11816:21:1;11873:1;11853:18;;;11846:29;-1:-1:-1;;;11891:18:1;;;11884:39;11940:18;;71860:59:0;11632:332:1;71860:59:0;71950:10;71938:23;;;;:11;:23;;;;;;68957:1;;71938:32;;71964:6;;71938:32;:::i;:::-;:47;;71930:74;;;;-1:-1:-1;;;71930:74:0;;9342:2:1;71930:74:0;;;9324:21:1;9381:2;9361:18;;;9354:30;-1:-1:-1;;;9400:18:1;;;9393:44;9454:18;;71930:74:0;9140:338:1;71930:74:0;69235:10;72023:15;:30;;72015:57;;;;-1:-1:-1;;;72015:57:0;;8592:2:1;72015:57:0;;;8574:21:1;8631:2;8611:18;;;8604:30;-1:-1:-1;;;8650:18:1;;;8643:44;8704:18;;72015:57:0;8390:338:1;72015:57:0;72107:15;69291:10;72091:31;;72083:59;;;;-1:-1:-1;;;72083:59:0;;8592:2:1;72083:59:0;;;8574:21:1;8631:2;8611:18;;;8604:30;-1:-1:-1;;;8650:18:1;;;8643:44;8704:18;;72083:59:0;8390:338:1;72083:59:0;72190:10;72178:23;;;;:11;:23;;;;;:33;;;;;;72226:8;:18;;;;;;72268:25;;72205:6;72268:5;:25::i;35544:104::-;35600:13;35633:7;35626:14;;;;;:::i;70264:700::-;70394:28;;-1:-1:-1;;70411:10:0;6415:2:1;6411:15;6407:53;70394:28:0;;;6395:66:1;70363:61:0;;70377:5;;6477:12:1;;70394:28:0;;;;;;;;;;;;70384:39;;;;;;70363:13;:61::i;:::-;70355:80;;;;-1:-1:-1;;;70355:80:0;;11499:2:1;70355:80:0;;;11481:21:1;11538:1;11518:18;;;11511:29;11576:9;11556:18;;;11549:37;11603:18;;70355:80:0;11297:330:1;70355:80:0;70467:23;68686:10;70467:6;:23;:::i;:::-;70454:9;:36;;70446:57;;;;-1:-1:-1;;;70446:57:0;;10462:2:1;70446:57:0;;;10444:21:1;10501:1;10481:18;;;10474:29;-1:-1:-1;;;10519:18:1;;;10512:39;10568:18;;70446:57:0;10260:332:1;70446:57:0;70534:10;70522:23;;;;:11;:23;;;;;;68859:1;;70522:32;;70548:6;;70522:32;:::i;:::-;:51;;70514:78;;;;-1:-1:-1;;;70514:78:0;;9342:2:1;70514:78:0;;;9324:21:1;9381:2;9361:18;;;9354:30;-1:-1:-1;;;9400:18:1;;;9393:44;9454:18;;70514:78:0;9140:338:1;70514:78:0;69058:4;70622:6;70611:8;;:17;;;;:::i;:::-;:41;;70603:63;;;;-1:-1:-1;;;70603:63:0;;11834:2:1;70603:63:0;;;11816:21:1;11873:1;11853:18;;;11846:29;-1:-1:-1;;;11891:18:1;;;11884:39;11940:18;;70603:63:0;11632:332:1;70603:63:0;69235:10;70685:15;:30;;70677:58;;;;-1:-1:-1;;;70677:58:0;;8592:2:1;70677:58:0;;;8574:21:1;8631:2;8611:18;;;8604:30;-1:-1:-1;;;8650:18:1;;;8643:44;8704:18;;70677:58:0;8390:338:1;70677:58:0;70770:15;69291:10;70754:31;;70746:59;;;;-1:-1:-1;;;70746:59:0;;8592:2:1;70746:59:0;;;8574:21:1;8631:2;8611:18;;;8604:30;-1:-1:-1;;;8650:18:1;;;8643:44;8704:18;;70746:59:0;8390:338:1;70746:59:0;70853:10;70841:23;;;;:11;:23;;;;;:33;;;;;;70889:8;:18;;;;;;70931:25;;70868:6;70931:5;:25::i;74260:300::-;-1:-1:-1;;;;;74410:33:0;;;;;;:23;:33;;;;;;;;74409:34;74387:111;;;;-1:-1:-1;;;74387:111:0;;11143:2:1;74387:111:0;;;11125:21:1;11182:2;11162:18;;;11155:30;11221:29;11201:18;;;11194:57;11268:18;;74387:111:0;10941:351:1;74387:111:0;74509:43;74533:8;74543;74509:23;:43::i;49210:407::-;49385:31;49398:4;49404:2;49408:7;49385:12;:31::i;:::-;-1:-1:-1;;;;;49431:14:0;;;:19;49427:183;;49470:56;49501:4;49507:2;49511:7;49520:5;49470:30;:56::i;:::-;49465:145;;49554:40;;-1:-1:-1;;;49554:40:0;;;;;;;;;;;49465:145;49210:407;;;;:::o;74681:494::-;74782:13;74835:16;74843:7;74835;:16::i;:::-;74813:113;;;;-1:-1:-1;;;74813:113:0;;10046:2:1;74813:113:0;;;10028:21:1;10085:2;10065:18;;;10058:30;10124:34;10104:18;;;10097:62;10195:17;10175:18;;;10168:45;10230:19;;74813:113:0;9844:411:1;74813:113:0;74937:21;74961:10;:8;:10::i;:::-;75022:15;;75008:51;;;;;;;;7795:25:1;;;74937:34:0;;-1:-1:-1;74982:23:0;;-1:-1:-1;;;;;75022:15:0;;;;75008:42;;7768:18:1;;75008:51:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;75008:51:0;;;;;;;;;;;;:::i;:::-;74982:77;;75096:7;75090:21;75115:1;75090:26;;:77;;;;;;;;;;;;;;;;;75136:9;75090:77;75070:97;74681:494;-1:-1:-1;;;;74681:494:0:o;69450:26::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;72809:184::-;72918:4;72947:38;72966:5;72973;;72980:4;72947:18;:38::i;15541:201::-;14521:13;:11;:13::i;:::-;-1:-1:-1;;;;;15630:22:0;::::1;15622:73;;;::::0;-1:-1:-1;;;15622:73:0;;8935:2:1;15622:73:0::1;::::0;::::1;8917:21:1::0;8974:2;8954:18;;;8947:30;9013:34;8993:18;;;8986:62;9084:8;9064:18;;;9057:36;9110:19;;15622:73:0::1;8733:402:1::0;15622:73:0::1;15706:28;15725:8;15706:18;:28::i;73713:103::-:0;14521:13;:11;:13::i;:::-;73782:15:::1;:26:::0;;-1:-1:-1;;73782:26:0::1;-1:-1:-1::0;;;;;73782:26:0;;;::::1;::::0;;;::::1;::::0;;73713:103::o;1222:190::-;1347:4;1400;1371:25;1384:5;1391:4;1371:12;:25::i;:::-;:33;;1222:190;-1:-1:-1;;;;1222:190:0:o;43230:282::-;43295:4;43351:7;75267:1;43332:26;;:66;;;;;43385:13;;43375:7;:23;43332:66;:153;;;;-1:-1:-1;;43436:26:0;;;;:17;:26;;;;;;-1:-1:-1;;;43436:44:0;:49;;43230:282::o;41292:408::-;41381:13;41397:16;41405:7;41397;:16::i;:::-;41381:32;-1:-1:-1;65625:10:0;-1:-1:-1;;;;;41430:28:0;;;41426:175;;41478:44;41495:5;65625:10;42808:164;:::i;41478:44::-;41473:128;;41550:35;;;;;;;;;;;;;;41473:128;41613:24;;;;:15;:24;;;;;;:35;;-1:-1:-1;;41613:35:0;-1:-1:-1;;;;;41613:35:0;;;;;;;;;41664:28;;41613:24;;41664:28;;;;;;;41370:330;41292:408;;:::o;37916:1275::-;37983:7;38018;;75267:1;38067:23;38063:1061;;38120:13;;38113:4;:20;38109:1015;;;38158:14;38175:23;;;:17;:23;;;;;;-1:-1:-1;;;38264:24:0;;38260:845;;38929:113;38936:11;38929:113;;-1:-1:-1;;;39007:6:0;38989:25;;;;:17;:25;;;;;;38929:113;;38260:845;38135:989;38109:1015;39152:31;;;;;;;;;;;;;;14800:132;14708:6;;-1:-1:-1;;;;;14708:6:0;65625:10;14864:23;14856:68;;;;-1:-1:-1;;;14856:68:0;;9685:2:1;14856:68:0;;;9667:21:1;;;9704:18;;;9697:30;9763:34;9743:18;;;9736:62;9815:18;;14856:68:0;9483:356:1;52879:2966:0;52952:20;52975:13;53003;52999:44;;53025:18;;;;;;;;;;;;;;52999:44;-1:-1:-1;;;;;53531:22:0;;;;;;:18;:22;;;;26600:2;53531:22;;;:71;;53569:32;53557:45;;53531:71;;;53845:31;;;:17;:31;;;;;-1:-1:-1;40581:15:0;;40555:24;40551:46;40150:11;40125:23;40121:41;40118:52;40108:63;;53845:173;;54080:23;;;;53845:31;;53531:22;;54845:25;53531:22;;54698:335;55359:1;55345:12;55341:20;55299:346;55400:3;55391:7;55388:16;55299:346;;55618:7;55608:8;55605:1;55578:25;55575:1;55572;55567:59;55453:1;55440:15;55299:346;;;-1:-1:-1;55678:13:0;55674:45;;55700:19;;;;;;;;;;;;;;55674:45;55736:13;:19;-1:-1:-1;73678:19:0::1;73601:104:::0;;:::o;15902:191::-;15995:6;;;-1:-1:-1;;;;;16012:17:0;;;-1:-1:-1;;16012:17:0;;;;;;;16045:40;;15995:6;;;16012:17;15995:6;;16045:40;;15976:16;;16045:40;15965:128;15902:191;:::o;42417:234::-;65625:10;42512:39;;;;:18;:39;;;;;;;;-1:-1:-1;;;;;42512:49:0;;;;;;;;;;;;:60;;-1:-1:-1;;42512:60:0;;;;;;;;;;42588:55;;7597:41:1;;;42512:49:0;;65625:10;42588:55;;7570:18:1;42588:55:0;;;;;;;42417:234;;:::o;51701:716::-;51885:88;;-1:-1:-1;;;51885:88:0;;51864:4;;-1:-1:-1;;;;;51885:45:0;;;;;:88;;65625:10;;51952:4;;51958:7;;51967:5;;51885:88;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;51885:88:0;;;;;;;;-1:-1:-1;;51885:88:0;;;;;;;;;;;;:::i;:::-;;;51881:529;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;52168:13:0;;52164:235;;52214:40;;-1:-1:-1;;;52214:40:0;;;;;;;;;;;52164:235;52357:6;52351:13;52342:6;52338:2;52334:15;52327:38;51881:529;-1:-1:-1;;;;;;52044:64:0;-1:-1:-1;;;52044:64:0;;-1:-1:-1;51701:716:0;;;;;;:::o;74568:105::-;74620:13;74653:12;74646:19;;;;;:::i;2089:296::-;2172:7;2215:4;2172:7;2230:118;2254:5;:12;2250:1;:16;2230:118;;;2303:33;2313:12;2327:5;2333:1;2327:8;;;;;;;;:::i;:::-;;;;;;;2303:9;:33::i;:::-;2288:48;-1:-1:-1;2268:3:0;;;;:::i;:::-;;;;2230:118;;;-1:-1:-1;2365:12:0;2089:296;-1:-1:-1;;;2089:296:0:o;9129:149::-;9192:7;9223:1;9219;:5;:51;;9354:13;9448:15;;;9484:4;9477:15;;;9531:4;9515:21;;9219:51;;;9354:13;9448:15;;;9484:4;9477:15;;;9531:4;9515:21;;9227:20;9286:268;-1:-1:-1;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;:::o;:::-;;;;;;;;;;;;;;;14:196:1;82:20;;-1:-1:-1;;;;;131:54:1;;121:65;;111:93;;200:1;197;190:12;111:93;14:196;;;:::o;215:723::-;269:5;322:3;315:4;307:6;303:17;299:27;289:55;;340:1;337;330:12;289:55;376:6;363:20;402:4;425:18;421:2;418:26;415:52;;;447:18;;:::i;:::-;493:2;490:1;486:10;516:28;540:2;536;532:11;516:28;:::i;:::-;578:15;;;609:12;;;;641:15;;;675;;;671:24;;668:33;-1:-1:-1;665:53:1;;;714:1;711;704:12;665:53;736:1;727:10;;746:163;760:2;757:1;754:9;746:163;;;817:17;;805:30;;778:1;771:9;;;;;855:12;;;;887;;746:163;;;-1:-1:-1;927:5:1;215:723;-1:-1:-1;;;;;;;215:723:1:o;943:186::-;1002:6;1055:2;1043:9;1034:7;1030:23;1026:32;1023:52;;;1071:1;1068;1061:12;1023:52;1094:29;1113:9;1094:29;:::i;1134:260::-;1202:6;1210;1263:2;1251:9;1242:7;1238:23;1234:32;1231:52;;;1279:1;1276;1269:12;1231:52;1302:29;1321:9;1302:29;:::i;:::-;1292:39;;1350:38;1384:2;1373:9;1369:18;1350:38;:::i;:::-;1340:48;;1134:260;;;;;:::o;1399:328::-;1476:6;1484;1492;1545:2;1533:9;1524:7;1520:23;1516:32;1513:52;;;1561:1;1558;1551:12;1513:52;1584:29;1603:9;1584:29;:::i;:::-;1574:39;;1632:38;1666:2;1655:9;1651:18;1632:38;:::i;:::-;1622:48;;1717:2;1706:9;1702:18;1689:32;1679:42;;1399:328;;;;;:::o;1732:888::-;1827:6;1835;1843;1851;1904:3;1892:9;1883:7;1879:23;1875:33;1872:53;;;1921:1;1918;1911:12;1872:53;1944:29;1963:9;1944:29;:::i;:::-;1934:39;;1992:38;2026:2;2015:9;2011:18;1992:38;:::i;:::-;1982:48;;2077:2;2066:9;2062:18;2049:32;2039:42;;2132:2;2121:9;2117:18;2104:32;2159:18;2151:6;2148:30;2145:50;;;2191:1;2188;2181:12;2145:50;2214:22;;2267:4;2259:13;;2255:27;-1:-1:-1;2245:55:1;;2296:1;2293;2286:12;2245:55;2332:2;2319:16;2357:48;2373:31;2401:2;2373:31;:::i;:::-;2357:48;:::i;:::-;2428:2;2421:5;2414:17;2468:7;2463:2;2458;2454;2450:11;2446:20;2443:33;2440:53;;;2489:1;2486;2479:12;2440:53;2544:2;2539;2535;2531:11;2526:2;2519:5;2515:14;2502:45;2588:1;2583:2;2578;2571:5;2567:14;2563:23;2556:34;2609:5;2599:15;;;;;1732:888;;;;;;;:::o;2625:347::-;2690:6;2698;2751:2;2739:9;2730:7;2726:23;2722:32;2719:52;;;2767:1;2764;2757:12;2719:52;2790:29;2809:9;2790:29;:::i;:::-;2780:39;;2869:2;2858:9;2854:18;2841:32;2916:5;2909:13;2902:21;2895:5;2892:32;2882:60;;2938:1;2935;2928:12;2882:60;2961:5;2951:15;;;2625:347;;;;;:::o;2977:254::-;3045:6;3053;3106:2;3094:9;3085:7;3081:23;3077:32;3074:52;;;3122:1;3119;3112:12;3074:52;3145:29;3164:9;3145:29;:::i;:::-;3135:39;3221:2;3206:18;;;;3193:32;;-1:-1:-1;;;2977:254:1:o;3236:416::-;3329:6;3337;3390:2;3378:9;3369:7;3365:23;3361:32;3358:52;;;3406:1;3403;3396:12;3358:52;3446:9;3433:23;3479:18;3471:6;3468:30;3465:50;;;3511:1;3508;3501:12;3465:50;3534:61;3587:7;3578:6;3567:9;3563:22;3534:61;:::i;:::-;3524:71;3642:2;3627:18;;;;3614:32;;-1:-1:-1;;;;3236:416:1:o;3657:245::-;3715:6;3768:2;3756:9;3747:7;3743:23;3739:32;3736:52;;;3784:1;3781;3774:12;3736:52;3823:9;3810:23;3842:30;3866:5;3842:30;:::i;3907:249::-;3976:6;4029:2;4017:9;4008:7;4004:23;4000:32;3997:52;;;4045:1;4042;4035:12;3997:52;4077:9;4071:16;4096:30;4120:5;4096:30;:::i;4161:592::-;4232:6;4240;4293:2;4281:9;4272:7;4268:23;4264:32;4261:52;;;4309:1;4306;4299:12;4261:52;4349:9;4336:23;4378:18;4419:2;4411:6;4408:14;4405:34;;;4435:1;4432;4425:12;4405:34;4473:6;4462:9;4458:22;4448:32;;4518:7;4511:4;4507:2;4503:13;4499:27;4489:55;;4540:1;4537;4530:12;4489:55;4580:2;4567:16;4606:2;4598:6;4595:14;4592:34;;;4622:1;4619;4612:12;4592:34;4667:7;4662:2;4653:6;4649:2;4645:15;4641:24;4638:37;4635:57;;;4688:1;4685;4678:12;4635:57;4719:2;4711:11;;;;;4741:6;;-1:-1:-1;4161:592:1;;-1:-1:-1;;;;4161:592:1:o;4758:635::-;4838:6;4891:2;4879:9;4870:7;4866:23;4862:32;4859:52;;;4907:1;4904;4897:12;4859:52;4940:9;4934:16;4973:18;4965:6;4962:30;4959:50;;;5005:1;5002;4995:12;4959:50;5028:22;;5081:4;5073:13;;5069:27;-1:-1:-1;5059:55:1;;5110:1;5107;5100:12;5059:55;5139:2;5133:9;5164:48;5180:31;5208:2;5180:31;:::i;5164:48::-;5235:2;5228:5;5221:17;5275:7;5270:2;5265;5261;5257:11;5253:20;5250:33;5247:53;;;5296:1;5293;5286:12;5247:53;5309:54;5360:2;5355;5348:5;5344:14;5339:2;5335;5331:11;5309:54;:::i;:::-;5382:5;4758:635;-1:-1:-1;;;;;4758:635:1:o;5398:180::-;5457:6;5510:2;5498:9;5489:7;5485:23;5481:32;5478:52;;;5526:1;5523;5516:12;5478:52;-1:-1:-1;5549:23:1;;5398:180;-1:-1:-1;5398:180:1:o;5583:416::-;5676:6;5684;5737:2;5725:9;5716:7;5712:23;5708:32;5705:52;;;5753:1;5750;5743:12;5705:52;5789:9;5776:23;5766:33;;5850:2;5839:9;5835:18;5822:32;5877:18;5869:6;5866:30;5863:50;;;5909:1;5906;5899:12;5863:50;5932:61;5985:7;5976:6;5965:9;5961:22;5932:61;:::i;:::-;5922:71;;;5583:416;;;;;:::o;6004:257::-;6045:3;6083:5;6077:12;6110:6;6105:3;6098:19;6126:63;6182:6;6175:4;6170:3;6166:14;6159:4;6152:5;6148:16;6126:63;:::i;:::-;6243:2;6222:15;-1:-1:-1;;6218:29:1;6209:39;;;;6250:4;6205:50;;6004:257;-1:-1:-1;;6004:257:1:o;6941:511::-;7135:4;-1:-1:-1;;;;;7245:2:1;7237:6;7233:15;7222:9;7215:34;7297:2;7289:6;7285:15;7280:2;7269:9;7265:18;7258:43;;7337:6;7332:2;7321:9;7317:18;7310:34;7380:3;7375:2;7364:9;7360:18;7353:31;7401:45;7441:3;7430:9;7426:19;7418:6;7401:45;:::i;:::-;7393:53;6941:511;-1:-1:-1;;;;;;6941:511:1:o;7831:219::-;7980:2;7969:9;7962:21;7943:4;8000:44;8040:2;8029:9;8025:18;8017:6;8000:44;:::i;12486:275::-;12557:2;12551:9;12622:2;12603:13;;-1:-1:-1;;12599:27:1;12587:40;;12657:18;12642:34;;12678:22;;;12639:62;12636:88;;;12704:18;;:::i;:::-;12740:2;12733:22;12486:275;;-1:-1:-1;12486:275:1:o;12766:186::-;12814:4;12847:18;12839:6;12836:30;12833:56;;;12869:18;;:::i;:::-;-1:-1:-1;12935:2:1;12914:15;-1:-1:-1;;12910:29:1;12941:4;12906:40;;12766:186::o;12957:128::-;12997:3;13028:1;13024:6;13021:1;13018:13;13015:39;;;13034:18;;:::i;:::-;-1:-1:-1;13070:9:1;;12957:128::o;13090:168::-;13130:7;13196:1;13192;13188:6;13184:14;13181:1;13178:21;13173:1;13166:9;13159:17;13155:45;13152:71;;;13203:18;;:::i;:::-;-1:-1:-1;13243:9:1;;13090:168::o;13263:258::-;13335:1;13345:113;13359:6;13356:1;13353:13;13345:113;;;13435:11;;;13429:18;13416:11;;;13409:39;13381:2;13374:10;13345:113;;;13476:6;13473:1;13470:13;13467:48;;;-1:-1:-1;;13511:1:1;13493:16;;13486:27;13263:258::o;13526:437::-;13605:1;13601:12;;;;13648;;;13669:61;;13723:4;13715:6;13711:17;13701:27;;13669:61;13776:2;13768:6;13765:14;13745:18;13742:38;13739:218;;;-1:-1:-1;;;13810:1:1;13803:88;13914:4;13911:1;13904:15;13942:4;13939:1;13932:15;13739:218;;13526:437;;;:::o;13968:135::-;14007:3;-1:-1:-1;;14028:17:1;;14025:43;;;14048:18;;:::i;:::-;-1:-1:-1;14095:1:1;14084:13;;13968:135::o;14108:184::-;-1:-1:-1;;;14157:1:1;14150:88;14257:4;14254:1;14247:15;14281:4;14278:1;14271:15;14297:184;-1:-1:-1;;;14346:1:1;14339:88;14446:4;14443:1;14436:15;14470:4;14467:1;14460:15;14486:184;-1:-1:-1;;;14535:1:1;14528:88;14635:4;14632:1;14625:15;14659:4;14656:1;14649:15;14675:177;-1:-1:-1;;;;;;14753:5:1;14749:78;14742:5;14739:89;14729:117;;14842:1;14839;14832:12

Swarm Source

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