ETH Price: $3,432.31 (-1.55%)

Token

Kanyudunks ($KNY)
 

Overview

Max Total Supply

87 $KNY

Holders

21

Market

Volume (24H)

N/A

Min Price (24H)

N/A

Max Price (24H)

N/A
Filtered by Token Holder
*0️⃣-3️⃣-0️⃣.eth
Balance
1 $KNY
0xbab6defc57704da6797ca735a89ef6614cae6d93
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:
Kanyudunks

Compiler Version
v0.8.19+commit.7dd6d404

Optimization Enabled:
Yes with 200 runs

Other Settings:
default evmVersion, MIT license

Contract Source Code (Solidity)

/**
 *Submitted for verification at Etherscan.io on 2023-03-19
*/

// SPDX-License-Identifier: MIT
// File: @openzeppelin/contracts/utils/cryptography/MerkleProof.sol


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

pragma solidity 0.8.19;

/**
 * @dev These functions deal with verification of Merkle Tree proofs.
 *
 * The proofs can be generated using the JavaScript library
 * https://github.com/miguelmota/merkletreejs[merkletreejs].
 * Note: the hashing algorithm should be keccak256 and pair sorting should be enabled.
 *
 * See `test/utils/cryptography/MerkleProof.test.js` for some examples.
 *
 * WARNING: You should avoid using leaf values that are 64 bytes long prior to
 * hashing, or use a hash function other than keccak256 for hashing leaves.
 * This is because the concatenation of a sorted pair of internal nodes in
 * the merkle tree could be reinterpreted as a leaf value.
 */
library MerkleProof {
    /**
     * @dev Returns true if a `leaf` can be proved to be a part of a Merkle tree
     * defined by `root`. For this, a `proof` must be provided, containing
     * sibling hashes on the branch from the leaf to the root of the tree. Each
     * pair of leaves and each pair of pre-images are assumed to be sorted.
     */
    function verify(
        bytes32[] memory proof,
        bytes32 root,
        bytes32 leaf
    ) internal pure returns (bool) {
        return processProof(proof, leaf) == root;
    }

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

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

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

    /**
     * @dev Returns true if the `leaves` can be proved to be a part of a Merkle tree defined by
     * `root`, according to `proof` and `proofFlags` as described in {processMultiProof}.
     *
     * _Available since v4.7._
     */
    function multiProofVerify(
        bytes32[] memory proof,
        bool[] memory proofFlags,
        bytes32 root,
        bytes32[] memory leaves
    ) internal pure returns (bool) {
        return processMultiProof(proof, proofFlags, leaves) == root;
    }

    /**
     * @dev Calldata version of {multiProofVerify}
     *
     * _Available since v4.7._
     */
    function multiProofVerifyCalldata(
        bytes32[] calldata proof,
        bool[] calldata proofFlags,
        bytes32 root,
        bytes32[] memory leaves
    ) internal pure returns (bool) {
        return processMultiProofCalldata(proof, proofFlags, leaves) == root;
    }

    /**
     * @dev Returns the root of a tree reconstructed from `leaves` and the sibling nodes in `proof`,
     * consuming from one or the other at each step according to the instructions given by
     * `proofFlags`.
     *
     * _Available since v4.7._
     */
    function processMultiProof(
        bytes32[] memory proof,
        bool[] memory proofFlags,
        bytes32[] memory leaves
    ) internal pure returns (bytes32 merkleRoot) {
        // This function rebuild the root hash by traversing the tree up from the leaves. The root is rebuilt by
        // consuming and producing values on a queue. The queue starts with the `leaves` array, then goes onto the
        // `hashes` array. At the end of the process, the last hash in the `hashes` array should contain the root of
        // the merkle tree.
        uint256 leavesLen = leaves.length;
        uint256 totalHashes = proofFlags.length;

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

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

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

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

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

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

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

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

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

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


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

pragma solidity 0.8.19;

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

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

    uint256 private _status;

    constructor() {
        _status = _NOT_ENTERED;
    }

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

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

        _;

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

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


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

pragma solidity 0.8.19;

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


/**
 * @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: contracts/SurgeCollection.sol


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

pragma solidity 0.8.19;




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

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

    // Base URI
    string internal _uri;

    // 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.selector);
        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.selector);

        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 _uri;
    }

    // =============================================================
    //                     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 Returns whether the ownership slot at `index` is initialized.
     * An uninitialized slot does not necessarily mean that the slot has no owner.
     */
    function _ownershipIsInitialized(uint256 index)
        internal
        view
        virtual
        returns (bool)
    {
        return _packedOwnerships[index] != 0;
    }

    /**
     * @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 packed)
    {
        if (_startTokenId() <= tokenId) {
            packed = _packedOwnerships[tokenId];
            // If the data at the starting slot does not exist, start the scan.
            if (packed == 0) {
                if (tokenId >= _currentIndex)
                    _revert(OwnerQueryForNonexistentToken.selector);
                // 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, `tokenId` will not underflow.
                //
                // We can directly compare the packed value.
                // If the address is zero, packed will be zero.
                for (;;) {
                    unchecked {
                        packed = _packedOwnerships[--tokenId];
                    }
                    if (packed == 0) continue;
                    if (packed & _BITMASK_BURNED == 0) return packed;
                    // Otherwise, the token is burned, and we must revert.
                    // This handles the case of batch burned tokens, where only the burned bit
                    // of the starting slot is set, and remaining slots are left uninitialized.
                    _revert(OwnerQueryForNonexistentToken.selector);
                }
            }
            // Otherwise, the data exists and we can skip the scan.
            // This is possible because we have already achieved the target condition.
            // This saves 2143 gas on transfers of initialized tokens.
            // If the token is not burned, return `packed`. Otherwise, revert.
            if (packed & _BITMASK_BURNED == 0) return packed;
        }
        _revert(OwnerQueryForNonexistentToken.selector);
    }

    /**
     * @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. See {ERC721A-_approve}.
     *
     * Requirements:
     *
     * - The caller must own the token or be an approved operator.
     */
    function approve(address to, uint256 tokenId)
        public
        payable
        virtual
        override
    {
        _approve(to, tokenId, true);
    }

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

        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 result)
    {
        if (_startTokenId() <= tokenId) {
            if (tokenId < _currentIndex) {
                uint256 packed;
                while ((packed = _packedOwnerships[tokenId]) == 0) --tokenId;
                result = packed & _BITMASK_BURNED == 0;
            }
        }
    }

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

        // Mask `from` to the lower 160 bits, in case the upper bits somehow aren't clean.
        from = address(uint160(uint256(uint160(from)) & _BITMASK_ADDRESS));

        if (address(uint160(prevOwnershipPacked)) != from)
            _revert(TransferFromIncorrectOwner.selector);

        (
            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.selector);

        _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;
                    }
                }
            }
        }

        // Mask `to` to the lower 160 bits, in case the upper bits somehow aren't clean.
        uint256 toMasked = uint256(uint160(to)) & _BITMASK_ADDRESS;
        assembly {
            // 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.
                from, // `from`.
                toMasked, // `to`.
                tokenId // `tokenId`.
            )
        }
        if (toMasked == 0) _revert(TransferToZeroAddress.selector);

        _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.selector);
            }
    }

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

        _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:
            // - `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)
            );

            // Updates:
            // - `balance += quantity`.
            // - `numberMinted += quantity`.
            //
            // We can directly add to the `balance` and `numberMinted`.
            _packedAddressData[to] +=
                quantity *
                ((1 << _BITPOS_NUMBER_MINTED) | 1);

            // Mask `to` to the lower 160 bits, in case the upper bits somehow aren't clean.
            uint256 toMasked = uint256(uint160(to)) & _BITMASK_ADDRESS;

            if (toMasked == 0) _revert(MintToZeroAddress.selector);

            uint256 end = startTokenId + quantity;
            uint256 tokenId = startTokenId;

            do {
                assembly {
                    // 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`.
                        tokenId // `tokenId`.
                    )
                }
                // The `!=` check ensures that large values of `quantity`
                // that overflows uint256 will make the loop run out of gas.
            } while (++tokenId != end);

            _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.selector);
        if (quantity == 0) _revert(MintZeroQuantity.selector);
        if (quantity > _MAX_MINT_ERC2309_QUANTITY_LIMIT)
            _revert(MintERC2309QuantityExceedsLimit.selector);

        _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.selector
                        );
                    }
                } while (index < end);
                // Reentrancy protection.
                if (_currentIndex != end) _revert(bytes4(0));
            }
        }
    }

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

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

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

    /**
     * @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:
     *
     * - `tokenId` must exist.
     *
     * Emits an {Approval} event.
     */
    function _approve(
        address to,
        uint256 tokenId,
        bool approvalCheck
    ) internal virtual {
        address owner = ownerOf(tokenId);

        if (approvalCheck && _msgSenderERC721A() != owner)
            if (!isApprovedForAll(owner, _msgSenderERC721A())) {
                _revert(ApprovalCallerNotOwnerNorApproved.selector);
            }

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

    // =============================================================
    //                        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.selector);
        }

        _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.selector);
        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)
        }
    }

    /**
     * @dev For more efficient reverts.
     */
    function _revert(bytes4 errorSelector) internal pure {
        assembly {
            mstore(0x00, errorSelector)
            revert(0x00, 0x04)
        }
    }
}

/*
     __    __   ______   __    __  __      __  __    __  _______   __    __  __    __  __    __   ______  
    |  \  /  \ /      \ |  \  |  \|  \    /  \|  \  |  \|       \ |  \  |  \|  \  |  \|  \  /  \ /      \ 
    | $$ /  $$|  $$$$$$\| $$\ | $$ \$$\  /  $$| $$  | $$| $$$$$$$\| $$  | $$| $$\ | $$| $$ /  $$|  $$$$$$\
    | $$/  $$ | $$__| $$| $$$\| $$  \$$\/  $$ | $$  | $$| $$  | $$| $$  | $$| $$$\| $$| $$/  $$ | $$___\$$
    | $$  $$  | $$    $$| $$$$\ $$   \$$  $$  | $$  | $$| $$  | $$| $$  | $$| $$$$\ $$| $$  $$   \$$    \ 
    | $$$$$\  | $$$$$$$$| $$\$$ $$    \$$$$   | $$  | $$| $$  | $$| $$  | $$| $$\$$ $$| $$$$$\   _\$$$$$$\
    | $$ \$$\ | $$  | $$| $$ \$$$$    | $$    | $$__/ $$| $$__/ $$| $$__/ $$| $$ \$$$$| $$ \$$\ |  \__| $$
    | $$  \$$\| $$  | $$| $$  \$$$    | $$     \$$    $$| $$    $$ \$$    $$| $$  \$$$| $$  \$$\ \$$    $$
     \$$   \$$ \$$   \$$ \$$   \$$     \$$      \$$$$$$  \$$$$$$$   \$$$$$$  \$$   \$$ \$$   \$$  \$$$$$$ 
                                                                                                                                                                                                       
*/

