ETH Price: $3,445.28 (-1.02%)
Gas: 12 Gwei

Token

DemonParty (DEMONS)
 

Overview

Max Total Supply

240 DEMONS

Holders

112

Market

Volume (24H)

N/A

Min Price (24H)

N/A

Max Price (24H)

N/A

Other Info

Balance
3 DEMONS
0x0b47b1ec9d415d88d4de4577c82f66d904d2c4d3
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:
DemonParty

Compiler Version
v0.8.6+commit.11564f7e

Optimization Enabled:
Yes with 200 runs

Other Settings:
default evmVersion, MIT license

Contract Source Code (Solidity)

/**
 *Submitted for verification at Etherscan.io on 2022-06-14
*/

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


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

pragma solidity ^0.8.0;

/**
 * @dev These functions deal with verification of Merkle Trees 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 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++) {
            bytes32 proofElement = proof[i];
            if (computedHash <= proofElement) {
                // Hash(current computed hash + current element of the proof)
                computedHash = _efficientHash(computedHash, proofElement);
            } else {
                // Hash(current element of the proof + current computed hash)
                computedHash = _efficientHash(proofElement, computedHash);
            }
        }
        return computedHash;
    }

    function _efficientHash(bytes32 a, bytes32 b) private pure returns (bytes32 value) {
        assembly {
            mstore(0x00, a)
            mstore(0x20, b)
            value := keccak256(0x00, 0x40)
        }
    }
}

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


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

pragma solidity ^0.8.0;

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

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

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

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

    /**
     * @dev Converts a `uint256` to its ASCII `string` hexadecimal representation with fixed length.
     */
    function toHexString(uint256 value, uint256 length) internal pure returns (string memory) {
        bytes memory buffer = new bytes(2 * length + 2);
        buffer[0] = "0";
        buffer[1] = "x";
        for (uint256 i = 2 * length + 1; i > 1; --i) {
            buffer[i] = _HEX_SYMBOLS[value & 0xf];
            value >>= 4;
        }
        require(value == 0, "Strings: hex length insufficient");
        return string(buffer);
    }
}

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


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

pragma solidity ^0.8.0;

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

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

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


// OpenZeppelin Contracts v4.4.1 (access/Ownable.sol)

pragma solidity ^0.8.0;


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

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

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

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

    /**
     * @dev Throws if called by any account other than the owner.
     */
    modifier onlyOwner() {
        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/IERC721A.sol


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

pragma solidity ^0.8.4;

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

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

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

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

    struct TokenOwnership {
        // The address of the owner.
        address addr;
        // Keeps track of the start time of ownership with minimal overhead for tokenomics.
        uint64 startTimestamp;
        // Whether the token has been burned.
        bool burned;
    }

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

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

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

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

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

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

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

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

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

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

    // ==============================
    //        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);
}
// File: contracts/ERC721A.sol


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