contract Kanyudunks is ERC721A, Ownable, ReentrancyGuard {
    // ------------------------------------------------------------------------------------------------------- //
    // ---------------------------------------------- INIZIALIZATION ----------------------------------------- //
    // ------------------------------------------------------------------------------------------------------- //

    constructor() ERC721A("Kanyudunks", "$KNY") {
        _mint(0x32ddc17C67BEb8ea8f225f016Af50bB89065079c, 55);
        _transferOwnership(0x32ddc17C67BEb8ea8f225f016Af50bB89065079c);
        _uri = "ipfs://bafybeidaqdhajj7jdzosxvrxcitebkpncn55ou4j42aebsriite5mllzw4/";
    }

    // ------------------------------------------------------------------------------------------------------- //
    // ------------------------------------------------ VARIABLES -------------------------------------------- //
    // ------------------------------------------------------------------------------------------------------- //

    uint256 private maxSupply = 5555;

    uint256 private publicPrice = 0.038 ether;
    uint256 private whitelistPrice = 0.03 ether;

    uint256 private ogStart = 1679252385;
    uint256 private publicStart = 1679254845;
    uint256 private dunklistStart = 1679253645;

    uint256 private maxPerTxPublic = 3;
    uint256 private maxPerTxWhitelist = 2;
    uint256 private maxPerWalletPublic = 3;
    uint256 private maxPerWalletWhitelist = 2;

    string private uriExtension = ".json";

    bytes32 private dunklistMerkleRoot =
        0x23b51651f3a9f971bcb9c3526e2eb44361d7f6fb75206f1536f3447fca9c7ad3;
    bytes32 private ogMerkleRoot =
        0x39eb2f200dedc8855e68f5201a7269918f93e412e707ce7171badd9b43c8e7ba;

    // ------------------------------------------------------------------------------------------------------- //
    // ------------------------------------------------ MODIFIERS -------------------------------------------- //
    // ------------------------------------------------------------------------------------------------------- //

    modifier onlyWhitelisted(
        bytes32 merkleRoot,
        bytes32[] calldata merkleProof
    ) {
        bytes32 leaf = keccak256(abi.encodePacked(msg.sender));
        require(
            MerkleProof.verify(merkleProof, merkleRoot, leaf),
            "NOT_WHITELISTED!"
        );
        _;
    }

    modifier checkMaxSupply(uint256 amount) {
        uint256 supplyAfterPurchase = _totalMinted() + amount;
        require(supplyAfterPurchase <= maxSupply, "EXCEEDS_MAX_SUPPLY!");
        _;
    }

    modifier checkWhitelistPrice(uint256 amount) {
        uint256 price = whitelistPrice * amount;
        require(msg.value == whitelistPrice * amount, "INCORRECT_VALUE!");
        _;
    }

    // ------------------------------------------------------------------------------------------------------- //
    // ------------------------------------------------ MAPPINGS --------------------------------------------- //
    // ------------------------------------------------------------------------------------------------------- //

    mapping(address => uint256) private _dlMinted;
    mapping(address => uint256) private _ogMinted;
    mapping(address => uint256) private _publicMinted;

    // ------------------------------------------------------------------------------------------------------- //
    // ------------------------------------------------- GETTERS --------------------------------------------- //
    // ------------------------------------------------------------------------------------------------------- //

    function getPhase() public view returns (uint256) {
        if (block.timestamp < ogStart) return 0;
        else if (block.timestamp >= ogStart && block.timestamp < dunklistStart)
            return 1;
        else if (
            block.timestamp >= dunklistStart && block.timestamp < publicStart
        ) return 2;
        else return 3;
    }

    function getOgMinted(address wallet) public view returns (uint256) {
        return _ogMinted[wallet];
    }

    function getDlMinted(address wallet) public view returns (uint256) {
        return _dlMinted[wallet];
    }

    function getPublicMinted(address wallet) public view returns (uint256) {
        return _publicMinted[wallet];
    }

    function getPublicPrice() public view returns (uint256) {
        return publicPrice;
    }

    function getWhitelistPrice() public view returns (uint256) {
        return whitelistPrice;
    }

    function getMaxSupply() public view returns (uint256) {
        return maxSupply;
    }

    function getWhitelists() public view returns (bytes32, bytes32) {
        return (ogMerkleRoot, dunklistMerkleRoot);
    }

    function isOgWhitelisted(bytes32[] calldata merkleProof)
        public
        view
        returns (bool)
    {
        bytes32 leaf = keccak256(abi.encodePacked(msg.sender));
        return MerkleProof.verify(merkleProof, ogMerkleRoot, leaf);
    }

    function isDunklistWhitelisted(bytes32[] calldata merkleProof)
        public
        view
        returns (bool)
    {
        bytes32 leaf = keccak256(abi.encodePacked(msg.sender));
        return MerkleProof.verify(merkleProof, dunklistMerkleRoot, leaf);
    }

    function getSaleLimits()
        public
        view
        returns (
            uint256,
            uint256,
            uint256,
            uint256
        )
    {
        return (
            maxPerTxPublic,
            maxPerTxWhitelist,
            maxPerWalletPublic,
            maxPerWalletWhitelist
        );
    }

    function getSaleTimestamps()
        public
        view
        returns (
            uint256,
            uint256,
            uint256
        )
    {
        return (ogStart, dunklistStart, publicStart);
    }

    // ------------------------------------------------------------------------------------------------------- //
    // ------------------------------------------------- SETTERS --------------------------------------------- //
    // ------------------------------------------------------------------------------------------------------- //

    /* ----------------------------------------------- CENTRALIZED ------------------------------------------- */

    function setBaseURI(string calldata uri) external onlyOwner {
        _uri = uri;
    }

    function setMaxSupply(uint256 _maxSupply) external onlyOwner {
        maxSupply = _maxSupply;
    }

    function setUriExtension(string calldata _uriExtension) external onlyOwner {
        uriExtension = _uriExtension;
    }

    function ownerMint(uint256 amount)
        external
        onlyOwner
        checkMaxSupply(amount)
    {
        _mint(msg.sender, amount);
    }

    function setSaleTimestamps(
        uint256 _ogStart,
        uint256 _dunklistStart,
        uint256 _publicStart
    ) external onlyOwner {
        ogStart = _ogStart;
        publicStart = _publicStart;
        dunklistStart = _dunklistStart;
    }

    function setSaleLimits(
        uint256 _maxPerTxPublic,
        uint256 _maxPerTxWhitelist,
        uint256 _maxPerWalletPublic,
        uint256 _maxPerWalletWhitelist
    ) external onlyOwner {
        maxPerTxPublic = _maxPerTxPublic;
        maxPerTxWhitelist = _maxPerTxWhitelist;
        maxPerWalletPublic = _maxPerWalletPublic;
        maxPerWalletWhitelist = _maxPerWalletWhitelist;
    }

    function setPrices(uint256 _whitelistPrice, uint256 _publicPrice)
        external
        onlyOwner
    {
        whitelistPrice = _whitelistPrice;
        publicPrice = _publicPrice;
    }

    function setWhitelists(bytes32 _ogMerkleRoot, bytes32 _dunklistMerkleRoot)
        external
        onlyOwner
    {
        ogMerkleRoot = _ogMerkleRoot;
        dunklistMerkleRoot = _dunklistMerkleRoot;
    }

    function withdraw() external onlyOwner {
        payable(msg.sender).transfer(address(this).balance);
    }

    /* ------------------------------------------------- PUBLIC ---------------------------------------------- */

    function dunklistMint(uint256 amount, bytes32[] calldata merkleProof)
        external
        payable
        nonReentrant
        checkMaxSupply(amount)
        checkWhitelistPrice(amount)
        onlyWhitelisted(dunklistMerkleRoot, merkleProof)
    {
        uint256 minted = _dlMinted[msg.sender] + amount;

        require(amount <= maxPerTxWhitelist, "EXCEEDS_MAX_PER_TX!");
        require(msg.value == whitelistPrice * amount, "INCORRECT_VALUE!");
        require(minted <= maxPerWalletWhitelist, "EXCEEDS_MAX_PER_WALLET!");

        _dlMinted[msg.sender] += amount;

        _mint(msg.sender, amount);
    }

    function ogMint(uint256 amount, bytes32[] calldata merkleProof)
        external
        payable
        nonReentrant
        checkMaxSupply(amount)
        checkWhitelistPrice(amount)
        onlyWhitelisted(ogMerkleRoot, merkleProof)
    {
        uint256 minted = _ogMinted[msg.sender] + amount;

        require(amount <= maxPerTxWhitelist, "EXCEEDS_MAX_PER_TX!");
        require(minted <= maxPerWalletWhitelist, "EXCEEDS_MAX_PER_WALLET!");

        _ogMinted[msg.sender] += amount;

        _mint(msg.sender, amount);
    }

    function publicMint(uint256 amount)
        external
        payable
        nonReentrant
        checkMaxSupply(amount)
    {
        uint256 minted = _publicMinted[msg.sender] + amount;
        uint256 price = publicPrice * amount;

        require(msg.value == price, "INCORRECT_VALUE!");
        require(amount <= maxPerTxPublic, "EXCEEDS_MAX_PER_TX!");
        require(minted <= maxPerWalletPublic, "EXCEEDS_MAX_PER_WALLET!");

        _publicMinted[msg.sender] += amount;

        _mint(msg.sender, amount);
    }

    // ------------------------------------------------------------------------------------------------------- //
    // ------------------------------------------------- OVERRIDES ------------------------------------------- //
    // ------------------------------------------------------------------------------------------------------- //

    function tokenURI(uint256 tokenId)
        public
        view
        virtual
        override
        returns (string memory)
    {
        if (!_exists(tokenId)) _revert(URIQueryForNonexistentToken.selector);

        string memory baseURI = _baseURI();
        return
            bytes(baseURI).length != 0
                ? string(
                    abi.encodePacked(baseURI, _toString(tokenId), uriExtension)
                )
                : "";
    }
}

Contract Security Audit

Contract ABI

[{"inputs":[],"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":[{"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":[{"internalType":"uint256","name":"amount","type":"uint256"},{"internalType":"bytes32[]","name":"merkleProof","type":"bytes32[]"}],"name":"dunklistMint","outputs":[],"stateMutability":"payable","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":"wallet","type":"address"}],"name":"getDlMinted","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"getMaxSupply","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"wallet","type":"address"}],"name":"getOgMinted","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"getPhase","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"wallet","type":"address"}],"name":"getPublicMinted","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"getPublicPrice","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"getSaleLimits","outputs":[{"internalType":"uint256","name":"","type":"uint256"},{"internalType":"uint256","name":"","type":"uint256"},{"internalType":"uint256","name":"","type":"uint256"},{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"getSaleTimestamps","outputs":[{"internalType":"uint256","name":"","type":"uint256"},{"internalType":"uint256","name":"","type":"uint256"},{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"getWhitelistPrice","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"getWhitelists","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"},{"internalType":"bytes32","name":"","type":"bytes32"}],"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":"merkleProof","type":"bytes32[]"}],"name":"isDunklistWhitelisted","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"bytes32[]","name":"merkleProof","type":"bytes32[]"}],"name":"isOgWhitelisted","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"name","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"amount","type":"uint256"},{"internalType":"bytes32[]","name":"merkleProof","type":"bytes32[]"}],"name":"ogMint","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"owner","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"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":[{"internalType":"uint256","name":"amount","type":"uint256"}],"name":"publicMint","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"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":"setBaseURI","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_maxSupply","type":"uint256"}],"name":"setMaxSupply","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_whitelistPrice","type":"uint256"},{"internalType":"uint256","name":"_publicPrice","type":"uint256"}],"name":"setPrices","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_maxPerTxPublic","type":"uint256"},{"internalType":"uint256","name":"_maxPerTxWhitelist","type":"uint256"},{"internalType":"uint256","name":"_maxPerWalletPublic","type":"uint256"},{"internalType":"uint256","name":"_maxPerWalletWhitelist","type":"uint256"}],"name":"setSaleLimits","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_ogStart","type":"uint256"},{"internalType":"uint256","name":"_dunklistStart","type":"uint256"},{"internalType":"uint256","name":"_publicStart","type":"uint256"}],"name":"setSaleTimestamps","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"_uriExtension","type":"string"}],"name":"setUriExtension","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"_ogMerkleRoot","type":"bytes32"},{"internalType":"bytes32","name":"_dunklistMerkleRoot","type":"bytes32"}],"name":"setWhitelists","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":"nonpayable","type":"function"}]

6115b3600b55668700cc75770000600c55666a94d74f430000600d556364175ba1600e55636417653d600f55636417608d601055600360118190556002601281905560139190915560145560c06040526005608090815264173539b7b760d91b60a0526015906200007190826200037a565b507f23b51651f3a9f971bcb9c3526e2eb44361d7f6fb75206f1536f3447fca9c7ad36016557f39eb2f200dedc8855e68f5201a7269918f93e412e707ce7171badd9b43c8e7ba601755348015620000c757600080fd5b506040518060400160405280600a8152602001694b616e797564756e6b7360b01b81525060405180604001604052806004815260200163244b4e5960e01b81525081600290816200011991906200037a565b5060036200012882826200037a565b505060008055506200013a33620001af565b6001600a55620001607332ddc17c67beb8ea8f225f016af50bb89065079c603762000201565b6200017f7332ddc17c67beb8ea8f225f016af50bb89065079c620001af565b6040518060800160405280604381526020016200256160439139600490620001a890826200037a565b5062000446565b600980546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b600080549082900362000220576200022063b562e8dd60e01b620002cc565b60008181526005602090815260408083206001600160a01b0387164260a01b6001881460e11b17811790915580845260069092528220805468010000000000000001860201905590819003620002815762000281622e076360e81b620002cc565b818301825b808360007fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a481816001019150810362000286575060005550505050565b505050565b8060005260046000fd5b634e487b7160e01b600052604160045260246000fd5b600181811c908216806200030157607f821691505b6020821081036200032257634e487b7160e01b600052602260045260246000fd5b50919050565b601f821115620002c757600081815260208120601f850160051c81016020861015620003515750805b601f850160051c820191505b8181101562000372578281556001016200035d565b505050505050565b81516001600160401b03811115620003965762000396620002d6565b620003ae81620003a78454620002ec565b8462000328565b602080601f831160018114620003e65760008415620003cd5750858301515b600019600386901b1c1916600185901b17855562000372565b600085815260208120601f198616915b828110156200041757888601518255948401946001909101908401620003f6565b5085821015620004365787850151600019600388901b60f8161c191681555b5050505050600190811b01905550565b61210b80620004566000396000f3fe6080604052600436106102465760003560e01c8063547e83161161013957806395d89b41116100b6578063c87b56dd1161007a578063c87b56dd146106a7578063e985e9c5146106c7578063eced028014610710578063f19e75d414610725578063f2fde38b14610745578063fad569781461076557600080fd5b806395d89b4114610617578063a22cb4651461062c578063b88d4fde1461064c578063bed2b4f11461065f578063c35dcf901461067f57600080fd5b8063715018a6116100fd578063715018a6146105915780637872f77f146105a65780637c538955146105c65780637db8d3d2146105e65780638da5cb5b146105f957600080fd5b8063547e8316146104db57806355f804b3146105115780636352211e146105315780636f8b44b01461055157806370a082311461057157600080fd5b806325f4fac6116101c75780633a9a37d81161018b5780633a9a37d8146104455780633ccfd60b1461046557806342842e0e1461047a57806346b4627a1461048d5780634c0f38c2146104c657600080fd5b806325f4fac6146103ca5780632b314dc6146103ea5780632ce9af50146103fd5780632db115441461041d578063363e86fe1461043057600080fd5b8063095ea7b31161020e578063095ea7b3146103405780630da51cd7146103535780631715c4731461036857806318160ddd1461039e57806323b872dd146103b757600080fd5b806301ffc9a71461024b57806304ad2d481461028057806305fefda7146102c457806306fdde03146102e6578063081812fc14610308575b600080fd5b34801561025757600080fd5b5061026b61026636600461189f565b610796565b60405190151581526020015b60405180910390f35b34801561028c57600080fd5b506102b661029b3660046118d3565b6001600160a01b03166000908152601a602052604090205490565b604051908152602001610277565b3480156102d057600080fd5b506102e46102df3660046118ee565b6107e8565b005b3480156102f257600080fd5b506102fb6107fb565b6040516102779190611960565b34801561031457600080fd5b50610328610323366004611973565b61088d565b6040516001600160a01b039091168152602001610277565b6102e461034e36600461198c565b6108c8565b34801561035f57600080fd5b50600d546102b6565b34801561037457600080fd5b506102b66103833660046118d3565b6001600160a01b031660009081526018602052604090205490565b3480156103aa57600080fd5b50600154600054036102b6565b6102e46103c53660046119b6565b6108d8565b3480156103d657600080fd5b5061026b6103e5366004611a3e565b610a3d565b6102e46103f8366004611a80565b610ab2565b34801561040957600080fd5b506102e4610418366004611acc565b610cae565b6102e461042b366004611973565b610cc8565b34801561043c57600080fd5b50600c546102b6565b34801561045157600080fd5b506102e4610460366004611b3e565b610df7565b34801561047157600080fd5b506102e4610e10565b6102e46104883660046119b6565b610e47565b34801561049957600080fd5b50601154601254601354601454604080519485526020850193909352918301526060820152608001610277565b3480156104d257600080fd5b50600b546102b6565b3480156104e757600080fd5b506102b66104f63660046118d3565b6001600160a01b031660009081526019602052604090205490565b34801561051d57600080fd5b506102e461052c366004611acc565b610e62565b34801561053d57600080fd5b5061032861054c366004611973565b610e77565b34801561055d57600080fd5b506102e461056c366004611973565b610e82565b34801561057d57600080fd5b506102b661058c3660046118d3565b610e8f565b34801561059d57600080fd5b506102e4610ed5565b3480156105b257600080fd5b506102e46105c13660046118ee565b610ee9565b3480156105d257600080fd5b506102e46105e1366004611b6a565b610efc565b6102e46105f4366004611a80565b610f18565b34801561060557600080fd5b506009546001600160a01b0316610328565b34801561062357600080fd5b506102fb611114565b34801561063857600080fd5b506102e4610647366004611b9c565b611123565b6102e461065a366004611bee565b61118f565b34801561066b57600080fd5b5061026b61067a366004611a3e565b6111d0565b34801561068b57600080fd5b5060175460165460408051928352602083019190915201610277565b3480156106b357600080fd5b506102fb6106c2366004611973565b61123d565b3480156106d357600080fd5b5061026b6106e2366004611cca565b6001600160a01b03918216600090815260086020908152604080832093909416825291909152205460ff1690565b34801561071c57600080fd5b506102b66112bb565b34801561073157600080fd5b506102e4610740366004611973565b61130f565b34801561075157600080fd5b506102e46107603660046118d3565b61135c565b34801561077157600080fd5b50600e54601054600f5460408051938452602084019290925290820152606001610277565b60006301ffc9a760e01b6001600160e01b0319831614806107c757506380ac58cd60e01b6001600160e01b03198316145b806107e25750635b5e139f60e01b6001600160e01b03198316145b92915050565b6107f06113d2565b600d91909155600c55565b60606002805461080a90611cfd565b80601f016020809104026020016040519081016040528092919081815260200182805461083690611cfd565b80156108835780601f1061085857610100808354040283529160200191610883565b820191906000526020600020905b81548152906001019060200180831161086657829003601f168201915b5050505050905090565b60006108988261142c565b6108ac576108ac6333d1c03960e21b611471565b506000908152600760205260409020546001600160a01b031690565b6108d48282600161147b565b5050565b60006108e38261151e565b6001600160a01b0394851694909150811684146109095761090962a1148160e81b611471565b60008281526007602052604090208054338082146001600160a01b0388169091141761094d5761093986336106e2565b61094d5761094d632ce44b5f60e11b611471565b801561095857600082555b6001600160a01b038681166000908152600660205260408082208054600019019055918716808252919020805460010190554260a01b17600160e11b17600085815260056020526040812091909155600160e11b841690036109ea576001840160008181526005602052604081205490036109e85760005481146109e85760008181526005602052604090208490555b505b6001600160a01b0385168481887fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a480600003610a3457610a34633a954ecd60e21b611471565b50505050505050565b60008033604051602001610a519190611d37565b604051602081830303815290604052805190602001209050610aaa8484808060200260200160405190810160405280939291908181526020018383602002808284376000920191909152505060175491508490506115b4565b949350505050565b6002600a5403610add5760405162461bcd60e51b8152600401610ad490611d54565b60405180910390fd5b6002600a5582600081610aef60005490565b610af99190611da1565b9050600b54811115610b1d5760405162461bcd60e51b8152600401610ad490611db4565b84600081600d54610b2e9190611de1565b905081600d54610b3e9190611de1565b3414610b5c5760405162461bcd60e51b8152600401610ad490611df8565b6017548686600033604051602001610b749190611d37565b604051602081830303815290604052805190602001209050610bcc8383808060200260200160405190810160405280939291908181526020018383602002808284376000920191909152508892508591506115b49050565b610c0b5760405162461bcd60e51b815260206004820152601060248201526f4e4f545f57484954454c49535445442160801b6044820152606401610ad4565b33600090815260196020526040812054610c26908d90611da1565b90506012548c1115610c4a5760405162461bcd60e51b8152600401610ad490611e22565b601454811115610c6c5760405162461bcd60e51b8152600401610ad490611e4f565b33600090815260196020526040812080548e9290610c8b908490611da1565b90915550610c9b9050338d6115ca565b50506001600a5550505050505050505050565b610cb66113d2565b6015610cc3828483611ed4565b505050565b6002600a5403610cea5760405162461bcd60e51b8152600401610ad490611d54565b6002600a5580600081610cfc60005490565b610d069190611da1565b9050600b54811115610d2a5760405162461bcd60e51b8152600401610ad490611db4565b336000908152601a6020526040812054610d45908590611da1565b9050600084600c54610d579190611de1565b9050803414610d785760405162461bcd60e51b8152600401610ad490611df8565b601154851115610d9a5760405162461bcd60e51b8152600401610ad490611e22565b601354821115610dbc5760405162461bcd60e51b8152600401610ad490611e4f565b336000908152601a602052604081208054879290610ddb908490611da1565b90915550610deb905033866115ca565b50506001600a55505050565b610dff6113d2565b600e92909255600f91909155601055565b610e186113d2565b60405133904780156108fc02916000818181858888f19350505050158015610e44573d6000803e3d6000fd5b50565b610cc38383836040518060200160405280600081525061118f565b610e6a6113d2565b6004610cc3828483611ed4565b60006107e28261151e565b610e8a6113d2565b600b55565b60006001600160a01b038216610eaf57610eaf6323d3ad8160e21b611471565b506001600160a01b031660009081526006602052604090205467ffffffffffffffff1690565b610edd6113d2565b610ee76000611689565b565b610ef16113d2565b601791909155601655565b610f046113d2565b601193909355601291909155601355601455565b6002600a5403610f3a5760405162461bcd60e51b8152600401610ad490611d54565b6002600a5582600081610f4c60005490565b610f569190611da1565b9050600b54811115610f7a5760405162461bcd60e51b8152600401610ad490611db4565b84600081600d54610f8b9190611de1565b905081600d54610f9b9190611de1565b3414610fb95760405162461bcd60e51b8152600401610ad490611df8565b6016548686600033604051602001610fd19190611d37565b6040516020818303038152906040528051906020012090506110298383808060200260200160405190810160405280939291908181526020018383602002808284376000920191909152508892508591506115b49050565b6110685760405162461bcd60e51b815260206004820152601060248201526f4e4f545f57484954454c49535445442160801b6044820152606401610ad4565b33600090815260186020526040812054611083908d90611da1565b90506012548c11156110a75760405162461bcd60e51b8152600401610ad490611e22565b8b600d546110b59190611de1565b34146110d35760405162461bcd60e51b8152600401610ad490611df8565b6014548111156110f55760405162461bcd60e51b8152600401610ad490611e4f565b33600090815260186020526040812080548e9290610c8b908490611da1565b60606003805461080a90611cfd565b3360008181526008602090815260408083206001600160a01b03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b61119a8484846108d8565b6001600160a01b0383163b156111ca576111b6848484846116db565b6111ca576111ca6368d2bf6b60e11b611471565b50505050565b600080336040516020016111e49190611d37565b604051602081830303815290604052805190602001209050610aaa8484808060200260200160405190810160405280939291908181526020018383602002808284376000920191909152505060165491508490506115b4565b60606112488261142c565b61125c5761125c630a14c4b560e41b611471565b60006112666117bd565b9050805160000361128657604051806020016040528060008152506112b4565b80611290846117cc565b60156040516020016112a493929190611f95565b6040516020818303038152906040525b9392505050565b6000600e544210156112cd5750600090565b600e5442101580156112e0575060105442105b156112eb5750600190565b60105442101580156112fe5750600f5442105b156113095750600290565b50600390565b6113176113d2565b8060008161132460005490565b61132e9190611da1565b9050600b548111156113525760405162461bcd60e51b8152600401610ad490611db4565b610cc333846115ca565b6113646113d2565b6001600160a01b0381166113c95760405162461bcd60e51b815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201526564647265737360d01b6064820152608401610ad4565b610e4481611689565b6009546001600160a01b03163314610ee75760405162461bcd60e51b815260206004820181905260248201527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e65726044820152606401610ad4565b6000805482101561146c5760005b50600082815260056020526040812054908190036114625761145b83612035565b925061143a565b600160e01b161590505b919050565b8060005260046000fd5b600061148683610e77565b905081801561149e5750336001600160a01b03821614155b156114c1576114ad81336106e2565b6114c1576114c16367d9dca160e11b611471565b60008381526007602052604080822080546001600160a01b0319166001600160a01b0388811691821790925591518693918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a450505050565b6000818152600560205260408120549081900361159157600054821061154e5761154e636f96cda160e11b611471565b5b5060001901600081815260056020526040902054801561154f57600160e01b811660000361157c57919050565b61158c636f96cda160e11b611471565b61154f565b600160e01b81166000036115a457919050565b61146c636f96cda160e11b611471565b6000826115c18584611810565b14949350505050565b60008054908290036115e6576115e663b562e8dd60e01b611471565b60008181526005602090815260408083206001600160a01b0387164260a01b6001881460e11b1781179091558084526006909252822080546801000000000000000186020190559081900361164457611644622e076360e81b611471565b818301825b808360007fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a4818160010191508103611649575060005550505050565b600980546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b604051630a85bd0160e11b81526000906001600160a01b0385169063150b7a029061171090339089908890889060040161204c565b6020604051808303816000875af192505050801561174b575060408051601f3d908101601f1916820190925261174891810190612089565b60015b6117a0573d808015611779576040519150601f19603f3d011682016040523d82523d6000602084013e61177e565b606091505b508051600003611798576117986368d2bf6b60e11b611471565b805181602001fd5b6001600160e01b031916630a85bd0160e11b149050949350505050565b60606004805461080a90611cfd565b606060a06040510180604052602081039150506000815280825b600183039250600a81066030018353600a9004806117e65750819003601f19909101908152919050565b600081815b84518110156118555761184182868381518110611834576118346120a6565b602002602001015161185d565b91508061184d816120bc565b915050611815565b509392505050565b60008183106118795760008281526020849052604090206112b4565b5060009182526020526040902090565b6001600160e01b031981168114610e4457600080fd5b6000602082840312156118b157600080fd5b81356112b481611889565b80356001600160a01b038116811461146c57600080fd5b6000602082840312156118e557600080fd5b6112b4826118bc565b6000806040838503121561190157600080fd5b50508035926020909101359150565b60005b8381101561192b578181015183820152602001611913565b50506000910152565b6000815180845261194c816020860160208601611910565b601f01601f19169290920160200192915050565b6020815260006112b46020830184611934565b60006020828403121561198557600080fd5b5035919050565b6000806040838503121561199f57600080fd5b6119a8836118bc565b946020939093013593505050565b6000806000606084860312156119cb57600080fd5b6119d4846118bc565b92506119e2602085016118bc565b9150604084013590509250925092565b60008083601f840112611a0457600080fd5b50813567ffffffffffffffff811115611a1c57600080fd5b6020830191508360208260051b8501011115611a3757600080fd5b9250929050565b60008060208385031215611a5157600080fd5b823567ffffffffffffffff811115611a6857600080fd5b611a74858286016119f2565b90969095509350505050565b600080600060408486031215611a9557600080fd5b83359250602084013567ffffffffffffffff811115611ab357600080fd5b611abf868287016119f2565b9497909650939450505050565b60008060208385031215611adf57600080fd5b823567ffffffffffffffff80821115611af757600080fd5b818501915085601f830112611b0b57600080fd5b813581811115611b1a57600080fd5b866020828501011115611b2c57600080fd5b60209290920196919550909350505050565b600080600060608486031215611b5357600080fd5b505081359360208301359350604090920135919050565b60008060008060808587031215611b8057600080fd5b5050823594602084013594506040840135936060013592509050565b60008060408385031215611baf57600080fd5b611bb8836118bc565b915060208301358015158114611bcd57600080fd5b809150509250929050565b634e487b7160e01b600052604160045260246000fd5b60008060008060808587031215611c0457600080fd5b611c0d856118bc565b9350611c1b602086016118bc565b925060408501359150606085013567ffffffffffffffff80821115611c3f57600080fd5b818701915087601f830112611c5357600080fd5b813581811115611c6557611c65611bd8565b604051601f8201601f19908116603f01168101908382118183101715611c8d57611c8d611bd8565b816040528281528a6020848701011115611ca657600080fd5b82602086016020830137600060208483010152809550505050505092959194509250565b60008060408385031215611cdd57600080fd5b611ce6836118bc565b9150611cf4602084016118bc565b90509250929050565b600181811c90821680611d1157607f821691505b602082108103611d3157634e487b7160e01b600052602260045260246000fd5b50919050565b60609190911b6bffffffffffffffffffffffff1916815260140190565b6020808252601f908201527f5265656e7472616e637947756172643a207265656e7472616e742063616c6c00604082015260600190565b634e487b7160e01b600052601160045260246000fd5b808201808211156107e2576107e2611d8b565b602080825260139082015272455843454544535f4d41585f535550504c592160681b604082015260600190565b80820281158282048414176107e2576107e2611d8b565b60208082526010908201526f494e434f52524543545f56414c55452160801b604082015260600190565b602080825260139082015272455843454544535f4d41585f5045525f54582160681b604082015260600190565b60208082526017908201527f455843454544535f4d41585f5045525f57414c4c455421000000000000000000604082015260600190565b601f821115610cc357600081815260208120601f850160051c81016020861015611ead5750805b601f850160051c820191505b81811015611ecc57828155600101611eb9565b505050505050565b67ffffffffffffffff831115611eec57611eec611bd8565b611f0083611efa8354611cfd565b83611e86565b6000601f841160018114611f345760008515611f1c5750838201355b600019600387901b1c1916600186901b178355611f8e565b600083815260209020601f19861690835b82811015611f655786850135825560209485019460019092019101611f45565b5086821015611f825760001960f88860031b161c19848701351681555b505060018560011b0183555b5050505050565b600084516020611fa88285838a01611910565b855191840191611fbb8184848a01611910565b8554920191600090611fcc81611cfd565b60018281168015611fe45760018114611ff957612025565b60ff1984168752821515830287019450612025565b896000528560002060005b8481101561201d57815489820152908301908701612004565b505082870194505b50929a9950505050505050505050565b60008161204457612044611d8b565b506000190190565b6001600160a01b038581168252841660208201526040810183905260806060820181905260009061207f90830184611934565b9695505050505050565b60006020828403121561209b57600080fd5b81516112b481611889565b634e487b7160e01b600052603260045260246000fd5b6000600182016120ce576120ce611d8b565b506001019056fea26469706673582212208894028f7ac0f5544a476324fd5a60017fa9bae2d3d1bb6be153646e8d3d0d7e64736f6c63430008130033697066733a2f2f626166796265696461716468616a6a376a647a6f737876727863697465626b706e636e35356f75346a3432616562737269697465356d6c6c7a77342f