pragma solidity ^0.8.4;


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

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

    // The number of tokens burned.
    uint256 private _burnCounter;

    // Token name
    string private _name;

    // Token symbol
    string private _symbol;

    // Mapping from token ID to ownership details
    // An empty struct value does not necessarily mean the token is unowned.
    // See `_packedOwnershipOf` implementation for details.
    //
    // Bits Layout:
    // - [0..159]   `addr`
    // - [160..223] `startTimestamp`
    // - [224]      `burned`
    // - [225]      `nextInitialized`
    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 => address) private _tokenApprovals;

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

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

    /**
     * @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 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 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 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 returns (uint256) {
        return _burnCounter;
    }

    /**
     * @dev See {IERC165-supportsInterface}.
     */
    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: 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.
    }

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

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

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

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

    /**
     * Sets the auxiliary data for `owner`. (e.g. number of whitelist mint slots used).
     * If there are multiple variables, please pack them into a uint64.
     */
    function _setAux(address owner, uint64 aux) internal {
        uint256 packed = _packedAddressData[owner];
        uint256 auxCasted;
        assembly {
            // Cast aux without masking.
            auxCasted := aux
        }
        packed = (packed & BITMASK_AUX_COMPLEMENT) | (auxCasted << BITPOS_AUX);
        _packedAddressData[owner] = packed;
    }

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

        unchecked {
            if (_startTokenId() <= curr)
                if (curr < _currentIndex) {
                    uint256 packed = _packedOwnerships[curr];
                    // If not burned.
                    if (packed & BITMASK_BURNED == 0) {
                        // Invariant:
                        // There will always be an ownership that has an address and is not burned
                        // before an ownership that does not have an address and is not burned.
                        // Hence, curr will not underflow.
                        //
                        // We can directly compare the packed value.
                        // If the address is zero, packed is zero.
                        while (packed == 0) {
                            packed = _packedOwnerships[--curr];
                        }
                        return packed;
                    }
                }
        }
        revert OwnerQueryForNonexistentToken();
    }

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

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

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

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

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

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

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

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

        string memory baseURI = _baseURI();
        return bytes(baseURI).length != 0 ? string(abi.encodePacked(baseURI, _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 '';
    }

    /**
     * @dev Casts the address to uint256 without masking.
     */
    function _addressToUint256(address value) private pure returns (uint256 result) {
        assembly {
            result := value
        }
    }

    /**
     * @dev Casts the boolean to uint256 without branching.
     */
    function _boolToUint256(bool value) private pure returns (uint256 result) {
        assembly {
            result := value
        }
    }

    /**
     * @dev See {IERC721-approve}.
     */
    function approve(address to, uint256 tokenId) public override {
        address owner = address(uint160(_packedOwnershipOf(tokenId)));

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

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

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

        return _tokenApprovals[tokenId];
    }

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

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

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

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

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

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

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

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

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

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

    /**
     * @dev 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 {
        uint256 startTokenId = _currentIndex;
        if (_addressToUint256(to) == 0) revert MintToZeroAddress();
        if (quantity == 0) revert MintZeroQuantity();

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

        // Overflows are incredibly unrealistic.
        // balance or numberMinted overflow if current value of either + quantity > 1.8e19 (2**64) - 1
        // updatedIndex overflows if _currentIndex + quantity > 1.2e77 (2**256) - 1
        unchecked {
            // Updates:
            // - `balance += quantity`.
            // - `numberMinted += quantity`.
            //
            // We can directly add to the balance and number minted.
            _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] =
                _addressToUint256(to) |
                (block.timestamp << BITPOS_START_TIMESTAMP) |
                (_boolToUint256(quantity == 1) << BITPOS_NEXT_INITIALIZED);

            uint256 offset;
            do {
                emit Transfer(address(0), to, startTokenId + offset++);
            } while (offset < quantity);

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

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

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

        address approvedAddress = _tokenApprovals[tokenId];

        bool isApprovedOrOwner = (_msgSenderERC721A() == from ||
            isApprovedForAll(from, _msgSenderERC721A()) ||
            approvedAddress == _msgSenderERC721A());

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

        _beforeTokenTransfers(from, to, tokenId, 1);

        // Clear approvals from the previous owner.
        if (_addressToUint256(approvedAddress) != 0) {
            delete _tokenApprovals[tokenId];
        }

        // 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] =
                _addressToUint256(to) |
                (block.timestamp << BITPOS_START_TIMESTAMP) |
                BITMASK_NEXT_INITIALIZED;

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

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

    /**
     * @dev Equivalent to `_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));
        address approvedAddress = _tokenApprovals[tokenId];

        if (approvalCheck) {
            bool isApprovedOrOwner = (_msgSenderERC721A() == from ||
                isApprovedForAll(from, _msgSenderERC721A()) ||
                approvedAddress == _msgSenderERC721A());

            if (!isApprovedOrOwner) revert TransferCallerNotOwnerNorApproved();
        }

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

        // Clear approvals from the previous owner.
        if (_addressToUint256(approvedAddress) != 0) {
            delete _tokenApprovals[tokenId];
        }

        // 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] =
                _addressToUint256(from) |
                (block.timestamp << BITPOS_START_TIMESTAMP) |
                BITMASK_BURNED |
                BITMASK_NEXT_INITIALIZED;

            // 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++;
        }
    }

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

    /**
     * @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 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 returns (string memory ptr) {
        assembly {
            // The maximum value of a uint256 contains 78 digits (1 byte per digit),
            // but we allocate 128 bytes to keep the free memory pointer 32-byte word aliged.
            // We will need 1 32-byte word to store the length,
            // and 3 32-byte words to store a maximum of 78 digits. Total: 32 + 3 * 32 = 128.
            ptr := add(mload(0x40), 128)
            // Update the free memory pointer to allocate.
            mstore(0x40, ptr)

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

            // We write the string from the rightmost digit to the leftmost digit.
            // The following is essentially a do-while loop that also handles the zero case.
            // Costs a bit more than early returning for the zero case,
            // but cheaper in terms of deployment and overall runtime costs.
            for {
                // Initialize and perform the first pass without check.
                let temp := value
                // Move the pointer 1 byte leftwards to point to an empty character slot.
                ptr := sub(ptr, 1)
                // Write the character to the pointer. 48 is the ASCII index of '0'.
                mstore8(ptr, add(48, mod(temp, 10)))
                temp := div(temp, 10)
            } temp {
                // Keep dividing `temp` until zero.
                temp := div(temp, 10)
            } {
                // Body of the for loop.
                ptr := sub(ptr, 1)
                mstore8(ptr, add(48, mod(temp, 10)))
            }

            let length := sub(end, ptr)
            // Move the pointer 32 bytes leftwards to make room for the length.
            ptr := sub(ptr, 32)
            // Store the length.
            mstore(ptr, length)
        }
    }
}
// File: contracts/DemonParty.sol


pragma solidity ^0.8.6;





contract DemonParty is ERC721A, Ownable {
  
  uint public constant NFT_PRICE = 0.0666 ether;
  uint public constant MAX_WHITELIST_MINT = 3;
  uint public constant MAX_PUBLIC_MINT = 5;
  uint public MAX_SUPPLY = 4000;
  uint public SEASON_MAX = 1000;
  uint public SEASONAL_GIFTS = 0;

  bool public active = false;

  uint8 public CURRENT_SEASON = 1;

  string public baseURI;

  bytes32 public root;

  mapping (uint => mapping (address => uint)) public minters;

  constructor(string memory _baseURI) ERC721A("DemonParty", "DEMONS") {
    baseURI = _baseURI;
  }

  function mint(uint amount) public payable {
    require(active, "SALE_NOT_ACTIVE");
    require(amount * NFT_PRICE == msg.value, "WRONG_ETH_AMOUNT");
    require(_totalMinted() + amount <= SEASON_MAX, "SEASON_MAX_SUPPLY");

    minters[CURRENT_SEASON][msg.sender] += amount;
    require(minters[CURRENT_SEASON][msg.sender] <= MAX_PUBLIC_MINT, "ADDRESS_MAX_REACHED");

    _mint(msg.sender, amount);
  }

  function premint(address account, uint amount, uint discount, bytes32[] calldata proof) public payable {
    bytes32 leaf = keccak256(abi.encode(account, discount));
    require(MerkleProof.verify(proof, root, leaf), "INVALID_MERKLE_PROOF");

    uint price = amount * NFT_PRICE;
    if (minters[CURRENT_SEASON][account] == 0) {
      price -= discount;
    }

    require(msg.value == price, "WRONG_ETH_AMOUNT");
    require(_totalMinted() + amount <= SEASON_MAX, "SEASON_MAX_SUPPLY");

    minters[CURRENT_SEASON][account] += amount;
    require(minters[CURRENT_SEASON][account] <= MAX_WHITELIST_MINT, "ADDRESS_MAX_REACHED");

    _mint(account, amount);
  }

  function burn(uint id) public {
    _burn(id, true);
  }

  function setActive() public onlyOwner {
    active = !active;
  }

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

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

  function endMinting() public onlyOwner {
    MAX_SUPPLY = totalSupply();
  }

  function gift(address[] calldata receivers) external onlyOwner {
    require(_totalMinted() + receivers.length <= SEASON_MAX, "TOO_MANY_MINTS");

    SEASONAL_GIFTS += receivers.length;
    require(SEASONAL_GIFTS <= 100, "NO_MORE_GIFTS");

    for(uint i = 0; i < receivers.length; i++) {
      _mint(receivers[i], 1);
    }
  }

  function bumpSeason(uint newSupply) public onlyOwner {
    require(newSupply > totalSupply(), "SUPPLY_TOO_LOW");
    require(newSupply <= MAX_SUPPLY, "SUPPLY_TOO_HIGH");

    root = 0x0;
    CURRENT_SEASON += 1;
    SEASON_MAX = newSupply;
    SEASONAL_GIFTS = 0;
  }

  address internal payout1 = address(0x08D4bCe80056c95b1C9bc38fEC63901e3b563186); // 24.5%
  address internal payout2 = address(0x3ECB3a23e78fD8846f9fA96b88911dBd96031c85); // 19%
  address internal payout3 = address(0x3966638835B46E0A2e952F6F70F9Fa1e4f553E55); // 19%
  address internal payout4 = address(0xcdB417221225fa9B623A056a06B3b1E7860f1c50); // 19%
  address internal payout5 = address(0x8b88130e3B6d99aC05e382C17bD28dcaD2F86D41); // 15%
  address internal payout6 = address(0x5687ad526924123A4939928F22022e467828Ba1a); // 1%
  address internal payout7 = address(0x57092EaD84D25cc4123b96100d52baEF026987e9); // 1%
  address internal payout8 = address(0xf751F674843F5BF8802C6E373a2FD2fC0027cD85); // 1%
  address internal payout9 = address(0x4A505A49f25f5B24D7ac9504fDbf2dfADa49668d); // 0.5%

  function withdraw() public onlyOwner {
    uint balance = address(this).balance;
    uint amount24_5 = balance * 245 / 1000;
    uint amount19 = balance * 190 / 1000;
    uint amount15 = balance * 150 / 1000;
    uint amount1 = balance * 10 / 1000;
    uint amount0_5 = balance * 5 / 1000;

    (bool sent1, ) = payable(payout1).call{value: amount24_5}("");
    require(sent1, "Failed to send Ether1");
    (bool sent2, ) = payable(payout2).call{value: amount19}("");
    require(sent2, "Failed to send Ether2");
    (bool sent3, ) = payable(payout3).call{value: amount19}("");
    require(sent3, "Failed to send Ether3");
    (bool sent4, ) = payable(payout4).call{value: amount19}("");
    require(sent4, "Failed to send Ether4");
    (bool sent5, ) = payable(payout5).call{value: amount15}("");
    require(sent5, "Failed to send Ether5");
    (bool sent6, ) = payable(payout6).call{value: amount1}("");
    require(sent6, "Failed to send Ether6");
    (bool sent7, ) = payable(payout7).call{value: amount1}("");
    require(sent7, "Failed to send Ether7");
    (bool sent8, ) = payable(payout8).call{value: amount1}("");
    require(sent8, "Failed to send Ether8");
    (bool sent9, ) = payable(payout9).call{value: amount0_5}("");
    require(sent9, "Failed to send Ether9");
  }
}

Contract Security Audit

Contract ABI

[{"inputs":[{"internalType":"string","name":"_baseURI","type":"string"}],"stateMutability":"nonpayable","type":"constructor"},{"inputs":[],"name":"ApprovalCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"ApprovalQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"ApproveToCaller","type":"error"},{"inputs":[],"name":"BalanceQueryForZeroAddress","type":"error"},{"inputs":[],"name":"MintToZeroAddress","type":"error"},{"inputs":[],"name":"MintZeroQuantity","type":"error"},{"inputs":[],"name":"OwnerQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"TransferCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"TransferFromIncorrectOwner","type":"error"},{"inputs":[],"name":"TransferToNonERC721ReceiverImplementer","type":"error"},{"inputs":[],"name":"TransferToZeroAddress","type":"error"},{"inputs":[],"name":"URIQueryForNonexistentToken","type":"error"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"approved","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Approval","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"operator","type":"address"},{"indexed":false,"internalType":"bool","name":"approved","type":"bool"}],"name":"ApprovalForAll","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"previousOwner","type":"address"},{"indexed":true,"internalType":"address","name":"newOwner","type":"address"}],"name":"OwnershipTransferred","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Transfer","type":"event"},{"inputs":[],"name":"CURRENT_SEASON","outputs":[{"internalType":"uint8","name":"","type":"uint8"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"MAX_PUBLIC_MINT","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"MAX_SUPPLY","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"MAX_WHITELIST_MINT","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"NFT_PRICE","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"SEASONAL_GIFTS","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"SEASON_MAX","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"active","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"approve","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"}],"name":"balanceOf","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"baseURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"newSupply","type":"uint256"}],"name":"bumpSeason","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"id","type":"uint256"}],"name":"burn","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"endMinting","outputs":[],"stateMutability":"nonpayable","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":"receivers","type":"address[]"}],"name":"gift","outputs":[],"stateMutability":"nonpayable","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":"uint256","name":"amount","type":"uint256"}],"name":"mint","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"uint256","name":"","type":"uint256"},{"internalType":"address","name":"","type":"address"}],"name":"minters","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"name","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"owner","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"ownerOf","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"account","type":"address"},{"internalType":"uint256","name":"amount","type":"uint256"},{"internalType":"uint256","name":"discount","type":"uint256"},{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"}],"name":"premint","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"root","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"},{"internalType":"bytes","name":"_data","type":"bytes"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"setActive","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"operator","type":"address"},{"internalType":"bool","name":"approved","type":"bool"}],"name":"setApprovalForAll","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"uri","type":"string"}],"name":"setBaseURI","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"merkleRoot","type":"bytes32"}],"name":"setMerkleRoot","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"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":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"newOwner","type":"address"}],"name":"transferOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"withdraw","outputs":[],"stateMutability":"nonpayable","type":"function"}]

6080604052610fa06009556103e8600a556000600b55600c805461ffff1916610100179055601080546001600160a01b03199081167308d4bce80056c95b1c9bc38fec63901e3b56318617909155601180548216733ecb3a23e78fd8846f9fa96b88911dbd96031c85179055601280548216733966638835b46e0a2e952f6f70f9fa1e4f553e5517905560138054821673cdb417221225fa9b623a056a06b3b1e7860f1c50179055601480548216738b88130e3b6d99ac05e382c17bd28dcad2f86d41179055601580548216735687ad526924123a4939928f22022e467828ba1a1790556016805482167357092ead84d25cc4123b96100d52baef026987e917905560178054821673f751f674843f5bf8802c6e373a2fd2fc0027cd8517905560188054909116734a505a49f25f5b24d7ac9504fdbf2dfada49668d1790553480156200014b57600080fd5b5060405162002b0738038062002b078339810160408190526200016e91620002fb565b604080518082018252600a81526944656d6f6e506172747960b01b60208083019182528351808501909452600684526544454d4f4e5360d01b908401528151919291620001be9160029162000255565b508051620001d490600390602084019062000255565b50506000805550620001e63362000203565b8051620001fb90600d90602084019062000255565b50506200042a565b600880546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b8280546200026390620003d7565b90600052602060002090601f016020900481019282620002875760008555620002d2565b82601f10620002a257805160ff1916838001178555620002d2565b82800160010185558215620002d2579182015b82811115620002d2578251825591602001919060010190620002b5565b50620002e0929150620002e4565b5090565b5b80821115620002e05760008155600101620002e5565b600060208083850312156200030f57600080fd5b82516001600160401b03808211156200032757600080fd5b818501915085601f8301126200033c57600080fd5b81518181111562000351576200035162000414565b604051601f8201601f19908116603f011681019083821181831017156200037c576200037c62000414565b8160405282815288868487010111156200039557600080fd5b600093505b82841015620003b957848401860151818501870152928501926200039a565b82841115620003cb5760008684830101525b98975050505050505050565b600181811c90821680620003ec57607f821691505b602082108114156200040e57634e487b7160e01b600052602260045260246000fd5b50919050565b634e487b7160e01b600052604160045260246000fd5b6126cd806200043a6000396000f3fe6080604052600436106102255760003560e01c806370a0823111610123578063a72c41cf116100ab578063e942bdd21161006f578063e942bdd2146105fd578063e985e9c514610635578063ebf0c7171461067e578063ef70aebf14610694578063f2fde38b146106a957600080fd5b8063a72c41cf14610561578063b88d4fde14610577578063c08dfd3c14610597578063c20deccf146105ac578063c87b56dd146105dd57600080fd5b80638da5cb5b116100f25780638da5cb5b146104db57806395d89b41146104f9578063a0712d681461050e578063a22cb46514610521578063a417f2971461054157600080fd5b806370a0823114610471578063715018a614610491578063760a8c2a146104a65780637cb64759146104bb57600080fd5b80633ccfd60b116101b15780636352211e116101755780636352211e146103f657806365f1309714610416578063676dd5631461042b5780636c0360eb146104465780636cec3bb01461045b57600080fd5b80633ccfd60b1461036e57806342842e0e1461038357806342966c68146103a35780634cca3f1c146103c357806355f804b3146103d657600080fd5b8063095ea7b3116101f8578063095ea7b3146102d3578063163e1e61146102f557806318160ddd1461031557806323b872dd1461033857806332cb6b0c1461035857600080fd5b806301ffc9a71461022a57806302fb0c5e1461025f57806306fdde0314610279578063081812fc1461029b575b600080fd5b34801561023657600080fd5b5061024a6102453660046123a2565b6106c9565b60405190151581526020015b60405180910390f35b34801561026b57600080fd5b50600c5461024a9060ff1681565b34801561028557600080fd5b5061028e61071b565b60405161025691906124e0565b3480156102a757600080fd5b506102bb6102b6366004612389565b6107ad565b6040516001600160a01b039091168152602001610256565b3480156102df57600080fd5b506102f36102ee3660046122b5565b6107f1565b005b34801561030157600080fd5b506102f3610310366004612347565b610891565b34801561032157600080fd5b50600154600054035b604051908152602001610256565b34801561034457600080fd5b506102f36103533660046121c1565b6109ca565b34801561036457600080fd5b5061032a60095481565b34801561037a57600080fd5b506102f36109d5565b34801561038f57600080fd5b506102f361039e3660046121c1565b611013565b3480156103af57600080fd5b506102f36103be366004612389565b61102e565b6102f36103d13660046122df565b61103c565b3480156103e257600080fd5b506102f36103f13660046123dc565b6112b0565b34801561040257600080fd5b506102bb610411366004612389565b6112f1565b34801561042257600080fd5b5061032a600581565b34801561043757600080fd5b5061032a66ec9c58de0a800081565b34801561045257600080fd5b5061028e6112fc565b34801561046757600080fd5b5061032a600b5481565b34801561047d57600080fd5b5061032a61048c366004612173565b61138a565b34801561049d57600080fd5b506102f36113d0565b3480156104b257600080fd5b506102f3611406565b3480156104c757600080fd5b506102f36104d6366004612389565b611444565b3480156104e757600080fd5b506008546001600160a01b03166102bb565b34801561050557600080fd5b5061028e611473565b6102f361051c366004612389565b611482565b34801561052d57600080fd5b506102f361053c366004612279565b61161f565b34801561054d57600080fd5b506102f361055c366004612389565b6116b5565b34801561056d57600080fd5b5061032a600a5481565b34801561058357600080fd5b506102f36105923660046121fd565b6117b2565b3480156105a357600080fd5b5061032a600381565b3480156105b857600080fd5b50600c546105cb90610100900460ff1681565b60405160ff9091168152602001610256565b3480156105e957600080fd5b5061028e6105f8366004612389565b6117fc565b34801561060957600080fd5b5061032a610618366004612425565b600f60209081526000928352604080842090915290825290205481565b34801561064157600080fd5b5061024a61065036600461218e565b6001600160a01b03918216600090815260076020908152604080832093909416825291909152205460ff1690565b34801561068a57600080fd5b5061032a600e5481565b3480156106a057600080fd5b506102f361188e565b3480156106b557600080fd5b506102f36106c4366004612173565b6118c4565b60006301ffc9a760e01b6001600160e01b0319831614806106fa57506380ac58cd60e01b6001600160e01b03198316145b806107155750635b5e139f60e01b6001600160e01b03198316145b92915050565b60606002805461072a906125e9565b80601f0160208091040260200160405190810160405280929190818152602001828054610756906125e9565b80156107a35780601f10610778576101008083540402835291602001916107a3565b820191906000526020600020905b81548152906001019060200180831161078657829003601f168201915b5050505050905090565b60006107b88261195c565b6107d5576040516333d1c03960e21b815260040160405180910390fd5b506000908152600660205260409020546001600160a01b031690565b60006107fc82611983565b9050336001600160a01b03821614610835576108188133610650565b610835576040516367d9dca160e11b815260040160405180910390fd5b60008281526006602052604080822080546001600160a01b0319166001600160a01b0387811691821790925591518593918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a4505050565b6008546001600160a01b031633146108c45760405162461bcd60e51b81526004016108bb906124f3565b60405180910390fd5b600a54816108d160005490565b6108db9190612528565b111561091a5760405162461bcd60e51b815260206004820152600e60248201526d544f4f5f4d414e595f4d494e545360901b60448201526064016108bb565b81819050600b600082825461092f9190612528565b9091555050600b54606410156109775760405162461bcd60e51b815260206004820152600d60248201526c4e4f5f4d4f52455f474946545360981b60448201526064016108bb565b60005b818110156109c5576109b383838381811061099757610997612655565b90506020020160208101906109ac9190612173565b60016119e4565b806109bd81612624565b91505061097a565b505050565b6109c5838383611ab6565b6008546001600160a01b031633146109ff5760405162461bcd60e51b81526004016108bb906124f3565b4760006103e8610a108360f5612587565b610a1a9190612565565b905060006103e8610a2c8460be612587565b610a369190612565565b905060006103e8610a48856096612587565b610a529190612565565b905060006103e8610a6486600a612587565b610a6e9190612565565b905060006103e8610a80876005612587565b610a8a9190612565565b6010546040519192506000916001600160a01b039091169087908381818185875af1925050503d8060008114610adc576040519150601f19603f3d011682016040523d82523d6000602084013e610ae1565b606091505b5050905080610b2a5760405162461bcd60e51b81526020600482015260156024820152744661696c656420746f2073656e642045746865723160581b60448201526064016108bb565b6011546040516000916001600160a01b03169087908381818185875af1925050503d8060008114610b77576040519150601f19603f3d011682016040523d82523d6000602084013e610b7c565b606091505b5050905080610bc55760405162461bcd60e51b81526020600482015260156024820152742330b4b632b2103a379039b2b7321022ba3432b91960591b60448201526064016108bb565b6012546040516000916001600160a01b03169088908381818185875af1925050503d8060008114610c12576040519150601f19603f3d011682016040523d82523d6000602084013e610c17565b606091505b5050905080610c605760405162461bcd60e51b81526020600482015260156024820152744661696c656420746f2073656e642045746865723360581b60448201526064016108bb565b6013546040516000916001600160a01b03169089908381818185875af1925050503d8060008114610cad576040519150601f19603f3d011682016040523d82523d6000602084013e610cb2565b606091505b5050905080610cfb5760405162461bcd60e51b815260206004820152601560248201527411985a5b1959081d1bc81cd95b9908115d1a195c8d605a1b60448201526064016108bb565b6014546040516000916001600160a01b03169089908381818185875af1925050503d8060008114610d48576040519150601f19603f3d011682016040523d82523d6000602084013e610d4d565b606091505b5050905080610d965760405162461bcd60e51b81526020600482015260156024820152744661696c656420746f2073656e642045746865723560581b60448201526064016108bb565b6015546040516000916001600160a01b03169089908381818185875af1925050503d8060008114610de3576040519150601f19603f3d011682016040523d82523d6000602084013e610de8565b606091505b5050905080610e315760405162461bcd60e51b81526020600482015260156024820152742330b4b632b2103a379039b2b7321022ba3432b91b60591b60448201526064016108bb565b6016546040516000916001600160a01b0316908a908381818185875af1925050503d8060008114610e7e576040519150601f19603f3d011682016040523d82523d6000602084013e610e83565b606091505b5050905080610ecc5760405162461bcd60e51b81526020600482015260156024820152744661696c656420746f2073656e642045746865723760581b60448201526064016108bb565b6017546040516000916001600160a01b0316908b908381818185875af1925050503d8060008114610f19576040519150601f19603f3d011682016040523d82523d6000602084013e610f1e565b606091505b5050905080610f675760405162461bcd60e51b815260206004820152601560248201527408cc2d2d8cac840e8de40e6cadcc8408ae8d0cae47605b1b60448201526064016108bb565b6018546040516000916001600160a01b0316908b908381818185875af1925050503d8060008114610fb4576040519150601f19603f3d011682016040523d82523d6000602084013e610fb9565b606091505b50509050806110025760405162461bcd60e51b81526020600482015260156024820152744661696c656420746f2073656e642045746865723960581b60448201526064016108bb565b505050505050505050505050505050565b6109c5838383604051806020016040528060008152506117b2565b611039816001611c66565b50565b604080516001600160a01b03871660208201529081018490526000906060016040516020818303038152906040528051906020012090506110b483838080602002602001604051908101604052809392919081815260200183836020028082843760009201919091525050600e549150849050611dd9565b6110f75760405162461bcd60e51b815260206004820152601460248201527324a72b20a624a22fa6a2a925a622afa82927a7a360611b60448201526064016108bb565b600061110a66ec9c58de0a800087612587565b600c54610100900460ff166000908152600f602090815260408083206001600160a01b038c16845290915290205490915061114c5761114985826125a6565b90505b80341461118e5760405162461bcd60e51b815260206004820152601060248201526f15d493d391d7d1551217d05353d5539560821b60448201526064016108bb565b600a548661119b60005490565b6111a59190612528565b11156111e75760405162461bcd60e51b8152602060048201526011602482015270534541534f4e5f4d41585f535550504c5960781b60448201526064016108bb565b600c54610100900460ff166000908152600f602090815260408083206001600160a01b038b16845290915281208054889290611224908490612528565b9091555050600c54610100900460ff166000908152600f602090815260408083206001600160a01b038b1684529091529020546003101561129d5760405162461bcd60e51b8152602060048201526013602482015272105111149154d4d7d3505617d4915050d21151606a1b60448201526064016108bb565b6112a787876119e4565b50505050505050565b6008546001600160a01b031633146112da5760405162461bcd60e51b81526004016108bb906124f3565b80516112ed90600d906020840190611ffc565b5050565b600061071582611983565b600d8054611309906125e9565b80601f0160208091040260200160405190810160405280929190818152602001828054611335906125e9565b80156113825780601f1061135757610100808354040283529160200191611382565b820191906000526020600020905b81548152906001019060200180831161136557829003601f168201915b505050505081565b6000816113aa576040516323d3ad8160e21b815260040160405180910390fd5b506001600160a01b031660009081526005602052604090205467ffffffffffffffff1690565b6008546001600160a01b031633146113fa5760405162461bcd60e51b81526004016108bb906124f3565b6114046000611def565b565b6008546001600160a01b031633146114305760405162461bcd60e51b81526004016108bb906124f3565b600c805460ff19811660ff90911615179055565b6008546001600160a01b0316331461146e5760405162461bcd60e51b81526004016108bb906124f3565b600e55565b60606003805461072a906125e9565b600c5460ff166114c65760405162461bcd60e51b815260206004820152600f60248201526e53414c455f4e4f545f41435449564560881b60448201526064016108bb565b346114d866ec9c58de0a800083612587565b146115185760405162461bcd60e51b815260206004820152601060248201526f15d493d391d7d1551217d05353d5539560821b60448201526064016108bb565b600a548161152560005490565b61152f9190612528565b11156115715760405162461bcd60e51b8152602060048201526011602482015270534541534f4e5f4d41585f535550504c5960781b60448201526064016108bb565b600c54610100900460ff166000908152600f60209081526040808320338452909152812080548392906115a5908490612528565b9091555050600c54610100900460ff166000908152600f60209081526040808320338452909152902054600510156116155760405162461bcd60e51b8152602060048201526013602482015272105111149154d4d7d3505617d4915050d21151606a1b60448201526064016108bb565b61103933826119e4565b6001600160a01b0382163314156116495760405163b06307db60e01b815260040160405180910390fd5b3360008181526007602090815260408083206001600160a01b03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b6008546001600160a01b031633146116df5760405162461bcd60e51b81526004016108bb906124f3565b6001546000540381116117255760405162461bcd60e51b815260206004820152600e60248201526d535550504c595f544f4f5f4c4f5760901b60448201526064016108bb565b6009548111156117695760405162461bcd60e51b815260206004820152600f60248201526e0a6aaa0a098b2bea89e9ebe90928e9608b1b60448201526064016108bb565b6000600e55600c805460019190829061178b908290610100900460ff16612540565b825460ff9182166101009390930a928302919092021990911617905550600a556000600b55565b6117bd848484611ab6565b6001600160a01b0383163b156117f6576117d984848484611e41565b6117f6576040516368d2bf6b60e11b815260040160405180910390fd5b50505050565b60606118078261195c565b61182457604051630a14c4b560e41b815260040160405180910390fd5b600061183b60408051602081019091526000815290565b905080516000141561185c5760405180602001604052806000815250611887565b8061186684611f39565b604051602001611877929190612474565b6040516020818303038152906040525b9392505050565b6008546001600160a01b031633146118b85760405162461bcd60e51b81526004016108bb906124f3565b60015460005403600955565b6008546001600160a01b031633146118ee5760405162461bcd60e51b81526004016108bb906124f3565b6001600160a01b0381166119535760405162461bcd60e51b815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201526564647265737360d01b60648201526084016108bb565b61103981611def565b6000805482108015610715575050600090815260046020526040902054600160e01b161590565b6000816000548110156119cb57600081815260046020526040902054600160e01b81166119c9575b806118875750600019016000818152600460205260409020546119ab565b505b604051636f96cda160e11b815260040160405180910390fd5b60005482611a0457604051622e076360e81b815260040160405180910390fd5b81611a225760405163b562e8dd60e01b815260040160405180910390fd5b6001600160a01b03831660009081526005602090815260408083208054680100000000000000018702019055838352600490915281204260a01b85176001851460e11b1790555b60405160018201918301906001600160a01b038616906000907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef908290a4828110611a6957500160005550565b6000611ac182611983565b9050836001600160a01b0316816001600160a01b031614611af45760405162a1148160e81b815260040160405180910390fd5b6000828152600660205260408120546001600160a01b0390811691908616331480611b245750611b248633610650565b80611b3757506001600160a01b03821633145b905080611b5757604051632ce44b5f60e11b815260040160405180910390fd5b84611b7557604051633a954ecd60e21b815260040160405180910390fd5b8115611b9857600084815260066020526040902080546001600160a01b03191690555b6001600160a01b03868116600090815260056020908152604080832080546000190190559288168252828220805460010190558682526004905220600160e11b4260a01b871781179091558316611c1d5760018401600081815260046020526040902054611c1b576000548114611c1b5760008181526004602052604090208490555b505b83856001600160a01b0316876001600160a01b03167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4505050505050565b6000611c7183611983565b60008481526006602052604090205490915081906001600160a01b03168315611ce7576000336001600160a01b0384161480611cb25750611cb28333610650565b80611cc557506001600160a01b03821633145b905080611ce557604051632ce44b5f60e11b815260040160405180910390fd5b505b8015611d0a57600085815260066020526040902080546001600160a01b03191690555b6001600160a01b038216600090815260056020908152604080832080546fffffffffffffffffffffffffffffffff01905587835260049091529020600360e01b4260a01b8417179055600160e11b8316611d925760018501600081815260046020526040902054611d90576000548114611d905760008181526004602052604090208490555b505b60405185906000906001600160a01b038516907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef908390a450506001805481019055505050565b600082611de68584611f88565b14949350505050565b600880546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b604051630a85bd0160e11b81526000906001600160a01b0385169063150b7a0290611e769033908990889088906004016124a3565b602060405180830381600087803b158015611e9057600080fd5b505af1925050508015611ec0575060408051601f3d908101601f19168201909252611ebd918101906123bf565b60015b611f1b573d808015611eee576040519150601f19603f3d011682016040523d82523d6000602084013e611ef3565b606091505b508051611f13576040516368d2bf6b60e11b815260040160405180910390fd5b805181602001fd5b6001600160e01b031916630a85bd0160e11b1490505b949350505050565b604080516080810191829052607f0190826030600a8206018353600a90045b8015611f7657600183039250600a81066030018353600a9004611f58565b50819003601f19909101908152919050565b600081815b8451811015611ff4576000858281518110611faa57611faa612655565b60200260200101519050808311611fd05760008381526020829052604090209250611fe1565b600081815260208490526040902092505b5080611fec81612624565b915050611f8d565b509392505050565b828054612008906125e9565b90600052602060002090601f01602090048101928261202a5760008555612070565b82601f1061204357805160ff1916838001178555612070565b82800160010185558215612070579182015b82811115612070578251825591602001919060010190612055565b5061207c929150612080565b5090565b5b8082111561207c5760008155600101612081565b600067ffffffffffffffff808411156120b0576120b061266b565b604051601f8501601f19908116603f011681019082821181831017156120d8576120d861266b565b816040528093508581528686860111156120f157600080fd5b858560208301376000602087830101525050509392505050565b80356001600160a01b038116811461212257600080fd5b919050565b60008083601f84011261213957600080fd5b50813567ffffffffffffffff81111561215157600080fd5b6020830191508360208260051b850101111561216c57600080fd5b9250929050565b60006020828403121561218557600080fd5b6118878261210b565b600080604083850312156121a157600080fd5b6121aa8361210b565b91506121b86020840161210b565b90509250929050565b6000806000606084860312156121d657600080fd5b6121df8461210b565b92506121ed6020850161210b565b9150604084013590509250925092565b6000806000806080858703121561221357600080fd5b61221c8561210b565b935061222a6020860161210b565b925060408501359150606085013567ffffffffffffffff81111561224d57600080fd5b8501601f8101871361225e57600080fd5b61226d87823560208401612095565b91505092959194509250565b6000806040838503121561228c57600080fd5b6122958361210b565b9150602083013580151581146122aa57600080fd5b809150509250929050565b600080604083850312156122c857600080fd5b6122d18361210b565b946020939093013593505050565b6000806000806000608086880312156122f757600080fd5b6123008661210b565b94506020860135935060408601359250606086013567ffffffffffffffff81111561232a57600080fd5b61233688828901612127565b969995985093965092949392505050565b6000806020838503121561235a57600080fd5b823567ffffffffffffffff81111561237157600080fd5b61237d85828601612127565b90969095509350505050565b60006020828403121561239b57600080fd5b5035919050565b6000602082840312156123b457600080fd5b813561188781612681565b6000602082840312156123d157600080fd5b815161188781612681565b6000602082840312156123ee57600080fd5b813567ffffffffffffffff81111561240557600080fd5b8201601f8101841361241657600080fd5b611f3184823560208401612095565b6000806040838503121561243857600080fd5b823591506121b86020840161210b565b600081518084526124608160208601602086016125bd565b601f01601f19169290920160200192915050565b600083516124868184602088016125bd565b83519083019061249a8183602088016125bd565b01949350505050565b6001600160a01b03858116825284166020820152604081018390526080606082018190526000906124d690830184612448565b9695505050505050565b6020815260006118876020830184612448565b6020808252818101527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572604082015260600190565b6000821982111561253b5761253b61263f565b500190565b600060ff821660ff84168060ff0382111561255d5761255d61263f565b019392505050565b60008261258257634e487b7160e01b600052601260045260246000fd5b500490565b60008160001904831182151516156125a1576125a161263f565b500290565b6000828210156125b8576125b861263f565b500390565b60005b838110156125d85781810151838201526020016125c0565b838111156117f65750506000910152565b600181811c908216806125fd57607f821691505b6020821081141561261e57634e487b7160e01b600052602260045260246000fd5b50919050565b60006000198214156126385761263861263f565b5060010190565b634e487b7160e01b600052601160045260246000fd5b634e487b7160e01b600052603260045260246000fd5b634e487b7160e01b600052604160045260246000fd5b6001600160e01b03198116811461103957600080fdfea264697066735822122032b2fe5f787506f6976b72f8013c2e5b00900b07aab7adf77290e147c963a68e64736f6c6343000806003300000000000000000000000000000000000000000000000000000000000000200000000000000000000000000000000000000000000000000000000000000000

Deployed Bytecode

0x6080604052600436106102255760003560e01c806370a0823111610123578063a72c41cf116100ab578063e942bdd21161006f578063e942bdd2146105fd578063e985e9c514610635578063ebf0c7171461067e578063ef70aebf14610694578063f2fde38b146106a957600080fd5b8063a72c41cf14610561578063b88d4fde14610577578063c08dfd3c14610597578063c20deccf146105ac578063c87b56dd146105dd57600080fd5b80638da5cb5b116100f25780638da5cb5b146104db57806395d89b41146104f9578063a0712d681461050e578063a22cb46514610521578063a417f2971461054157600080fd5b806370a0823114610471578063715018a614610491578063760a8c2a146104a65780637cb64759146104bb57600080fd5b80633ccfd60b116101b15780636352211e116101755780636352211e146103f657806365f1309714610416578063676dd5631461042b5780636c0360eb146104465780636cec3bb01461045b57600080fd5b80633ccfd60b1461036e57806342842e0e1461038357806342966c68146103a35780634cca3f1c146103c357806355f804b3146103d657600080fd5b8063095ea7b3116101f8578063095ea7b3146102d3578063163e1e61146102f557806318160ddd1461031557806323b872dd1461033857806332cb6b0c1461035857600080fd5b806301ffc9a71461022a57806302fb0c5e1461025f57806306fdde0314610279578063081812fc1461029b575b600080fd5b34801561023657600080fd5b5061024a6102453660046123a2565b6106c9565b60405190151581526020015b60405180910390f35b34801561026b57600080fd5b50600c5461024a9060ff1681565b34801561028557600080fd5b5061028e61071b565b60405161025691906124e0565b3480156102a757600080fd5b506102bb6102b6366004612389565b6107ad565b6040516001600160a01b039091168152602001610256565b3480156102df57600080fd5b506102f36102ee3660046122b5565b6107f1565b005b34801561030157600080fd5b506102f3610310366004612347565b610891565b34801561032157600080fd5b50600154600054035b604051908152602001610256565b34801561034457600080fd5b506102f36103533660046121c1565b6109ca565b34801561036457600080fd5b5061032a60095481565b34801561037a57600080fd5b506102f36109d5565b34801561038f57600080fd5b506102f361039e3660046121c1565b611013565b3480156103af57600080fd5b506102f36103be366004612389565b61102e565b6102f36103d13660046122df565b61103c565b3480156103e257600080fd5b506102f36103f13660046123dc565b6112b0565b34801561040257600080fd5b506102bb610411366004612389565b6112f1565b34801561042257600080fd5b5061032a600581565b34801561043757600080fd5b5061032a66ec9c58de0a800081565b34801561045257600080fd5b5061028e6112fc565b34801561046757600080fd5b5061032a600b5481565b34801561047d57600080fd5b5061032a61048c366004612173565b61138a565b34801561049d57600080fd5b506102f36113d0565b3480156104b257600080fd5b506102f3611406565b3480156104c757600080fd5b506102f36104d6366004612389565b611444565b3480156104e757600080fd5b506008546001600160a01b03166102bb565b34801561050557600080fd5b5061028e611473565b6102f361051c366004612389565b611482565b34801561052d57600080fd5b506102f361053c366004612279565b61161f565b34801561054d57600080fd5b506102f361055c366004612389565b6116b5565b34801561056d57600080fd5b5061032a600a5481565b34801561058357600080fd5b506102f36105923660046121fd565b6117b2565b3480156105a357600080fd5b5061032a600381565b3480156105b857600080fd5b50600c546105cb90610100900460ff1681565b60405160ff9091168152602001610256565b3480156105e957600080fd5b5061028e6105f8366004612389565b6117fc565b34801561060957600080fd5b5061032a610618366004612425565b600f60209081526000928352604080842090915290825290205481565b34801561064157600080fd5b5061024a61065036600461218e565b6001600160a01b03918216600090815260076020908152604080832093909416825291909152205460ff1690565b34801561068a57600080fd5b5061032a600e5481565b3480156106a057600080fd5b506102f361188e565b3480156106b557600080fd5b506102f36106c4366004612173565b6118c4565b60006301ffc9a760e01b6001600160e01b0319831614806106fa57506380ac58cd60e01b6001600160e01b03198316145b806107155750635b5e139f60e01b6001600160e01b03198316145b92915050565b60606002805461072a906125e9565b80601f0160208091040260200160405190810160405280929190818152602001828054610756906125e9565b80156107a35780601f10610778576101008083540402835291602001916107a3565b820191906000526020600020905b81548152906001019060200180831161078657829003601f168201915b5050505050905090565b60006107b88261195c565b6107d5576040516333d1c03960e21b815260040160405180910390fd5b506000908152600660205260409020546001600160a01b031690565b60006107fc82611983565b9050336001600160a01b03821614610835576108188133610650565b610835576040516367d9dca160e11b815260040160405180910390fd5b60008281526006602052604080822080546001600160a01b0319166001600160a01b0387811691821790925591518593918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a4505050565b6008546001600160a01b031633146108c45760405162461bcd60e51b81526004016108bb906124f3565b60405180910390fd5b600a54816108d160005490565b6108db9190612528565b111561091a5760405162461bcd60e51b815260206004820152600e60248201526d544f4f5f4d414e595f4d494e545360901b60448201526064016108bb565b81819050600b600082825461092f9190612528565b9091555050600b54606410156109775760405162461bcd60e51b815260206004820152600d60248201526c4e4f5f4d4f52455f474946545360981b60448201526064016108bb565b60005b818110156109c5576109b383838381811061099757610997612655565b90506020020160208101906109ac9190612173565b60016119e4565b806109bd81612624565b91505061097a565b505050565b6109c5838383611ab6565b6008546001600160a01b031633146109ff5760405162461bcd60e51b81526004016108bb906124f3565b4760006103e8610a108360f5612587565b610a1a9190612565565b905060006103e8610a2c8460be612587565b610a369190612565565b905060006103e8610a48856096612587565b610a529190612565565b905060006103e8610a6486600a612587565b610a6e9190612565565b905060006103e8610a80876005612587565b610a8a9190612565565b6010546040519192506000916001600160a01b039091169087908381818185875af1925050503d8060008114610adc576040519150601f19603f3d011682016040523d82523d6000602084013e610ae1565b606091505b5050905080610b2a5760405162461bcd60e51b81526020600482015260156024820152744661696c656420746f2073656e642045746865723160581b60448201526064016108bb565b6011546040516000916001600160a01b03169087908381818185875af1925050503d8060008114610b77576040519150601f19603f3d011682016040523d82523d6000602084013e610b7c565b606091505b5050905080610bc55760405162461bcd60e51b81526020600482015260156024820152742330b4b632b2103a379039b2b7321022ba3432b91960591b60448201526064016108bb565b6012546040516000916001600160a01b03169088908381818185875af1925050503d8060008114610c12576040519150601f19603f3d011682016040523d82523d6000602084013e610c17565b606091505b5050905080610c605760405162461bcd60e51b81526020600482015260156024820152744661696c656420746f2073656e642045746865723360581b60448201526064016108bb565b6013546040516000916001600160a01b03169089908381818185875af1925050503d8060008114610cad576040519150601f19603f3d011682016040523d82523d6000602084013e610cb2565b606091505b5050905080610cfb5760405162461bcd60e51b815260206004820152601560248201527411985a5b1959081d1bc81cd95b9908115d1a195c8d605a1b60448201526064016108bb565b6014546040516000916001600160a01b03169089908381818185875af1925050503d8060008114610d48576040519150601f19603f3d011682016040523d82523d6000602084013e610d4d565b606091505b5050905080610d965760405162461bcd60e51b81526020600482015260156024820152744661696c656420746f2073656e642045746865723560581b60448201526064016108bb565b6015546040516000916001600160a01b03169089908381818185875af1925050503d8060008114610de3576040519150601f19603f3d011682016040523d82523d6000602084013e610de8565b606091505b5050905080610e315760405162461bcd60e51b81526020600482015260156024820152742330b4b632b2103a379039b2b7321022ba3432b91b60591b60448201526064016108bb565b6016546040516000916001600160a01b0316908a908381818185875af1925050503d8060008114610e7e576040519150601f19603f3d011682016040523d82523d6000602084013e610e83565b606091505b5050905080610ecc5760405162461bcd60e51b81526020600482015260156024820152744661696c656420746f2073656e642045746865723760581b60448201526064016108bb565b6017546040516000916001600160a01b0316908b908381818185875af1925050503d8060008114610f19576040519150601f19603f3d011682016040523d82523d6000602084013e610f1e565b606091505b5050905080610f675760405162461bcd60e51b815260206004820152601560248201527408cc2d2d8cac840e8de40e6cadcc8408ae8d0cae47605b1b60448201526064016108bb565b6018546040516000916001600160a01b0316908b908381818185875af1925050503d8060008114610fb4576040519150601f19603f3d011682016040523d82523d6000602084013e610fb9565b606091505b50509050806110025760405162461bcd60e51b81526020600482015260156024820152744661696c656420746f2073656e642045746865723960581b60448201526064016108bb565b505050505050505050505050505050565b6109c5838383604051806020016040528060008152506117b2565b611039816001611c66565b50565b604080516001600160a01b03871660208201529081018490526000906060016040516020818303038152906040528051906020012090506110b483838080602002602001604051908101604052809392919081815260200183836020028082843760009201919091525050600e549150849050611dd9565b6110f75760405162461bcd60e51b815260206004820152601460248201527324a72b20a624a22fa6a2a925a622afa82927a7a360611b60448201526064016108bb565b600061110a66ec9c58de0a800087612587565b600c54610100900460ff166000908152600f602090815260408083206001600160a01b038c16845290915290205490915061114c5761114985826125a6565b90505b80341461118e5760405162461bcd60e51b815260206004820152601060248201526f15d493d391d7d1551217d05353d5539560821b60448201526064016108bb565b600a548661119b60005490565b6111a59190612528565b11156111e75760405162461bcd60e51b8152602060048201526011602482015270534541534f4e5f4d41585f535550504c5960781b60448201526064016108bb565b600c54610100900460ff166000908152600f602090815260408083206001600160a01b038b16845290915281208054889290611224908490612528565b9091555050600c54610100900460ff166000908152600f602090815260408083206001600160a01b038b1684529091529020546003101561129d5760405162461bcd60e51b8152602060048201526013602482015272105111149154d4d7d3505617d4915050d21151606a1b60448201526064016108bb565b6112a787876119e4565b50505050505050565b6008546001600160a01b031633146112da5760405162461bcd60e51b81526004016108bb906124f3565b80516112ed90600d906020840190611ffc565b5050565b600061071582611983565b600d8054611309906125e9565b80601f0160208091040260200160405190810160405280929190818152602001828054611335906125e9565b80156113825780601f1061135757610100808354040283529160200191611382565b820191906000526020600020905b81548152906001019060200180831161136557829003601f168201915b505050505081565b6000816113aa576040516323d3ad8160e21b815260040160405180910390fd5b506001600160a01b031660009081526005602052604090205467ffffffffffffffff1690565b6008546001600160a01b031633146113fa5760405162461bcd60e51b81526004016108bb906124f3565b6114046000611def565b565b6008546001600160a01b031633146114305760405162461bcd60e51b81526004016108bb906124f3565b600c805460ff19811660ff90911615179055565b6008546001600160a01b0316331461146e5760405162461bcd60e51b81526004016108bb906124f3565b600e55565b60606003805461072a906125e9565b600c5460ff166114c65760405162461bcd60e51b815260206004820152600f60248201526e53414c455f4e4f545f41435449564560881b60448201526064016108bb565b346114d866ec9c58de0a800083612587565b146115185760405162461bcd60e51b815260206004820152601060248201526f15d493d391d7d1551217d05353d5539560821b60448201526064016108bb565b600a548161152560005490565b61152f9190612528565b11156115715760405162461bcd60e51b8152602060048201526011602482015270534541534f4e5f4d41585f535550504c5960781b60448201526064016108bb565b600c54610100900460ff166000908152600f60209081526040808320338452909152812080548392906115a5908490612528565b9091555050600c54610100900460ff166000908152600f60209081526040808320338452909152902054600510156116155760405162461bcd60e51b8152602060048201526013602482015272105111149154d4d7d3505617d4915050d21151606a1b60448201526064016108bb565b61103933826119e4565b6001600160a01b0382163314156116495760405163b06307db60e01b815260040160405180910390fd5b3360008181526007602090815260408083206001600160a01b03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b6008546001600160a01b031633146116df5760405162461bcd60e51b81526004016108bb906124f3565b6001546000540381116117255760405162461bcd60e51b815260206004820152600e60248201526d535550504c595f544f4f5f4c4f5760901b60448201526064016108bb565b6009548111156117695760405162461bcd60e51b815260206004820152600f60248201526e0a6aaa0a098b2bea89e9ebe90928e9608b1b60448201526064016108bb565b6000600e55600c805460019190829061178b908290610100900460ff16612540565b825460ff9182166101009390930a928302919092021990911617905550600a556000600b55565b6117bd848484611ab6565b6001600160a01b0383163b156117f6576117d984848484611e41565b6117f6576040516368d2bf6b60e11b815260040160405180910390fd5b50505050565b60606118078261195c565b61182457604051630a14c4b560e41b815260040160405180910390fd5b600061183b60408051602081019091526000815290565b905080516000141561185c5760405180602001604052806000815250611887565b8061186684611f39565b604051602001611877929190612474565b6040516020818303038152906040525b9392505050565b6008546001600160a01b031633146118b85760405162461bcd60e51b81526004016108bb906124f3565b60015460005403600955565b6008546001600160a01b031633146118ee5760405162461bcd60e51b81526004016108bb906124f3565b6001600160a01b0381166119535760405162461bcd60e51b815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201526564647265737360d01b60648201526084016108bb565b61103981611def565b6000805482108015610715575050600090815260046020526040902054600160e01b161590565b6000816000548110156119cb57600081815260046020526040902054600160e01b81166119c9575b806118875750600019016000818152600460205260409020546119ab565b505b604051636f96cda160e11b815260040160405180910390fd5b60005482611a0457604051622e076360e81b815260040160405180910390fd5b81611a225760405163b562e8dd60e01b815260040160405180910390fd5b6001600160a01b03831660009081526005602090815260408083208054680100000000000000018702019055838352600490915281204260a01b85176001851460e11b1790555b60405160018201918301906001600160a01b038616906000907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef908290a4828110611a6957500160005550565b6000611ac182611983565b9050836001600160a01b0316816001600160a01b031614611af45760405162a1148160e81b815260040160405180910390fd5b6000828152600660205260408120546001600160a01b0390811691908616331480611b245750611b248633610650565b80611b3757506001600160a01b03821633145b905080611b5757604051632ce44b5f60e11b815260040160405180910390fd5b84611b7557604051633a954ecd60e21b815260040160405180910390fd5b8115611b9857600084815260066020526040902080546001600160a01b03191690555b6001600160a01b03868116600090815260056020908152604080832080546000190190559288168252828220805460010190558682526004905220600160e11b4260a01b871781179091558316611c1d5760018401600081815260046020526040902054611c1b576000548114611c1b5760008181526004602052604090208490555b505b83856001600160a01b0316876001600160a01b03167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4505050505050565b6000611c7183611983565b60008481526006602052604090205490915081906001600160a01b03168315611ce7576000336001600160a01b0384161480611cb25750611cb28333610650565b80611cc557506001600160a01b03821633145b905080611ce557604051632ce44b5f60e11b815260040160405180910390fd5b505b8015611d0a57600085815260066020526040902080546001600160a01b03191690555b6001600160a01b038216600090815260056020908152604080832080546fffffffffffffffffffffffffffffffff01905587835260049091529020600360e01b4260a01b8417179055600160e11b8316611d925760018501600081815260046020526040902054611d90576000548114611d905760008181526004602052604090208490555b505b60405185906000906001600160a01b038516907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef908390a450506001805481019055505050565b600082611de68584611f88565b14949350505050565b600880546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b604051630a85bd0160e11b81526000906001600160a01b0385169063150b7a0290611e769033908990889088906004016124a3565b602060405180830381600087803b158015611e9057600080fd5b505af1925050508015611ec0575060408051601f3d908101601f19168201909252611ebd918101906123bf565b60015b611f1b573d808015611eee576040519150601f19603f3d011682016040523d82523d6000602084013e611ef3565b606091505b508051611f13576040516368d2bf6b60e11b815260040160405180910390fd5b805181602001fd5b6001600160e01b031916630a85bd0160e11b1490505b949350505050565b604080516080810191829052607f0190826030600a8206018353600a90045b8015611f7657600183039250600a81066030018353600a9004611f58565b50819003601f19909101908152919050565b600081815b8451811015611ff4576000858281518110611faa57611faa612655565b60200260200101519050808311611fd05760008381526020829052604090209250611fe1565b600081815260208490526040902092505b5080611fec81612624565b915050611f8d565b509392505050565b828054612008906125e9565b90600052602060002090601f01602090048101928261202a5760008555612070565b82601f1061204357805160ff1916838001178555612070565b82800160010185558215612070579182015b82811115612070578251825591602001919060010190612055565b5061207c929150612080565b5090565b5b8082111561207c5760008155600101612081565b600067ffffffffffffffff808411156120b0576120b061266b565b604051601f8501601f19908116603f011681019082821181831017156120d8576120d861266b565b816040528093508581528686860111156120f157600080fd5b858560208301376000602087830101525050509392505050565b80356001600160a01b038116811461212257600080fd5b919050565b60008083601f84011261213957600080fd5b50813567ffffffffffffffff81111561215157600080fd5b6020830191508360208260051b850101111561216c57600080fd5b9250929050565b60006020828403121561218557600080fd5b6118878261210b565b600080604083850312156121a157600080fd5b6121aa8361210b565b91506121b86020840161210b565b90509250929050565b6000806000606084860312156121d657600080fd5b6121df8461210b565b92506121ed6020850161210b565b9150604084013590509250925092565b6000806000806080858703121561221357600080fd5b61221c8561210b565b935061222a6020860161210b565b925060408501359150606085013567ffffffffffffffff81111561224d57600080fd5b8501601f8101871361225e57600080fd5b61226d87823560208401612095565b91505092959194509250565b6000806040838503121561228c57600080fd5b6122958361210b565b9150602083013580151581146122aa57600080fd5b809150509250929050565b600080604083850312156122c857600080fd5b6122d18361210b565b946020939093013593505050565b6000806000806000608086880312156122f757600080fd5b6123008661210b565b94506020860135935060408601359250606086013567ffffffffffffffff81111561232a57600080fd5b61233688828901612127565b969995985093965092949392505050565b6000806020838503121561235a57600080fd5b823567ffffffffffffffff81111561237157600080fd5b61237d85828601612127565b90969095509350505050565b60006020828403121561239b57600080fd5b5035919050565b6000602082840312156123b457600080fd5b813561188781612681565b6000602082840312156123d157600080fd5b815161188781612681565b6000602082840312156123ee57600080fd5b813567ffffffffffffffff81111561240557600080fd5b8201601f8101841361241657600080fd5b611f3184823560208401612095565b6000806040838503121561243857600080fd5b823591506121b86020840161210b565b600081518084526124608160208601602086016125bd565b601f01601f19169290920160200192915050565b600083516124868184602088016125bd565b83519083019061249a8183602088016125bd565b01949350505050565b6001600160a01b03858116825284166020820152604081018390526080606082018190526000906124d690830184612448565b9695505050505050565b6020815260006118876020830184612448565b6020808252818101527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572604082015260600190565b6000821982111561253b5761253b61263f565b500190565b600060ff821660ff84168060ff0382111561255d5761255d61263f565b019392505050565b60008261258257634e487b7160e01b600052601260045260246000fd5b500490565b60008160001904831182151516156125a1576125a161263f565b500290565b6000828210156125b8576125b861263f565b500390565b60005b838110156125d85781810151838201526020016125c0565b838111156117f65750506000910152565b600181811c908216806125fd57607f821691505b6020821081141561261e57634e487b7160e01b600052602260045260246000fd5b50919050565b60006000198214156126385761263861263f565b5060010190565b634e487b7160e01b600052601160045260246000fd5b634e487b7160e01b600052603260045260246000fd5b634e487b7160e01b600052604160045260246000fd5b6001600160e01b03198116811461103957600080fdfea264697066735822122032b2fe5f787506f6976b72f8013c2e5b00900b07aab7adf77290e147c963a68e64736f6c63430008060033

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

00000000000000000000000000000000000000000000000000000000000000200000000000000000000000000000000000000000000000000000000000000000

-----Decoded View---------------
Arg [0] : _baseURI (string):

-----Encoded View---------------
2 Constructor Arguments found :
Arg [0] : 0000000000000000000000000000000000000000000000000000000000000020
Arg [1] : 0000000000000000000000000000000000000000000000000000000000000000


Deployed Bytecode Sourcemap

45175:4845:0:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;21168:615;;;;;;;;;;-1:-1:-1;21168:615:0;;;;;:::i;:::-;;:::i;:::-;;;8046:14:1;;8039:22;8021:41;;8009:2;7994:18;21168:615:0;;;;;;;;45472:26;;;;;;;;;;-1:-1:-1;45472:26:0;;;;;;;;26204:100;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;28217:204::-;;;;;;;;;;-1:-1:-1;28217:204:0;;;;;:::i;:::-;;:::i;:::-;;;-1:-1:-1;;;;;7065:32:1;;;7047:51;;7035:2;7020:18;28217:204:0;7002:102:1;27736:415:0;;;;;;;;;;-1:-1:-1;27736:415:0;;;;;:::i;:::-;;:::i;:::-;;47271:337;;;;;;;;;;-1:-1:-1;47271:337:0;;;;;:::i;:::-;;:::i;20222:315::-;;;;;;;;;;-1:-1:-1;20488:12:0;;20275:7;20472:13;:28;20222:315;;;8219:25:1;;;8207:2;8192:18;20222:315:0;8174:76:1;29103:170:0;;;;;;;;;;-1:-1:-1;29103:170:0;;;;;:::i;:::-;;:::i;45367:29::-;;;;;;;;;;;;;;;;48707:1310;;;;;;;;;;;;;:::i;29344:185::-;;;;;;;;;;-1:-1:-1;29344:185:0;;;;;:::i;:::-;;:::i;46866:58::-;;;;;;;;;;-1:-1:-1;46866:58:0;;;;;:::i;:::-;;:::i;46184:676::-;;;;;;:::i;:::-;;:::i;47099:82::-;;;;;;;;;;-1:-1:-1;47099:82:0;;;;;:::i;:::-;;:::i;25993:144::-;;;;;;;;;;-1:-1:-1;25993:144:0;;;;;:::i;:::-;;:::i;45322:40::-;;;;;;;;;;;;45361:1;45322:40;;45224:45;;;;;;;;;;;;45257:12;45224:45;;45543:21;;;;;;;;;;;;;:::i;45435:30::-;;;;;;;;;;;;;;;;21847:234;;;;;;;;;;-1:-1:-1;21847:234:0;;;;;:::i;:::-;;:::i;7415:103::-;;;;;;;;;;;;;:::i;46930:67::-;;;;;;;;;;;;;:::i;47003:90::-;;;;;;;;;;-1:-1:-1;47003:90:0;;;;;:::i;:::-;;:::i;6764:87::-;;;;;;;;;;-1:-1:-1;6837:6:0;;-1:-1:-1;;;;;6837:6:0;6764:87;;26373:104;;;;;;;;;;;;;:::i;45767:411::-;;;;;;:::i;:::-;;:::i;28493:308::-;;;;;;;;;;-1:-1:-1;28493:308:0;;;;;:::i;:::-;;:::i;47614:275::-;;;;;;;;;;-1:-1:-1;47614:275:0;;;;;:::i;:::-;;:::i;45401:29::-;;;;;;;;;;;;;;;;29600:396;;;;;;;;;;-1:-1:-1;29600:396:0;;;;;:::i;:::-;;:::i;45274:43::-;;;;;;;;;;;;45316:1;45274:43;;45505:31;;;;;;;;;;-1:-1:-1;45505:31:0;;;;;;;;;;;;;;15855:4:1;15843:17;;;15825:36;;15813:2;15798:18;45505:31:0;15780:87:1;26548:318:0;;;;;;;;;;-1:-1:-1;26548:318:0;;;;;:::i;:::-;;:::i;45597:58::-;;;;;;;;;;-1:-1:-1;45597:58:0;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;28872:164;;;;;;;;;;-1:-1:-1;28872:164:0;;;;;:::i;:::-;-1:-1:-1;;;;;28993:25:0;;;28969:4;28993:25;;;:18;:25;;;;;;;;:35;;;;;;;;;;;;;;;28872:164;45571:19;;;;;;;;;;;;;;;;47187:78;;;;;;;;;;;;;:::i;7673:201::-;;;;;;;;;;-1:-1:-1;7673:201:0;;;;;:::i;:::-;;:::i;21168:615::-;21253:4;-1:-1:-1;;;;;;;;;21553:25:0;;;;:102;;-1:-1:-1;;;;;;;;;;21630:25:0;;;21553:102;:179;;;-1:-1:-1;;;;;;;;;;21707:25:0;;;21553:179;21533:199;21168:615;-1:-1:-1;;21168:615:0:o;26204:100::-;26258:13;26291:5;26284:12;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;26204:100;:::o;28217:204::-;28285:7;28310:16;28318:7;28310;:16::i;:::-;28305:64;;28335:34;;-1:-1:-1;;;28335:34:0;;;;;;;;;;;28305:64;-1:-1:-1;28389:24:0;;;;:15;:24;;;;;;-1:-1:-1;;;;;28389:24:0;;28217:204::o;27736:415::-;27809:13;27841:27;27860:7;27841:18;:27::i;:::-;27809:61;-1:-1:-1;43012:10:0;-1:-1:-1;;;;;27887:28:0;;;27883:175;;27935:44;27952:5;43012:10;28872:164;:::i;27935:44::-;27930:128;;28007:35;;-1:-1:-1;;;28007:35:0;;;;;;;;;;;27930:128;28070:24;;;;:15;:24;;;;;;:29;;-1:-1:-1;;;;;;28070:29:0;-1:-1:-1;;;;;28070:29:0;;;;;;;;;28115:28;;28070:24;;28115:28;;;;;;;27798:353;27736:415;;:::o;47271:337::-;6837:6;;-1:-1:-1;;;;;6837:6:0;43012:10;6984:23;6976:68;;;;-1:-1:-1;;;6976:68:0;;;;;;;:::i;:::-;;;;;;;;;47386:10:::1;::::0;47366:9;47349:14:::1;20682:7:::0;20870:13;;20635:285;47349:14:::1;:33;;;;:::i;:::-;:47;;47341:74;;;::::0;-1:-1:-1;;;47341:74:0;;8681:2:1;47341:74:0::1;::::0;::::1;8663:21:1::0;8720:2;8700:18;;;8693:30;-1:-1:-1;;;8739:18:1;;;8732:44;8793:18;;47341:74:0::1;8653:164:1::0;47341:74:0::1;47442:9;;:16;;47424:14;;:34;;;;;;;:::i;:::-;::::0;;;-1:-1:-1;;47473:14:0::1;::::0;47491:3:::1;-1:-1:-1::0;47473:21:0::1;47465:47;;;::::0;-1:-1:-1;;;47465:47:0;;15361:2:1;47465:47:0::1;::::0;::::1;15343:21:1::0;15400:2;15380:18;;;15373:30;-1:-1:-1;;;15419:18:1;;;15412:43;15472:18;;47465:47:0::1;15333:163:1::0;47465:47:0::1;47525:6;47521:82;47537:20:::0;;::::1;47521:82;;;47573:22;47579:9;;47589:1;47579:12;;;;;;;:::i;:::-;;;;;;;;;;;;;;:::i;:::-;47593:1;47573:5;:22::i;:::-;47559:3:::0;::::1;::::0;::::1;:::i;:::-;;;;47521:82;;;;47271:337:::0;;:::o;29103:170::-;29237:28;29247:4;29253:2;29257:7;29237:9;:28::i;48707:1310::-;6837:6;;-1:-1:-1;;;;;6837:6:0;43012:10;6984:23;6976:68;;;;-1:-1:-1;;;6976:68:0;;;;;;;:::i;:::-;48766:21:::1;48751:12;48828:4;48812:13;48766:21:::0;48822:3:::1;48812:13;:::i;:::-;:20;;;;:::i;:::-;48794:38:::0;-1:-1:-1;48839:13:0::1;48871:4;48855:13;:7:::0;48865:3:::1;48855:13;:::i;:::-;:20;;;;:::i;:::-;48839:36:::0;-1:-1:-1;48882:13:0::1;48914:4;48898:13;:7:::0;48908:3:::1;48898:13;:::i;:::-;:20;;;;:::i;:::-;48882:36:::0;-1:-1:-1;48925:12:0::1;48955:4;48940:12;:7:::0;48950:2:::1;48940:12;:::i;:::-;:19;;;;:::i;:::-;48925:34:::0;-1:-1:-1;48966:14:0::1;48997:4;48983:11;:7:::0;48993:1:::1;48983:11;:::i;:::-;:18;;;;:::i;:::-;49035:7;::::0;49027:44:::1;::::0;48966:35;;-1:-1:-1;49011:10:0::1;::::0;-1:-1:-1;;;;;49035:7:0;;::::1;::::0;49056:10;;49011;49027:44;49011:10;49027:44;49056:10;49035:7;49027:44:::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;49010:61;;;49086:5;49078:39;;;::::0;-1:-1:-1;;;49078:39:0;;9722:2:1;49078:39:0::1;::::0;::::1;9704:21:1::0;9761:2;9741:18;;;9734:30;-1:-1:-1;;;9780:18:1;;;9773:51;9841:18;;49078:39:0::1;9694:171:1::0;49078:39:0::1;49149:7;::::0;49141:42:::1;::::0;49125:10:::1;::::0;-1:-1:-1;;;;;49149:7:0::1;::::0;49170:8;;49125:10;49141:42;49125:10;49141:42;49170:8;49149:7;49141:42:::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;49124:59;;;49198:5;49190:39;;;::::0;-1:-1:-1;;;49190:39:0;;10072:2:1;49190:39:0::1;::::0;::::1;10054:21:1::0;10111:2;10091:18;;;10084:30;-1:-1:-1;;;10130:18:1;;;10123:51;10191:18;;49190:39:0::1;10044:171:1::0;49190:39:0::1;49261:7;::::0;49253:42:::1;::::0;49237:10:::1;::::0;-1:-1:-1;;;;;49261:7:0::1;::::0;49282:8;;49237:10;49253:42;49237:10;49253:42;49282:8;49261:7;49253:42:::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;49236:59;;;49310:5;49302:39;;;::::0;-1:-1:-1;;;49302:39:0;;11878:2:1;49302:39:0::1;::::0;::::1;11860:21:1::0;11917:2;11897:18;;;11890:30;-1:-1:-1;;;11936:18:1;;;11929:51;11997:18;;49302:39:0::1;11850:171:1::0;49302:39:0::1;49373:7;::::0;49365:42:::1;::::0;49349:10:::1;::::0;-1:-1:-1;;;;;49373:7:0::1;::::0;49394:8;;49349:10;49365:42;49349:10;49365:42;49394:8;49373:7;49365:42:::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;49348:59;;;49422:5;49414:39;;;::::0;-1:-1:-1;;;49414:39:0;;9372:2:1;49414:39:0::1;::::0;::::1;9354:21:1::0;9411:2;9391:18;;;9384:30;-1:-1:-1;;;9430:18:1;;;9423:51;9491:18;;49414:39:0::1;9344:171:1::0;49414:39:0::1;49485:7;::::0;49477:42:::1;::::0;49461:10:::1;::::0;-1:-1:-1;;;;;49485:7:0::1;::::0;49506:8;;49461:10;49477:42;49461:10;49477:42;49506:8;49485:7;49477:42:::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;49460:59;;;49534:5;49526:39;;;::::0;-1:-1:-1;;;49526:39:0;;12228:2:1;49526:39:0::1;::::0;::::1;12210:21:1::0;12267:2;12247:18;;;12240:30;-1:-1:-1;;;12286:18:1;;;12279:51;12347:18;;49526:39:0::1;12200:171:1::0;49526:39:0::1;49597:7;::::0;49589:41:::1;::::0;49573:10:::1;::::0;-1:-1:-1;;;;;49597:7:0::1;::::0;49618;;49573:10;49589:41;49573:10;49589:41;49618:7;49597;49589:41:::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;49572:58;;;49645:5;49637:39;;;::::0;-1:-1:-1;;;49637:39:0;;11178:2:1;49637:39:0::1;::::0;::::1;11160:21:1::0;11217:2;11197:18;;;11190:30;-1:-1:-1;;;11236:18:1;;;11229:51;11297:18;;49637:39:0::1;11150:171:1::0;49637:39:0::1;49708:7;::::0;49700:41:::1;::::0;49684:10:::1;::::0;-1:-1:-1;;;;;49708:7:0::1;::::0;49729;;49684:10;49700:41;49684:10;49700:41;49729:7;49708;49700:41:::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;49683:58;;;49756:5;49748:39;;;::::0;-1:-1:-1;;;49748:39:0;;11528:2:1;49748:39:0::1;::::0;::::1;11510:21:1::0;11567:2;11547:18;;;11540:30;-1:-1:-1;;;11586:18:1;;;11579:51;11647:18;;49748:39:0::1;11500:171:1::0;49748:39:0::1;49819:7;::::0;49811:41:::1;::::0;49795:10:::1;::::0;-1:-1:-1;;;;;49819:7:0::1;::::0;49840;;49795:10;49811:41;49795:10;49811:41;49840:7;49819;49811:41:::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;49794:58;;;49867:5;49859:39;;;::::0;-1:-1:-1;;;49859:39:0;;14315:2:1;49859:39:0::1;::::0;::::1;14297:21:1::0;14354:2;14334:18;;;14327:30;-1:-1:-1;;;14373:18:1;;;14366:51;14434:18;;49859:39:0::1;14287:171:1::0;49859:39:0::1;49930:7;::::0;49922:43:::1;::::0;49906:10:::1;::::0;-1:-1:-1;;;;;49930:7:0::1;::::0;49951:9;;49906:10;49922:43;49906:10;49922:43;49951:9;49930:7;49922:43:::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;49905:60;;;49980:5;49972:39;;;::::0;-1:-1:-1;;;49972:39:0;;14665:2:1;49972:39:0::1;::::0;::::1;14647:21:1::0;14704:2;14684:18;;;14677:30;-1:-1:-1;;;14723:18:1;;;14716:51;14784:18;;49972:39:0::1;14637:171:1::0;49972:39:0::1;48744:1273;;;;;;;;;;;;;;;48707:1310::o:0;29344:185::-;29482:39;29499:4;29505:2;29509:7;29482:39;;;;;;;;;;;;:16;:39::i;46866:58::-;46903:15;46909:2;46913:4;46903:5;:15::i;:::-;46866:58;:::o;46184:676::-;46319:29;;;-1:-1:-1;;;;;7794:32:1;;46319:29:0;;;7776:51:1;7843:18;;;7836:34;;;46294:12:0;;7749:18:1;;46319:29:0;;;;;;;;;;;;46309:40;;;;;;46294:55;;46364:37;46383:5;;46364:37;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;46390:4:0;;;-1:-1:-1;46396:4:0;;-1:-1:-1;46364:18:0;:37::i;:::-;46356:70;;;;-1:-1:-1;;;46356:70:0;;10829:2:1;46356:70:0;;;10811:21:1;10868:2;10848:18;;;10841:30;-1:-1:-1;;;10887:18:1;;;10880:50;10947:18;;46356:70:0;10801:170:1;46356:70:0;46435:10;46448:18;45257:12;46448:6;:18;:::i;:::-;46485:14;;;;;;;46477:23;;;;:7;:23;;;;;;;;-1:-1:-1;;;;;46477:32:0;;;;;;;;;;46435:31;;-1:-1:-1;46473:77:0;;46525:17;46534:8;46525:17;;:::i;:::-;;;46473:77;46579:5;46566:9;:18;46558:47;;;;-1:-1:-1;;;46558:47:0;;12939:2:1;46558:47:0;;;12921:21:1;12978:2;12958:18;;;12951:30;-1:-1:-1;;;12997:18:1;;;12990:46;13053:18;;46558:47:0;12911:166:1;46558:47:0;46647:10;;46637:6;46620:14;20682:7;20870:13;;20635:285;46620:14;:23;;;;:::i;:::-;:37;;46612:67;;;;-1:-1:-1;;;46612:67:0;;15015:2:1;46612:67:0;;;14997:21:1;15054:2;15034:18;;;15027:30;-1:-1:-1;;;15073:18:1;;;15066:47;15130:18;;46612:67:0;14987:167:1;46612:67:0;46696:14;;;;;;;46688:23;;;;:7;:23;;;;;;;;-1:-1:-1;;;;;46688:32:0;;;;;;;;;:42;;46724:6;;46688:23;:42;;46724:6;;46688:42;:::i;:::-;;;;-1:-1:-1;;46753:14:0;;;;;;;46745:23;;;;:7;:23;;;;;;;;-1:-1:-1;;;;;46745:32:0;;;;;;;;;;45316:1;-1:-1:-1;46745:54:0;46737:86;;;;-1:-1:-1;;;46737:86:0;;9024:2:1;46737:86:0;;;9006:21:1;9063:2;9043:18;;;9036:30;-1:-1:-1;;;9082:18:1;;;9075:49;9141:18;;46737:86:0;8996:169:1;46737:86:0;46832:22;46838:7;46847:6;46832:5;:22::i;:::-;46287:573;;46184:676;;;;;:::o;47099:82::-;6837:6;;-1:-1:-1;;;;;6837:6:0;43012:10;6984:23;6976:68;;;;-1:-1:-1;;;6976:68:0;;;;;;;:::i;:::-;47162:13;;::::1;::::0;:7:::1;::::0;:13:::1;::::0;::::1;::::0;::::1;:::i;:::-;;47099:82:::0;:::o;25993:144::-;26057:7;26100:27;26119:7;26100:18;:27::i;45543:21::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;21847:234::-;21911:7;21953:5;21931:70;;21973:28;;-1:-1:-1;;;21973:28:0;;;;;;;;;;;21931:70;-1:-1:-1;;;;;;22019:25:0;;;;;:18;:25;;;;;;17192:13;22019:54;;21847:234::o;7415:103::-;6837:6;;-1:-1:-1;;;;;6837:6:0;43012:10;6984:23;6976:68;;;;-1:-1:-1;;;6976:68:0;;;;;;;:::i;:::-;7480:30:::1;7507:1;7480:18;:30::i;:::-;7415:103::o:0;46930:67::-;6837:6;;-1:-1:-1;;;;;6837:6:0;43012:10;6984:23;6976:68;;;;-1:-1:-1;;;6976:68:0;;;;;;;:::i;:::-;46985:6:::1;::::0;;-1:-1:-1;;46975:16:0;::::1;46985:6;::::0;;::::1;46984:7;46975:16;::::0;;46930:67::o;47003:90::-;6837:6;;-1:-1:-1;;;;;6837:6:0;43012:10;6984:23;6976:68;;;;-1:-1:-1;;;6976:68:0;;;;;;;:::i;:::-;47070:4:::1;:17:::0;47003:90::o;26373:104::-;26429:13;26462:7;26455:14;;;;;:::i;45767:411::-;45824:6;;;;45816:34;;;;-1:-1:-1;;;45816:34:0;;13284:2:1;45816:34:0;;;13266:21:1;13323:2;13303:18;;;13296:30;-1:-1:-1;;;13342:18:1;;;13335:45;13397:18;;45816:34:0;13256:165:1;45816:34:0;45887:9;45865:18;45257:12;45865:6;:18;:::i;:::-;:31;45857:60;;;;-1:-1:-1;;;45857:60:0;;12939:2:1;45857:60:0;;;12921:21:1;12978:2;12958:18;;;12951:30;-1:-1:-1;;;12997:18:1;;;12990:46;13053:18;;45857:60:0;12911:166:1;45857:60:0;45959:10;;45949:6;45932:14;20682:7;20870:13;;20635:285;45932:14;:23;;;;:::i;:::-;:37;;45924:67;;;;-1:-1:-1;;;45924:67:0;;15015:2:1;45924:67:0;;;14997:21:1;15054:2;15034:18;;;15027:30;-1:-1:-1;;;15073:18:1;;;15066:47;15130:18;;45924:67:0;14987:167:1;45924:67:0;46008:14;;;;;;;46000:23;;;;:7;:23;;;;;;;;46024:10;46000:35;;;;;;;:45;;46039:6;;46000:23;:45;;46039:6;;46000:45;:::i;:::-;;;;-1:-1:-1;;46068:14:0;;;;;;;46060:23;;;;:7;:23;;;;;;;;46084:10;46060:35;;;;;;;;45361:1;-1:-1:-1;46060:54:0;46052:86;;;;-1:-1:-1;;;46052:86:0;;9024:2:1;46052:86:0;;;9006:21:1;9063:2;9043:18;;;9036:30;-1:-1:-1;;;9082:18:1;;;9075:49;9141:18;;46052:86:0;8996:169:1;46052:86:0;46147:25;46153:10;46165:6;46147:5;:25::i;28493:308::-;-1:-1:-1;;;;;28592:31:0;;43012:10;28592:31;28588:61;;;28632:17;;-1:-1:-1;;;28632:17:0;;;;;;;;;;;28588:61;43012:10;28662:39;;;;:18;:39;;;;;;;;-1:-1:-1;;;;;28662:49:0;;;;;;;;;;;;:60;;-1:-1:-1;;28662:60:0;;;;;;;;;;28738:55;;8021:41:1;;;28662:49:0;;43012:10;28738:55;;7994:18:1;28738:55:0;;;;;;;28493:308;;:::o;47614:275::-;6837:6;;-1:-1:-1;;;;;6837:6:0;43012:10;6984:23;6976:68;;;;-1:-1:-1;;;6976:68:0;;;;;;;:::i;:::-;20488:12;;20275:7;20472:13;:28;47682:9:::1;:25;47674:52;;;::::0;-1:-1:-1;;;47674:52:0;;13628:2:1;47674:52:0::1;::::0;::::1;13610:21:1::0;13667:2;13647:18;;;13640:30;-1:-1:-1;;;13686:18:1;;;13679:44;13740:18;;47674:52:0::1;13600:164:1::0;47674:52:0::1;47754:10;;47741:9;:23;;47733:51;;;::::0;-1:-1:-1;;;47733:51:0;;13971:2:1;47733:51:0::1;::::0;::::1;13953:21:1::0;14010:2;13990:18;;;13983:30;-1:-1:-1;;;14029:18:1;;;14022:45;14084:18;;47733:51:0::1;13943:165:1::0;47733:51:0::1;47800:3;47793:4;:10:::0;47810:14:::1;:19:::0;;47828:1:::1;::::0;47810:14;47828:1;;47810:19:::1;::::0;47828:1;;47810:19:::1;::::0;::::1;;;;:::i;:::-;::::0;;::::1;::::0;;::::1;;::::0;;;::::1;::::0;;::::1;::::0;;;::::1;;::::0;;::::1;;::::0;;-1:-1:-1;47836:10:0::1;:22:::0;-1:-1:-1;47865:14:0::1;:18:::0;47614:275::o;29600:396::-;29767:28;29777:4;29783:2;29787:7;29767:9;:28::i;:::-;-1:-1:-1;;;;;29810:14:0;;;:19;29806:183;;29849:56;29880:4;29886:2;29890:7;29899:5;29849:30;:56::i;:::-;29844:145;;29933:40;;-1:-1:-1;;;29933:40:0;;;;;;;;;;;29844:145;29600:396;;;;:::o;26548:318::-;26621:13;26652:16;26660:7;26652;:16::i;:::-;26647:59;;26677:29;;-1:-1:-1;;;26677:29:0;;;;;;;;;;;26647:59;26719:21;26743:10;27195:9;;;;;;;;;-1:-1:-1;27195:9:0;;;27118:94;26743:10;26719:34;;26777:7;26771:21;26796:1;26771:26;;:87;;;;;;;;;;;;;;;;;26824:7;26833:18;26843:7;26833:9;:18::i;:::-;26807:45;;;;;;;;;:::i;:::-;;;;;;;;;;;;;26771:87;26764:94;26548:318;-1:-1:-1;;;26548:318:0:o;47187:78::-;6837:6;;-1:-1:-1;;;;;6837:6:0;43012:10;6984:23;6976:68;;;;-1:-1:-1;;;6976:68:0;;;;;;;:::i;:::-;20488:12;;20275:7;20472:13;:28;47233:10:::1;:26:::0;47187:78::o;7673:201::-;6837:6;;-1:-1:-1;;;;;6837:6:0;43012:10;6984:23;6976:68;;;;-1:-1:-1;;;6976:68:0;;;;;;;:::i;:::-;-1:-1:-1;;;;;7762:22:0;::::1;7754:73;;;::::0;-1:-1:-1;;;7754:73:0;;10422:2:1;7754:73:0::1;::::0;::::1;10404:21:1::0;10461:2;10441:18;;;10434:30;10500:34;10480:18;;;10473:62;-1:-1:-1;;;10551:18:1;;;10544:36;10597:19;;7754:73:0::1;10394:228:1::0;7754:73:0::1;7838:28;7857:8;7838:18;:28::i;30251:273::-:0;30308:4;30398:13;;30388:7;:23;30345:152;;;;-1:-1:-1;;30449:26:0;;;;:17;:26;;;;;;-1:-1:-1;;;30449:43:0;:48;;30251:273::o;23508:1129::-;23575:7;23610;23712:13;;23705:4;:20;23701:869;;;23750:14;23767:23;;;:17;:23;;;;;;-1:-1:-1;;;23856:23:0;;23852:699;;24375:113;24382:11;24375:113;;-1:-1:-1;;;24453:6:0;24435:25;;;;:17;:25;;;;;;24375:113;;23852:699;23727:843;23701:869;24598:31;;-1:-1:-1;;;24598:31:0;;;;;;;;;;;32053:1610;32118:20;32141:13;32187:2;32165:58;;32204:19;;-1:-1:-1;;;32204:19:0;;;;;;;;;;;32165:58;32238:13;32234:44;;32260:18;;-1:-1:-1;;;32260:18:0;;;;;;;;;;;32234:44;-1:-1:-1;;;;;32827:22:0;;;;;;:18;:22;;;;17329:2;32827:22;;;:70;;32865:31;32853:44;;32827:70;;;33140:31;;;:17;:31;;;;;33233:15;17846:3;33233:41;33191:84;;-1:-1:-1;33311:13:0;;18105:3;33296:56;33191:162;33140:213;;33399:119;33426:49;;33466:8;;;;33451:23;;;-1:-1:-1;;;;;33426:49:0;;;33443:1;;33426:49;;33443:1;;33426:49;33508:8;33499:6;:17;33399:119;;-1:-1:-1;33550:23:0;33534:13;:39;-1:-1:-1;47271:337:0:o;33917:2654::-;34032:27;34062;34081:7;34062:18;:27::i;:::-;34032:57;;34147:4;-1:-1:-1;;;;;34106:45:0;34122:19;-1:-1:-1;;;;;34106:45:0;;34102:86;;34160:28;;-1:-1:-1;;;34160:28:0;;;;;;;;;;;34102:86;34201:23;34227:24;;;:15;:24;;;;;;-1:-1:-1;;;;;34227:24:0;;;;34201:23;34290:27;;43012:10;34290:27;;:87;;-1:-1:-1;34334:43:0;34351:4;43012:10;28872:164;:::i;34334:43::-;34290:142;;;-1:-1:-1;;;;;;34394:38:0;;43012:10;34394:38;34290:142;34264:169;;34451:17;34446:66;;34477:35;;-1:-1:-1;;;34477:35:0;;;;;;;;;;;34446:66;34545:2;34523:62;;34562:23;;-1:-1:-1;;;34562:23:0;;;;;;;;;;;34523:62;34729:15;34711:39;34707:103;;34774:24;;;;:15;:24;;;;;34767:31;;-1:-1:-1;;;;;;34767:31:0;;;34707:103;-1:-1:-1;;;;;35177:24:0;;;;;;;:18;:24;;;;;;;;35175:26;;-1:-1:-1;;35175:26:0;;;35246:22;;;;;;;;35244:24;;-1:-1:-1;35244:24:0;;;35539:26;;;:17;:26;;;-1:-1:-1;;;35627:15:0;17846:3;35627:41;35585:84;;:128;;35539:174;;;35833:46;;35829:626;;35937:1;35927:11;;35905:19;36060:30;;;:17;:30;;;;;;36056:384;;36198:13;;36183:11;:28;36179:242;;36345:30;;;;:17;:30;;;;;:52;;;36179:242;35886:569;35829:626;36502:7;36498:2;-1:-1:-1;;;;;36483:27:0;36492:4;-1:-1:-1;;;;;36483:27:0;;;;;;;;;;;34021:2550;;;33917:2654;;;:::o;36967:2935::-;37047:27;37077;37096:7;37077:18;:27::i;:::-;37117:12;37206:24;;;:15;:24;;;;;;37047:57;;-1:-1:-1;37047:57:0;;-1:-1:-1;;;;;37206:24:0;37243:306;;;;37277:22;43012:10;-1:-1:-1;;;;;37303:27:0;;;;:91;;-1:-1:-1;37351:43:0;37368:4;43012:10;28872:164;:::i;37351:43::-;37303:150;;;-1:-1:-1;;;;;;37415:38:0;;43012:10;37415:38;37303:150;37277:177;;37476:17;37471:66;;37502:35;;-1:-1:-1;;;37502:35:0;;;;;;;;;;;37471:66;37262:287;37243:306;37700:15;37682:39;37678:103;;37745:24;;;;:15;:24;;;;;37738:31;;-1:-1:-1;;;;;;37738:31:0;;;37678:103;-1:-1:-1;;;;;38369:24:0;;;;;;:18;:24;;;;;;;;:59;;38397:31;38369:59;;;38666:26;;;:17;:26;;;;;-1:-1:-1;;;38756:15:0;17846:3;38756:41;38712:86;;:164;38666:210;;-1:-1:-1;;;38996:46:0;;38992:626;;39100:1;39090:11;;39068:19;39223:30;;;:17;:30;;;;;;39219:384;;39361:13;;39346:11;:28;39342:242;;39508:30;;;;:17;:30;;;;;:52;;;39342:242;39049:569;38992:626;39646:35;;39673:7;;39669:1;;-1:-1:-1;;;;;39646:35:0;;;;;39669:1;;39646:35;-1:-1:-1;;39869:12:0;:14;;;;;;-1:-1:-1;;;36967:2935:0:o;1220:190::-;1345:4;1398;1369:25;1382:5;1389:4;1369:12;:25::i;:::-;:33;;1220:190;-1:-1:-1;;;;1220:190:0:o;8034:191::-;8127:6;;;-1:-1:-1;;;;;8144:17:0;;;-1:-1:-1;;;;;;8144:17:0;;;;;;;8177:40;;8127:6;;;8144:17;8127:6;;8177:40;;8108:16;;8177:40;8097:128;8034:191;:::o;40394:716::-;40578:88;;-1:-1:-1;;;40578:88:0;;40557:4;;-1:-1:-1;;;;;40578:45:0;;;;;:88;;43012:10;;40645:4;;40651:7;;40660:5;;40578:88;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;40578:88:0;;;;;;;;-1:-1:-1;;40578:88:0;;;;;;;;;;;;:::i;:::-;;;40574:529;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;40861:13:0;;40857:235;;40907:40;;-1:-1:-1;;;40907:40:0;;;;;;;;;;;40857:235;41050:6;41044:13;41035:6;41031:2;41027:15;41020:38;40574:529;-1:-1:-1;;;;;;40737:64:0;-1:-1:-1;;;40737:64:0;;-1:-1:-1;40574:529:0;40394:716;;;;;;:::o;43136:1960::-;43605:4;43599:11;;43612:3;43595:21;;43690:17;;;;44386:11;;;44265:5;44518:2;44532;44522:13;;44514:22;44386:11;44501:36;44573:2;44563:13;;44157:697;44592:4;44157:697;;;44783:1;44778:3;44774:11;44767:18;;44834:2;44828:4;44824:13;44820:2;44816:22;44811:3;44803:36;44687:2;44677:13;;44157:697;;;-1:-1:-1;44884:13:0;;;-1:-1:-1;;44999:12:0;;;45059:19;;;44999:12;43136:1960;-1:-1:-1;43136:1960:0:o;1771:675::-;1854:7;1897:4;1854:7;1912:497;1936:5;:12;1932:1;:16;1912:497;;;1970:20;1993:5;1999:1;1993:8;;;;;;;;:::i;:::-;;;;;;;1970:31;;2036:12;2020;:28;2016:382;;2522:13;2572:15;;;2608:4;2601:15;;;2655:4;2639:21;;2148:57;;2016:382;;;2522:13;2572:15;;;2608:4;2601:15;;;2655:4;2639:21;;2325:57;;2016:382;-1:-1:-1;1950:3:0;;;;:::i;:::-;;;;1912:497;;;-1:-1:-1;2426:12:0;1771:675;-1:-1:-1;;;1771:675:0:o;-1:-1:-1:-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;:::o;:::-;;;;;;;;;;;;;;;14:631:1;78:5;108:18;149:2;141:6;138:14;135:2;;;155:18;;:::i;:::-;230:2;224:9;198:2;284:15;;-1:-1:-1;;280:24:1;;;306:2;276:33;272:42;260:55;;;330:18;;;350:22;;;327:46;324:2;;;376:18;;:::i;:::-;416:10;412:2;405:22;445:6;436:15;;475:6;467;460:22;515:3;506:6;501:3;497:16;494:25;491:2;;;532:1;529;522:12;491:2;582:6;577:3;570:4;562:6;558:17;545:44;637:1;630:4;621:6;613;609:19;605:30;598:41;;;;88:557;;;;;:::o;650:173::-;718:20;;-1:-1:-1;;;;;767:31:1;;757:42;;747:2;;813:1;810;803:12;747:2;699:124;;;:::o;828:367::-;891:8;901:6;955:3;948:4;940:6;936:17;932:27;922:2;;973:1;970;963:12;922:2;-1:-1:-1;996:20:1;;1039:18;1028:30;;1025:2;;;1071:1;1068;1061:12;1025:2;1108:4;1100:6;1096:17;1084:29;;1168:3;1161:4;1151:6;1148:1;1144:14;1136:6;1132:27;1128:38;1125:47;1122:2;;;1185:1;1182;1175:12;1122:2;912:283;;;;;:::o;1200:186::-;1259:6;1312:2;1300:9;1291:7;1287:23;1283:32;1280:2;;;1328:1;1325;1318:12;1280:2;1351:29;1370:9;1351:29;:::i;1391:260::-;1459:6;1467;1520:2;1508:9;1499:7;1495:23;1491:32;1488:2;;;1536:1;1533;1526:12;1488:2;1559:29;1578:9;1559:29;:::i;:::-;1549:39;;1607:38;1641:2;1630:9;1626:18;1607:38;:::i;:::-;1597:48;;1478:173;;;;;:::o;1656:328::-;1733:6;1741;1749;1802:2;1790:9;1781:7;1777:23;1773:32;1770:2;;;1818:1;1815;1808:12;1770:2;1841:29;1860:9;1841:29;:::i;:::-;1831:39;;1889:38;1923:2;1912:9;1908:18;1889:38;:::i;:::-;1879:48;;1974:2;1963:9;1959:18;1946:32;1936:42;;1760:224;;;;;:::o;1989:666::-;2084:6;2092;2100;2108;2161:3;2149:9;2140:7;2136:23;2132:33;2129:2;;;2178:1;2175;2168:12;2129:2;2201:29;2220:9;2201:29;:::i;:::-;2191:39;;2249:38;2283:2;2272:9;2268:18;2249:38;:::i;:::-;2239:48;;2334:2;2323:9;2319:18;2306:32;2296:42;;2389:2;2378:9;2374:18;2361:32;2416:18;2408:6;2405:30;2402:2;;;2448:1;2445;2438:12;2402:2;2471:22;;2524:4;2516:13;;2512:27;-1:-1:-1;2502:2:1;;2553:1;2550;2543:12;2502:2;2576:73;2641:7;2636:2;2623:16;2618:2;2614;2610:11;2576:73;:::i;:::-;2566:83;;;2119:536;;;;;;;:::o;2660:347::-;2725:6;2733;2786:2;2774:9;2765:7;2761:23;2757:32;2754:2;;;2802:1;2799;2792:12;2754:2;2825:29;2844:9;2825:29;:::i;:::-;2815:39;;2904:2;2893:9;2889:18;2876:32;2951:5;2944:13;2937:21;2930:5;2927:32;2917:2;;2973:1;2970;2963:12;2917:2;2996:5;2986:15;;;2744:263;;;;;:::o;3012:254::-;3080:6;3088;3141:2;3129:9;3120:7;3116:23;3112:32;3109:2;;;3157:1;3154;3147:12;3109:2;3180:29;3199:9;3180:29;:::i;:::-;3170:39;3256:2;3241:18;;;;3228:32;;-1:-1:-1;;;3099:167:1:o;3271:648::-;3384:6;3392;3400;3408;3416;3469:3;3457:9;3448:7;3444:23;3440:33;3437:2;;;3486:1;3483;3476:12;3437:2;3509:29;3528:9;3509:29;:::i;:::-;3499:39;;3585:2;3574:9;3570:18;3557:32;3547:42;;3636:2;3625:9;3621:18;3608:32;3598:42;;3691:2;3680:9;3676:18;3663:32;3718:18;3710:6;3707:30;3704:2;;;3750:1;3747;3740:12;3704:2;3789:70;3851:7;3842:6;3831:9;3827:22;3789:70;:::i;:::-;3427:492;;;;-1:-1:-1;3427:492:1;;-1:-1:-1;3878:8:1;;3763:96;3427:492;-1:-1:-1;;;3427:492:1:o;3924:437::-;4010:6;4018;4071:2;4059:9;4050:7;4046:23;4042:32;4039:2;;;4087:1;4084;4077:12;4039:2;4127:9;4114:23;4160:18;4152:6;4149:30;4146:2;;;4192:1;4189;4182:12;4146:2;4231:70;4293:7;4284:6;4273:9;4269:22;4231:70;:::i;:::-;4320:8;;4205:96;;-1:-1:-1;4029:332:1;-1:-1:-1;;;;4029:332:1:o;4366:180::-;4425:6;4478:2;4466:9;4457:7;4453:23;4449:32;4446:2;;;4494:1;4491;4484:12;4446:2;-1:-1:-1;4517:23:1;;4436:110;-1:-1:-1;4436:110:1:o;4551:245::-;4609:6;4662:2;4650:9;4641:7;4637:23;4633:32;4630:2;;;4678:1;4675;4668:12;4630:2;4717:9;4704:23;4736:30;4760:5;4736:30;:::i;4801:249::-;4870:6;4923:2;4911:9;4902:7;4898:23;4894:32;4891:2;;;4939:1;4936;4929:12;4891:2;4971:9;4965:16;4990:30;5014:5;4990:30;:::i;5055:450::-;5124:6;5177:2;5165:9;5156:7;5152:23;5148:32;5145:2;;;5193:1;5190;5183:12;5145:2;5233:9;5220:23;5266:18;5258:6;5255:30;5252:2;;;5298:1;5295;5288:12;5252:2;5321:22;;5374:4;5366:13;;5362:27;-1:-1:-1;5352:2:1;;5403:1;5400;5393:12;5352:2;5426:73;5491:7;5486:2;5473:16;5468:2;5464;5460:11;5426:73;:::i;5695:254::-;5763:6;5771;5824:2;5812:9;5803:7;5799:23;5795:32;5792:2;;;5840:1;5837;5830:12;5792:2;5876:9;5863:23;5853:33;;5905:38;5939:2;5928:9;5924:18;5905:38;:::i;5954:257::-;5995:3;6033:5;6027:12;6060:6;6055:3;6048:19;6076:63;6132:6;6125:4;6120:3;6116:14;6109:4;6102:5;6098:16;6076:63;:::i;:::-;6193:2;6172:15;-1:-1:-1;;6168:29:1;6159:39;;;;6200:4;6155:50;;6003:208;-1:-1:-1;;6003:208:1:o;6216:470::-;6395:3;6433:6;6427:13;6449:53;6495:6;6490:3;6483:4;6475:6;6471:17;6449:53;:::i;:::-;6565:13;;6524:16;;;;6587:57;6565:13;6524:16;6621:4;6609:17;;6587:57;:::i;:::-;6660:20;;6403:283;-1:-1:-1;;;;6403:283:1:o;7109:488::-;-1:-1:-1;;;;;7378:15:1;;;7360:34;;7430:15;;7425:2;7410:18;;7403:43;7477:2;7462:18;;7455:34;;;7525:3;7520:2;7505:18;;7498:31;;;7303:4;;7546:45;;7571:19;;7563:6;7546:45;:::i;:::-;7538:53;7312:285;-1:-1:-1;;;;;;7312:285:1:o;8255:219::-;8404:2;8393:9;8386:21;8367:4;8424:44;8464:2;8453:9;8449:18;8441:6;8424:44;:::i;12376:356::-;12578:2;12560:21;;;12597:18;;;12590:30;12656:34;12651:2;12636:18;;12629:62;12723:2;12708:18;;12550:182::o;15872:128::-;15912:3;15943:1;15939:6;15936:1;15933:13;15930:2;;;15949:18;;:::i;:::-;-1:-1:-1;15985:9:1;;15920:80::o;16005:204::-;16043:3;16079:4;16076:1;16072:12;16111:4;16108:1;16104:12;16146:3;16140:4;16136:14;16131:3;16128:23;16125:2;;;16154:18;;:::i;:::-;16190:13;;16051:158;-1:-1:-1;;;16051:158:1:o;16214:217::-;16254:1;16280;16270:2;;16324:10;16319:3;16315:20;16312:1;16305:31;16359:4;16356:1;16349:15;16387:4;16384:1;16377:15;16270:2;-1:-1:-1;16416:9:1;;16260:171::o;16436:168::-;16476:7;16542:1;16538;16534:6;16530:14;16527:1;16524:21;16519:1;16512:9;16505:17;16501:45;16498:2;;;16549:18;;:::i;:::-;-1:-1:-1;16589:9:1;;16488:116::o;16609:125::-;16649:4;16677:1;16674;16671:8;16668:2;;;16682:18;;:::i;:::-;-1:-1:-1;16719:9:1;;16658:76::o;16739:258::-;16811:1;16821:113;16835:6;16832:1;16829:13;16821:113;;;16911:11;;;16905:18;16892:11;;;16885:39;16857:2;16850:10;16821:113;;;16952:6;16949:1;16946:13;16943:2;;;-1:-1:-1;;16987:1:1;16969:16;;16962:27;16792:205::o;17002:380::-;17081:1;17077:12;;;;17124;;;17145:2;;17199:4;17191:6;17187:17;17177:27;;17145:2;17252;17244:6;17241:14;17221:18;17218:38;17215:2;;;17298:10;17293:3;17289:20;17286:1;17279:31;17333:4;17330:1;17323:15;17361:4;17358:1;17351:15;17215:2;;17057:325;;;:::o;17387:135::-;17426:3;-1:-1:-1;;17447:17:1;;17444:2;;;17467:18;;:::i;:::-;-1:-1:-1;17514:1:1;17503:13;;17434:88::o;17527:127::-;17588:10;17583:3;17579:20;17576:1;17569:31;17619:4;17616:1;17609:15;17643:4;17640:1;17633:15;17659:127;17720:10;17715:3;17711:20;17708:1;17701:31;17751:4;17748:1;17741:15;17775:4;17772:1;17765:15;17791:127;17852:10;17847:3;17843:20;17840:1;17833:31;17883:4;17880:1;17873:15;17907:4;17904:1;17897:15;17923:131;-1:-1:-1;;;;;;17997:32:1;;17987:43;;17977:2;;18044:1;18041;18034:12

Swarm Source

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