Deployed Bytecode

0x6080604052600436106102465760003560e01c8063547e83161161013957806395d89b41116100b6578063c87b56dd1161007a578063c87b56dd146106a7578063e985e9c5146106c7578063eced028014610710578063f19e75d414610725578063f2fde38b14610745578063fad569781461076557600080fd5b806395d89b4114610617578063a22cb4651461062c578063b88d4fde1461064c578063bed2b4f11461065f578063c35dcf901461067f57600080fd5b8063715018a6116100fd578063715018a6146105915780637872f77f146105a65780637c538955146105c65780637db8d3d2146105e65780638da5cb5b146105f957600080fd5b8063547e8316146104db57806355f804b3146105115780636352211e146105315780636f8b44b01461055157806370a082311461057157600080fd5b806325f4fac6116101c75780633a9a37d81161018b5780633a9a37d8146104455780633ccfd60b1461046557806342842e0e1461047a57806346b4627a1461048d5780634c0f38c2146104c657600080fd5b806325f4fac6146103ca5780632b314dc6146103ea5780632ce9af50146103fd5780632db115441461041d578063363e86fe1461043057600080fd5b8063095ea7b31161020e578063095ea7b3146103405780630da51cd7146103535780631715c4731461036857806318160ddd1461039e57806323b872dd146103b757600080fd5b806301ffc9a71461024b57806304ad2d481461028057806305fefda7146102c457806306fdde03146102e6578063081812fc14610308575b600080fd5b34801561025757600080fd5b5061026b61026636600461189f565b610796565b60405190151581526020015b60405180910390f35b34801561028c57600080fd5b506102b661029b3660046118d3565b6001600160a01b03166000908152601a602052604090205490565b604051908152602001610277565b3480156102d057600080fd5b506102e46102df3660046118ee565b6107e8565b005b3480156102f257600080fd5b506102fb6107fb565b6040516102779190611960565b34801561031457600080fd5b50610328610323366004611973565b61088d565b6040516001600160a01b039091168152602001610277565b6102e461034e36600461198c565b6108c8565b34801561035f57600080fd5b50600d546102b6565b34801561037457600080fd5b506102b66103833660046118d3565b6001600160a01b031660009081526018602052604090205490565b3480156103aa57600080fd5b50600154600054036102b6565b6102e46103c53660046119b6565b6108d8565b3480156103d657600080fd5b5061026b6103e5366004611a3e565b610a3d565b6102e46103f8366004611a80565b610ab2565b34801561040957600080fd5b506102e4610418366004611acc565b610cae565b6102e461042b366004611973565b610cc8565b34801561043c57600080fd5b50600c546102b6565b34801561045157600080fd5b506102e4610460366004611b3e565b610df7565b34801561047157600080fd5b506102e4610e10565b6102e46104883660046119b6565b610e47565b34801561049957600080fd5b50601154601254601354601454604080519485526020850193909352918301526060820152608001610277565b3480156104d257600080fd5b50600b546102b6565b3480156104e757600080fd5b506102b66104f63660046118d3565b6001600160a01b031660009081526019602052604090205490565b34801561051d57600080fd5b506102e461052c366004611acc565b610e62565b34801561053d57600080fd5b5061032861054c366004611973565b610e77565b34801561055d57600080fd5b506102e461056c366004611973565b610e82565b34801561057d57600080fd5b506102b661058c3660046118d3565b610e8f565b34801561059d57600080fd5b506102e4610ed5565b3480156105b257600080fd5b506102e46105c13660046118ee565b610ee9565b3480156105d257600080fd5b506102e46105e1366004611b6a565b610efc565b6102e46105f4366004611a80565b610f18565b34801561060557600080fd5b506009546001600160a01b0316610328565b34801561062357600080fd5b506102fb611114565b34801561063857600080fd5b506102e4610647366004611b9c565b611123565b6102e461065a366004611bee565b61118f565b34801561066b57600080fd5b5061026b61067a366004611a3e565b6111d0565b34801561068b57600080fd5b5060175460165460408051928352602083019190915201610277565b3480156106b357600080fd5b506102fb6106c2366004611973565b61123d565b3480156106d357600080fd5b5061026b6106e2366004611cca565b6001600160a01b03918216600090815260086020908152604080832093909416825291909152205460ff1690565b34801561071c57600080fd5b506102b66112bb565b34801561073157600080fd5b506102e4610740366004611973565b61130f565b34801561075157600080fd5b506102e46107603660046118d3565b61135c565b34801561077157600080fd5b50600e54601054600f5460408051938452602084019290925290820152606001610277565b60006301ffc9a760e01b6001600160e01b0319831614806107c757506380ac58cd60e01b6001600160e01b03198316145b806107e25750635b5e139f60e01b6001600160e01b03198316145b92915050565b6107f06113d2565b600d91909155600c55565b60606002805461080a90611cfd565b80601f016020809104026020016040519081016040528092919081815260200182805461083690611cfd565b80156108835780601f1061085857610100808354040283529160200191610883565b820191906000526020600020905b81548152906001019060200180831161086657829003601f168201915b5050505050905090565b60006108988261142c565b6108ac576108ac6333d1c03960e21b611471565b506000908152600760205260409020546001600160a01b031690565b6108d48282600161147b565b5050565b60006108e38261151e565b6001600160a01b0394851694909150811684146109095761090962a1148160e81b611471565b60008281526007602052604090208054338082146001600160a01b0388169091141761094d5761093986336106e2565b61094d5761094d632ce44b5f60e11b611471565b801561095857600082555b6001600160a01b038681166000908152600660205260408082208054600019019055918716808252919020805460010190554260a01b17600160e11b17600085815260056020526040812091909155600160e11b841690036109ea576001840160008181526005602052604081205490036109e85760005481146109e85760008181526005602052604090208490555b505b6001600160a01b0385168481887fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a480600003610a3457610a34633a954ecd60e21b611471565b50505050505050565b60008033604051602001610a519190611d37565b604051602081830303815290604052805190602001209050610aaa8484808060200260200160405190810160405280939291908181526020018383602002808284376000920191909152505060175491508490506115b4565b949350505050565b6002600a5403610add5760405162461bcd60e51b8152600401610ad490611d54565b60405180910390fd5b6002600a5582600081610aef60005490565b610af99190611da1565b9050600b54811115610b1d5760405162461bcd60e51b8152600401610ad490611db4565b84600081600d54610b2e9190611de1565b905081600d54610b3e9190611de1565b3414610b5c5760405162461bcd60e51b8152600401610ad490611df8565b6017548686600033604051602001610b749190611d37565b604051602081830303815290604052805190602001209050610bcc8383808060200260200160405190810160405280939291908181526020018383602002808284376000920191909152508892508591506115b49050565b610c0b5760405162461bcd60e51b815260206004820152601060248201526f4e4f545f57484954454c49535445442160801b6044820152606401610ad4565b33600090815260196020526040812054610c26908d90611da1565b90506012548c1115610c4a5760405162461bcd60e51b8152600401610ad490611e22565b601454811115610c6c5760405162461bcd60e51b8152600401610ad490611e4f565b33600090815260196020526040812080548e9290610c8b908490611da1565b90915550610c9b9050338d6115ca565b50506001600a5550505050505050505050565b610cb66113d2565b6015610cc3828483611ed4565b505050565b6002600a5403610cea5760405162461bcd60e51b8152600401610ad490611d54565b6002600a5580600081610cfc60005490565b610d069190611da1565b9050600b54811115610d2a5760405162461bcd60e51b8152600401610ad490611db4565b336000908152601a6020526040812054610d45908590611da1565b9050600084600c54610d579190611de1565b9050803414610d785760405162461bcd60e51b8152600401610ad490611df8565b601154851115610d9a5760405162461bcd60e51b8152600401610ad490611e22565b601354821115610dbc5760405162461bcd60e51b8152600401610ad490611e4f565b336000908152601a602052604081208054879290610ddb908490611da1565b90915550610deb905033866115ca565b50506001600a55505050565b610dff6113d2565b600e92909255600f91909155601055565b610e186113d2565b60405133904780156108fc02916000818181858888f19350505050158015610e44573d6000803e3d6000fd5b50565b610cc38383836040518060200160405280600081525061118f565b610e6a6113d2565b6004610cc3828483611ed4565b60006107e28261151e565b610e8a6113d2565b600b55565b60006001600160a01b038216610eaf57610eaf6323d3ad8160e21b611471565b506001600160a01b031660009081526006602052604090205467ffffffffffffffff1690565b610edd6113d2565b610ee76000611689565b565b610ef16113d2565b601791909155601655565b610f046113d2565b601193909355601291909155601355601455565b6002600a5403610f3a5760405162461bcd60e51b8152600401610ad490611d54565b6002600a5582600081610f4c60005490565b610f569190611da1565b9050600b54811115610f7a5760405162461bcd60e51b8152600401610ad490611db4565b84600081600d54610f8b9190611de1565b905081600d54610f9b9190611de1565b3414610fb95760405162461bcd60e51b8152600401610ad490611df8565b6016548686600033604051602001610fd19190611d37565b6040516020818303038152906040528051906020012090506110298383808060200260200160405190810160405280939291908181526020018383602002808284376000920191909152508892508591506115b49050565b6110685760405162461bcd60e51b815260206004820152601060248201526f4e4f545f57484954454c49535445442160801b6044820152606401610ad4565b33600090815260186020526040812054611083908d90611da1565b90506012548c11156110a75760405162461bcd60e51b8152600401610ad490611e22565b8b600d546110b59190611de1565b34146110d35760405162461bcd60e51b8152600401610ad490611df8565b6014548111156110f55760405162461bcd60e51b8152600401610ad490611e4f565b33600090815260186020526040812080548e9290610c8b908490611da1565b60606003805461080a90611cfd565b3360008181526008602090815260408083206001600160a01b03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b61119a8484846108d8565b6001600160a01b0383163b156111ca576111b6848484846116db565b6111ca576111ca6368d2bf6b60e11b611471565b50505050565b600080336040516020016111e49190611d37565b604051602081830303815290604052805190602001209050610aaa8484808060200260200160405190810160405280939291908181526020018383602002808284376000920191909152505060165491508490506115b4565b60606112488261142c565b61125c5761125c630a14c4b560e41b611471565b60006112666117bd565b9050805160000361128657604051806020016040528060008152506112b4565b80611290846117cc565b60156040516020016112a493929190611f95565b6040516020818303038152906040525b9392505050565b6000600e544210156112cd5750600090565b600e5442101580156112e0575060105442105b156112eb5750600190565b60105442101580156112fe5750600f5442105b156113095750600290565b50600390565b6113176113d2565b8060008161132460005490565b61132e9190611da1565b9050600b548111156113525760405162461bcd60e51b8152600401610ad490611db4565b610cc333846115ca565b6113646113d2565b6001600160a01b0381166113c95760405162461bcd60e51b815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201526564647265737360d01b6064820152608401610ad4565b610e4481611689565b6009546001600160a01b03163314610ee75760405162461bcd60e51b815260206004820181905260248201527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e65726044820152606401610ad4565b6000805482101561146c5760005b50600082815260056020526040812054908190036114625761145b83612035565b925061143a565b600160e01b161590505b919050565b8060005260046000fd5b600061148683610e77565b905081801561149e5750336001600160a01b03821614155b156114c1576114ad81336106e2565b6114c1576114c16367d9dca160e11b611471565b60008381526007602052604080822080546001600160a01b0319166001600160a01b0388811691821790925591518693918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a450505050565b6000818152600560205260408120549081900361159157600054821061154e5761154e636f96cda160e11b611471565b5b5060001901600081815260056020526040902054801561154f57600160e01b811660000361157c57919050565b61158c636f96cda160e11b611471565b61154f565b600160e01b81166000036115a457919050565b61146c636f96cda160e11b611471565b6000826115c18584611810565b14949350505050565b60008054908290036115e6576115e663b562e8dd60e01b611471565b60008181526005602090815260408083206001600160a01b0387164260a01b6001881460e11b1781179091558084526006909252822080546801000000000000000186020190559081900361164457611644622e076360e81b611471565b818301825b808360007fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a4818160010191508103611649575060005550505050565b600980546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b604051630a85bd0160e11b81526000906001600160a01b0385169063150b7a029061171090339089908890889060040161204c565b6020604051808303816000875af192505050801561174b575060408051601f3d908101601f1916820190925261174891810190612089565b60015b6117a0573d808015611779576040519150601f19603f3d011682016040523d82523d6000602084013e61177e565b606091505b508051600003611798576117986368d2bf6b60e11b611471565b805181602001fd5b6001600160e01b031916630a85bd0160e11b149050949350505050565b60606004805461080a90611cfd565b606060a06040510180604052602081039150506000815280825b600183039250600a81066030018353600a9004806117e65750819003601f19909101908152919050565b600081815b84518110156118555761184182868381518110611834576118346120a6565b602002602001015161185d565b91508061184d816120bc565b915050611815565b509392505050565b60008183106118795760008281526020849052604090206112b4565b5060009182526020526040902090565b6001600160e01b031981168114610e4457600080fd5b6000602082840312156118b157600080fd5b81356112b481611889565b80356001600160a01b038116811461146c57600080fd5b6000602082840312156118e557600080fd5b6112b4826118bc565b6000806040838503121561190157600080fd5b50508035926020909101359150565b60005b8381101561192b578181015183820152602001611913565b50506000910152565b6000815180845261194c816020860160208601611910565b601f01601f19169290920160200192915050565b6020815260006112b46020830184611934565b60006020828403121561198557600080fd5b5035919050565b6000806040838503121561199f57600080fd5b6119a8836118bc565b946020939093013593505050565b6000806000606084860312156119cb57600080fd5b6119d4846118bc565b92506119e2602085016118bc565b9150604084013590509250925092565b60008083601f840112611a0457600080fd5b50813567ffffffffffffffff811115611a1c57600080fd5b6020830191508360208260051b8501011115611a3757600080fd5b9250929050565b60008060208385031215611a5157600080fd5b823567ffffffffffffffff811115611a6857600080fd5b611a74858286016119f2565b90969095509350505050565b600080600060408486031215611a9557600080fd5b83359250602084013567ffffffffffffffff811115611ab357600080fd5b611abf868287016119f2565b9497909650939450505050565b60008060208385031215611adf57600080fd5b823567ffffffffffffffff80821115611af757600080fd5b818501915085601f830112611b0b57600080fd5b813581811115611b1a57600080fd5b866020828501011115611b2c57600080fd5b60209290920196919550909350505050565b600080600060608486031215611b5357600080fd5b505081359360208301359350604090920135919050565b60008060008060808587031215611b8057600080fd5b5050823594602084013594506040840135936060013592509050565b60008060408385031215611baf57600080fd5b611bb8836118bc565b915060208301358015158114611bcd57600080fd5b809150509250929050565b634e487b7160e01b600052604160045260246000fd5b60008060008060808587031215611c0457600080fd5b611c0d856118bc565b9350611c1b602086016118bc565b925060408501359150606085013567ffffffffffffffff80821115611c3f57600080fd5b818701915087601f830112611c5357600080fd5b813581811115611c6557611c65611bd8565b604051601f8201601f19908116603f01168101908382118183101715611c8d57611c8d611bd8565b816040528281528a6020848701011115611ca657600080fd5b82602086016020830137600060208483010152809550505050505092959194509250565b60008060408385031215611cdd57600080fd5b611ce6836118bc565b9150611cf4602084016118bc565b90509250929050565b600181811c90821680611d1157607f821691505b602082108103611d3157634e487b7160e01b600052602260045260246000fd5b50919050565b60609190911b6bffffffffffffffffffffffff1916815260140190565b6020808252601f908201527f5265656e7472616e637947756172643a207265656e7472616e742063616c6c00604082015260600190565b634e487b7160e01b600052601160045260246000fd5b808201808211156107e2576107e2611d8b565b602080825260139082015272455843454544535f4d41585f535550504c592160681b604082015260600190565b80820281158282048414176107e2576107e2611d8b565b60208082526010908201526f494e434f52524543545f56414c55452160801b604082015260600190565b602080825260139082015272455843454544535f4d41585f5045525f54582160681b604082015260600190565b60208082526017908201527f455843454544535f4d41585f5045525f57414c4c455421000000000000000000604082015260600190565b601f821115610cc357600081815260208120601f850160051c81016020861015611ead5750805b601f850160051c820191505b81811015611ecc57828155600101611eb9565b505050505050565b67ffffffffffffffff831115611eec57611eec611bd8565b611f0083611efa8354611cfd565b83611e86565b6000601f841160018114611f345760008515611f1c5750838201355b600019600387901b1c1916600186901b178355611f8e565b600083815260209020601f19861690835b82811015611f655786850135825560209485019460019092019101611f45565b5086821015611f825760001960f88860031b161c19848701351681555b505060018560011b0183555b5050505050565b600084516020611fa88285838a01611910565b855191840191611fbb8184848a01611910565b8554920191600090611fcc81611cfd565b60018281168015611fe45760018114611ff957612025565b60ff1984168752821515830287019450612025565b896000528560002060005b8481101561201d57815489820152908301908701612004565b505082870194505b50929a9950505050505050505050565b60008161204457612044611d8b565b506000190190565b6001600160a01b038581168252841660208201526040810183905260806060820181905260009061207f90830184611934565b9695505050505050565b60006020828403121561209b57600080fd5b81516112b481611889565b634e487b7160e01b600052603260045260246000fd5b6000600182016120ce576120ce611d8b565b506001019056fea26469706673582212208894028f7ac0f5544a476324fd5a60017fa9bae2d3d1bb6be153646e8d3d0d7e64736f6c63430008130033

Deployed Bytecode Sourcemap

71975:10872:0:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;33773:689;;;;;;;;;;-1:-1:-1;33773:689:0;;;;;:::i;:::-;;:::i;:::-;;;565:14:1;;558:22;540:41;;528:2;513:18;33773:689:0;;;;;;;;76288:118;;;;;;;;;;-1:-1:-1;76288:118:0;;;;;:::i;:::-;-1:-1:-1;;;;;76377:21:0;76350:7;76377:21;;;:13;:21;;;;;;;76288:118;;;;1107:25:1;;;1095:2;1080:18;76288:118:0;961:177:1;79621:196:0;;;;;;;;;;-1:-1:-1;79621:196:0;;;;;:::i;:::-;;:::i;:::-;;34725:100;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;42270:290::-;;;;;;;;;;-1:-1:-1;42270:290:0;;;;;:::i;:::-;;:::i;:::-;;;-1:-1:-1;;;;;2501:32:1;;;2483:51;;2471:2;2456:18;42270:290:0;2337:203:1;41946:165:0;;;;;;:::i;:::-;;:::i;76515:99::-;;;;;;;;;;-1:-1:-1;76592:14:0;;76515:99;;76170:110;;;;;;;;;;-1:-1:-1;76170:110:0;;;;;:::i;:::-;-1:-1:-1;;;;;76255:17:0;76228:7;76255:17;;;:9;:17;;;;;;;76170:110;30289:323;;;;;;;;;;-1:-1:-1;30563:12:0;;30350:7;30547:13;:28;30289:323;;46190:3701;;;;;;:::i;:::-;;:::i;76851:258::-;;;;;;;;;;-1:-1:-1;76851:258:0;;;;;:::i;:::-;;:::i;80923:545::-;;;;;;:::i;:::-;;:::i;78648:122::-;;;;;;;;;;-1:-1:-1;78648:122:0;;;;;:::i;:::-;;:::i;81476:535::-;;;;;;:::i;:::-;;:::i;76414:93::-;;;;;;;;;;-1:-1:-1;76488:11:0;;76414:93;;78939:259;;;;;;;;;;-1:-1:-1;78939:259:0;;;;;:::i;:::-;;:::i;80048:109::-;;;;;;;;;;;;;:::i;49987:193::-;;;;;;:::i;:::-;;:::i;77395:344::-;;;;;;;;;;-1:-1:-1;77605:14:0;;77634:17;;77666:18;;77699:21;;77395:344;;;5610:25:1;;;5666:2;5651:18;;5644:34;;;;5694:18;;;5687:34;5752:2;5737:18;;5730:34;5597:3;5582:19;77395:344:0;5379:391:1;76622:89:0;;;;;;;;;;-1:-1:-1;76694:9:0;;76622:89;;76052:110;;;;;;;;;;-1:-1:-1;76052:110:0;;;;;:::i;:::-;-1:-1:-1;;;;;76137:17:0;76110:7;76137:17;;;:9;:17;;;;;;;76052:110;78441:89;;;;;;;;;;-1:-1:-1;78441:89:0;;;;;:::i;:::-;;:::i;36226:202::-;;;;;;;;;;-1:-1:-1;36226:202:0;;;;;:::i;:::-;;:::i;78538:102::-;;;;;;;;;;-1:-1:-1;78538:102:0;;;;;:::i;:::-;;:::i;31473:292::-;;;;;;;;;;-1:-1:-1;31473:292:0;;;;;:::i;:::-;;:::i;14293:103::-;;;;;;;;;;;;;:::i;79825:215::-;;;;;;;;;;-1:-1:-1;79825:215:0;;;;;:::i;:::-;;:::i;79206:407::-;;;;;;;;;;-1:-1:-1;79206:407:0;;;;;:::i;:::-;;:::i;80282:633::-;;;;;;:::i;:::-;;:::i;13645:87::-;;;;;;;;;;-1:-1:-1;13718:6:0;;-1:-1:-1;;;;;13718:6:0;13645:87;;34901:104;;;;;;;;;;;;;:::i;42900:266::-;;;;;;;;;;-1:-1:-1;42900:266:0;;;;;:::i;:::-;;:::i;50778:416::-;;;;;;:::i;:::-;;:::i;77117:270::-;;;;;;;;;;-1:-1:-1;77117:270:0;;;;;:::i;:::-;;:::i;76719:124::-;;;;;;;;;;-1:-1:-1;76802:12:0;;76816:18;;76719:124;;;8219:25:1;;;8275:2;8260:18;;8253:34;;;;8192:18;76719:124:0;8045:248:1;82366:478:0;;;;;;;;;;-1:-1:-1;82366:478:0;;;;;:::i;:::-;;:::i;43323:214::-;;;;;;;;;;-1:-1:-1;43323:214:0;;;;;:::i;:::-;-1:-1:-1;;;;;43494:25:0;;;43465:4;43494:25;;;:18;:25;;;;;;;;:35;;;;;;;;;;;;;;;43323:214;75689:355;;;;;;;;;;;;;:::i;78778:153::-;;;;;;;;;;-1:-1:-1;78778:153:0;;;;;:::i;:::-;;:::i;14551:201::-;;;;;;;;;;-1:-1:-1;14551:201:0;;;;;:::i;:::-;;:::i;77747:222::-;;;;;;;;;;-1:-1:-1;77925:7:0;;77934:13;;77949:11;;77747:222;;;8765:25:1;;;8821:2;8806:18;;8799:34;;;;8849:18;;;8842:34;8753:2;8738:18;77747:222:0;8563:319:1;33773:689:0;33903:4;-1:-1:-1;;;;;;;;;34232:25:0;;;;:102;;-1:-1:-1;;;;;;;;;;34309:25:0;;;34232:102;:179;;;-1:-1:-1;;;;;;;;;;34386:25:0;;;34232:179;34212:199;33773:689;-1:-1:-1;;33773:689:0:o;79621:196::-;13531:13;:11;:13::i;:::-;79740:14:::1;:32:::0;;;;79783:11:::1;:26:::0;79621:196::o;34725:100::-;34779:13;34812:5;34805:12;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;34725:100;:::o;42270:290::-;42391:7;42421:16;42429:7;42421;:16::i;:::-;42416:86;;42452:50;-1:-1:-1;;;42452:7:0;:50::i;:::-;-1:-1:-1;42522:24:0;;;;:15;:24;;;;;:30;-1:-1:-1;;;;;42522:30:0;;42270:290::o;41946:165::-;42076:27;42085:2;42089:7;42098:4;42076:8;:27::i;:::-;41946:165;;:::o;46190:3701::-;46332:27;46362;46381:7;46362:18;:27::i;:::-;-1:-1:-1;;;;;46517:22:0;;;;46332:57;;-1:-1:-1;46577:45:0;;;;46573:108;;46637:44;-1:-1:-1;;;46637:7:0;:44::i;:::-;46709:27;45298:24;;;:15;:24;;;;;45526:26;;68647:10;44923:30;;;-1:-1:-1;;;;;44616:28:0;;44901:20;;;44898:56;46918:296;;47101:43;47118:4;68647:10;43323:214;:::i;47101:43::-;47096:118;;47163:51;-1:-1:-1;;;47163:7:0;:51::i;:::-;47363:15;47360:160;;;47503:1;47482:19;47475:30;47360:160;-1:-1:-1;;;;;47900:24:0;;;;;;;:18;:24;;;;;;47898:26;;-1:-1:-1;;47898:26:0;;;47969:22;;;;;;;;;47967:24;;-1:-1:-1;47967:24:0;;;41002:11;40977:23;40973:41;40925:112;-1:-1:-1;;;40925:112:0;48262:26;;;;:17;:26;;;;;:196;;;;-1:-1:-1;;;48578:47:0;;:52;;48574:627;;48683:1;48673:11;;48651:19;48806:30;;;:17;:30;;;;;;:35;;48802:384;;48944:13;;48929:11;:28;48925:242;;49091:30;;;;:17;:30;;;;;:52;;;48925:242;48632:569;48574:627;-1:-1:-1;;;;;49333:20:0;;49713:7;49333:20;49643:4;49585:25;49314:16;;49450:299;49774:8;49786:1;49774:13;49770:58;;49789:39;-1:-1:-1;;;49789:7:0;:39::i;:::-;46321:3570;;;;46190:3701;;;:::o;76851:258::-;76956:4;76978:12;77020:10;77003:28;;;;;;;;:::i;:::-;;;;;;;;;;;;;76993:39;;;;;;76978:54;;77050:51;77069:11;;77050:51;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;77082:12:0;;;-1:-1:-1;77096:4:0;;-1:-1:-1;77050:18:0;:51::i;:::-;77043:58;76851:258;-1:-1:-1;;;;76851:258:0:o;80923:545::-;10570:1;11168:7;;:19;11160:63;;;;-1:-1:-1;;;11160:63:0;;;;;;;:::i;:::-;;;;;;;;;10570:1;11301:7;:18;81068:6;74478:27:::1;81068:6:::0;74508:14:::1;30765:7:::0;30956:13;;30710:296;74508:14:::1;:23;;;;:::i;:::-;74478:53;;74573:9;;74550:19;:32;;74542:64;;;;-1:-1:-1::0;;;74542:64:0::1;;;;;;;:::i;:::-;81105:6:::2;74690:13;74723:6;74706:14;;:23;;;;:::i;:::-;74690:39;;74778:6;74761:14;;:23;;;;:::i;:::-;74748:9;:36;74740:65;;;;-1:-1:-1::0;;;74740:65:0::2;;;;;;;:::i;:::-;81138:12:::3;;81152:11;;74219:12;74261:10;74244:28;;;;;;;;:::i;:::-;;;;;;;;;;;;;74234:39;;;;;;74219:54;;74306:49;74325:11;;74306:49;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;::::0;::::3;::::0;;;;-1:-1:-1;74338:10:0;;-1:-1:-1;74350:4:0;;-1:-1:-1;74306:18:0::3;::::0;-1:-1:-1;74306:49:0:i:3;:::-;74284:115;;;::::0;-1:-1:-1;;;74284:115:0;;11196:2:1;74284:115:0::3;::::0;::::3;11178:21:1::0;11235:2;11215:18;;;11208:30;-1:-1:-1;;;11254:18:1;;;11247:46;11310:18;;74284:115:0::3;10994:340:1::0;74284:115:0::3;81208:10:::4;81181:14;81198:21:::0;;;:9:::4;:21;::::0;;;;;:30:::4;::::0;81222:6;;81198:30:::4;:::i;:::-;81181:47;;81259:17;;81249:6;:27;;81241:59;;;;-1:-1:-1::0;;;81241:59:0::4;;;;;;;:::i;:::-;81329:21;;81319:6;:31;;81311:67;;;;-1:-1:-1::0;;;81311:67:0::4;;;;;;;:::i;:::-;81401:10;81391:21;::::0;;;:9:::4;:21;::::0;;;;:31;;81416:6;;81391:21;:31:::4;::::0;81416:6;;81391:31:::4;:::i;:::-;::::0;;;-1:-1:-1;81435:25:0::4;::::0;-1:-1:-1;81441:10:0::4;81453:6:::0;81435:5:::4;:25::i;:::-;-1:-1:-1::0;;10526:1:0;11480:7;:22;-1:-1:-1;;;;;;;;;;80923:545:0:o;78648:122::-;13531:13;:11;:13::i;:::-;78734:12:::1;:28;78749:13:::0;;78734:12;:28:::1;:::i;:::-;;78648:122:::0;;:::o;81476:535::-;10570:1;11168:7;;:19;11160:63;;;;-1:-1:-1;;;11160:63:0;;;;;;;:::i;:::-;10570:1;11301:7;:18;81593:6;74478:27:::1;81593:6:::0;74508:14:::1;30765:7:::0;30956:13;;30710:296;74508:14:::1;:23;;;;:::i;:::-;74478:53;;74573:9;;74550:19;:32;;74542:64;;;;-1:-1:-1::0;;;74542:64:0::1;;;;;;;:::i;:::-;81648:10:::2;81617:14;81634:25:::0;;;:13:::2;:25;::::0;;;;;:34:::2;::::0;81662:6;;81634:34:::2;:::i;:::-;81617:51;;81679:13;81709:6;81695:11;;:20;;;;:::i;:::-;81679:36;;81749:5;81736:9;:18;81728:47;;;;-1:-1:-1::0;;;81728:47:0::2;;;;;;;:::i;:::-;81804:14;;81794:6;:24;;81786:56;;;;-1:-1:-1::0;;;81786:56:0::2;;;;;;;:::i;:::-;81871:18;;81861:6;:28;;81853:64;;;;-1:-1:-1::0;;;81853:64:0::2;;;;;;;:::i;:::-;81944:10;81930:25;::::0;;;:13:::2;:25;::::0;;;;:35;;81959:6;;81930:25;:35:::2;::::0;81959:6;;81930:35:::2;:::i;:::-;::::0;;;-1:-1:-1;81978:25:0::2;::::0;-1:-1:-1;81984:10:0::2;81996:6:::0;81978:5:::2;:25::i;:::-;-1:-1:-1::0;;10526:1:0;11480:7;:22;-1:-1:-1;;;81476:535:0:o;78939:259::-;13531:13;:11;:13::i;:::-;79094:7:::1;:18:::0;;;;79123:11:::1;:26:::0;;;;79160:13:::1;:30:::0;78939:259::o;80048:109::-;13531:13;:11;:13::i;:::-;80098:51:::1;::::0;80106:10:::1;::::0;80127:21:::1;80098:51:::0;::::1;;;::::0;::::1;::::0;;;80127:21;80106:10;80098:51;::::1;;;;;;;;;;;;;::::0;::::1;;;;;;80048:109::o:0;49987:193::-;50133:39;50150:4;50156:2;50160:7;50133:39;;;;;;;;;;;;:16;:39::i;78441:89::-;13531:13;:11;:13::i;:::-;78512:4:::1;:10;78519:3:::0;;78512:4;:10:::1;:::i;36226:202::-:0;36343:7;36391:27;36410:7;36391:18;:27::i;78538:102::-;13531:13;:11;:13::i;:::-;78610:9:::1;:22:::0;78538:102::o;31473:292::-;31590:7;-1:-1:-1;;;;;31619:19:0;;31615:69;;31640:44;-1:-1:-1;;;31640:7:0;:44::i;:::-;-1:-1:-1;;;;;;31702:25:0;;;;;:18;:25;;;;;;25586:13;31702:55;;31473:292::o;14293:103::-;13531:13;:11;:13::i;:::-;14358:30:::1;14385:1;14358:18;:30::i;:::-;14293:103::o:0;79825:215::-;13531:13;:11;:13::i;:::-;79953:12:::1;:28:::0;;;;79992:18:::1;:40:::0;79825:215::o;79206:407::-;13531:13;:11;:13::i;:::-;79416:14:::1;:32:::0;;;;79459:17:::1;:38:::0;;;;79508:18:::1;:40:::0;79559:21:::1;:46:::0;79206:407::o;80282:633::-;10570:1;11168:7;;:19;11160:63;;;;-1:-1:-1;;;11160:63:0;;;;;;;:::i;:::-;10570:1;11301:7;:18;80433:6;74478:27:::1;80433:6:::0;74508:14:::1;30765:7:::0;30956:13;;30710:296;74508:14:::1;:23;;;;:::i;:::-;74478:53;;74573:9;;74550:19;:32;;74542:64;;;;-1:-1:-1::0;;;74542:64:0::1;;;;;;;:::i;:::-;80470:6:::2;74690:13;74723:6;74706:14;;:23;;;;:::i;:::-;74690:39;;74778:6;74761:14;;:23;;;;:::i;:::-;74748:9;:36;74740:65;;;;-1:-1:-1::0;;;74740:65:0::2;;;;;;;:::i;:::-;80503:18:::3;;80523:11;;74219:12;74261:10;74244:28;;;;;;;;:::i;:::-;;;;;;;;;;;;;74234:39;;;;;;74219:54;;74306:49;74325:11;;74306:49;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;::::0;::::3;::::0;;;;-1:-1:-1;74338:10:0;;-1:-1:-1;74350:4:0;;-1:-1:-1;74306:18:0::3;::::0;-1:-1:-1;74306:49:0:i:3;:::-;74284:115;;;::::0;-1:-1:-1;;;74284:115:0;;11196:2:1;74284:115:0::3;::::0;::::3;11178:21:1::0;11235:2;11215:18;;;11208:30;-1:-1:-1;;;11254:18:1;;;11247:46;11310:18;;74284:115:0::3;10994:340:1::0;74284:115:0::3;80579:10:::4;80552:14;80569:21:::0;;;:9:::4;:21;::::0;;;;;:30:::4;::::0;80593:6;;80569:30:::4;:::i;:::-;80552:47;;80630:17;;80620:6;:27;;80612:59;;;;-1:-1:-1::0;;;80612:59:0::4;;;;;;;:::i;:::-;80720:6;80703:14;;:23;;;;:::i;:::-;80690:9;:36;80682:65;;;;-1:-1:-1::0;;;80682:65:0::4;;;;;;;:::i;:::-;80776:21;;80766:6;:31;;80758:67;;;;-1:-1:-1::0;;;80758:67:0::4;;;;;;;:::i;:::-;80848:10;80838:21;::::0;;;:9:::4;:21;::::0;;;;:31;;80863:6;;80838:21;:31:::4;::::0;80863:6;;80838:31:::4;:::i;34901:104::-:0;34957:13;34990:7;34983:14;;;;;:::i;42900:266::-;68647:10;43027:39;;;;:18;:39;;;;;;;;-1:-1:-1;;;;;43027:49:0;;;;;;;;;;;;:60;;-1:-1:-1;;43027:60:0;;;;;;;;;;43103:55;;540:41:1;;;43027:49:0;;68647:10;43103:55;;513:18:1;43103:55:0;;;;;;;42900:266;;:::o;50778:416::-;50953:31;50966:4;50972:2;50976:7;50953:12;:31::i;:::-;-1:-1:-1;;;;;50999:14:0;;;:19;50995:192;;51038:56;51069:4;51075:2;51079:7;51088:5;51038:30;:56::i;:::-;51033:154;;51115:56;-1:-1:-1;;;51115:7:0;:56::i;:::-;50778:416;;;;:::o;77117:270::-;77228:4;77250:12;77292:10;77275:28;;;;;;;;:::i;:::-;;;;;;;;;;;;;77265:39;;;;;;77250:54;;77322:57;77341:11;;77322:57;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;77354:18:0;;;-1:-1:-1;77374:4:0;;-1:-1:-1;77322:18:0;:57::i;82366:478::-;82484:13;82520:16;82528:7;82520;:16::i;:::-;82515:68;;82538:45;-1:-1:-1;;;82538:7:0;:45::i;:::-;82596:21;82620:10;:8;:10::i;:::-;82596:34;;82667:7;82661:21;82686:1;82661:26;:175;;;;;;;;;;;;;;;;;82753:7;82762:18;82772:7;82762:9;:18::i;:::-;82782:12;82736:59;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;82661:175;82641:195;82366:478;-1:-1:-1;;;82366:478:0:o;75689:355::-;75730:7;75772;;75754:15;:25;75750:286;;;-1:-1:-1;75788:1:0;;75689:355::o;75750:286::-;75828:7;;75809:15;:26;;:61;;;;;75857:13;;75839:15;:31;75809:61;75805:231;;;-1:-1:-1;75892:1:0;;75689:355::o;75805:231::-;75946:13;;75927:15;:32;;:65;;;;;75981:11;;75963:15;:29;75927:65;75909:127;;;-1:-1:-1;76011:1:0;;75689:355::o;75909:127::-;-1:-1:-1;76035:1:0;;75689:355::o;78778:153::-;13531:13;:11;:13::i;:::-;78874:6:::1;74478:27;74525:6;74508:14;30765:7:::0;30956:13;;30710:296;74508:14:::1;:23;;;;:::i;:::-;74478:53;;74573:9;;74550:19;:32;;74542:64;;;;-1:-1:-1::0;;;74542:64:0::1;;;;;;;:::i;:::-;78898:25:::2;78904:10;78916:6;78898:5;:25::i;14551:201::-:0;13531:13;:11;:13::i;:::-;-1:-1:-1;;;;;14640:22:0;::::1;14632:73;;;::::0;-1:-1:-1;;;14632:73:0;;15560:2:1;14632:73:0::1;::::0;::::1;15542:21:1::0;15599:2;15579:18;;;15572:30;15638:34;15618:18;;;15611:62;-1:-1:-1;;;15689:18:1;;;15682:36;15735:19;;14632:73:0::1;15358:402:1::0;14632:73:0::1;14716:28;14735:8;14716:18;:28::i;13810:132::-:0;13718:6;;-1:-1:-1;;;;;13718:6:0;68647:10;13874:23;13866:68;;;;-1:-1:-1;;;13866:68:0;;15967:2:1;13866:68:0;;;15949:21:1;;;15986:18;;;15979:30;16045:34;16025:18;;;16018:62;16097:18;;13866:68:0;15765:356:1;43795:409:0;43896:11;43986:13;;43976:7;:23;43972:214;;;44020:14;44053:60;-1:-1:-1;44070:26:0;;;;:17;:26;;;;;;;44060:42;;;44053:60;;44104:9;;;:::i;:::-;;;44053:60;;;-1:-1:-1;;;44141:24:0;:29;;-1:-1:-1;43972:214:0;43795:409;;;:::o;70620:165::-;70721:13;70715:4;70708:27;70762:4;70756;70749:18;61793:474;61922:13;61938:16;61946:7;61938;:16::i;:::-;61922:32;;61971:13;:45;;;;-1:-1:-1;68647:10:0;-1:-1:-1;;;;;61988:28:0;;;;61971:45;61967:201;;;62036:44;62053:5;68647:10;43323:214;:::i;62036:44::-;62031:137;;62101:51;-1:-1:-1;;;62101:7:0;:51::i;:::-;62180:24;;;;:15;:24;;;;;;:35;;-1:-1:-1;;;;;;62180:35:0;-1:-1:-1;;;;;62180:35:0;;;;;;;;;62231:28;;62180:24;;62231:28;;;;;;;61911:356;61793:474;;;:::o;37879:2065::-;38061:26;;;;:17;:26;;;;;;;38187:11;;;38183:1313;;38234:13;;38223:7;:24;38219:98;;38270:47;-1:-1:-1;;;38270:7:0;:47::i;:::-;38874:607;-1:-1:-1;;;38970:9:0;38952:28;;;;:17;:28;;;;;;39026:25;;38874:607;39026:25;-1:-1:-1;;;39078:6:0;:24;39106:1;39078:29;39074:48;;37879:2065;;;:::o;39074:48::-;39414:47;-1:-1:-1;;;39414:7:0;:47::i;:::-;38874:607;;38183:1313;-1:-1:-1;;;39823:6:0;:24;39851:1;39823:29;39819:48;;37879:2065;;;:::o;39819:48::-;39889:47;-1:-1:-1;;;39889:7:0;:47::i;1252:190::-;1377:4;1430;1401:25;1414:5;1421:4;1401:12;:25::i;:::-;:33;;1252:190;-1:-1:-1;;;;1252:190:0:o;54546:2360::-;54619:20;54642:13;;;54670;;;54666:53;;54685:34;-1:-1:-1;;;54685:7:0;:34::i;:::-;55232:31;;;;:17;:31;;;;;;;;-1:-1:-1;;;;;40793:28:0;;41002:11;40977:23;40973:41;41492:1;41479:15;;41453:24;41449:46;40970:52;40925:112;;55232:194;;;55644:22;;;:18;:22;;;;;:105;;55716:32;55687:62;;55644:105;;;40793:28;55939:13;;;55935:54;;55954:35;-1:-1:-1;;;55954:7:0;:35::i;:::-;56020:23;;;:12;56105:676;56524:7;56480:8;56435:1;56369:25;56306:1;56241;56210:358;56776:3;56763:9;;;;;;:16;56105:676;;-1:-1:-1;56797:13:0;:19;-1:-1:-1;78734:28:0::1;78648:122:::0;;:::o;14912:191::-;15005:6;;;-1:-1:-1;;;;;15022:17:0;;;-1:-1:-1;;;;;;15022:17:0;;;;;;;15055:40;;15005:6;;;15022:17;15005:6;;15055:40;;14986:16;;15055:40;14975:128;14912:191;:::o;53278:806::-;53475:171;;-1:-1:-1;;;53475:171:0;;53441:4;;-1:-1:-1;;;;;53475:45:0;;;;;:171;;68647:10;;53577:4;;53600:7;;53626:5;;53475:171;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;-1:-1:-1;53475:171:0;;;;;;;;-1:-1:-1;;53475:171:0;;;;;;;;;;;;:::i;:::-;;;53458:619;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;53860:6;:13;53877:1;53860:18;53856:115;;53899:56;-1:-1:-1;;;53899:7:0;:56::i;:::-;54043:6;54037:13;54028:6;54024:2;54020:15;54013:38;53458:619;-1:-1:-1;;;;;;53719:81:0;-1:-1:-1;;;53719:81:0;;-1:-1:-1;53278:806:0;;;;;;:::o;35787:96::-;35838:13;35871:4;35864:11;;;;;:::i;68767:1786::-;68868:17;69307:4;69300;69294:11;69290:22;69399:1;69393:4;69386:15;69474:4;69471:1;69467:12;69460:19;;;69556:1;69551:3;69544:14;69660:3;69899:5;69881:428;69947:1;69942:3;69938:11;69931:18;;70118:2;70112:4;70108:13;70104:2;70100:22;70095:3;70087:36;70212:2;70202:13;;70269:25;69881:428;70269:25;-1:-1:-1;70339:13:0;;;-1:-1:-1;;70454:14:0;;;70516:19;;;70454:14;68767:1786;-1:-1:-1;68767:1786:0:o;2119:296::-;2202:7;2245:4;2202:7;2260:118;2284:5;:12;2280:1;:16;2260:118;;;2333:33;2343:12;2357:5;2363:1;2357:8;;;;;;;;:::i;:::-;;;;;;;2333:9;:33::i;:::-;2318:48;-1:-1:-1;2298:3:0;;;;:::i;:::-;;;;2260:118;;;-1:-1:-1;2395:12:0;2119:296;-1:-1:-1;;;2119:296:0:o;8326:149::-;8389:7;8420:1;8416;:5;:51;;8551:13;8645:15;;;8681:4;8674:15;;;8728:4;8712:21;;8416:51;;;-1:-1:-1;8551:13:0;8645:15;;;8681:4;8674:15;8728:4;8712:21;;;8326:149::o;14:131:1:-;-1:-1:-1;;;;;;88:32:1;;78:43;;68:71;;135:1;132;125:12;150:245;208:6;261:2;249:9;240:7;236:23;232:32;229:52;;;277:1;274;267:12;229:52;316:9;303:23;335:30;359:5;335:30;:::i;592:173::-;660:20;;-1:-1:-1;;;;;709:31:1;;699:42;;689:70;;755:1;752;745:12;770:186;829:6;882:2;870:9;861:7;857:23;853:32;850:52;;;898:1;895;888:12;850:52;921:29;940:9;921:29;:::i;1143:248::-;1211:6;1219;1272:2;1260:9;1251:7;1247:23;1243:32;1240:52;;;1288:1;1285;1278:12;1240:52;-1:-1:-1;;1311:23:1;;;1381:2;1366:18;;;1353:32;;-1:-1:-1;1143:248:1:o;1396:250::-;1481:1;1491:113;1505:6;1502:1;1499:13;1491:113;;;1581:11;;;1575:18;1562:11;;;1555:39;1527:2;1520:10;1491:113;;;-1:-1:-1;;1638:1:1;1620:16;;1613:27;1396:250::o;1651:271::-;1693:3;1731:5;1725:12;1758:6;1753:3;1746:19;1774:76;1843:6;1836:4;1831:3;1827:14;1820:4;1813:5;1809:16;1774:76;:::i;:::-;1904:2;1883:15;-1:-1:-1;;1879:29:1;1870:39;;;;1911:4;1866:50;;1651:271;-1:-1:-1;;1651:271:1:o;1927:220::-;2076:2;2065:9;2058:21;2039:4;2096:45;2137:2;2126:9;2122:18;2114:6;2096:45;:::i;2152:180::-;2211:6;2264:2;2252:9;2243:7;2239:23;2235:32;2232:52;;;2280:1;2277;2270:12;2232:52;-1:-1:-1;2303:23:1;;2152:180;-1:-1:-1;2152:180:1:o;2545:254::-;2613:6;2621;2674:2;2662:9;2653:7;2649:23;2645:32;2642:52;;;2690:1;2687;2680:12;2642:52;2713:29;2732:9;2713:29;:::i;:::-;2703:39;2789:2;2774:18;;;;2761:32;;-1:-1:-1;;;2545:254:1:o;2804:328::-;2881:6;2889;2897;2950:2;2938:9;2929:7;2925:23;2921:32;2918:52;;;2966:1;2963;2956:12;2918:52;2989:29;3008:9;2989:29;:::i;:::-;2979:39;;3037:38;3071:2;3060:9;3056:18;3037:38;:::i;:::-;3027:48;;3122:2;3111:9;3107:18;3094:32;3084:42;;2804:328;;;;;:::o;3137:367::-;3200:8;3210:6;3264:3;3257:4;3249:6;3245:17;3241:27;3231:55;;3282:1;3279;3272:12;3231:55;-1:-1:-1;3305:20:1;;3348:18;3337:30;;3334:50;;;3380:1;3377;3370:12;3334:50;3417:4;3409:6;3405:17;3393:29;;3477:3;3470:4;3460:6;3457:1;3453:14;3445:6;3441:27;3437:38;3434:47;3431:67;;;3494:1;3491;3484:12;3431:67;3137:367;;;;;:::o;3509:437::-;3595:6;3603;3656:2;3644:9;3635:7;3631:23;3627:32;3624:52;;;3672:1;3669;3662:12;3624:52;3712:9;3699:23;3745:18;3737:6;3734:30;3731:50;;;3777:1;3774;3767:12;3731:50;3816:70;3878:7;3869:6;3858:9;3854:22;3816:70;:::i;:::-;3905:8;;3790:96;;-1:-1:-1;3509:437:1;-1:-1:-1;;;;3509:437:1:o;3951:505::-;4046:6;4054;4062;4115:2;4103:9;4094:7;4090:23;4086:32;4083:52;;;4131:1;4128;4121:12;4083:52;4167:9;4154:23;4144:33;;4228:2;4217:9;4213:18;4200:32;4255:18;4247:6;4244:30;4241:50;;;4287:1;4284;4277:12;4241:50;4326:70;4388:7;4379:6;4368:9;4364:22;4326:70;:::i;:::-;3951:505;;4415:8;;-1:-1:-1;4300:96:1;;-1:-1:-1;;;;3951:505:1:o;4461:592::-;4532:6;4540;4593:2;4581:9;4572:7;4568:23;4564:32;4561:52;;;4609:1;4606;4599:12;4561:52;4649:9;4636:23;4678:18;4719:2;4711:6;4708:14;4705:34;;;4735:1;4732;4725:12;4705:34;4773:6;4762:9;4758:22;4748:32;;4818:7;4811:4;4807:2;4803:13;4799:27;4789:55;;4840:1;4837;4830:12;4789:55;4880:2;4867:16;4906:2;4898:6;4895:14;4892:34;;;4922:1;4919;4912:12;4892:34;4967:7;4962:2;4953:6;4949:2;4945:15;4941:24;4938:37;4935:57;;;4988:1;4985;4978:12;4935:57;5019:2;5011:11;;;;;5041:6;;-1:-1:-1;4461:592:1;;-1:-1:-1;;;;4461:592:1:o;5058:316::-;5135:6;5143;5151;5204:2;5192:9;5183:7;5179:23;5175:32;5172:52;;;5220:1;5217;5210:12;5172:52;-1:-1:-1;;5243:23:1;;;5313:2;5298:18;;5285:32;;-1:-1:-1;5364:2:1;5349:18;;;5336:32;;5058:316;-1:-1:-1;5058:316:1:o;6028:385::-;6114:6;6122;6130;6138;6191:3;6179:9;6170:7;6166:23;6162:33;6159:53;;;6208:1;6205;6198:12;6159:53;-1:-1:-1;;6231:23:1;;;6301:2;6286:18;;6273:32;;-1:-1:-1;6352:2:1;6337:18;;6324:32;;6403:2;6388:18;6375:32;;-1:-1:-1;6028:385:1;-1:-1:-1;6028:385:1:o;6418:347::-;6483:6;6491;6544:2;6532:9;6523:7;6519:23;6515:32;6512:52;;;6560:1;6557;6550:12;6512:52;6583:29;6602:9;6583:29;:::i;:::-;6573:39;;6662:2;6651:9;6647:18;6634:32;6709:5;6702:13;6695:21;6688:5;6685:32;6675:60;;6731:1;6728;6721:12;6675:60;6754:5;6744:15;;;6418:347;;;;;:::o;6770:127::-;6831:10;6826:3;6822:20;6819:1;6812:31;6862:4;6859:1;6852:15;6886:4;6883:1;6876:15;6902:1138;6997:6;7005;7013;7021;7074:3;7062:9;7053:7;7049:23;7045:33;7042:53;;;7091:1;7088;7081:12;7042:53;7114:29;7133:9;7114:29;:::i;:::-;7104:39;;7162:38;7196:2;7185:9;7181:18;7162:38;:::i;:::-;7152:48;;7247:2;7236:9;7232:18;7219:32;7209:42;;7302:2;7291:9;7287:18;7274:32;7325:18;7366:2;7358:6;7355:14;7352:34;;;7382:1;7379;7372:12;7352:34;7420:6;7409:9;7405:22;7395:32;;7465:7;7458:4;7454:2;7450:13;7446:27;7436:55;;7487:1;7484;7477:12;7436:55;7523:2;7510:16;7545:2;7541;7538:10;7535:36;;;7551:18;;:::i;:::-;7626:2;7620:9;7594:2;7680:13;;-1:-1:-1;;7676:22:1;;;7700:2;7672:31;7668:40;7656:53;;;7724:18;;;7744:22;;;7721:46;7718:72;;;7770:18;;:::i;:::-;7810:10;7806:2;7799:22;7845:2;7837:6;7830:18;7885:7;7880:2;7875;7871;7867:11;7863:20;7860:33;7857:53;;;7906:1;7903;7896:12;7857:53;7962:2;7957;7953;7949:11;7944:2;7936:6;7932:15;7919:46;8007:1;8002:2;7997;7989:6;7985:15;7981:24;7974:35;8028:6;8018:16;;;;;;;6902:1138;;;;;;;:::o;8298:260::-;8366:6;8374;8427:2;8415:9;8406:7;8402:23;8398:32;8395:52;;;8443:1;8440;8433:12;8395:52;8466:29;8485:9;8466:29;:::i;:::-;8456:39;;8514:38;8548:2;8537:9;8533:18;8514:38;:::i;:::-;8504:48;;8298:260;;;;;:::o;8887:380::-;8966:1;8962:12;;;;9009;;;9030:61;;9084:4;9076:6;9072:17;9062:27;;9030:61;9137:2;9129:6;9126:14;9106:18;9103:38;9100:161;;9183:10;9178:3;9174:20;9171:1;9164:31;9218:4;9215:1;9208:15;9246:4;9243:1;9236:15;9100:161;;8887:380;;;:::o;9272:229::-;9421:2;9417:15;;;;-1:-1:-1;;9413:53:1;9401:66;;9492:2;9483:12;;9272:229::o;9506:355::-;9708:2;9690:21;;;9747:2;9727:18;;;9720:30;9786:33;9781:2;9766:18;;9759:61;9852:2;9837:18;;9506:355::o;9866:127::-;9927:10;9922:3;9918:20;9915:1;9908:31;9958:4;9955:1;9948:15;9982:4;9979:1;9972:15;9998:125;10063:9;;;10084:10;;;10081:36;;;10097:18;;:::i;10128:343::-;10330:2;10312:21;;;10369:2;10349:18;;;10342:30;-1:-1:-1;;;10403:2:1;10388:18;;10381:49;10462:2;10447:18;;10128:343::o;10476:168::-;10549:9;;;10580;;10597:15;;;10591:22;;10577:37;10567:71;;10618:18;;:::i;10649:340::-;10851:2;10833:21;;;10890:2;10870:18;;;10863:30;-1:-1:-1;;;10924:2:1;10909:18;;10902:46;10980:2;10965:18;;10649:340::o;11339:343::-;11541:2;11523:21;;;11580:2;11560:18;;;11553:30;-1:-1:-1;;;11614:2:1;11599:18;;11592:49;11673:2;11658:18;;11339:343::o;11687:347::-;11889:2;11871:21;;;11928:2;11908:18;;;11901:30;11967:25;11962:2;11947:18;;11940:53;12025:2;12010:18;;11687:347::o;12165:545::-;12267:2;12262:3;12259:11;12256:448;;;12303:1;12328:5;12324:2;12317:17;12373:4;12369:2;12359:19;12443:2;12431:10;12427:19;12424:1;12420:27;12414:4;12410:38;12479:4;12467:10;12464:20;12461:47;;;-1:-1:-1;12502:4:1;12461:47;12557:2;12552:3;12548:12;12545:1;12541:20;12535:4;12531:31;12521:41;;12612:82;12630:2;12623:5;12620:13;12612:82;;;12675:17;;;12656:1;12645:13;12612:82;;;12616:3;;;12165:545;;;:::o;12886:1206::-;13010:18;13005:3;13002:27;12999:53;;;13032:18;;:::i;:::-;13061:94;13151:3;13111:38;13143:4;13137:11;13111:38;:::i;:::-;13105:4;13061:94;:::i;:::-;13181:1;13206:2;13201:3;13198:11;13223:1;13218:616;;;;13878:1;13895:3;13892:93;;;-1:-1:-1;13951:19:1;;;13938:33;13892:93;-1:-1:-1;;12843:1:1;12839:11;;;12835:24;12831:29;12821:40;12867:1;12863:11;;;12818:57;13998:78;;13191:895;;13218:616;12112:1;12105:14;;;12149:4;12136:18;;-1:-1:-1;;13254:17:1;;;13355:9;13377:229;13391:7;13388:1;13385:14;13377:229;;;13480:19;;;13467:33;13452:49;;13587:4;13572:20;;;;13540:1;13528:14;;;;13407:12;13377:229;;;13381:3;13634;13625:7;13622:16;13619:159;;;13758:1;13754:6;13748:3;13742;13739:1;13735:11;13731:21;13727:34;13723:39;13710:9;13705:3;13701:19;13688:33;13684:79;13676:6;13669:95;13619:159;;;13821:1;13815:3;13812:1;13808:11;13804:19;13798:4;13791:33;13191:895;;;12886:1206;;;:::o;14097:1256::-;14321:3;14359:6;14353:13;14385:4;14398:64;14455:6;14450:3;14445:2;14437:6;14433:15;14398:64;:::i;:::-;14525:13;;14484:16;;;;14547:68;14525:13;14484:16;14582:15;;;14547:68;:::i;:::-;14704:13;;14637:20;;;14677:1;;14742:36;14704:13;14742:36;:::i;:::-;14797:1;14814:18;;;14841:141;;;;14996:1;14991:337;;;;14807:521;;14841:141;-1:-1:-1;;14876:24:1;;14862:39;;14953:16;;14946:24;14932:39;;14921:51;;;-1:-1:-1;14841:141:1;;14991:337;15022:6;15019:1;15012:17;15070:2;15067:1;15057:16;15095:1;15109:169;15123:8;15120:1;15117:15;15109:169;;;15205:14;;15190:13;;;15183:37;15248:16;;;;15140:10;;15109:169;;;15113:3;;15309:8;15302:5;15298:20;15291:27;;14807:521;-1:-1:-1;15344:3:1;;14097:1256;-1:-1:-1;;;;;;;;;;14097:1256:1:o;16126:136::-;16165:3;16193:5;16183:39;;16202:18;;:::i;:::-;-1:-1:-1;;;16238:18:1;;16126:136::o;16267:489::-;-1:-1:-1;;;;;16536:15:1;;;16518:34;;16588:15;;16583:2;16568:18;;16561:43;16635:2;16620:18;;16613:34;;;16683:3;16678:2;16663:18;;16656:31;;;16461:4;;16704:46;;16730:19;;16722:6;16704:46;:::i;:::-;16696:54;16267:489;-1:-1:-1;;;;;;16267:489:1:o;16761:249::-;16830:6;16883:2;16871:9;16862:7;16858:23;16854:32;16851:52;;;16899:1;16896;16889:12;16851:52;16931:9;16925:16;16950:30;16974:5;16950:30;:::i;17015:127::-;17076:10;17071:3;17067:20;17064:1;17057:31;17107:4;17104:1;17097:15;17131:4;17128:1;17121:15;17147:135;17186:3;17207:17;;;17204:43;;17227:18;;:::i;:::-;-1:-1:-1;17274:1:1;17263:13;;17147:135::o

Swarm Source

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