ETH Price: $3,404.77 (+1.39%)
Gas: 8 Gwei

Token

Pee Pee (Pee)
 

Overview

Max Total Supply

3,358 Pee

Holders

508

Market

Volume (24H)

N/A

Min Price (24H)

N/A

Max Price (24H)

N/A
Balance
13 Pee
0xc59dc5b9906728a19070bed06f10e31da2313ac6
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:
Pee

Compiler Version
v0.8.9+commit.e5eed63a

Optimization Enabled:
Yes with 200 runs

Other Settings:
default evmVersion, MIT license

Contract Source Code (Solidity Multiple files format)

File 9 of 11: Pee.sol
// SPDX-License-Identifier: MIT

pragma solidity >=0.8.9 <0.9.0;

import './ERC721AQueryable.sol';
import './Ownable.sol';
import './MerkleProof.sol';
import './ReentrancyGuard.sol';
import './Strings.sol';


interface IERC20 {
    function totalSupply() external view returns (uint256);
    function balanceOf(address account) external view returns (uint256);
    function transfer(address recipient, uint256 amount) external returns (bool);
    function allowance(address owner, address spender) external view returns (uint256);
    function approve(address spender, uint256 amount) external returns (bool);
    function transferFrom(address sender, address recipient, uint256 amount) external returns (bool);

    function mint(address to, uint256 amount) external returns (bool);
    function burn(uint256 amount) external returns (bool);

    event Transfer(address indexed from, address indexed to, uint256 value);
    event Approval(address indexed owner, address indexed spender, uint256 value);
}

contract Pee is ERC721AQueryable, Ownable, ReentrancyGuard {

  using Strings for uint256;

  bytes32 public merkleRoot;
  mapping(address => bool) public whitelistClaimed;
  mapping(address => uint256)public mintedAmount;
  mapping(address =>bool)public isfree;
  mapping(uint256=>bool)public isClaim;
  IERC20 public PeeCoinContract;
  address public Peeaddress;
  bool public holderClaim_state = false;
  uint   public maxPerFree = 1;
  uint   public whitelistPerFree = 3;
  string public uriPrefix = '';
  string public uriSuffix = '.json';
  string public hiddenMetadataUri;
  uint public totalFreeMinted = 0;
  uint256 public cost;
  uint256 public maxSupply;
  uint256 public maxMintAmountPerTx;

  bool public paused = true;
  bool public whitelistMintEnabled = false;
  bool public revealed = false;

  constructor(
    string memory _tokenName,
    string memory _tokenSymbol,
    uint256 _cost,
    uint256 _maxSupply,
    uint256 _maxMintAmountPerTx,
    string memory _hiddenMetadataUri
  ) ERC721A(_tokenName, _tokenSymbol) {
    setCost(_cost);

    maxSupply = _maxSupply;
    Peeaddress = address(this);
    setMaxMintAmountPerTx(_maxMintAmountPerTx);
    setHiddenMetadataUri(_hiddenMetadataUri);
  }




  function whitelistMint(uint256 _mintAmount, bytes32[] calldata _merkleProof) public payable {
    require(_mintAmount > 0 && _mintAmount <= maxMintAmountPerTx, 'Invalid mint amount!');
    require(totalSupply() + _mintAmount <= maxSupply, 'Max supply exceeded!');
    require(msg.value >= cost * _mintAmount - cost*whitelistPerFree, 'Insufficient funds!');
    require(whitelistMintEnabled, 'The whitelist sale is not enabled!');
    require(!whitelistClaimed[_msgSender()], 'Address already claimed!');
    bytes32 leaf = keccak256(abi.encodePacked(_msgSender()));
    require(_msgSender()==tx.origin,'The minter is another contract');
    require(MerkleProof.verify(_merkleProof, merkleRoot, leaf), 'Invalid proof!');
    require(mintedAmount[_msgSender()]<20,'Maximum number of wallets is 20');
    require(mintedAmount[_msgSender()]+_mintAmount<=20,'Maximum number of wallets is 20');
    totalFreeMinted += whitelistPerFree;
    whitelistClaimed[_msgSender()] = true;
    isfree[_msgSender()]=true;
    mintedAmount[_msgSender()] +=_mintAmount;
    _safeMint(_msgSender(), _mintAmount);
  }

  function setPeecoinaddress(address Peeadd_) public onlyOwner {
      PeeCoinContract = IERC20(Peeadd_);
  }

 function holderClaim(uint256[] memory tokenIds) external {
    require(holderClaim_state, 'Activity redemption has not yet started');
    uint256 claimAmount = 5000*10**18;
    uint256 tokenCount = tokenIds.length;
    address sender = msg.sender;
    for (uint256 i = 0; i < tokenCount; i++) {
        uint256 tokenId = tokenIds[i];
        require(ownerOf(tokenId) == sender, "You don't own this token");
        if (!isClaim[tokenId]) {
            isClaim[tokenId] = true;
            PeeCoinContract.transfer(sender, claimAmount);
        }
    }
}
  function setholderClaimstate(bool _state)public onlyOwner{
    holderClaim_state=_state;
  }


 function mint(uint256 _mintAmount) public payable {
    require(_mintAmount > 0 && _mintAmount <= maxMintAmountPerTx, 'Invalid mint amount!');
    require(totalSupply() + _mintAmount <= maxSupply, 'Max supply exceeded!');
    require(!paused, 'The contract is paused!');
    require(_msgSender()==tx.origin,'The minter is another contract');
    require(mintedAmount[_msgSender()]+_mintAmount<=20,'Maximum number of wallets is 20');
    if (!isfree[_msgSender()]) {
        require(msg.value >= (_mintAmount * cost) - cost*maxPerFree, 'Insufficient funds!');
        totalFreeMinted += maxPerFree;
        mintedAmount[_msgSender()] += _mintAmount;
        isfree[_msgSender()] = true;
    } else {
        require(msg.value >= (_mintAmount * cost), 'Insufficient funds!');
        mintedAmount[_msgSender()] += _mintAmount;
    }
    _safeMint(_msgSender(), _mintAmount);
}

  
  function mintForAddress(uint256 _mintAmount, address _receiver) public onlyOwner {
    require(_mintAmount > 0 && _mintAmount <= maxMintAmountPerTx, 'Invalid mint amount!');
    require(totalSupply() + _mintAmount <= maxSupply, 'Max supply exceeded!');
    _safeMint(_receiver, _mintAmount);
  }

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


  function tokenURI(uint256 _tokenId) public view virtual override returns (string memory) {
    require(_exists(_tokenId), 'ERC721Metadata: URI query for nonexistent token');

    if (revealed == false) {
      return hiddenMetadataUri;
    }

  
    string memory currentBaseURI = _baseURI();
    return bytes(currentBaseURI).length > 0
        ? string(abi.encodePacked(currentBaseURI, _tokenId.toString(), uriSuffix))
        : '';
  }

  function setRevealed(bool _state) public onlyOwner {
    revealed = _state;
  }

  function setCost(uint256 _cost) public onlyOwner {
    cost = _cost;
  }

  function setMaxPerFree(uint freenum_)public onlyOwner{
    maxPerFree = freenum_;
  }
  function setWhitelistPerFree(uint freenum)public onlyOwner{
    whitelistPerFree = freenum;
  }
  function setMaxMintAmountPerTx(uint256 _maxMintAmountPerTx) public onlyOwner {
    maxMintAmountPerTx = _maxMintAmountPerTx;
  }

  function setHiddenMetadataUri(string memory _hiddenMetadataUri) public onlyOwner {
    hiddenMetadataUri = _hiddenMetadataUri;
  }

  function setUriPrefix(string memory _uriPrefix) public onlyOwner {
    uriPrefix = _uriPrefix;
  }

  function setUriSuffix(string memory _uriSuffix) public onlyOwner {
    uriSuffix = _uriSuffix;
  }

  function setPaused(bool _state) public onlyOwner {
    paused = _state;
  }

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

  function setWhitelistMintEnabled(bool _state) public onlyOwner {
    whitelistMintEnabled = _state;
  }

  function withdraw() public onlyOwner nonReentrant {


    (bool os, ) = payable(owner()).call{value: address(this).balance}('');
    require(os);

  }
  
  function withdrawPeetoken(uint Amount_) public onlyOwner {
    PeeCoinContract.transfer(owner(), Amount_);

  }

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

File 1 of 11: Context.sol
// SPDX-License-Identifier: MIT
// 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 2 of 11: ERC721A.sol
// SPDX-License-Identifier: MIT
// ERC721A Contracts v4.2.3
// Creator: Chiru Labs

pragma solidity ^0.8.4;

import './IERC721A.sol';

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

    // Token name
    string private _name;

    // Token symbol
    string private _symbol;

    // Mapping from token ID to ownership details
    // An empty struct value does not necessarily mean the token is unowned.
    // See {_packedOwnershipOf} implementation for details.
    //
    // Bits Layout:
    // - [0..159]   `addr`
    // - [160..223] `startTimestamp`
    // - [224]      `burned`
    // - [225]      `nextInitialized`
    // - [232..255] `extraData`
    mapping(uint256 => uint256) private _packedOwnerships;

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

    /**
     * @dev Returns the Uniform Resource Identifier (URI) for `tokenId` token.
     */
    function tokenURI(uint256 tokenId) public view virtual override returns (string memory) {
        if (!_exists(tokenId)) _revert(URIQueryForNonexistentToken.selector);

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

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

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

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

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

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

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

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

    /**
     * Returns the packed ownership data of `tokenId`.
     */
    function _packedOwnershipOf(uint256 tokenId) private view returns (uint256 packed) {
        if (_startTokenId() <= tokenId) {
            packed = _packedOwnerships[tokenId];
            // If the data at the starting slot does not exist, start the scan.
            if (packed == 0) {
                if (tokenId >= _currentIndex) _revert(OwnerQueryForNonexistentToken.selector);
                // Invariant:
                // There will always be an initialized ownership slot
                // (i.e. `ownership.addr != address(0) && ownership.burned == false`)
                // before an unintialized ownership slot
                // (i.e. `ownership.addr == address(0) && ownership.burned == false`)
                // Hence, `tokenId` will not underflow.
                //
                // We can directly compare the packed value.
                // If the address is zero, packed will be zero.
                for (;;) {
                    unchecked {
                        packed = _packedOwnerships[--tokenId];
                    }
                    if (packed == 0) continue;
                    if (packed & _BITMASK_BURNED == 0) return packed;
                    // Otherwise, the token is burned, and we must revert.
                    // This handles the case of batch burned tokens, where only the burned bit
                    // of the starting slot is set, and remaining slots are left uninitialized.
                    _revert(OwnerQueryForNonexistentToken.selector);
                }
            }
            // Otherwise, the data exists and we can skip the scan.
            // This is possible because we have already achieved the target condition.
            // This saves 2143 gas on transfers of initialized tokens.
            // If the token is not burned, return `packed`. Otherwise, revert.
            if (packed & _BITMASK_BURNED == 0) return packed;
        }
        _revert(OwnerQueryForNonexistentToken.selector);
    }

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

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

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

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

    /**
     * @dev Gives permission to `to` to transfer `tokenId` token to another account. See {ERC721A-_approve}.
     *
     * Requirements:
     *
     * - The caller must own the token or be an approved operator.
     */
    function approve(address to, uint256 tokenId) public payable virtual override {
        _approve(to, tokenId, true);
    }

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

        return _tokenApprovals[tokenId].value;
    }

    /**
     * @dev Approve or remove `operator` as an operator for the caller.
     * Operators can call {transferFrom} or {safeTransferFrom}
     * for any token owned by the caller.
     *
     * Requirements:
     *
     * - The `operator` cannot be the caller.
     *
     * Emits an {ApprovalForAll} event.
     */
    function setApprovalForAll(address operator, bool approved) public virtual override {
        _operatorApprovals[_msgSenderERC721A()][operator] = approved;
        emit ApprovalForAll(_msgSenderERC721A(), operator, approved);
    }

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

    /**
     * @dev Returns whether `tokenId` exists.
     *
     * Tokens can be managed by their owner or approved accounts via {approve} or {setApprovalForAll}.
     *
     * Tokens start existing when they are minted. See {_mint}.
     */
    function _exists(uint256 tokenId) internal view virtual returns (bool result) {
        if (_startTokenId() <= tokenId) {
            if (tokenId < _currentIndex) {
                uint256 packed;
                while ((packed = _packedOwnerships[tokenId]) == 0) --tokenId;
                result = packed & _BITMASK_BURNED == 0;
            }
        }
    }

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

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

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

    /**
     * @dev Transfers `tokenId` from `from` to `to`.
     *
     * Requirements:
     *
     * - `from` cannot be the zero address.
     * - `to` cannot be the zero address.
     * - `tokenId` token must be owned by `from`.
     * - If the caller is not `from`, it must be approved to move this token
     * by either {approve} or {setApprovalForAll}.
     *
     * Emits a {Transfer} event.
     */
    function transferFrom(
        address from,
        address to,
        uint256 tokenId
    ) public payable virtual override {
        uint256 prevOwnershipPacked = _packedOwnershipOf(tokenId);

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

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

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

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

        _beforeTokenTransfers(from, to, tokenId, 1);

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

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

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

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

        // Mask `to` to the lower 160 bits, in case the upper bits somehow aren't clean.
        uint256 toMasked = uint256(uint160(to)) & _BITMASK_ADDRESS;
        assembly {
            // Emit the `Transfer` event.
            log4(
                0, // Start of data (0, since no data).
                0, // End of data (0, since no data).
                _TRANSFER_EVENT_SIGNATURE, // Signature.
                from, // `from`.
                toMasked, // `to`.
                tokenId // `tokenId`.
            )
        }
        if (toMasked == 0) _revert(TransferToZeroAddress.selector);

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

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

    /**
     * @dev Safely transfers `tokenId` token from `from` to `to`.
     *
     * Requirements:
     *
     * - `from` cannot be the zero address.
     * - `to` cannot be the zero address.
     * - `tokenId` token must exist and be owned by `from`.
     * - If the caller is not `from`, it must be approved to move this token
     * by either {approve} or {setApprovalForAll}.
     * - If `to` refers to a smart contract, it must implement
     * {IERC721Receiver-onERC721Received}, which is called upon a safe transfer.
     *
     * Emits a {Transfer} event.
     */
    function safeTransferFrom(
        address from,
        address to,
        uint256 tokenId,
        bytes memory _data
    ) public payable virtual override {
        transferFrom(from, to, tokenId);
        if (to.code.length != 0)
            if (!_checkContractOnERC721Received(from, to, tokenId, _data)) {
                _revert(TransferToNonERC721ReceiverImplementer.selector);
            }
    }

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

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

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

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

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

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

        // Overflows are incredibly unrealistic.
        // `balance` and `numberMinted` have a maximum limit of 2**64.
        // `tokenId` has a maximum limit of 2**256.
        unchecked {
            // Updates:
            // - `address` to the owner.
            // - `startTimestamp` to the timestamp of minting.
            // - `burned` to `false`.
            // - `nextInitialized` to `quantity == 1`.
            _packedOwnerships[startTokenId] = _packOwnershipData(
                to,
                _nextInitializedFlag(quantity) | _nextExtraData(address(0), to, 0)
            );

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

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

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

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

            do {
                assembly {
                    // Emit the `Transfer` event.
                    log4(
                        0, // Start of data (0, since no data).
                        0, // End of data (0, since no data).
                        _TRANSFER_EVENT_SIGNATURE, // Signature.
                        0, // `address(0)`.
                        toMasked, // `to`.
                        tokenId // `tokenId`.
                    )
                }
                // The `!=` check ensures that large values of `quantity`
                // that overflows uint256 will make the loop run out of gas.
            } while (++tokenId != end);

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

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

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

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

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

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

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

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

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

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

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

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

    /**
     * @dev Gives permission to `to` to transfer `tokenId` token to another account.
     * The approval is cleared when the token is transferred.
     *
     * Only a single account can be approved at a time, so approving the
     * zero address clears previous approvals.
     *
     * Requirements:
     *
     * - `tokenId` must exist.
     *
     * Emits an {Approval} event.
     */
    function _approve(
        address to,
        uint256 tokenId,
        bool approvalCheck
    ) internal virtual {
        address owner = ownerOf(tokenId);

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

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

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

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

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

        address from = address(uint160(prevOwnershipPacked));

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

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

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

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

        // Underflow of the sender's balance is impossible because we check for
        // ownership above and the recipient's balance can't realistically overflow.
        // Counter overflow is incredibly unrealistic as `tokenId` would have to be 2**256.
        unchecked {
            // Updates:
            // - `balance -= 1`.
            // - `numberBurned += 1`.
            //
            // We can directly decrement the balance, and increment the number burned.
            // This is equivalent to `packed -= 1; packed += 1 << _BITPOS_NUMBER_BURNED;`.
            _packedAddressData[from] += (1 << _BITPOS_NUMBER_BURNED) - 1;

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

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

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

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

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

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

    /**
     * @dev Called during each token transfer to set the 24bit `extraData` field.
     * Intended to be overridden by the cosumer contract.
     *
     * `previousExtraData` - the value of `extraData` before transfer.
     *
     * Calling conditions:
     *
     * - When `from` and `to` are both non-zero, `from`'s `tokenId` will be
     * transferred to `to`.
     * - When `from` is zero, `tokenId` will be minted for `to`.
     * - When `to` is zero, `tokenId` will be burned by `from`.
     * - `from` and `to` are never both zero.
     */
    function _extraData(
        address from,
        address to,
        uint24 previousExtraData
    ) internal view virtual returns (uint24) {}

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

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

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

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

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

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

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

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

File 3 of 11: ERC721AQueryable.sol
// SPDX-License-Identifier: MIT
// ERC721A Contracts v4.2.3
// Creator: Chiru Labs

pragma solidity ^0.8.4;

import './IERC721AQueryable.sol';
import './ERC721A.sol';

/**
 * @title ERC721AQueryable.
 *
 * @dev ERC721A subclass with convenience query functions.
 */
abstract contract ERC721AQueryable is ERC721A, IERC721AQueryable {
    /**
     * @dev Returns the `TokenOwnership` struct at `tokenId` without reverting.
     *
     * If the `tokenId` is out of bounds:
     *
     * - `addr = address(0)`
     * - `startTimestamp = 0`
     * - `burned = false`
     * - `extraData = 0`
     *
     * If the `tokenId` is burned:
     *
     * - `addr = <Address of owner before token was burned>`
     * - `startTimestamp = <Timestamp when token was burned>`
     * - `burned = true`
     * - `extraData = <Extra data when token was burned>`
     *
     * Otherwise:
     *
     * - `addr = <Address of owner>`
     * - `startTimestamp = <Timestamp of start of ownership>`
     * - `burned = false`
     * - `extraData = <Extra data at start of ownership>`
     */
    function explicitOwnershipOf(uint256 tokenId)
        public
        view
        virtual
        override
        returns (TokenOwnership memory ownership)
    {
        unchecked {
            if (tokenId >= _startTokenId()) {
                if (tokenId < _nextTokenId()) {
                    // If the `tokenId` is within bounds,
                    // scan backwards for the initialized ownership slot.
                    while (!_ownershipIsInitialized(tokenId)) --tokenId;
                    return _ownershipAt(tokenId);
                }
            }
        }
    }

    /**
     * @dev Returns an array of `TokenOwnership` structs at `tokenIds` in order.
     * See {ERC721AQueryable-explicitOwnershipOf}
     */
    function explicitOwnershipsOf(uint256[] calldata tokenIds)
        external
        view
        virtual
        override
        returns (TokenOwnership[] memory)
    {
        TokenOwnership[] memory ownerships;
        uint256 i = tokenIds.length;
        assembly {
            // Grab the free memory pointer.
            ownerships := mload(0x40)
            // Store the length.
            mstore(ownerships, i)
            // Allocate one word for the length,
            // `tokenIds.length` words for the pointers.
            i := shl(5, i) // Multiply `i` by 32.
            mstore(0x40, add(add(ownerships, 0x20), i))
        }
        while (i != 0) {
            uint256 tokenId;
            assembly {
                i := sub(i, 0x20)
                tokenId := calldataload(add(tokenIds.offset, i))
            }
            TokenOwnership memory ownership = explicitOwnershipOf(tokenId);
            assembly {
                // Store the pointer of `ownership` in the `ownerships` array.
                mstore(add(add(ownerships, 0x20), i), ownership)
            }
        }
        return ownerships;
    }

    /**
     * @dev Returns an array of token IDs owned by `owner`,
     * in the range [`start`, `stop`)
     * (i.e. `start <= tokenId < stop`).
     *
     * This function allows for tokens to be queried if the collection
     * grows too big for a single call of {ERC721AQueryable-tokensOfOwner}.
     *
     * Requirements:
     *
     * - `start < stop`
     */
    function tokensOfOwnerIn(
        address owner,
        uint256 start,
        uint256 stop
    ) external view virtual override returns (uint256[] memory) {
        return _tokensOfOwnerIn(owner, start, stop);
    }

    /**
     * @dev Returns an array of token IDs owned by `owner`.
     *
     * This function scans the ownership mapping and is O(`totalSupply`) in complexity.
     * It is meant to be called off-chain.
     *
     * See {ERC721AQueryable-tokensOfOwnerIn} for splitting the scan into
     * multiple smaller scans if the collection is large enough to cause
     * an out-of-gas error (10K collections should be fine).
     */
    function tokensOfOwner(address owner) external view virtual override returns (uint256[] memory) {
        uint256 start = _startTokenId();
        uint256 stop = _nextTokenId();
        uint256[] memory tokenIds;
        if (start != stop) tokenIds = _tokensOfOwnerIn(owner, start, stop);
        return tokenIds;
    }

    /**
     * @dev Helper function for returning an array of token IDs owned by `owner`.
     *
     * Note that this function is optimized for smaller bytecode size over runtime gas,
     * since it is meant to be called off-chain.
     */
    function _tokensOfOwnerIn(
        address owner,
        uint256 start,
        uint256 stop
    ) private view returns (uint256[] memory) {
        unchecked {
            if (start >= stop) _revert(InvalidQueryRange.selector);
            // Set `start = max(start, _startTokenId())`.
            if (start < _startTokenId()) {
                start = _startTokenId();
            }
            uint256 stopLimit = _nextTokenId();
            // Set `stop = min(stop, stopLimit)`.
            if (stop >= stopLimit) {
                stop = stopLimit;
            }
            uint256[] memory tokenIds;
            uint256 tokenIdsMaxLength = balanceOf(owner);
            bool startLtStop = start < stop;
            assembly {
                // Set `tokenIdsMaxLength` to zero if `start` is less than `stop`.
                tokenIdsMaxLength := mul(tokenIdsMaxLength, startLtStop)
            }
            if (tokenIdsMaxLength != 0) {
                // Set `tokenIdsMaxLength = min(balanceOf(owner), stop - start)`,
                // to cater for cases where `balanceOf(owner)` is too big.
                if (stop - start <= tokenIdsMaxLength) {
                    tokenIdsMaxLength = stop - start;
                }
                assembly {
                    // Grab the free memory pointer.
                    tokenIds := mload(0x40)
                    // Allocate one word for the length, and `tokenIdsMaxLength` words
                    // for the data. `shl(5, x)` is equivalent to `mul(32, x)`.
                    mstore(0x40, add(tokenIds, shl(5, add(tokenIdsMaxLength, 1))))
                }
                // We need to call `explicitOwnershipOf(start)`,
                // because the slot at `start` may not be initialized.
                TokenOwnership memory ownership = explicitOwnershipOf(start);
                address currOwnershipAddr;
                // If the starting slot exists (i.e. not burned),
                // initialize `currOwnershipAddr`.
                // `ownership.address` will not be zero,
                // as `start` is clamped to the valid token ID range.
                if (!ownership.burned) {
                    currOwnershipAddr = ownership.addr;
                }
                uint256 tokenIdsIdx;
                // Use a do-while, which is slightly more efficient for this case,
                // as the array will at least contain one element.
                do {
                    ownership = _ownershipAt(start);
                    assembly {
                        switch mload(add(ownership, 0x40))
                        // if `ownership.burned == false`.
                        case 0 {
                            // if `ownership.addr != address(0)`.
                            // The `addr` already has it's upper 96 bits clearned,
                            // since it is written to memory with regular Solidity.
                            if mload(ownership) {
                                currOwnershipAddr := mload(ownership)
                            }
                            // if `currOwnershipAddr == owner`.
                            // The `shl(96, x)` is to make the comparison agnostic to any
                            // dirty upper 96 bits in `owner`.
                            if iszero(shl(96, xor(currOwnershipAddr, owner))) {
                                tokenIdsIdx := add(tokenIdsIdx, 1)
                                mstore(add(tokenIds, shl(5, tokenIdsIdx)), start)
                            }
                        }
                        // Otherwise, reset `currOwnershipAddr`.
                        // This handles the case of batch burned tokens
                        // (burned bit of first slot set, remaining slots left uninitialized).
                        default {
                            currOwnershipAddr := 0
                        }
                        start := add(start, 1)
                    }
                } while (!(start == stop || tokenIdsIdx == tokenIdsMaxLength));
                // Store the length of the array.
                assembly {
                    mstore(tokenIds, tokenIdsIdx)
                }
            }
            return tokenIds;
        }
    }
}

File 4 of 11: IERC721A.sol
// SPDX-License-Identifier: MIT
// ERC721A Contracts v4.2.3
// Creator: Chiru Labs

pragma solidity ^0.8.4;

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

    /**
     * @dev Emitted when `tokenId` token is transferred from `from` to `to`.
     */
    event Transfer(address indexed from, address indexed to, uint256 indexed tokenId);

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

File 5 of 11: IERC721AQueryable.sol
// SPDX-License-Identifier: MIT
// ERC721A Contracts v4.2.3
// Creator: Chiru Labs

pragma solidity ^0.8.4;

import './IERC721A.sol';

/**
 * @dev Interface of ERC721AQueryable.
 */
interface IERC721AQueryable is IERC721A {
    /**
     * Invalid query range (`start` >= `stop`).
     */
    error InvalidQueryRange();

    /**
     * @dev Returns the `TokenOwnership` struct at `tokenId` without reverting.
     *
     * If the `tokenId` is out of bounds:
     *
     * - `addr = address(0)`
     * - `startTimestamp = 0`
     * - `burned = false`
     * - `extraData = 0`
     *
     * If the `tokenId` is burned:
     *
     * - `addr = <Address of owner before token was burned>`
     * - `startTimestamp = <Timestamp when token was burned>`
     * - `burned = true`
     * - `extraData = <Extra data when token was burned>`
     *
     * Otherwise:
     *
     * - `addr = <Address of owner>`
     * - `startTimestamp = <Timestamp of start of ownership>`
     * - `burned = false`
     * - `extraData = <Extra data at start of ownership>`
     */
    function explicitOwnershipOf(uint256 tokenId) external view returns (TokenOwnership memory);

    /**
     * @dev Returns an array of `TokenOwnership` structs at `tokenIds` in order.
     * See {ERC721AQueryable-explicitOwnershipOf}
     */
    function explicitOwnershipsOf(uint256[] memory tokenIds) external view returns (TokenOwnership[] memory);

    /**
     * @dev Returns an array of token IDs owned by `owner`,
     * in the range [`start`, `stop`)
     * (i.e. `start <= tokenId < stop`).
     *
     * This function allows for tokens to be queried if the collection
     * grows too big for a single call of {ERC721AQueryable-tokensOfOwner}.
     *
     * Requirements:
     *
     * - `start < stop`
     */
    function tokensOfOwnerIn(
        address owner,
        uint256 start,
        uint256 stop
    ) external view returns (uint256[] memory);

    /**
     * @dev Returns an array of token IDs owned by `owner`.
     *
     * This function scans the ownership mapping and is O(`totalSupply`) in complexity.
     * It is meant to be called off-chain.
     *
     * See {ERC721AQueryable-tokensOfOwnerIn} for splitting the scan into
     * multiple smaller scans if the collection is large enough to cause
     * an out-of-gas error (10K collections should be fine).
     */
    function tokensOfOwner(address owner) external view returns (uint256[] memory);
}

File 6 of 11: Math.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts (last updated v4.8.0) (utils/math/Math.sol)

pragma solidity ^0.8.0;

/**
 * @dev Standard math utilities missing in the Solidity language.
 */
library Math {
    enum Rounding {
        Down, // Toward negative infinity
        Up, // Toward infinity
        Zero // Toward zero
    }

    /**
     * @dev Returns the largest of two numbers.
     */
    function max(uint256 a, uint256 b) internal pure returns (uint256) {
        return a > b ? a : b;
    }

    /**
     * @dev Returns the smallest of two numbers.
     */
    function min(uint256 a, uint256 b) internal pure returns (uint256) {
        return a < b ? a : b;
    }

    /**
     * @dev Returns the average of two numbers. The result is rounded towards
     * zero.
     */
    function average(uint256 a, uint256 b) internal pure returns (uint256) {
        // (a + b) / 2 can overflow.
        return (a & b) + (a ^ b) / 2;
    }

    /**
     * @dev Returns the ceiling of the division of two numbers.
     *
     * This differs from standard division with `/` in that it rounds up instead
     * of rounding down.
     */
    function ceilDiv(uint256 a, uint256 b) internal pure returns (uint256) {
        // (a + b - 1) / b can overflow on addition, so we distribute.
        return a == 0 ? 0 : (a - 1) / b + 1;
    }

    /**
     * @notice Calculates floor(x * y / denominator) with full precision. Throws if result overflows a uint256 or denominator == 0
     * @dev Original credit to Remco Bloemen under MIT license (https://xn--2-umb.com/21/muldiv)
     * with further edits by Uniswap Labs also under MIT license.
     */
    function mulDiv(
        uint256 x,
        uint256 y,
        uint256 denominator
    ) internal pure returns (uint256 result) {
        unchecked {
            // 512-bit multiply [prod1 prod0] = x * y. Compute the product mod 2^256 and mod 2^256 - 1, then use
            // use the Chinese Remainder Theorem to reconstruct the 512 bit result. The result is stored in two 256
            // variables such that product = prod1 * 2^256 + prod0.
            uint256 prod0; // Least significant 256 bits of the product
            uint256 prod1; // Most significant 256 bits of the product
            assembly {
                let mm := mulmod(x, y, not(0))
                prod0 := mul(x, y)
                prod1 := sub(sub(mm, prod0), lt(mm, prod0))
            }

            // Handle non-overflow cases, 256 by 256 division.
            if (prod1 == 0) {
                return prod0 / denominator;
            }

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

            ///////////////////////////////////////////////
            // 512 by 256 division.
            ///////////////////////////////////////////////

            // Make division exact by subtracting the remainder from [prod1 prod0].
            uint256 remainder;
            assembly {
                // Compute remainder using mulmod.
                remainder := mulmod(x, y, denominator)

                // Subtract 256 bit number from 512 bit number.
                prod1 := sub(prod1, gt(remainder, prod0))
                prod0 := sub(prod0, remainder)
            }

            // Factor powers of two out of denominator and compute largest power of two divisor of denominator. Always >= 1.
            // See https://cs.stackexchange.com/q/138556/92363.

            // Does not overflow because the denominator cannot be zero at this stage in the function.
            uint256 twos = denominator & (~denominator + 1);
            assembly {
                // Divide denominator by twos.
                denominator := div(denominator, twos)

                // Divide [prod1 prod0] by twos.
                prod0 := div(prod0, twos)

                // Flip twos such that it is 2^256 / twos. If twos is zero, then it becomes one.
                twos := add(div(sub(0, twos), twos), 1)
            }

            // Shift in bits from prod1 into prod0.
            prod0 |= prod1 * twos;

            // Invert denominator mod 2^256. Now that denominator is an odd number, it has an inverse modulo 2^256 such
            // that denominator * inv = 1 mod 2^256. Compute the inverse by starting with a seed that is correct for
            // four bits. That is, denominator * inv = 1 mod 2^4.
            uint256 inverse = (3 * denominator) ^ 2;

            // Use the Newton-Raphson iteration to improve the precision. Thanks to Hensel's lifting lemma, this also works
            // in modular arithmetic, doubling the correct bits in each step.
            inverse *= 2 - denominator * inverse; // inverse mod 2^8
            inverse *= 2 - denominator * inverse; // inverse mod 2^16
            inverse *= 2 - denominator * inverse; // inverse mod 2^32
            inverse *= 2 - denominator * inverse; // inverse mod 2^64
            inverse *= 2 - denominator * inverse; // inverse mod 2^128
            inverse *= 2 - denominator * inverse; // inverse mod 2^256

            // Because the division is now exact we can divide by multiplying with the modular inverse of denominator.
            // This will give us the correct result modulo 2^256. Since the preconditions guarantee that the outcome is
            // less than 2^256, this is the final result. We don't need to compute the high bits of the result and prod1
            // is no longer required.
            result = prod0 * inverse;
            return result;
        }
    }

    /**
     * @notice Calculates x * y / denominator with full precision, following the selected rounding direction.
     */
    function mulDiv(
        uint256 x,
        uint256 y,
        uint256 denominator,
        Rounding rounding
    ) internal pure returns (uint256) {
        uint256 result = mulDiv(x, y, denominator);
        if (rounding == Rounding.Up && mulmod(x, y, denominator) > 0) {
            result += 1;
        }
        return result;
    }

    /**
     * @dev Returns the square root of a number. If the number is not a perfect square, the value is rounded down.
     *
     * Inspired by Henry S. Warren, Jr.'s "Hacker's Delight" (Chapter 11).
     */
    function sqrt(uint256 a) internal pure returns (uint256) {
        if (a == 0) {
            return 0;
        }

        // For our first guess, we get the biggest power of 2 which is smaller than the square root of the target.
        //
        // We know that the "msb" (most significant bit) of our target number `a` is a power of 2 such that we have
        // `msb(a) <= a < 2*msb(a)`. This value can be written `msb(a)=2**k` with `k=log2(a)`.
        //
        // This can be rewritten `2**log2(a) <= a < 2**(log2(a) + 1)`
        // → `sqrt(2**k) <= sqrt(a) < sqrt(2**(k+1))`
        // → `2**(k/2) <= sqrt(a) < 2**((k+1)/2) <= 2**(k/2 + 1)`
        //
        // Consequently, `2**(log2(a) / 2)` is a good first approximation of `sqrt(a)` with at least 1 correct bit.
        uint256 result = 1 << (log2(a) >> 1);

        // At this point `result` is an estimation with one bit of precision. We know the true value is a uint128,
        // since it is the square root of a uint256. Newton's method converges quadratically (precision doubles at
        // every iteration). We thus need at most 7 iteration to turn our partial result with one bit of precision
        // into the expected uint128 result.
        unchecked {
            result = (result + a / result) >> 1;
            result = (result + a / result) >> 1;
            result = (result + a / result) >> 1;
            result = (result + a / result) >> 1;
            result = (result + a / result) >> 1;
            result = (result + a / result) >> 1;
            result = (result + a / result) >> 1;
            return min(result, a / result);
        }
    }

    /**
     * @notice Calculates sqrt(a), following the selected rounding direction.
     */
    function sqrt(uint256 a, Rounding rounding) internal pure returns (uint256) {
        unchecked {
            uint256 result = sqrt(a);
            return result + (rounding == Rounding.Up && result * result < a ? 1 : 0);
        }
    }

    /**
     * @dev Return the log in base 2, rounded down, of a positive value.
     * Returns 0 if given 0.
     */
    function log2(uint256 value) internal pure returns (uint256) {
        uint256 result = 0;
        unchecked {
            if (value >> 128 > 0) {
                value >>= 128;
                result += 128;
            }
            if (value >> 64 > 0) {
                value >>= 64;
                result += 64;
            }
            if (value >> 32 > 0) {
                value >>= 32;
                result += 32;
            }
            if (value >> 16 > 0) {
                value >>= 16;
                result += 16;
            }
            if (value >> 8 > 0) {
                value >>= 8;
                result += 8;
            }
            if (value >> 4 > 0) {
                value >>= 4;
                result += 4;
            }
            if (value >> 2 > 0) {
                value >>= 2;
                result += 2;
            }
            if (value >> 1 > 0) {
                result += 1;
            }
        }
        return result;
    }

    /**
     * @dev Return the log in base 2, following the selected rounding direction, of a positive value.
     * Returns 0 if given 0.
     */
    function log2(uint256 value, Rounding rounding) internal pure returns (uint256) {
        unchecked {
            uint256 result = log2(value);
            return result + (rounding == Rounding.Up && 1 << result < value ? 1 : 0);
        }
    }

    /**
     * @dev Return the log in base 10, rounded down, of a positive value.
     * Returns 0 if given 0.
     */
    function log10(uint256 value) internal pure returns (uint256) {
        uint256 result = 0;
        unchecked {
            if (value >= 10**64) {
                value /= 10**64;
                result += 64;
            }
            if (value >= 10**32) {
                value /= 10**32;
                result += 32;
            }
            if (value >= 10**16) {
                value /= 10**16;
                result += 16;
            }
            if (value >= 10**8) {
                value /= 10**8;
                result += 8;
            }
            if (value >= 10**4) {
                value /= 10**4;
                result += 4;
            }
            if (value >= 10**2) {
                value /= 10**2;
                result += 2;
            }
            if (value >= 10**1) {
                result += 1;
            }
        }
        return result;
    }

    /**
     * @dev Return the log in base 10, following the selected rounding direction, of a positive value.
     * Returns 0 if given 0.
     */
    function log10(uint256 value, Rounding rounding) internal pure returns (uint256) {
        unchecked {
            uint256 result = log10(value);
            return result + (rounding == Rounding.Up && 10**result < value ? 1 : 0);
        }
    }

    /**
     * @dev Return the log in base 256, rounded down, of a positive value.
     * Returns 0 if given 0.
     *
     * Adding one to the result gives the number of pairs of hex symbols needed to represent `value` as a hex string.
     */
    function log256(uint256 value) internal pure returns (uint256) {
        uint256 result = 0;
        unchecked {
            if (value >> 128 > 0) {
                value >>= 128;
                result += 16;
            }
            if (value >> 64 > 0) {
                value >>= 64;
                result += 8;
            }
            if (value >> 32 > 0) {
                value >>= 32;
                result += 4;
            }
            if (value >> 16 > 0) {
                value >>= 16;
                result += 2;
            }
            if (value >> 8 > 0) {
                result += 1;
            }
        }
        return result;
    }

    /**
     * @dev Return the log in base 10, following the selected rounding direction, of a positive value.
     * Returns 0 if given 0.
     */
    function log256(uint256 value, Rounding rounding) internal pure returns (uint256) {
        unchecked {
            uint256 result = log256(value);
            return result + (rounding == Rounding.Up && 1 << (result * 8) < value ? 1 : 0);
        }
    }
}

File 7 of 11: MerkleProof.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts (last updated v4.8.0) (utils/cryptography/MerkleProof.sol)

pragma solidity ^0.8.0;

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

File 8 of 11: Ownable.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts (last updated v4.7.0) (access/Ownable.sol)

pragma solidity ^0.8.0;

import "./Context.sol";

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

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

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

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

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

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

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

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

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

File 10 of 11: ReentrancyGuard.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts (last updated v4.8.0) (security/ReentrancyGuard.sol)

pragma solidity ^0.8.0;

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

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

    uint256 private _status;

    constructor() {
        _status = _NOT_ENTERED;
    }

    /**
     * @dev Prevents a contract from calling itself, directly or indirectly.
     * Calling a `nonReentrant` function from another `nonReentrant`
     * function is not supported. It is possible to prevent this from happening
     * by making the `nonReentrant` function external, and making it call a
     * `private` function that does the actual work.
     */
    modifier nonReentrant() {
        _nonReentrantBefore();
        _;
        _nonReentrantAfter();
    }

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

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

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

File 11 of 11: Strings.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts (last updated v4.8.0) (utils/Strings.sol)

pragma solidity ^0.8.0;

import "./Math.sol";

/**
 * @dev String operations.
 */
library Strings {
    bytes16 private constant _SYMBOLS = "0123456789abcdef";
    uint8 private constant _ADDRESS_LENGTH = 20;

    /**
     * @dev Converts a `uint256` to its ASCII `string` decimal representation.
     */
    function toString(uint256 value) internal pure returns (string memory) {
        unchecked {
            uint256 length = Math.log10(value) + 1;
            string memory buffer = new string(length);
            uint256 ptr;
            /// @solidity memory-safe-assembly
            assembly {
                ptr := add(buffer, add(32, length))
            }
            while (true) {
                ptr--;
                /// @solidity memory-safe-assembly
                assembly {
                    mstore8(ptr, byte(mod(value, 10), _SYMBOLS))
                }
                value /= 10;
                if (value == 0) break;
            }
            return buffer;
        }
    }

    /**
     * @dev Converts a `uint256` to its ASCII `string` hexadecimal representation.
     */
    function toHexString(uint256 value) internal pure returns (string memory) {
        unchecked {
            return toHexString(value, Math.log256(value) + 1);
        }
    }

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

    /**
     * @dev Converts an `address` with fixed length of 20 bytes to its not checksummed ASCII `string` hexadecimal representation.
     */
    function toHexString(address addr) internal pure returns (string memory) {
        return toHexString(uint256(uint160(addr)), _ADDRESS_LENGTH);
    }
}

Contract Security Audit

Contract ABI

[{"inputs":[{"internalType":"string","name":"_tokenName","type":"string"},{"internalType":"string","name":"_tokenSymbol","type":"string"},{"internalType":"uint256","name":"_cost","type":"uint256"},{"internalType":"uint256","name":"_maxSupply","type":"uint256"},{"internalType":"uint256","name":"_maxMintAmountPerTx","type":"uint256"},{"internalType":"string","name":"_hiddenMetadataUri","type":"string"}],"stateMutability":"nonpayable","type":"constructor"},{"inputs":[],"name":"ApprovalCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"ApprovalQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"BalanceQueryForZeroAddress","type":"error"},{"inputs":[],"name":"InvalidQueryRange","type":"error"},{"inputs":[],"name":"MintERC2309QuantityExceedsLimit","type":"error"},{"inputs":[],"name":"MintToZeroAddress","type":"error"},{"inputs":[],"name":"MintZeroQuantity","type":"error"},{"inputs":[],"name":"OwnerQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"OwnershipNotInitializedForExtraData","type":"error"},{"inputs":[],"name":"TransferCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"TransferFromIncorrectOwner","type":"error"},{"inputs":[],"name":"TransferToNonERC721ReceiverImplementer","type":"error"},{"inputs":[],"name":"TransferToZeroAddress","type":"error"},{"inputs":[],"name":"URIQueryForNonexistentToken","type":"error"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"approved","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Approval","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"operator","type":"address"},{"indexed":false,"internalType":"bool","name":"approved","type":"bool"}],"name":"ApprovalForAll","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"uint256","name":"fromTokenId","type":"uint256"},{"indexed":false,"internalType":"uint256","name":"toTokenId","type":"uint256"},{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"}],"name":"ConsecutiveTransfer","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"previousOwner","type":"address"},{"indexed":true,"internalType":"address","name":"newOwner","type":"address"}],"name":"OwnershipTransferred","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Transfer","type":"event"},{"inputs":[],"name":"PeeCoinContract","outputs":[{"internalType":"contract IERC20","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"Peeaddress","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"approve","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"}],"name":"balanceOf","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"cost","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"explicitOwnershipOf","outputs":[{"components":[{"internalType":"address","name":"addr","type":"address"},{"internalType":"uint64","name":"startTimestamp","type":"uint64"},{"internalType":"bool","name":"burned","type":"bool"},{"internalType":"uint24","name":"extraData","type":"uint24"}],"internalType":"struct IERC721A.TokenOwnership","name":"ownership","type":"tuple"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256[]","name":"tokenIds","type":"uint256[]"}],"name":"explicitOwnershipsOf","outputs":[{"components":[{"internalType":"address","name":"addr","type":"address"},{"internalType":"uint64","name":"startTimestamp","type":"uint64"},{"internalType":"bool","name":"burned","type":"bool"},{"internalType":"uint24","name":"extraData","type":"uint24"}],"internalType":"struct IERC721A.TokenOwnership[]","name":"","type":"tuple[]"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"getApproved","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"hiddenMetadataUri","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256[]","name":"tokenIds","type":"uint256[]"}],"name":"holderClaim","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"holderClaim_state","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"},{"internalType":"address","name":"operator","type":"address"}],"name":"isApprovedForAll","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"","type":"uint256"}],"name":"isClaim","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"isfree","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxMintAmountPerTx","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxPerFree","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxSupply","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"merkleRoot","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"_mintAmount","type":"uint256"}],"name":"mint","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_mintAmount","type":"uint256"},{"internalType":"address","name":"_receiver","type":"address"}],"name":"mintForAddress","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"mintedAmount","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"name","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"owner","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"ownerOf","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"paused","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"revealed","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"},{"internalType":"bytes","name":"_data","type":"bytes"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"address","name":"operator","type":"address"},{"internalType":"bool","name":"approved","type":"bool"}],"name":"setApprovalForAll","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_cost","type":"uint256"}],"name":"setCost","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"_hiddenMetadataUri","type":"string"}],"name":"setHiddenMetadataUri","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_maxMintAmountPerTx","type":"uint256"}],"name":"setMaxMintAmountPerTx","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"freenum_","type":"uint256"}],"name":"setMaxPerFree","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"_merkleRoot","type":"bytes32"}],"name":"setMerkleRoot","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bool","name":"_state","type":"bool"}],"name":"setPaused","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"Peeadd_","type":"address"}],"name":"setPeecoinaddress","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bool","name":"_state","type":"bool"}],"name":"setRevealed","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"_uriPrefix","type":"string"}],"name":"setUriPrefix","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"_uriSuffix","type":"string"}],"name":"setUriSuffix","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bool","name":"_state","type":"bool"}],"name":"setWhitelistMintEnabled","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"freenum","type":"uint256"}],"name":"setWhitelistPerFree","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bool","name":"_state","type":"bool"}],"name":"setholderClaimstate","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":[{"internalType":"address","name":"owner","type":"address"}],"name":"tokensOfOwner","outputs":[{"internalType":"uint256[]","name":"","type":"uint256[]"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"},{"internalType":"uint256","name":"start","type":"uint256"},{"internalType":"uint256","name":"stop","type":"uint256"}],"name":"tokensOfOwnerIn","outputs":[{"internalType":"uint256[]","name":"","type":"uint256[]"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"totalFreeMinted","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"totalSupply","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"transferFrom","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"address","name":"newOwner","type":"address"}],"name":"transferOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"uriPrefix","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"uriSuffix","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"whitelistClaimed","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"_mintAmount","type":"uint256"},{"internalType":"bytes32[]","name":"_merkleProof","type":"bytes32[]"}],"name":"whitelistMint","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"whitelistMintEnabled","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"whitelistPerFree","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"withdraw","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"Amount_","type":"uint256"}],"name":"withdrawPeetoken","outputs":[],"stateMutability":"nonpayable","type":"function"}]

6010805460ff60a01b191690556001601155600360125560a0604081905260006080819052620000329160139162000225565b5060408051808201909152600580825264173539b7b760d91b6020909201918252620000619160149162000225565b506000601655601a805462ffffff191660011790553480156200008357600080fd5b506040516200333638038062003336833981016040819052620000a69162000398565b855186908690620000bf90600290602085019062000225565b508051620000d590600390602084019062000225565b5050600160005550620000e83362000131565b6001600955620000f88462000183565b6018839055601080546001600160a01b031916301790556200011a8262000192565b6200012581620001a1565b50505050505062000482565b600880546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b6200018d620001c4565b601755565b6200019c620001c4565b601955565b620001ab620001c4565b8051620001c090601590602084019062000225565b5050565b6008546001600160a01b03163314620002235760405162461bcd60e51b815260206004820181905260248201527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572604482015260640160405180910390fd5b565b828054620002339062000445565b90600052602060002090601f016020900481019282620002575760008555620002a2565b82601f106200027257805160ff1916838001178555620002a2565b82800160010185558215620002a2579182015b82811115620002a257825182559160200191906001019062000285565b50620002b0929150620002b4565b5090565b5b80821115620002b05760008155600101620002b5565b634e487b7160e01b600052604160045260246000fd5b600082601f830112620002f357600080fd5b81516001600160401b0380821115620003105762000310620002cb565b604051601f8301601f19908116603f011681019082821181831017156200033b576200033b620002cb565b816040528381526020925086838588010111156200035857600080fd5b600091505b838210156200037c57858201830151818301840152908201906200035d565b838211156200038e5760008385830101525b9695505050505050565b60008060008060008060c08789031215620003b257600080fd5b86516001600160401b0380821115620003ca57600080fd5b620003d88a838b01620002e1565b97506020890151915080821115620003ef57600080fd5b620003fd8a838b01620002e1565b965060408901519550606089015194506080890151935060a08901519150808211156200042957600080fd5b506200043889828a01620002e1565b9150509295509295509295565b600181811c908216806200045a57607f821691505b602082108114156200047c57634e487b7160e01b600052602260045260246000fd5b50919050565b612ea480620004926000396000f3fe6080604052600436106103975760003560e01c80637cb64759116101dc578063c7c39ffc11610102578063e0a80853116100a0578063efbd73f41161006f578063efbd73f414610a7a578063f1a631ec14610a9a578063f2fde38b14610abb578063fbbf8cc314610adb57600080fd5b8063e0a80853146109d1578063e945971c146109f1578063e985e9c514610a11578063ef29948914610a5a57600080fd5b8063d5abeb01116100dc578063d5abeb0114610955578063dad7b5c91461096b578063db4bec4414610981578063dc8c3270146109b157600080fd5b8063c7c39ffc1461090c578063c87b56dd14610922578063d2cab0561461094257600080fd5b806399a2557a1161017a578063b071401b11610149578063b071401b1461088c578063b767a098146108ac578063b88d4fde146108cc578063c23dc68f146108df57600080fd5b806399a2557a14610824578063a0712d6814610844578063a22cb46514610857578063a45ba8e71461087757600080fd5b80638da5cb5b116101b65780638da5cb5b146107bb57806394354fd0146107d957806395d89b41146107ef57806398dfe50b1461080457600080fd5b80637cb647591461074e5780637ec4a6591461076e5780638462151c1461078e57600080fd5b80634fdd43cb116102c15780635c975abb1161025f5780636caede3d1161022e5780636caede3d146106ca57806370a08231146106e9578063715018a614610709578063745308e71461071e57600080fd5b80635c975abb1461065b57806362b99ad4146106755780636352211e1461068a57806364febc38146106aa57600080fd5b80635503a0e81161029b5780635503a0e8146105d957806357a2e24b146105ee57806359236f3a1461060e5780635bbb21771461062e57600080fd5b80634fdd43cb146105795780635183022714610599578063542d878b146105b957600080fd5b806316c38b3c116103395780633c4ed0ad116103085780633c4ed0ad1461051b5780633ccfd60b1461053157806342842e0e1461054657806344a0d68a1461055957600080fd5b806316c38b3c146104b457806318160ddd146104d457806323b872dd146104f25780632eb4a7ab1461050557600080fd5b8063081812fc11610375578063081812fc14610423578063095ea7b31461045b57806313faede61461047057806316ba10e01461049457600080fd5b806301ffc9a71461039c57806306fdde03146103d157806307cfa41b146103f3575b600080fd5b3480156103a857600080fd5b506103bc6103b73660046125bf565b610b08565b60405190151581526020015b60405180910390f35b3480156103dd57600080fd5b506103e6610b5a565b6040516103c89190612634565b3480156103ff57600080fd5b506103bc61040e366004612647565b600e6020526000908152604090205460ff1681565b34801561042f57600080fd5b5061044361043e366004612647565b610bec565b6040516001600160a01b0390911681526020016103c8565b61046e610469366004612677565b610c27565b005b34801561047c57600080fd5b5061048660175481565b6040519081526020016103c8565b3480156104a057600080fd5b5061046e6104af366004612740565b610c37565b3480156104c057600080fd5b5061046e6104cf366004612797565b610c52565b3480156104e057600080fd5b50610486600154600054036000190190565b61046e6105003660046127b4565b610c6d565b34801561051157600080fd5b50610486600a5481565b34801561052757600080fd5b5061048660125481565b34801561053d57600080fd5b5061046e610dc8565b61046e6105543660046127b4565b610e56565b34801561056557600080fd5b5061046e610574366004612647565b610e76565b34801561058557600080fd5b5061046e610594366004612740565b610e83565b3480156105a557600080fd5b50601a546103bc9062010000900460ff1681565b3480156105c557600080fd5b5061046e6105d4366004612647565b610e9e565b3480156105e557600080fd5b506103e6610eab565b3480156105fa57600080fd5b50600f54610443906001600160a01b031681565b34801561061a57600080fd5b5061046e6106293660046127f0565b610f39565b34801561063a57600080fd5b5061064e610649366004612857565b610f63565b6040516103c891906128d6565b34801561066757600080fd5b50601a546103bc9060ff1681565b34801561068157600080fd5b506103e6610faf565b34801561069657600080fd5b506104436106a5366004612647565b610fbc565b3480156106b657600080fd5b5061046e6106c5366004612918565b610fc7565b3480156106d657600080fd5b50601a546103bc90610100900460ff1681565b3480156106f557600080fd5b506104866107043660046127f0565b6111a8565b34801561071557600080fd5b5061046e6111ee565b34801561072a57600080fd5b506103bc6107393660046127f0565b600d6020526000908152604090205460ff1681565b34801561075a57600080fd5b5061046e610769366004612647565b611200565b34801561077a57600080fd5b5061046e610789366004612740565b61120d565b34801561079a57600080fd5b506107ae6107a93660046127f0565b611228565b6040516103c891906129be565b3480156107c757600080fd5b506008546001600160a01b0316610443565b3480156107e557600080fd5b5061048660195481565b3480156107fb57600080fd5b506103e661124f565b34801561081057600080fd5b5061046e61081f366004612797565b61125e565b34801561083057600080fd5b506107ae61083f3660046129f6565b611284565b61046e610852366004612647565b611291565b34801561086357600080fd5b5061046e610872366004612a29565b6114f1565b34801561088357600080fd5b506103e661155d565b34801561089857600080fd5b5061046e6108a7366004612647565b61156a565b3480156108b857600080fd5b5061046e6108c7366004612797565b611577565b61046e6108da366004612a60565b611599565b3480156108eb57600080fd5b506108ff6108fa366004612647565b6115da565b6040516103c89190612adc565b34801561091857600080fd5b5061048660115481565b34801561092e57600080fd5b506103e661093d366004612647565b61163e565b61046e610950366004612aea565b6117ae565b34801561096157600080fd5b5061048660185481565b34801561097757600080fd5b5061048660165481565b34801561098d57600080fd5b506103bc61099c3660046127f0565b600b6020526000908152604090205460ff1681565b3480156109bd57600080fd5b5061046e6109cc366004612647565b611b07565b3480156109dd57600080fd5b5061046e6109ec366004612797565b611bb2565b3480156109fd57600080fd5b5061046e610a0c366004612647565b611bd6565b348015610a1d57600080fd5b506103bc610a2c366004612b36565b6001600160a01b03918216600090815260076020908152604080832093909416825291909152205460ff1690565b348015610a6657600080fd5b50601054610443906001600160a01b031681565b348015610a8657600080fd5b5061046e610a95366004612b69565b611be3565b348015610aa657600080fd5b506010546103bc90600160a01b900460ff1681565b348015610ac757600080fd5b5061046e610ad63660046127f0565b611c60565b348015610ae757600080fd5b50610486610af63660046127f0565b600c6020526000908152604090205481565b60006301ffc9a760e01b6001600160e01b031983161480610b3957506380ac58cd60e01b6001600160e01b03198316145b80610b545750635b5e139f60e01b6001600160e01b03198316145b92915050565b606060028054610b6990612b8c565b80601f0160208091040260200160405190810160405280929190818152602001828054610b9590612b8c565b8015610be25780601f10610bb757610100808354040283529160200191610be2565b820191906000526020600020905b815481529060010190602001808311610bc557829003601f168201915b5050505050905090565b6000610bf782611cd6565b610c0b57610c0b6333d1c03960e21b611d1f565b506000908152600660205260409020546001600160a01b031690565b610c3382826001611d29565b5050565b610c3f611dcc565b8051610c33906014906020840190612510565b610c5a611dcc565b601a805460ff1916911515919091179055565b6000610c7882611e26565b6001600160a01b039485169490915081168414610c9e57610c9e62a1148160e81b611d1f565b60008281526006602052604090208054338082146001600160a01b03881690911417610ce257610cce8633610a2c565b610ce257610ce2632ce44b5f60e11b611d1f565b8015610ced57600082555b6001600160a01b038681166000908152600560205260408082208054600019019055918716808252919020805460010190554260a01b17600160e11b17600085815260046020526040902055600160e11b8316610d785760018401600081815260046020526040902054610d76576000548114610d765760008181526004602052604090208490555b505b6001600160a01b0385168481887fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a480610dbf57610dbf633a954ecd60e21b611d1f565b50505050505050565b610dd0611dcc565b610dd8611ec2565b6000610dec6008546001600160a01b031690565b6001600160a01b03164760405160006040518083038185875af1925050503d8060008114610e36576040519150601f19603f3d011682016040523d82523d6000602084013e610e3b565b606091505b5050905080610e4957600080fd5b50610e546001600955565b565b610e7183838360405180602001604052806000815250611599565b505050565b610e7e611dcc565b601755565b610e8b611dcc565b8051610c33906015906020840190612510565b610ea6611dcc565b601255565b60148054610eb890612b8c565b80601f0160208091040260200160405190810160405280929190818152602001828054610ee490612b8c565b8015610f315780601f10610f0657610100808354040283529160200191610f31565b820191906000526020600020905b815481529060010190602001808311610f1457829003601f168201915b505050505081565b610f41611dcc565b600f80546001600160a01b0319166001600160a01b0392909216919091179055565b60408051828152600583901b8082016020019092526060915b8015610fa757601f1980820191860101356000610f98826115da565b8484016020015250610f7c9050565b509392505050565b60138054610eb890612b8c565b6000610b5482611e26565b601054600160a01b900460ff166110355760405162461bcd60e51b815260206004820152602760248201527f416374697669747920726564656d7074696f6e20686173206e6f7420796574206044820152661cdd185c9d195960ca1b60648201526084015b60405180910390fd5b805169010f0cf064dd59200000903360005b828110156111a157600085828151811061106357611063612bc7565b60200260200101519050826001600160a01b031661108082610fbc565b6001600160a01b0316146110d65760405162461bcd60e51b815260206004820152601860248201527f596f7520646f6e2774206f776e207468697320746f6b656e0000000000000000604482015260640161102c565b6000818152600e602052604090205460ff1661118e576000818152600e602052604090819020805460ff19166001179055600f54905163a9059cbb60e01b81526001600160a01b038581166004830152602482018890529091169063a9059cbb90604401602060405180830381600087803b15801561115457600080fd5b505af1158015611168573d6000803e3d6000fd5b505050506040513d601f19601f8201168201806040525081019061118c9190612bdd565b505b508061119981612c10565b915050611047565b5050505050565b60006001600160a01b0382166111c8576111c86323d3ad8160e21b611d1f565b506001600160a01b031660009081526005602052604090205467ffffffffffffffff1690565b6111f6611dcc565b610e546000611f1c565b611208611dcc565b600a55565b611215611dcc565b8051610c33906013906020840190612510565b6000546060906001908282821461124757611244858484611f6e565b90505b949350505050565b606060038054610b6990612b8c565b611266611dcc565b60108054911515600160a01b0260ff60a01b19909216919091179055565b6060611247848484611f6e565b6000811180156112a357506019548111155b6112bf5760405162461bcd60e51b815260040161102c90612c2b565b601854816112d4600154600054036000190190565b6112de9190612c59565b11156112fc5760405162461bcd60e51b815260040161102c90612c71565b601a5460ff161561134f5760405162461bcd60e51b815260206004820152601760248201527f54686520636f6e74726163742069732070617573656421000000000000000000604482015260640161102c565b33321461139e5760405162461bcd60e51b815260206004820152601e60248201527f546865206d696e74657220697320616e6f7468657220636f6e74726163740000604482015260640161102c565b336000908152600c60205260409020546014906113bc908390612c59565b11156113da5760405162461bcd60e51b815260040161102c90612c9f565b336000908152600d602052604090205460ff16611493576011546017546114019190612cd6565b60175461140e9083612cd6565b6114189190612cf5565b3410156114375760405162461bcd60e51b815260040161102c90612d0c565b6011546016600082825461144b9190612c59565b9091555050336000908152600c60205260408120805483929061146f908490612c59565b9091555050336000908152600d60205260409020805460ff191660011790556114e4565b6017546114a09082612cd6565b3410156114bf5760405162461bcd60e51b815260040161102c90612d0c565b336000908152600c6020526040812080548392906114de908490612c59565b90915550505b6114ee338261206d565b50565b3360008181526007602090815260408083206001600160a01b03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b60158054610eb890612b8c565b611572611dcc565b601955565b61157f611dcc565b601a80549115156101000261ff0019909216919091179055565b6115a4848484610c6d565b6001600160a01b0383163b156115d4576115c084848484612087565b6115d4576115d46368d2bf6b60e11b611d1f565b50505050565b6040805160808101825260008082526020820181905291810182905260608101919091526001821061163957600054821015611639575b6000828152600460205260409020546116305760001990910190611611565b610b5482612175565b919050565b606061164982611cd6565b6116ad5760405162461bcd60e51b815260206004820152602f60248201527f4552433732314d657461646174613a2055524920717565727920666f72206e6f60448201526e3732bc34b9ba32b73a103a37b5b2b760891b606482015260840161102c565b601a5462010000900460ff1661174f57601580546116ca90612b8c565b80601f01602080910402602001604051908101604052809291908181526020018280546116f690612b8c565b80156117435780601f1061171857610100808354040283529160200191611743565b820191906000526020600020905b81548152906001019060200180831161172657829003601f168201915b50505050509050919050565b60006117596121f4565b9050600081511161177957604051806020016040528060008152506117a7565b8061178384612203565b601460405160200161179793929190612d39565b6040516020818303038152906040525b9392505050565b6000831180156117c057506019548311155b6117dc5760405162461bcd60e51b815260040161102c90612c2b565b601854836117f1600154600054036000190190565b6117fb9190612c59565b11156118195760405162461bcd60e51b815260040161102c90612c71565b6012546017546118299190612cd6565b836017546118379190612cd6565b6118419190612cf5565b3410156118605760405162461bcd60e51b815260040161102c90612d0c565b601a54610100900460ff166118c25760405162461bcd60e51b815260206004820152602260248201527f5468652077686974656c6973742073616c65206973206e6f7420656e61626c65604482015261642160f01b606482015260840161102c565b336000908152600b602052604090205460ff16156119225760405162461bcd60e51b815260206004820152601860248201527f4164647265737320616c726561647920636c61696d6564210000000000000000604482015260640161102c565b6040516bffffffffffffffffffffffff193360601b16602082015260009060340160408051808303601f19018152919052805160209091012090503332146119ac5760405162461bcd60e51b815260206004820152601e60248201527f546865206d696e74657220697320616e6f7468657220636f6e74726163740000604482015260640161102c565b6119ed83838080602002602001604051908101604052809392919081815260200183836020028082843760009201919091525050600a549150849050612298565b611a2a5760405162461bcd60e51b815260206004820152600e60248201526d496e76616c69642070726f6f662160901b604482015260640161102c565b336000908152600c6020526040902054601411611a595760405162461bcd60e51b815260040161102c90612c9f565b336000908152600c6020526040902054601490611a77908690612c59565b1115611a955760405162461bcd60e51b815260040161102c90612c9f565b60125460166000828254611aa99190612c59565b9091555050336000908152600b602090815260408083208054600160ff199182168117909255600d845282852080549091169091179055600c90915281208054869290611af7908490612c59565b909155506115d49050338561206d565b611b0f611dcc565b600f546001600160a01b031663a9059cbb611b326008546001600160a01b031690565b6040516001600160e01b031960e084901b1681526001600160a01b03909116600482015260248101849052604401602060405180830381600087803b158015611b7a57600080fd5b505af1158015611b8e573d6000803e3d6000fd5b505050506040513d601f19601f82011682018060405250810190610c339190612bdd565b611bba611dcc565b601a8054911515620100000262ff000019909216919091179055565b611bde611dcc565b601155565b611beb611dcc565b600082118015611bfd57506019548211155b611c195760405162461bcd60e51b815260040161102c90612c2b565b60185482611c2e600154600054036000190190565b611c389190612c59565b1115611c565760405162461bcd60e51b815260040161102c90612c71565b610c33818361206d565b611c68611dcc565b6001600160a01b038116611ccd5760405162461bcd60e51b815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201526564647265737360d01b606482015260840161102c565b6114ee81611f1c565b600081600111611639576000548210156116395760005b5060008281526004602052604090205480611d1257611d0b83612dfd565b9250611ced565b600160e01b161592915050565b8060005260046000fd5b6000611d3483610fbc565b9050818015611d4c5750336001600160a01b03821614155b15611d6f57611d5b8133610a2c565b611d6f57611d6f6367d9dca160e11b611d1f565b60008381526006602052604080822080546001600160a01b0319166001600160a01b0388811691821790925591518693918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a450505050565b6008546001600160a01b03163314610e545760405162461bcd60e51b815260206004820181905260248201527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572604482015260640161102c565b600081600111611eb2575060008181526004602052604090205480611ea2576000548210611e5e57611e5e636f96cda160e11b611d1f565b5b506000190160008181526004602052604090205480611e7d57611e5f565b600160e01b8116611e8d57919050565b611e9d636f96cda160e11b611d1f565b611e5f565b600160e01b8116611eb257919050565b611639636f96cda160e11b611d1f565b60026009541415611f155760405162461bcd60e51b815260206004820152601f60248201527f5265656e7472616e637947756172643a207265656e7472616e742063616c6c00604482015260640161102c565b6002600955565b600880546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b6060818310611f8757611f87631960ccad60e11b611d1f565b6001831015611f9557600192505b600054808310611fa3578092505b60606000611fb0876111a8565b85871090810291508115612061578187870311611fcd5786860391505b60405192506001820160051b83016040526000611fe9886115da565b905060008160400151611ffa575080515b60005b6120068a612175565b925060408301516000811461201e5760009250612043565b83511561202a57835192505b8b831860601b612043576001820191508a8260051b8801525b5060018a019950888a148061205757508481145b15611ffd57855250505b50909695505050505050565b610c338282604051806020016040528060008152506122ae565b604051630a85bd0160e11b81526000906001600160a01b0385169063150b7a02906120bc903390899088908890600401612e14565b602060405180830381600087803b1580156120d657600080fd5b505af1925050508015612106575060408051601f3d908101601f1916820190925261210391810190612e51565b60015b612158573d808015612134576040519150601f19603f3d011682016040523d82523d6000602084013e612139565b606091505b508051612150576121506368d2bf6b60e11b611d1f565b805181602001fd5b6001600160e01b031916630a85bd0160e11b149050949350505050565b604080516080810182526000808252602082018190529181018290526060810191909152600082815260046020526040902054610b5490604080516080810182526001600160a01b038316815260a083901c67ffffffffffffffff166020820152600160e01b831615159181019190915260e89190911c606082015290565b606060138054610b6990612b8c565b6060600061221083612310565b600101905060008167ffffffffffffffff811115612230576122306126a1565b6040519080825280601f01601f19166020018201604052801561225a576020820181803683370190505b5090508181016020015b600019016f181899199a1a9b1b9c1cb0b131b232b360811b600a86061a8153600a850494508461229357610fa7565b612264565b6000826122a585846123e8565b14949350505050565b6122b8838361242d565b6001600160a01b0383163b15610e71576000548281035b6122e26000868380600101945086612087565b6122f6576122f66368d2bf6b60e11b611d1f565b8181106122cf5781600054146111a1576111a16000611d1f565b60008072184f03e93ff9f4daa797ed6e38ed64bf6a1f0160401b831061234f5772184f03e93ff9f4daa797ed6e38ed64bf6a1f0160401b830492506040015b6d04ee2d6d415b85acef8100000000831061237b576d04ee2d6d415b85acef8100000000830492506020015b662386f26fc10000831061239957662386f26fc10000830492506010015b6305f5e10083106123b1576305f5e100830492506008015b61271083106123c557612710830492506004015b606483106123d7576064830492506002015b600a8310610b545760010192915050565b600081815b8451811015610fa7576124198286838151811061240c5761240c612bc7565b60200260200101516124e4565b91508061242581612c10565b9150506123ed565b600054816124455761244563b562e8dd60e01b611d1f565b60008181526004602090815260408083206001600160a01b0387164260a01b6001881460e11b17811790915580845260059092529091208054680100000000000000018502019055806124a1576124a1622e076360e81b611d1f565b818301825b808360007fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a4600101808214156124a6575060005550505050565b60008183106125005760008281526020849052604090206117a7565b5060009182526020526040902090565b82805461251c90612b8c565b90600052602060002090601f01602090048101928261253e5760008555612584565b82601f1061255757805160ff1916838001178555612584565b82800160010185558215612584579182015b82811115612584578251825591602001919060010190612569565b50612590929150612594565b5090565b5b808211156125905760008155600101612595565b6001600160e01b0319811681146114ee57600080fd5b6000602082840312156125d157600080fd5b81356117a7816125a9565b60005b838110156125f75781810151838201526020016125df565b838111156115d45750506000910152565b600081518084526126208160208601602086016125dc565b601f01601f19169290920160200192915050565b6020815260006117a76020830184612608565b60006020828403121561265957600080fd5b5035919050565b80356001600160a01b038116811461163957600080fd5b6000806040838503121561268a57600080fd5b61269383612660565b946020939093013593505050565b634e487b7160e01b600052604160045260246000fd5b604051601f8201601f1916810167ffffffffffffffff811182821017156126e0576126e06126a1565b604052919050565b600067ffffffffffffffff831115612702576127026126a1565b612715601f8401601f19166020016126b7565b905082815283838301111561272957600080fd5b828260208301376000602084830101529392505050565b60006020828403121561275257600080fd5b813567ffffffffffffffff81111561276957600080fd5b8201601f8101841361277a57600080fd5b611247848235602084016126e8565b80151581146114ee57600080fd5b6000602082840312156127a957600080fd5b81356117a781612789565b6000806000606084860312156127c957600080fd5b6127d284612660565b92506127e060208501612660565b9150604084013590509250925092565b60006020828403121561280257600080fd5b6117a782612660565b60008083601f84011261281d57600080fd5b50813567ffffffffffffffff81111561283557600080fd5b6020830191508360208260051b850101111561285057600080fd5b9250929050565b6000806020838503121561286a57600080fd5b823567ffffffffffffffff81111561288157600080fd5b61288d8582860161280b565b90969095509350505050565b80516001600160a01b0316825260208082015167ffffffffffffffff169083015260408082015115159083015260609081015162ffffff16910152565b6020808252825182820181905260009190848201906040850190845b8181101561206157612905838551612899565b92840192608092909201916001016128f2565b6000602080838503121561292b57600080fd5b823567ffffffffffffffff8082111561294357600080fd5b818501915085601f83011261295757600080fd5b813581811115612969576129696126a1565b8060051b915061297a8483016126b7565b818152918301840191848101908884111561299457600080fd5b938501935b838510156129b257843582529385019390850190612999565b98975050505050505050565b6020808252825182820181905260009190848201906040850190845b81811015612061578351835292840192918401916001016129da565b600080600060608486031215612a0b57600080fd5b612a1484612660565b95602085013595506040909401359392505050565b60008060408385031215612a3c57600080fd5b612a4583612660565b91506020830135612a5581612789565b809150509250929050565b60008060008060808587031215612a7657600080fd5b612a7f85612660565b9350612a8d60208601612660565b925060408501359150606085013567ffffffffffffffff811115612ab057600080fd5b8501601f81018713612ac157600080fd5b612ad0878235602084016126e8565b91505092959194509250565b60808101610b548284612899565b600080600060408486031215612aff57600080fd5b83359250602084013567ffffffffffffffff811115612b1d57600080fd5b612b298682870161280b565b9497909650939450505050565b60008060408385031215612b4957600080fd5b612b5283612660565b9150612b6060208401612660565b90509250929050565b60008060408385031215612b7c57600080fd5b82359150612b6060208401612660565b600181811c90821680612ba057607f821691505b60208210811415612bc157634e487b7160e01b600052602260045260246000fd5b50919050565b634e487b7160e01b600052603260045260246000fd5b600060208284031215612bef57600080fd5b81516117a781612789565b634e487b7160e01b600052601160045260246000fd5b6000600019821415612c2457612c24612bfa565b5060010190565b602080825260149082015273496e76616c6964206d696e7420616d6f756e742160601b604082015260600190565b60008219821115612c6c57612c6c612bfa565b500190565b6020808252601490820152734d617820737570706c792065786365656465642160601b604082015260600190565b6020808252601f908201527f4d6178696d756d206e756d626572206f662077616c6c65747320697320323000604082015260600190565b6000816000190483118215151615612cf057612cf0612bfa565b500290565b600082821015612d0757612d07612bfa565b500390565b602080825260139082015272496e73756666696369656e742066756e64732160681b604082015260600190565b600084516020612d4c8285838a016125dc565b855191840191612d5f8184848a016125dc565b8554920191600090600181811c9080831680612d7c57607f831692505b858310811415612d9a57634e487b7160e01b85526022600452602485fd5b808015612dae5760018114612dbf57612dec565b60ff19851688528388019550612dec565b60008b81526020902060005b85811015612de45781548a820152908401908801612dcb565b505083880195505b50939b9a5050505050505050505050565b600081612e0c57612e0c612bfa565b506000190190565b6001600160a01b0385811682528416602082015260408101839052608060608201819052600090612e4790830184612608565b9695505050505050565b600060208284031215612e6357600080fd5b81516117a7816125a956fea26469706673582212208618e0c8a68ec3a577d22999e1ffbfc6f6012574f509b5a2aa394f662957318764736f6c6343000809003300000000000000000000000000000000000000000000000000000000000000c00000000000000000000000000000000000000000000000000000000000000100000000000000000000000000000000000000000000000000006a94d74f4300000000000000000000000000000000000000000000000000000000000000001e6100000000000000000000000000000000000000000000000000000000000000140000000000000000000000000000000000000000000000000000000000000140000000000000000000000000000000000000000000000000000000000000000750656520506565000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000003506565000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000022727000000000000000000000000000000000000000000000000000000000000

Deployed Bytecode

0x6080604052600436106103975760003560e01c80637cb64759116101dc578063c7c39ffc11610102578063e0a80853116100a0578063efbd73f41161006f578063efbd73f414610a7a578063f1a631ec14610a9a578063f2fde38b14610abb578063fbbf8cc314610adb57600080fd5b8063e0a80853146109d1578063e945971c146109f1578063e985e9c514610a11578063ef29948914610a5a57600080fd5b8063d5abeb01116100dc578063d5abeb0114610955578063dad7b5c91461096b578063db4bec4414610981578063dc8c3270146109b157600080fd5b8063c7c39ffc1461090c578063c87b56dd14610922578063d2cab0561461094257600080fd5b806399a2557a1161017a578063b071401b11610149578063b071401b1461088c578063b767a098146108ac578063b88d4fde146108cc578063c23dc68f146108df57600080fd5b806399a2557a14610824578063a0712d6814610844578063a22cb46514610857578063a45ba8e71461087757600080fd5b80638da5cb5b116101b65780638da5cb5b146107bb57806394354fd0146107d957806395d89b41146107ef57806398dfe50b1461080457600080fd5b80637cb647591461074e5780637ec4a6591461076e5780638462151c1461078e57600080fd5b80634fdd43cb116102c15780635c975abb1161025f5780636caede3d1161022e5780636caede3d146106ca57806370a08231146106e9578063715018a614610709578063745308e71461071e57600080fd5b80635c975abb1461065b57806362b99ad4146106755780636352211e1461068a57806364febc38146106aa57600080fd5b80635503a0e81161029b5780635503a0e8146105d957806357a2e24b146105ee57806359236f3a1461060e5780635bbb21771461062e57600080fd5b80634fdd43cb146105795780635183022714610599578063542d878b146105b957600080fd5b806316c38b3c116103395780633c4ed0ad116103085780633c4ed0ad1461051b5780633ccfd60b1461053157806342842e0e1461054657806344a0d68a1461055957600080fd5b806316c38b3c146104b457806318160ddd146104d457806323b872dd146104f25780632eb4a7ab1461050557600080fd5b8063081812fc11610375578063081812fc14610423578063095ea7b31461045b57806313faede61461047057806316ba10e01461049457600080fd5b806301ffc9a71461039c57806306fdde03146103d157806307cfa41b146103f3575b600080fd5b3480156103a857600080fd5b506103bc6103b73660046125bf565b610b08565b60405190151581526020015b60405180910390f35b3480156103dd57600080fd5b506103e6610b5a565b6040516103c89190612634565b3480156103ff57600080fd5b506103bc61040e366004612647565b600e6020526000908152604090205460ff1681565b34801561042f57600080fd5b5061044361043e366004612647565b610bec565b6040516001600160a01b0390911681526020016103c8565b61046e610469366004612677565b610c27565b005b34801561047c57600080fd5b5061048660175481565b6040519081526020016103c8565b3480156104a057600080fd5b5061046e6104af366004612740565b610c37565b3480156104c057600080fd5b5061046e6104cf366004612797565b610c52565b3480156104e057600080fd5b50610486600154600054036000190190565b61046e6105003660046127b4565b610c6d565b34801561051157600080fd5b50610486600a5481565b34801561052757600080fd5b5061048660125481565b34801561053d57600080fd5b5061046e610dc8565b61046e6105543660046127b4565b610e56565b34801561056557600080fd5b5061046e610574366004612647565b610e76565b34801561058557600080fd5b5061046e610594366004612740565b610e83565b3480156105a557600080fd5b50601a546103bc9062010000900460ff1681565b3480156105c557600080fd5b5061046e6105d4366004612647565b610e9e565b3480156105e557600080fd5b506103e6610eab565b3480156105fa57600080fd5b50600f54610443906001600160a01b031681565b34801561061a57600080fd5b5061046e6106293660046127f0565b610f39565b34801561063a57600080fd5b5061064e610649366004612857565b610f63565b6040516103c891906128d6565b34801561066757600080fd5b50601a546103bc9060ff1681565b34801561068157600080fd5b506103e6610faf565b34801561069657600080fd5b506104436106a5366004612647565b610fbc565b3480156106b657600080fd5b5061046e6106c5366004612918565b610fc7565b3480156106d657600080fd5b50601a546103bc90610100900460ff1681565b3480156106f557600080fd5b506104866107043660046127f0565b6111a8565b34801561071557600080fd5b5061046e6111ee565b34801561072a57600080fd5b506103bc6107393660046127f0565b600d6020526000908152604090205460ff1681565b34801561075a57600080fd5b5061046e610769366004612647565b611200565b34801561077a57600080fd5b5061046e610789366004612740565b61120d565b34801561079a57600080fd5b506107ae6107a93660046127f0565b611228565b6040516103c891906129be565b3480156107c757600080fd5b506008546001600160a01b0316610443565b3480156107e557600080fd5b5061048660195481565b3480156107fb57600080fd5b506103e661124f565b34801561081057600080fd5b5061046e61081f366004612797565b61125e565b34801561083057600080fd5b506107ae61083f3660046129f6565b611284565b61046e610852366004612647565b611291565b34801561086357600080fd5b5061046e610872366004612a29565b6114f1565b34801561088357600080fd5b506103e661155d565b34801561089857600080fd5b5061046e6108a7366004612647565b61156a565b3480156108b857600080fd5b5061046e6108c7366004612797565b611577565b61046e6108da366004612a60565b611599565b3480156108eb57600080fd5b506108ff6108fa366004612647565b6115da565b6040516103c89190612adc565b34801561091857600080fd5b5061048660115481565b34801561092e57600080fd5b506103e661093d366004612647565b61163e565b61046e610950366004612aea565b6117ae565b34801561096157600080fd5b5061048660185481565b34801561097757600080fd5b5061048660165481565b34801561098d57600080fd5b506103bc61099c3660046127f0565b600b6020526000908152604090205460ff1681565b3480156109bd57600080fd5b5061046e6109cc366004612647565b611b07565b3480156109dd57600080fd5b5061046e6109ec366004612797565b611bb2565b3480156109fd57600080fd5b5061046e610a0c366004612647565b611bd6565b348015610a1d57600080fd5b506103bc610a2c366004612b36565b6001600160a01b03918216600090815260076020908152604080832093909416825291909152205460ff1690565b348015610a6657600080fd5b50601054610443906001600160a01b031681565b348015610a8657600080fd5b5061046e610a95366004612b69565b611be3565b348015610aa657600080fd5b506010546103bc90600160a01b900460ff1681565b348015610ac757600080fd5b5061046e610ad63660046127f0565b611c60565b348015610ae757600080fd5b50610486610af63660046127f0565b600c6020526000908152604090205481565b60006301ffc9a760e01b6001600160e01b031983161480610b3957506380ac58cd60e01b6001600160e01b03198316145b80610b545750635b5e139f60e01b6001600160e01b03198316145b92915050565b606060028054610b6990612b8c565b80601f0160208091040260200160405190810160405280929190818152602001828054610b9590612b8c565b8015610be25780601f10610bb757610100808354040283529160200191610be2565b820191906000526020600020905b815481529060010190602001808311610bc557829003601f168201915b5050505050905090565b6000610bf782611cd6565b610c0b57610c0b6333d1c03960e21b611d1f565b506000908152600660205260409020546001600160a01b031690565b610c3382826001611d29565b5050565b610c3f611dcc565b8051610c33906014906020840190612510565b610c5a611dcc565b601a805460ff1916911515919091179055565b6000610c7882611e26565b6001600160a01b039485169490915081168414610c9e57610c9e62a1148160e81b611d1f565b60008281526006602052604090208054338082146001600160a01b03881690911417610ce257610cce8633610a2c565b610ce257610ce2632ce44b5f60e11b611d1f565b8015610ced57600082555b6001600160a01b038681166000908152600560205260408082208054600019019055918716808252919020805460010190554260a01b17600160e11b17600085815260046020526040902055600160e11b8316610d785760018401600081815260046020526040902054610d76576000548114610d765760008181526004602052604090208490555b505b6001600160a01b0385168481887fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a480610dbf57610dbf633a954ecd60e21b611d1f565b50505050505050565b610dd0611dcc565b610dd8611ec2565b6000610dec6008546001600160a01b031690565b6001600160a01b03164760405160006040518083038185875af1925050503d8060008114610e36576040519150601f19603f3d011682016040523d82523d6000602084013e610e3b565b606091505b5050905080610e4957600080fd5b50610e546001600955565b565b610e7183838360405180602001604052806000815250611599565b505050565b610e7e611dcc565b601755565b610e8b611dcc565b8051610c33906015906020840190612510565b610ea6611dcc565b601255565b60148054610eb890612b8c565b80601f0160208091040260200160405190810160405280929190818152602001828054610ee490612b8c565b8015610f315780601f10610f0657610100808354040283529160200191610f31565b820191906000526020600020905b815481529060010190602001808311610f1457829003601f168201915b505050505081565b610f41611dcc565b600f80546001600160a01b0319166001600160a01b0392909216919091179055565b60408051828152600583901b8082016020019092526060915b8015610fa757601f1980820191860101356000610f98826115da565b8484016020015250610f7c9050565b509392505050565b60138054610eb890612b8c565b6000610b5482611e26565b601054600160a01b900460ff166110355760405162461bcd60e51b815260206004820152602760248201527f416374697669747920726564656d7074696f6e20686173206e6f7420796574206044820152661cdd185c9d195960ca1b60648201526084015b60405180910390fd5b805169010f0cf064dd59200000903360005b828110156111a157600085828151811061106357611063612bc7565b60200260200101519050826001600160a01b031661108082610fbc565b6001600160a01b0316146110d65760405162461bcd60e51b815260206004820152601860248201527f596f7520646f6e2774206f776e207468697320746f6b656e0000000000000000604482015260640161102c565b6000818152600e602052604090205460ff1661118e576000818152600e602052604090819020805460ff19166001179055600f54905163a9059cbb60e01b81526001600160a01b038581166004830152602482018890529091169063a9059cbb90604401602060405180830381600087803b15801561115457600080fd5b505af1158015611168573d6000803e3d6000fd5b505050506040513d601f19601f8201168201806040525081019061118c9190612bdd565b505b508061119981612c10565b915050611047565b5050505050565b60006001600160a01b0382166111c8576111c86323d3ad8160e21b611d1f565b506001600160a01b031660009081526005602052604090205467ffffffffffffffff1690565b6111f6611dcc565b610e546000611f1c565b611208611dcc565b600a55565b611215611dcc565b8051610c33906013906020840190612510565b6000546060906001908282821461124757611244858484611f6e565b90505b949350505050565b606060038054610b6990612b8c565b611266611dcc565b60108054911515600160a01b0260ff60a01b19909216919091179055565b6060611247848484611f6e565b6000811180156112a357506019548111155b6112bf5760405162461bcd60e51b815260040161102c90612c2b565b601854816112d4600154600054036000190190565b6112de9190612c59565b11156112fc5760405162461bcd60e51b815260040161102c90612c71565b601a5460ff161561134f5760405162461bcd60e51b815260206004820152601760248201527f54686520636f6e74726163742069732070617573656421000000000000000000604482015260640161102c565b33321461139e5760405162461bcd60e51b815260206004820152601e60248201527f546865206d696e74657220697320616e6f7468657220636f6e74726163740000604482015260640161102c565b336000908152600c60205260409020546014906113bc908390612c59565b11156113da5760405162461bcd60e51b815260040161102c90612c9f565b336000908152600d602052604090205460ff16611493576011546017546114019190612cd6565b60175461140e9083612cd6565b6114189190612cf5565b3410156114375760405162461bcd60e51b815260040161102c90612d0c565b6011546016600082825461144b9190612c59565b9091555050336000908152600c60205260408120805483929061146f908490612c59565b9091555050336000908152600d60205260409020805460ff191660011790556114e4565b6017546114a09082612cd6565b3410156114bf5760405162461bcd60e51b815260040161102c90612d0c565b336000908152600c6020526040812080548392906114de908490612c59565b90915550505b6114ee338261206d565b50565b3360008181526007602090815260408083206001600160a01b03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b60158054610eb890612b8c565b611572611dcc565b601955565b61157f611dcc565b601a80549115156101000261ff0019909216919091179055565b6115a4848484610c6d565b6001600160a01b0383163b156115d4576115c084848484612087565b6115d4576115d46368d2bf6b60e11b611d1f565b50505050565b6040805160808101825260008082526020820181905291810182905260608101919091526001821061163957600054821015611639575b6000828152600460205260409020546116305760001990910190611611565b610b5482612175565b919050565b606061164982611cd6565b6116ad5760405162461bcd60e51b815260206004820152602f60248201527f4552433732314d657461646174613a2055524920717565727920666f72206e6f60448201526e3732bc34b9ba32b73a103a37b5b2b760891b606482015260840161102c565b601a5462010000900460ff1661174f57601580546116ca90612b8c565b80601f01602080910402602001604051908101604052809291908181526020018280546116f690612b8c565b80156117435780601f1061171857610100808354040283529160200191611743565b820191906000526020600020905b81548152906001019060200180831161172657829003601f168201915b50505050509050919050565b60006117596121f4565b9050600081511161177957604051806020016040528060008152506117a7565b8061178384612203565b601460405160200161179793929190612d39565b6040516020818303038152906040525b9392505050565b6000831180156117c057506019548311155b6117dc5760405162461bcd60e51b815260040161102c90612c2b565b601854836117f1600154600054036000190190565b6117fb9190612c59565b11156118195760405162461bcd60e51b815260040161102c90612c71565b6012546017546118299190612cd6565b836017546118379190612cd6565b6118419190612cf5565b3410156118605760405162461bcd60e51b815260040161102c90612d0c565b601a54610100900460ff166118c25760405162461bcd60e51b815260206004820152602260248201527f5468652077686974656c6973742073616c65206973206e6f7420656e61626c65604482015261642160f01b606482015260840161102c565b336000908152600b602052604090205460ff16156119225760405162461bcd60e51b815260206004820152601860248201527f4164647265737320616c726561647920636c61696d6564210000000000000000604482015260640161102c565b6040516bffffffffffffffffffffffff193360601b16602082015260009060340160408051808303601f19018152919052805160209091012090503332146119ac5760405162461bcd60e51b815260206004820152601e60248201527f546865206d696e74657220697320616e6f7468657220636f6e74726163740000604482015260640161102c565b6119ed83838080602002602001604051908101604052809392919081815260200183836020028082843760009201919091525050600a549150849050612298565b611a2a5760405162461bcd60e51b815260206004820152600e60248201526d496e76616c69642070726f6f662160901b604482015260640161102c565b336000908152600c6020526040902054601411611a595760405162461bcd60e51b815260040161102c90612c9f565b336000908152600c6020526040902054601490611a77908690612c59565b1115611a955760405162461bcd60e51b815260040161102c90612c9f565b60125460166000828254611aa99190612c59565b9091555050336000908152600b602090815260408083208054600160ff199182168117909255600d845282852080549091169091179055600c90915281208054869290611af7908490612c59565b909155506115d49050338561206d565b611b0f611dcc565b600f546001600160a01b031663a9059cbb611b326008546001600160a01b031690565b6040516001600160e01b031960e084901b1681526001600160a01b03909116600482015260248101849052604401602060405180830381600087803b158015611b7a57600080fd5b505af1158015611b8e573d6000803e3d6000fd5b505050506040513d601f19601f82011682018060405250810190610c339190612bdd565b611bba611dcc565b601a8054911515620100000262ff000019909216919091179055565b611bde611dcc565b601155565b611beb611dcc565b600082118015611bfd57506019548211155b611c195760405162461bcd60e51b815260040161102c90612c2b565b60185482611c2e600154600054036000190190565b611c389190612c59565b1115611c565760405162461bcd60e51b815260040161102c90612c71565b610c33818361206d565b611c68611dcc565b6001600160a01b038116611ccd5760405162461bcd60e51b815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201526564647265737360d01b606482015260840161102c565b6114ee81611f1c565b600081600111611639576000548210156116395760005b5060008281526004602052604090205480611d1257611d0b83612dfd565b9250611ced565b600160e01b161592915050565b8060005260046000fd5b6000611d3483610fbc565b9050818015611d4c5750336001600160a01b03821614155b15611d6f57611d5b8133610a2c565b611d6f57611d6f6367d9dca160e11b611d1f565b60008381526006602052604080822080546001600160a01b0319166001600160a01b0388811691821790925591518693918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a450505050565b6008546001600160a01b03163314610e545760405162461bcd60e51b815260206004820181905260248201527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572604482015260640161102c565b600081600111611eb2575060008181526004602052604090205480611ea2576000548210611e5e57611e5e636f96cda160e11b611d1f565b5b506000190160008181526004602052604090205480611e7d57611e5f565b600160e01b8116611e8d57919050565b611e9d636f96cda160e11b611d1f565b611e5f565b600160e01b8116611eb257919050565b611639636f96cda160e11b611d1f565b60026009541415611f155760405162461bcd60e51b815260206004820152601f60248201527f5265656e7472616e637947756172643a207265656e7472616e742063616c6c00604482015260640161102c565b6002600955565b600880546001600160a01b038381166001600160a01b0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b6060818310611f8757611f87631960ccad60e11b611d1f565b6001831015611f9557600192505b600054808310611fa3578092505b60606000611fb0876111a8565b85871090810291508115612061578187870311611fcd5786860391505b60405192506001820160051b83016040526000611fe9886115da565b905060008160400151611ffa575080515b60005b6120068a612175565b925060408301516000811461201e5760009250612043565b83511561202a57835192505b8b831860601b612043576001820191508a8260051b8801525b5060018a019950888a148061205757508481145b15611ffd57855250505b50909695505050505050565b610c338282604051806020016040528060008152506122ae565b604051630a85bd0160e11b81526000906001600160a01b0385169063150b7a02906120bc903390899088908890600401612e14565b602060405180830381600087803b1580156120d657600080fd5b505af1925050508015612106575060408051601f3d908101601f1916820190925261210391810190612e51565b60015b612158573d808015612134576040519150601f19603f3d011682016040523d82523d6000602084013e612139565b606091505b508051612150576121506368d2bf6b60e11b611d1f565b805181602001fd5b6001600160e01b031916630a85bd0160e11b149050949350505050565b604080516080810182526000808252602082018190529181018290526060810191909152600082815260046020526040902054610b5490604080516080810182526001600160a01b038316815260a083901c67ffffffffffffffff166020820152600160e01b831615159181019190915260e89190911c606082015290565b606060138054610b6990612b8c565b6060600061221083612310565b600101905060008167ffffffffffffffff811115612230576122306126a1565b6040519080825280601f01601f19166020018201604052801561225a576020820181803683370190505b5090508181016020015b600019016f181899199a1a9b1b9c1cb0b131b232b360811b600a86061a8153600a850494508461229357610fa7565b612264565b6000826122a585846123e8565b14949350505050565b6122b8838361242d565b6001600160a01b0383163b15610e71576000548281035b6122e26000868380600101945086612087565b6122f6576122f66368d2bf6b60e11b611d1f565b8181106122cf5781600054146111a1576111a16000611d1f565b60008072184f03e93ff9f4daa797ed6e38ed64bf6a1f0160401b831061234f5772184f03e93ff9f4daa797ed6e38ed64bf6a1f0160401b830492506040015b6d04ee2d6d415b85acef8100000000831061237b576d04ee2d6d415b85acef8100000000830492506020015b662386f26fc10000831061239957662386f26fc10000830492506010015b6305f5e10083106123b1576305f5e100830492506008015b61271083106123c557612710830492506004015b606483106123d7576064830492506002015b600a8310610b545760010192915050565b600081815b8451811015610fa7576124198286838151811061240c5761240c612bc7565b60200260200101516124e4565b91508061242581612c10565b9150506123ed565b600054816124455761244563b562e8dd60e01b611d1f565b60008181526004602090815260408083206001600160a01b0387164260a01b6001881460e11b17811790915580845260059092529091208054680100000000000000018502019055806124a1576124a1622e076360e81b611d1f565b818301825b808360007fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef600080a4600101808214156124a6575060005550505050565b60008183106125005760008281526020849052604090206117a7565b5060009182526020526040902090565b82805461251c90612b8c565b90600052602060002090601f01602090048101928261253e5760008555612584565b82601f1061255757805160ff1916838001178555612584565b82800160010185558215612584579182015b82811115612584578251825591602001919060010190612569565b50612590929150612594565b5090565b5b808211156125905760008155600101612595565b6001600160e01b0319811681146114ee57600080fd5b6000602082840312156125d157600080fd5b81356117a7816125a9565b60005b838110156125f75781810151838201526020016125df565b838111156115d45750506000910152565b600081518084526126208160208601602086016125dc565b601f01601f19169290920160200192915050565b6020815260006117a76020830184612608565b60006020828403121561265957600080fd5b5035919050565b80356001600160a01b038116811461163957600080fd5b6000806040838503121561268a57600080fd5b61269383612660565b946020939093013593505050565b634e487b7160e01b600052604160045260246000fd5b604051601f8201601f1916810167ffffffffffffffff811182821017156126e0576126e06126a1565b604052919050565b600067ffffffffffffffff831115612702576127026126a1565b612715601f8401601f19166020016126b7565b905082815283838301111561272957600080fd5b828260208301376000602084830101529392505050565b60006020828403121561275257600080fd5b813567ffffffffffffffff81111561276957600080fd5b8201601f8101841361277a57600080fd5b611247848235602084016126e8565b80151581146114ee57600080fd5b6000602082840312156127a957600080fd5b81356117a781612789565b6000806000606084860312156127c957600080fd5b6127d284612660565b92506127e060208501612660565b9150604084013590509250925092565b60006020828403121561280257600080fd5b6117a782612660565b60008083601f84011261281d57600080fd5b50813567ffffffffffffffff81111561283557600080fd5b6020830191508360208260051b850101111561285057600080fd5b9250929050565b6000806020838503121561286a57600080fd5b823567ffffffffffffffff81111561288157600080fd5b61288d8582860161280b565b90969095509350505050565b80516001600160a01b0316825260208082015167ffffffffffffffff169083015260408082015115159083015260609081015162ffffff16910152565b6020808252825182820181905260009190848201906040850190845b8181101561206157612905838551612899565b92840192608092909201916001016128f2565b6000602080838503121561292b57600080fd5b823567ffffffffffffffff8082111561294357600080fd5b818501915085601f83011261295757600080fd5b813581811115612969576129696126a1565b8060051b915061297a8483016126b7565b818152918301840191848101908884111561299457600080fd5b938501935b838510156129b257843582529385019390850190612999565b98975050505050505050565b6020808252825182820181905260009190848201906040850190845b81811015612061578351835292840192918401916001016129da565b600080600060608486031215612a0b57600080fd5b612a1484612660565b95602085013595506040909401359392505050565b60008060408385031215612a3c57600080fd5b612a4583612660565b91506020830135612a5581612789565b809150509250929050565b60008060008060808587031215612a7657600080fd5b612a7f85612660565b9350612a8d60208601612660565b925060408501359150606085013567ffffffffffffffff811115612ab057600080fd5b8501601f81018713612ac157600080fd5b612ad0878235602084016126e8565b91505092959194509250565b60808101610b548284612899565b600080600060408486031215612aff57600080fd5b83359250602084013567ffffffffffffffff811115612b1d57600080fd5b612b298682870161280b565b9497909650939450505050565b60008060408385031215612b4957600080fd5b612b5283612660565b9150612b6060208401612660565b90509250929050565b60008060408385031215612b7c57600080fd5b82359150612b6060208401612660565b600181811c90821680612ba057607f821691505b60208210811415612bc157634e487b7160e01b600052602260045260246000fd5b50919050565b634e487b7160e01b600052603260045260246000fd5b600060208284031215612bef57600080fd5b81516117a781612789565b634e487b7160e01b600052601160045260246000fd5b6000600019821415612c2457612c24612bfa565b5060010190565b602080825260149082015273496e76616c6964206d696e7420616d6f756e742160601b604082015260600190565b60008219821115612c6c57612c6c612bfa565b500190565b6020808252601490820152734d617820737570706c792065786365656465642160601b604082015260600190565b6020808252601f908201527f4d6178696d756d206e756d626572206f662077616c6c65747320697320323000604082015260600190565b6000816000190483118215151615612cf057612cf0612bfa565b500290565b600082821015612d0757612d07612bfa565b500390565b602080825260139082015272496e73756666696369656e742066756e64732160681b604082015260600190565b600084516020612d4c8285838a016125dc565b855191840191612d5f8184848a016125dc565b8554920191600090600181811c9080831680612d7c57607f831692505b858310811415612d9a57634e487b7160e01b85526022600452602485fd5b808015612dae5760018114612dbf57612dec565b60ff19851688528388019550612dec565b60008b81526020902060005b85811015612de45781548a820152908401908801612dcb565b505083880195505b50939b9a5050505050505050505050565b600081612e0c57612e0c612bfa565b506000190190565b6001600160a01b0385811682528416602082015260408101839052608060608201819052600090612e4790830184612608565b9695505050505050565b600060208284031215612e6357600080fd5b81516117a7816125a956fea26469706673582212208618e0c8a68ec3a577d22999e1ffbfc6f6012574f509b5a2aa394f662957318764736f6c63430008090033

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

00000000000000000000000000000000000000000000000000000000000000c00000000000000000000000000000000000000000000000000000000000000100000000000000000000000000000000000000000000000000006a94d74f4300000000000000000000000000000000000000000000000000000000000000001e6100000000000000000000000000000000000000000000000000000000000000140000000000000000000000000000000000000000000000000000000000000140000000000000000000000000000000000000000000000000000000000000000750656520506565000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000003506565000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000022727000000000000000000000000000000000000000000000000000000000000

-----Decoded View---------------
Arg [0] : _tokenName (string): Pee Pee
Arg [1] : _tokenSymbol (string): Pee
Arg [2] : _cost (uint256): 30000000000000000
Arg [3] : _maxSupply (uint256): 7777
Arg [4] : _maxMintAmountPerTx (uint256): 20
Arg [5] : _hiddenMetadataUri (string): ''

-----Encoded View---------------
12 Constructor Arguments found :
Arg [0] : 00000000000000000000000000000000000000000000000000000000000000c0
Arg [1] : 0000000000000000000000000000000000000000000000000000000000000100
Arg [2] : 000000000000000000000000000000000000000000000000006a94d74f430000
Arg [3] : 0000000000000000000000000000000000000000000000000000000000001e61
Arg [4] : 0000000000000000000000000000000000000000000000000000000000000014
Arg [5] : 0000000000000000000000000000000000000000000000000000000000000140
Arg [6] : 0000000000000000000000000000000000000000000000000000000000000007
Arg [7] : 5065652050656500000000000000000000000000000000000000000000000000
Arg [8] : 0000000000000000000000000000000000000000000000000000000000000003
Arg [9] : 5065650000000000000000000000000000000000000000000000000000000000
Arg [10] : 0000000000000000000000000000000000000000000000000000000000000002
Arg [11] : 2727000000000000000000000000000000000000000000000000000000000000


Deployed Bytecode Sourcemap

1033:6469:8:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;9164:630:1;;;;;;;;;;-1:-1:-1;9164:630:1;;;;;:::i;:::-;;:::i;:::-;;;565:14:11;;558:22;540:41;;528:2;513:18;9164:630:1;;;;;;;;10048:98;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;1306:36:8:-;;;;;;;;;;-1:-1:-1;1306:36:8;;;;;:::i;:::-;;;;;;;;;;;;;;;;16911:223:1;;;;;;;;;;-1:-1:-1;16911:223:1;;;;;:::i;:::-;;:::i;:::-;;;-1:-1:-1;;;;;1692:32:11;;;1674:51;;1662:2;1647:18;16911:223:1;1528:203:11;16639:122:1;;;;;;:::i;:::-;;:::i;:::-;;1668:19:8;;;;;;;;;;;;;;;;;;;2319:25:11;;;2307:2;2292:18;1668:19:8;2173:177:11;6707:100:8;;;;;;;;;;-1:-1:-1;6707:100:8;;;;;:::i;:::-;;:::i;6813:77::-;;;;;;;;;;-1:-1:-1;6813:77:8;;;;;:::i;:::-;;:::i;5894:317:1:-;;;;;;;;;;;;5498:1:8;6164:12:1;5955:7;6148:13;:28;-1:-1:-1;;6148:46:1;;5894:317;20546:3447;;;;;;:::i;:::-;;:::i;1131:25:8:-;;;;;;;;;;;;;;;;1486:34;;;;;;;;;;;;;;;;7111:156;;;;;;;;;;;;;:::i;24084:187:1:-;;;;;;:::i;:::-;;:::i;6055:74:8:-;;;;;;;;;;-1:-1:-1;6055:74:8;;;;;:::i;:::-;;:::i;6463:132::-;;;;;;;;;;-1:-1:-1;6463:132:8;;;;;:::i;:::-;;:::i;1836:28::-;;;;;;;;;;-1:-1:-1;1836:28:8;;;;;;;;;;;6226:97;;;;;;;;;;-1:-1:-1;6226:97:8;;;;;:::i;:::-;;:::i;1558:33::-;;;;;;;;;;;;;:::i;1347:29::-;;;;;;;;;;-1:-1:-1;1347:29:8;;;;-1:-1:-1;;;;;1347:29:8;;;3420:109;;;;;;;;;;-1:-1:-1;3420:109:8;;;;;:::i;:::-;;:::i;1801:1131:2:-;;;;;;;;;;-1:-1:-1;1801:1131:2;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;1761:25:8:-;;;;;;;;;;-1:-1:-1;1761:25:8;;;;;;;;1525:28;;;;;;;;;;;;;:::i;11409:150:1:-;;;;;;;;;;-1:-1:-1;11409:150:1;;;;;:::i;:::-;;:::i;3534:566:8:-;;;;;;;;;;-1:-1:-1;3534:566:8;;;;;:::i;:::-;;:::i;1791:40::-;;;;;;;;;;-1:-1:-1;1791:40:8;;;;;;;;;;;7045:239:1;;;;;;;;;;-1:-1:-1;7045:239:1;;;;;:::i;:::-;;:::i;1824:101:7:-;;;;;;;;;;;;;:::i;1265:36:8:-;;;;;;;;;;-1:-1:-1;1265:36:8;;;;;:::i;:::-;;;;;;;;;;;;;;;;6896:98;;;;;;;;;;-1:-1:-1;6896:98:8;;;;;:::i;:::-;;:::i;6601:100::-;;;;;;;;;;-1:-1:-1;6601:100:8;;;;;:::i;:::-;;:::i;3958:319:2:-;;;;;;;;;;-1:-1:-1;3958:319:2;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;1194:85:7:-;;;;;;;;;;-1:-1:-1;1266:6:7;;-1:-1:-1;;;;;1266:6:7;1194:85;;1721:33:8;;;;;;;;;;;;;;;;10217:102:1;;;;;;;;;;;;;:::i;4104:94:8:-;;;;;;;;;;-1:-1:-1;4104:94:8;;;;;:::i;:::-;;:::i;3306:217:2:-;;;;;;;;;;-1:-1:-1;3306:217:2;;;;;:::i;:::-;;:::i;4205:890:8:-;;;;;;:::i;:::-;;:::i;17461:231:1:-;;;;;;;;;;-1:-1:-1;17461:231:1;;;;;:::i;:::-;;:::i;1596:31:8:-;;;;;;;;;;;;;:::i;6327:130::-;;;;;;;;;;-1:-1:-1;6327:130:8;;;;;:::i;:::-;;:::i;7000:105::-;;;;;;;;;;-1:-1:-1;7000:105:8;;;;;:::i;:::-;;:::i;24852:405:1:-;;;;;;:::i;:::-;;:::i;1069:579:2:-;;;;;;;;;;-1:-1:-1;1069:579:2;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;1453:28:8:-;;;;;;;;;;;;;;;;5513:449;;;;;;;;;;-1:-1:-1;5513:449:8;;;;;:::i;:::-;;:::i;2303:1111::-;;;;;;:::i;:::-;;:::i;1692:24::-;;;;;;;;;;;;;;;;1632:31;;;;;;;;;;;;;;;;1161:48;;;;;;;;;;-1:-1:-1;1161:48:8;;;;;:::i;:::-;;;;;;;;;;;;;;;;7275:114;;;;;;;;;;-1:-1:-1;7275:114:8;;;;;:::i;:::-;;:::i;5968:81::-;;;;;;;;;;-1:-1:-1;5968:81:8;;;;;:::i;:::-;;:::i;6135:87::-;;;;;;;;;;-1:-1:-1;6135:87:8;;;;;:::i;:::-;;:::i;17842:162:1:-;;;;;;;;;;-1:-1:-1;17842:162:1;;;;;:::i;:::-;-1:-1:-1;;;;;17962:25:1;;;17939:4;17962:25;;;:18;:25;;;;;;;;:35;;;;;;;;;;;;;;;17842:162;1381:25:8;;;;;;;;;;-1:-1:-1;1381:25:8;;;;-1:-1:-1;;;;;1381:25:8;;;5105:299;;;;;;;;;;-1:-1:-1;5105:299:8;;;;;:::i;:::-;;:::i;1411:37::-;;;;;;;;;;-1:-1:-1;1411:37:8;;;;-1:-1:-1;;;1411:37:8;;;;;;2074:198:7;;;;;;;;;;-1:-1:-1;2074:198:7;;;;;:::i;:::-;;:::i;1214:46:8:-;;;;;;;;;;-1:-1:-1;1214:46:8;;;;;:::i;:::-;;;;;;;;;;;;;;9164:630:1;9249:4;-1:-1:-1;;;;;;;;;9567:25:1;;;;:101;;-1:-1:-1;;;;;;;;;;9643:25:1;;;9567:101;:177;;;-1:-1:-1;;;;;;;;;;9719:25:1;;;9567:177;9548:196;9164:630;-1:-1:-1;;9164:630:1:o;10048:98::-;10102:13;10134:5;10127:12;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;10048:98;:::o;16911:223::-;16987:7;17011:16;17019:7;17011;:16::i;:::-;17006:73;;17029:50;-1:-1:-1;;;17029:7:1;:50::i;:::-;-1:-1:-1;17097:24:1;;;;:15;:24;;;;;:30;-1:-1:-1;;;;;17097:30:1;;16911:223::o;16639:122::-;16727:27;16736:2;16740:7;16749:4;16727:8;:27::i;:::-;16639:122;;:::o;6707:100:8:-;1087:13:7;:11;:13::i;:::-;6779:22:8;;::::1;::::0;:9:::1;::::0;:22:::1;::::0;::::1;::::0;::::1;:::i;6813:77::-:0;1087:13:7;:11;:13::i;:::-;6869:6:8::1;:15:::0;;-1:-1:-1;;6869:15:8::1;::::0;::::1;;::::0;;;::::1;::::0;;6813:77::o;20546:3447:1:-;20683:27;20713;20732:7;20713:18;:27::i;:::-;-1:-1:-1;;;;;20865:22:1;;;;20683:57;;-1:-1:-1;20923:45:1;;;;20919:95;;20970:44;-1:-1:-1;;;20970:7:1;:44::i;:::-;21026:27;19679:24;;;:15;:24;;;;;19903:26;;41487:10;19316:30;;;-1:-1:-1;;;;;19013:28:1;;19294:20;;;19291:56;21209:188;;21301:43;21318:4;41487:10;17842:162;:::i;21301:43::-;21296:101;;21346:51;-1:-1:-1;;;21346:7:1;:51::i;:::-;21540:15;21537:157;;;21678:1;21657:19;21650:30;21537:157;-1:-1:-1;;;;;22066:24:1;;;;;;;:18;:24;;;;;;22064:26;;-1:-1:-1;;22064:26:1;;;22134:22;;;;;;;;;22132:24;;-1:-1:-1;22132:24:1;;;15767:11;15742:23;15738:41;15725:63;-1:-1:-1;;;15725:63:1;22420:26;;;;:17;:26;;;;;:172;-1:-1:-1;;;22709:47:1;;22705:617;;22813:1;22803:11;;22781:19;22934:30;;;:17;:30;;;;;;22930:378;;23070:13;;23055:11;:28;23051:239;;23215:30;;;;:17;:30;;;;;:52;;;23051:239;22763:559;22705:617;-1:-1:-1;;;;;23450:20:1;;23821:7;23450:20;23753:4;23696:25;23431:16;;23564:292;23879:13;23875:58;;23894:39;-1:-1:-1;;;23894:7:1;:39::i;:::-;20673:3320;;;;20546:3447;;;:::o;7111:156:8:-;1087:13:7;:11;:13::i;:::-;2261:21:9::1;:19;:21::i;:::-;7173:7:8::2;7194;1266:6:7::0;;-1:-1:-1;;;;;1266:6:7;;1194:85;7194:7:8::2;-1:-1:-1::0;;;;;7186:21:8::2;7215;7186:55;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;7172:69;;;7256:2;7248:11;;;::::0;::::2;;7161:106;2303:20:9::1;1716:1:::0;2809:7;:22;2629:209;2303:20:::1;7111:156:8:o:0;24084:187:1:-;24225:39;24242:4;24248:2;24252:7;24225:39;;;;;;;;;;;;:16;:39::i;:::-;24084:187;;;:::o;6055:74:8:-;1087:13:7;:11;:13::i;:::-;6111:4:8::1;:12:::0;6055:74::o;6463:132::-;1087:13:7;:11;:13::i;:::-;6551:38:8;;::::1;::::0;:17:::1;::::0;:38:::1;::::0;::::1;::::0;::::1;:::i;6226:97::-:0;1087:13:7;:11;:13::i;:::-;6291:16:8::1;:26:::0;6226:97::o;1558:33::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;3420:109::-;1087:13:7;:11;:13::i;:::-;3490:15:8::1;:33:::0;;-1:-1:-1;;;;;;3490:33:8::1;-1:-1:-1::0;;;;;3490:33:8;;;::::1;::::0;;;::::1;::::0;;3420:109::o;1801:1131:2:-;2148:4;2142:11;;2199:21;;;2348:1;2344:9;;;2402:29;;;2422:4;2402:29;2389:43;;;1940:23;;2451:448;2458:6;;2451:448;;-1:-1:-1;;2541:12:2;;;;2594:23;;;2581:37;2480:15;2679:28;2581:37;2679:19;:28::i;:::-;2834:29;;;2854:4;2834:29;2827:48;-1:-1:-1;2451:448:2;;-1:-1:-1;2451:448:2;;-1:-1:-1;2915:10:2;1801:1131;-1:-1:-1;;;1801:1131:2:o;1525:28:8:-;;;;;;;:::i;11409:150:1:-;11481:7;11523:27;11542:7;11523:18;:27::i;3534:566:8:-;3606:17;;-1:-1:-1;;;3606:17:8;;;;3598:69;;;;-1:-1:-1;;;3598:69:8;;12026:2:11;3598:69:8;;;12008:21:11;12065:2;12045:18;;;12038:30;12104:34;12084:18;;;12077:62;-1:-1:-1;;;12155:18:11;;;12148:37;12202:19;;3598:69:8;;;;;;;;;3735:15;;3696:11;;3774:10;3674:19;3791:306;3815:10;3811:1;:14;3791:306;;;3843:15;3861:8;3870:1;3861:11;;;;;;;;:::i;:::-;;;;;;;3843:29;;3911:6;-1:-1:-1;;;;;3891:26:8;:16;3899:7;3891;:16::i;:::-;-1:-1:-1;;;;;3891:26:8;;3883:63;;;;-1:-1:-1;;;3883:63:8;;12566:2:11;3883:63:8;;;12548:21:11;12605:2;12585:18;;;12578:30;12644:26;12624:18;;;12617:54;12688:18;;3883:63:8;12364:348:11;3883:63:8;3962:16;;;;:7;:16;;;;;;;;3957:133;;3995:16;;;;:7;:16;;;;;;;:23;;-1:-1:-1;;3995:23:8;4014:4;3995:23;;;4033:15;;:45;;-1:-1:-1;;;4033:45:8;;-1:-1:-1;;;;;12909:32:11;;;4033:45:8;;;12891:51:11;12958:18;;;12951:34;;;4033:15:8;;;;:24;;12864:18:11;;4033:45:8;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;3957:133;-1:-1:-1;3827:3:8;;;;:::i;:::-;;;;3791:306;;;;3591:509;;;3534:566;:::o;7045:239:1:-;7117:7;-1:-1:-1;;;;;7140:19:1;;7136:69;;7161:44;-1:-1:-1;;;7161:7:1;:44::i;:::-;-1:-1:-1;;;;;;7222:25:1;;;;;:18;:25;;;;;;1360:13;7222:55;;7045:239::o;1824:101:7:-;1087:13;:11;:13::i;:::-;1888:30:::1;1915:1;1888:18;:30::i;6896:98:8:-:0;1087:13:7;:11;:13::i;:::-;6964:10:8::1;:24:::0;6896:98::o;6601:100::-;1087:13:7;:11;:13::i;:::-;6673:22:8;;::::1;::::0;:9:::1;::::0;:22:::1;::::0;::::1;::::0;::::1;:::i;3958:319:2:-:0;4064:13;5671::1;4036:16:2;;5498:1:8;;4036:16:2;4183:13;;;4179:66;;4209:36;4226:5;4233;4240:4;4209:16;:36::i;:::-;4198:47;;4179:66;4262:8;3958:319;-1:-1:-1;;;;3958:319:2:o;10217:102:1:-;10273:13;10305:7;10298:14;;;;;:::i;4104:94:8:-;1087:13:7;:11;:13::i;:::-;4168:17:8::1;:24:::0;;;::::1;;-1:-1:-1::0;;;4168:24:8::1;-1:-1:-1::0;;;;4168:24:8;;::::1;::::0;;;::::1;::::0;;4104:94::o;3306:217:2:-;3445:16;3480:36;3497:5;3504;3511:4;3480:16;:36::i;4205:890:8:-;4284:1;4270:11;:15;:52;;;;;4304:18;;4289:11;:33;;4270:52;4262:85;;;;-1:-1:-1;;;4262:85:8;;;;;;;:::i;:::-;4393:9;;4378:11;4362:13;5498:1;6164:12:1;5955:7;6148:13;:28;-1:-1:-1;;6148:46:1;;5894:317;4362:13:8;:27;;;;:::i;:::-;:40;;4354:73;;;;-1:-1:-1;;;4354:73:8;;;;;;;:::i;:::-;4443:6;;;;4442:7;4434:43;;;;-1:-1:-1;;;4434:43:8;;14551:2:11;4434:43:8;;;14533:21:11;14590:2;14570:18;;;14563:30;14629:25;14609:18;;;14602:53;14672:18;;4434:43:8;14349:347:11;4434:43:8;41487:10:1;4506:9:8;4492:23;4484:65;;;;-1:-1:-1;;;4484:65:8;;14903:2:11;4484:65:8;;;14885:21:11;14942:2;14922:18;;;14915:30;14981:32;14961:18;;;14954:60;15031:18;;4484:65:8;14701:354:11;4484:65:8;41487:10:1;4564:26:8;;;;:12;:26;;;;;;4604:2;;4564:38;;4591:11;;4564:38;:::i;:::-;:42;;4556:85;;;;-1:-1:-1;;;4556:85:8;;;;;;;:::i;:::-;41487:10:1;4653:20:8;;;;:6;:20;;;;;;;;4648:401;;4735:10;;4730:4;;:15;;;;:::i;:::-;4722:4;;4708:18;;:11;:18;:::i;:::-;4707:38;;;;:::i;:::-;4694:9;:51;;4686:83;;;;-1:-1:-1;;;4686:83:8;;;;;;;:::i;:::-;4799:10;;4780:15;;:29;;;;;;;:::i;:::-;;;;-1:-1:-1;;41487:10:1;4820:26:8;;;;:12;:26;;;;;:41;;4850:11;;4820:26;:41;;4850:11;;4820:41;:::i;:::-;;;;-1:-1:-1;;41487:10:1;4872:20:8;;;;:6;:20;;;;;:27;;-1:-1:-1;;4872:27:8;4895:4;4872:27;;;4648:401;;;4960:4;;4946:18;;:11;:18;:::i;:::-;4932:9;:33;;4924:65;;;;-1:-1:-1;;;4924:65:8;;;;;;;:::i;:::-;41487:10:1;5000:26:8;;;;:12;:26;;;;;:41;;5030:11;;5000:26;:41;;5030:11;;5000:41;:::i;:::-;;;;-1:-1:-1;;4648:401:8;5055:36;41487:10:1;5079:11:8;5055:9;:36::i;:::-;4205:890;:::o;17461:231:1:-;41487:10;17555:39;;;;:18;:39;;;;;;;;-1:-1:-1;;;;;17555:49:1;;;;;;;;;;;;:60;;-1:-1:-1;;17555:60:1;;;;;;;;;;17630:55;;540:41:11;;;17555:49:1;;41487:10;17630:55;;513:18:11;17630:55:1;;;;;;;17461:231;;:::o;1596:31:8:-;;;;;;;:::i;6327:130::-;1087:13:7;:11;:13::i;:::-;6411:18:8::1;:40:::0;6327:130::o;7000:105::-;1087:13:7;:11;:13::i;:::-;7070:20:8::1;:29:::0;;;::::1;;;;-1:-1:-1::0;;7070:29:8;;::::1;::::0;;;::::1;::::0;;7000:105::o;24852:405:1:-;25021:31;25034:4;25040:2;25044:7;25021:12;:31::i;:::-;-1:-1:-1;;;;;25066:14:1;;;:19;25062:189;;25104:56;25135:4;25141:2;25145:7;25154:5;25104:30;:56::i;:::-;25099:152;;25180:56;-1:-1:-1;;;25180:7:1;:56::i;:::-;24852:405;;;;:::o;1069:579:2:-;-1:-1:-1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;5498:1:8;1268:7:2;:26;1264:368;;5645:7:1;5671:13;1318:7:2;:24;1314:304;;;1498:51;12414:4:1;12437:24;;;:17;:24;;;;;;1498:51:2;;-1:-1:-1;;1540:9:2;;;;1498:51;;;1578:21;1591:7;1578:12;:21::i;1314:304::-;1069:579;;;:::o;5513:449:8:-;5587:13;5617:17;5625:8;5617:7;:17::i;:::-;5609:77;;;;-1:-1:-1;;;5609:77:8;;16273:2:11;5609:77:8;;;16255:21:11;16312:2;16292:18;;;16285:30;16351:34;16331:18;;;16324:62;-1:-1:-1;;;16402:18:11;;;16395:45;16457:19;;5609:77:8;16071:411:11;5609:77:8;5699:8;;;;;;;5695:64;;5734:17;5727:24;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;5513:449;;;:::o;5695:64::-;5771:28;5802:10;:8;:10::i;:::-;5771:41;;5857:1;5832:14;5826:28;:32;:130;;;;;;;;;;;;;;;;;5894:14;5910:19;:8;:17;:19::i;:::-;5931:9;5877:64;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;5826:130;5819:137;5513:449;-1:-1:-1;;;5513:449:8:o;2303:1111::-;2424:1;2410:11;:15;:52;;;;;2444:18;;2429:11;:33;;2410:52;2402:85;;;;-1:-1:-1;;;2402:85:8;;;;;;;:::i;:::-;2533:9;;2518:11;2502:13;5498:1;6164:12:1;5955:7;6148:13;:28;-1:-1:-1;;6148:46:1;;5894:317;2502:13:8;:27;;;;:::i;:::-;:40;;2494:73;;;;-1:-1:-1;;;2494:73:8;;;;;;;:::i;:::-;2621:16;;2616:4;;:21;;;;:::i;:::-;2602:11;2595:4;;:18;;;;:::i;:::-;:42;;;;:::i;:::-;2582:9;:55;;2574:87;;;;-1:-1:-1;;;2574:87:8;;;;;;;:::i;:::-;2676:20;;;;;;;2668:67;;;;-1:-1:-1;;;2668:67:8;;18347:2:11;2668:67:8;;;18329:21:11;18386:2;18366:18;;;18359:30;18425:34;18405:18;;;18398:62;-1:-1:-1;;;18476:18:11;;;18469:32;18518:19;;2668:67:8;18145:398:11;2668:67:8;41487:10:1;2751:30:8;;;;:16;:30;;;;;;;;2750:31;2742:68;;;;-1:-1:-1;;;2742:68:8;;18750:2:11;2742:68:8;;;18732:21:11;18789:2;18769:18;;;18762:30;18828:26;18808:18;;;18801:54;18872:18;;2742:68:8;18548:348:11;2742:68:8;2842:30;;-1:-1:-1;;41487:10:1;19050:2:11;19046:15;19042:53;2842:30:8;;;19030:66:11;2817:12:8;;19112::11;;2842:30:8;;;;;;-1:-1:-1;;2842:30:8;;;;;;2832:41;;2842:30;2832:41;;;;;-1:-1:-1;41487:10:1;2902:9:8;2888:23;2880:65;;;;-1:-1:-1;;;2880:65:8;;14903:2:11;2880:65:8;;;14885:21:11;14942:2;14922:18;;;14915:30;14981:32;14961:18;;;14954:60;15031:18;;2880:65:8;14701:354:11;2880:65:8;2960:50;2979:12;;2960:50;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;2993:10:8;;;-1:-1:-1;3005:4:8;;-1:-1:-1;2960:18:8;:50::i;:::-;2952:77;;;;-1:-1:-1;;;2952:77:8;;19337:2:11;2952:77:8;;;19319:21:11;19376:2;19356:18;;;19349:30;-1:-1:-1;;;19395:18:11;;;19388:44;19449:18;;2952:77:8;19135:338:11;2952:77:8;41487:10:1;3044:26:8;;;;:12;:26;;;;;;3071:2;-1:-1:-1;3036:72:8;;;;-1:-1:-1;;;3036:72:8;;;;;;;:::i;:::-;41487:10:1;3123:26:8;;;;:12;:26;;;;;;3163:2;;3123:38;;3150:11;;3123:38;:::i;:::-;:42;;3115:85;;;;-1:-1:-1;;;3115:85:8;;;;;;;:::i;:::-;3226:16;;3207:15;;:35;;;;;;;:::i;:::-;;;;-1:-1:-1;;41487:10:1;3249:30:8;;;;:16;:30;;;;;;;;:37;;3282:4;-1:-1:-1;;3249:37:8;;;;;;;;3293:6;:20;;;;;:25;;;;;;;;;;3325:12;:26;;;;;:40;;3354:11;;3249:30;3325:40;;3354:11;;3325:40;:::i;:::-;;;;-1:-1:-1;3372:36:8;;-1:-1:-1;41487:10:1;3396:11:8;3372:9;:36::i;7275:114::-;1087:13:7;:11;:13::i;:::-;7339:15:8::1;::::0;-1:-1:-1;;;;;7339:15:8::1;:24;7364:7;1266:6:7::0;;-1:-1:-1;;;;;1266:6:7;;1194:85;7364:7:8::1;7339:42;::::0;-1:-1:-1;;;;;;7339:42:8::1;::::0;;;;;;-1:-1:-1;;;;;12909:32:11;;;7339:42:8::1;::::0;::::1;12891:51:11::0;12958:18;;;12951:34;;;12864:18;;7339:42:8::1;;;;;;;;;;;;;;;;;::::0;::::1;;;;;;;;;;;;::::0;::::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;5968:81::-:0;1087:13:7;:11;:13::i;:::-;6026:8:8::1;:17:::0;;;::::1;;::::0;::::1;-1:-1:-1::0;;6026:17:8;;::::1;::::0;;;::::1;::::0;;5968:81::o;6135:87::-;1087:13:7;:11;:13::i;:::-;6195:10:8::1;:21:::0;6135:87::o;5105:299::-;1087:13:7;:11;:13::i;:::-;5215:1:8::1;5201:11;:15;:52;;;;;5235:18;;5220:11;:33;;5201:52;5193:85;;;;-1:-1:-1::0;;;5193:85:8::1;;;;;;;:::i;:::-;5324:9;;5309:11;5293:13;5498:1:::0;6164:12:1;5955:7;6148:13;:28;-1:-1:-1;;6148:46:1;;5894:317;5293:13:8::1;:27;;;;:::i;:::-;:40;;5285:73;;;;-1:-1:-1::0;;;5285:73:8::1;;;;;;;:::i;:::-;5365:33;5375:9;5386:11;5365:9;:33::i;2074:198:7:-:0;1087:13;:11;:13::i;:::-;-1:-1:-1;;;;;2162:22:7;::::1;2154:73;;;::::0;-1:-1:-1;;;2154:73:7;;19680:2:11;2154:73:7::1;::::0;::::1;19662:21:11::0;19719:2;19699:18;;;19692:30;19758:34;19738:18;;;19731:62;-1:-1:-1;;;19809:18:11;;;19802:36;19855:19;;2154:73:7::1;19478:402:11::0;2154:73:7::1;2237:28;2256:8;2237:18;:28::i;18253:360:1:-:0;18318:11;18364:7;5498:1:8;18345:26:1;18341:266;;18401:13;;18391:7;:23;18387:210;;;18434:14;18466:60;-1:-1:-1;18483:26:1;;;;:17;:26;;;;;;18473:42;18466:60;;18517:9;;;:::i;:::-;;;18466:60;;;-1:-1:-1;;;18553:24:1;:29;;18253:360;-1:-1:-1;;18253:360:1:o;43371:160::-;43470:13;43464:4;43457:27;43510:4;43504;43497:18;35019:460;35143:13;35159:16;35167:7;35159;:16::i;:::-;35143:32;;35190:13;:45;;;;-1:-1:-1;41487:10:1;-1:-1:-1;;;;;35207:28:1;;;;35190:45;35186:198;;;35254:44;35271:5;41487:10;17842:162;:::i;35254:44::-;35249:135;;35318:51;-1:-1:-1;;;35318:7:1;:51::i;:::-;35394:24;;;;:15;:24;;;;;;:35;;-1:-1:-1;;;;;;35394:35:1;-1:-1:-1;;;;;35394:35:1;;;;;;;;;35444:28;;35394:24;;35444:28;;;;;;;35133:346;35019:460;;;:::o;1352:130:7:-;1266:6;;-1:-1:-1;;;;;1266:6:7;41487:10:1;1415:23:7;1407:68;;;;-1:-1:-1;;;1407:68:7;;20228:2:11;1407:68:7;;;20210:21:11;;;20247:18;;;20240:30;20306:34;20286:18;;;20279:62;20358:18;;1407:68:7;20026:356:11;12850:1978:1;12917:14;12966:7;5498:1:8;12947:26:1;12943:1822;;-1:-1:-1;12998:26:1;;;;:17;:26;;;;;;13122:11;13118:1270;;13168:13;;13157:7;:24;13153:77;;13183:47;-1:-1:-1;;;13183:7:1;:47::i;:::-;13777:597;-1:-1:-1;;;13871:9:1;13853:28;;;;:17;:28;;;;;;13929:11;13925:25;;13777:597;;13925:25;-1:-1:-1;;;13976:24:1;;13972:48;;12850:1978;;;:::o;13972:48::-;14308:47;-1:-1:-1;;;14308:7:1;:47::i;:::-;13777:597;;13118:1270;-1:-1:-1;;;14710:24:1;;14706:48;;12850:1978;;;:::o;14706:48::-;14774:47;-1:-1:-1;;;14774:7:1;:47::i;2336:287:9:-;1759:1;2468:7;;:19;;2460:63;;;;-1:-1:-1;;;2460:63:9;;20589:2:11;2460:63:9;;;20571:21:11;20628:2;20608:18;;;20601:30;20667:33;20647:18;;;20640:61;20718:18;;2460:63:9;20387:355:11;2460:63:9;1759:1;2598:7;:18;2336:287::o;2426:187:7:-;2518:6;;;-1:-1:-1;;;;;2534:17:7;;;-1:-1:-1;;;;;;2534:17:7;;;;;;;2566:40;;2518:6;;;2534:17;2518:6;;2566:40;;2499:16;;2566:40;2489:124;2426:187;:::o;4525:4263:2:-;4647:16;4712:4;4703:5;:13;4699:54;;4718:35;-1:-1:-1;;;4718:7:2;:35::i;:::-;5498:1:8;4829:5:2;:23;4825:85;;;5498:1:8;4872:23:2;;4825:85;4923:17;5671:13:1;5025:17:2;;;5021:72;;5069:9;5062:16;;5021:72;5106:25;5145;5173:16;5183:5;5173:9;:16::i;:::-;5222:12;;;5379:35;;;;-1:-1:-1;5445:22:2;;5441:3302;;5664:17;5655:5;5648:4;:12;:33;5644:112;;5732:5;5725:4;:12;5705:32;;5644:112;5875:4;5869:11;5857:23;;6125:1;6106:17;6102:25;6099:1;6095:33;6085:8;6081:48;6075:4;6068:62;6301:31;6335:26;6355:5;6335:19;:26::i;:::-;6301:60;;6379:25;6671:9;:16;;;6666:98;;-1:-1:-1;6731:14:2;;6666:98;6781:19;6968:1616;7005:19;7018:5;7005:12;:19::i;:::-;6993:31;;7109:4;7098:9;7094:20;7088:27;7204:1;7199:893;;;;8408:1;8387:22;;7081:1354;;7199:893;7478:9;7472:16;7469:121;;;7550:9;7544:16;7523:37;;7469:121;7877:5;7858:17;7854:29;7850:2;7846:38;7836:230;;7952:1;7939:11;7935:19;7920:34;;8030:5;8015:11;8012:1;8008:19;7998:8;7994:34;7987:49;7836:230;7081:1354;8480:1;8473:5;8469:13;8460:22;;8541:4;8532:5;:13;:49;;;;8564:17;8549:11;:32;8532:49;8530:52;6968:1616;;8682:29;;-1:-1:-1;;5441:3302:2;-1:-1:-1;8763:8:2;;4525:4263;-1:-1:-1;;;;;;4525:4263:2:o;34129:110:1:-;34205:27;34215:2;34219:8;34205:27;;;;;;;;;;;;:9;:27::i;27283:673::-;27461:88;;-1:-1:-1;;;27461:88:1;;27441:4;;-1:-1:-1;;;;;27461:45:1;;;;;:88;;41487:10;;27528:4;;27534:7;;27543:5;;27461:88;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;27461:88:1;;;;;;;;-1:-1:-1;;27461:88:1;;;;;;;;;;;;:::i;:::-;;;27457:493;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;27739:13:1;;27735:113;;27777:56;-1:-1:-1;;;27777:7:1;:56::i;:::-;27918:6;27912:13;27903:6;27899:2;27895:15;27888:38;27457:493;-1:-1:-1;;;;;;27617:64:1;-1:-1:-1;;;27617:64:1;;-1:-1:-1;27283:673:1;;;;;;:::o;11997:159::-;-1:-1:-1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;12124:24:1;;;;:17;:24;;;;;;12105:44;;-1:-1:-1;;;;;;;;;;;;;15031:41:1;;;;2004:3;15116:33;;;15082:68;;-1:-1:-1;;;15082:68:1;-1:-1:-1;;;15179:24:1;;:29;;-1:-1:-1;;;15160:48:1;;;;2513:3;15247:28;;;;-1:-1:-1;;;15218:58:1;-1:-1:-1;14922:361:1;7395:104:8;7455:13;7484:9;7477:16;;;;;:::i;410:696:10:-;466:13;515:14;532:17;543:5;532:10;:17::i;:::-;552:1;532:21;515:38;;567:20;601:6;590:18;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;590:18:10;-1:-1:-1;567:41:10;-1:-1:-1;728:28:10;;;744:2;728:28;783:280;-1:-1:-1;;814:5:10;-1:-1:-1;;;948:2:10;937:14;;932:30;814:5;919:44;1007:2;998:11;;;-1:-1:-1;1031:10:10;1027:21;;1043:5;;1027:21;783:280;;1156:184:6;1277:4;1329;1300:25;1313:5;1320:4;1300:12;:25::i;:::-;:33;;1156:184;-1:-1:-1;;;;1156:184:6:o;33362:688:1:-;33488:19;33494:2;33498:8;33488:5;:19::i;:::-;-1:-1:-1;;;;;33546:14:1;;;:19;33542:492;;33585:11;33599:13;33646:14;;;33678:238;33708:62;33747:1;33751:2;33755:7;;;;;;33764:5;33708:30;:62::i;:::-;33703:174;;33798:56;-1:-1:-1;;;33798:7:1;:56::i;:::-;33911:3;33903:5;:11;33678:238;;33996:3;33979:13;;:20;33975:44;;34001:18;34016:1;34001:7;:18::i;9889:890:5:-;9942:7;;-1:-1:-1;;;10017:15:5;;10013:99;;-1:-1:-1;;;10052:15:5;;;-1:-1:-1;10095:2:5;10085:12;10013:99;10138:6;10129:5;:15;10125:99;;10173:6;10164:15;;;-1:-1:-1;10207:2:5;10197:12;10125:99;10250:6;10241:5;:15;10237:99;;10285:6;10276:15;;;-1:-1:-1;10319:2:5;10309:12;10237:99;10362:5;10353;:14;10349:96;;10396:5;10387:14;;;-1:-1:-1;10429:1:5;10419:11;10349:96;10471:5;10462;:14;10458:96;;10505:5;10496:14;;;-1:-1:-1;10538:1:5;10528:11;10458:96;10580:5;10571;:14;10567:96;;10614:5;10605:14;;;-1:-1:-1;10647:1:5;10637:11;10567:96;10689:5;10680;:14;10676:64;;10724:1;10714:11;10766:6;9889:890;-1:-1:-1;;9889:890:5:o;1994:290:6:-;2077:7;2119:4;2077:7;2133:116;2157:5;:12;2153:1;:16;2133:116;;;2205:33;2215:12;2229:5;2235:1;2229:8;;;;;;;;:::i;:::-;;;;;;;2205:9;:33::i;:::-;2190:48;-1:-1:-1;2171:3:6;;;;:::i;:::-;;;;2133:116;;28402:2251:1;28474:20;28497:13;28524;28520:53;;28539:34;-1:-1:-1;;;28539:7:1;:34::i;:::-;29073:31;;;;:17;:31;;;;;;;;-1:-1:-1;;;;;15595:28:1;;15767:11;15742:23;15738:41;16200:1;16187:15;;16161:24;16157:46;15735:52;15725:63;;29073:170;;;29454:22;;;:18;:22;;;;;;:71;;29492:32;29480:45;;29454:71;;;15595:28;29706:54;;29725:35;-1:-1:-1;;;29725:7:1;:35::i;:::-;29789:23;;;:12;29871:662;30281:7;30238:8;30194:1;30129:25;30067:1;30003;29973:351;30515:9;;:16;;;;29871:662;;-1:-1:-1;30547:13:1;:19;-1:-1:-1;24084:187:1;;;:::o;8879:147:6:-;8942:7;8972:1;8968;:5;:51;;9100:13;9191:15;;;9226:4;9219:15;;;9272:4;9256:21;;8968:51;;;-1:-1:-1;9100:13:6;9191:15;;;9226:4;9219:15;9272:4;9256:21;;;8879:147::o;-1:-1:-1:-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;:::o;:::-;;;;;;;;;;;;;;;14:131:11;-1:-1:-1;;;;;;88:32:11;;78:43;;68:71;;135:1;132;125:12;150:245;208:6;261:2;249:9;240:7;236:23;232:32;229:52;;;277:1;274;267:12;229:52;316:9;303:23;335:30;359:5;335:30;:::i;592:258::-;664:1;674:113;688:6;685:1;682:13;674:113;;;764:11;;;758:18;745:11;;;738:39;710:2;703:10;674:113;;;805:6;802:1;799:13;796:48;;;-1:-1:-1;;840:1:11;822:16;;815:27;592:258::o;855:::-;897:3;935:5;929:12;962:6;957:3;950:19;978:63;1034:6;1027:4;1022:3;1018:14;1011:4;1004:5;1000:16;978:63;:::i;:::-;1095:2;1074:15;-1:-1:-1;;1070:29:11;1061:39;;;;1102:4;1057:50;;855:258;-1:-1:-1;;855:258:11:o;1118:220::-;1267:2;1256:9;1249:21;1230:4;1287:45;1328:2;1317:9;1313:18;1305:6;1287:45;:::i;1343:180::-;1402:6;1455:2;1443:9;1434:7;1430:23;1426:32;1423:52;;;1471:1;1468;1461:12;1423:52;-1:-1:-1;1494:23:11;;1343:180;-1:-1:-1;1343:180:11:o;1736:173::-;1804:20;;-1:-1:-1;;;;;1853:31:11;;1843:42;;1833:70;;1899:1;1896;1889:12;1914:254;1982:6;1990;2043:2;2031:9;2022:7;2018:23;2014:32;2011:52;;;2059:1;2056;2049:12;2011:52;2082:29;2101:9;2082:29;:::i;:::-;2072:39;2158:2;2143:18;;;;2130:32;;-1:-1:-1;;;1914:254:11:o;2355:127::-;2416:10;2411:3;2407:20;2404:1;2397:31;2447:4;2444:1;2437:15;2471:4;2468:1;2461:15;2487:275;2558:2;2552:9;2623:2;2604:13;;-1:-1:-1;;2600:27:11;2588:40;;2658:18;2643:34;;2679:22;;;2640:62;2637:88;;;2705:18;;:::i;:::-;2741:2;2734:22;2487:275;;-1:-1:-1;2487:275:11:o;2767:407::-;2832:5;2866:18;2858:6;2855:30;2852:56;;;2888:18;;:::i;:::-;2926:57;2971:2;2950:15;;-1:-1:-1;;2946:29:11;2977:4;2942:40;2926:57;:::i;:::-;2917:66;;3006:6;2999:5;2992:21;3046:3;3037:6;3032:3;3028:16;3025:25;3022:45;;;3063:1;3060;3053:12;3022:45;3112:6;3107:3;3100:4;3093:5;3089:16;3076:43;3166:1;3159:4;3150:6;3143:5;3139:18;3135:29;3128:40;2767:407;;;;;:::o;3179:451::-;3248:6;3301:2;3289:9;3280:7;3276:23;3272:32;3269:52;;;3317:1;3314;3307:12;3269:52;3357:9;3344:23;3390:18;3382:6;3379:30;3376:50;;;3422:1;3419;3412:12;3376:50;3445:22;;3498:4;3490:13;;3486:27;-1:-1:-1;3476:55:11;;3527:1;3524;3517:12;3476:55;3550:74;3616:7;3611:2;3598:16;3593:2;3589;3585:11;3550:74;:::i;3635:118::-;3721:5;3714:13;3707:21;3700:5;3697:32;3687:60;;3743:1;3740;3733:12;3758:241;3814:6;3867:2;3855:9;3846:7;3842:23;3838:32;3835:52;;;3883:1;3880;3873:12;3835:52;3922:9;3909:23;3941:28;3963:5;3941:28;:::i;4004:328::-;4081:6;4089;4097;4150:2;4138:9;4129:7;4125:23;4121:32;4118:52;;;4166:1;4163;4156:12;4118:52;4189:29;4208:9;4189:29;:::i;:::-;4179:39;;4237:38;4271:2;4260:9;4256:18;4237:38;:::i;:::-;4227:48;;4322:2;4311:9;4307:18;4294:32;4284:42;;4004:328;;;;;:::o;4742:186::-;4801:6;4854:2;4842:9;4833:7;4829:23;4825:32;4822:52;;;4870:1;4867;4860:12;4822:52;4893:29;4912:9;4893:29;:::i;4933:367::-;4996:8;5006:6;5060:3;5053:4;5045:6;5041:17;5037:27;5027:55;;5078:1;5075;5068:12;5027:55;-1:-1:-1;5101:20:11;;5144:18;5133:30;;5130:50;;;5176:1;5173;5166:12;5130:50;5213:4;5205:6;5201:17;5189:29;;5273:3;5266:4;5256:6;5253:1;5249:14;5241:6;5237:27;5233:38;5230:47;5227:67;;;5290:1;5287;5280:12;5227:67;4933:367;;;;;:::o;5305:437::-;5391:6;5399;5452:2;5440:9;5431:7;5427:23;5423:32;5420:52;;;5468:1;5465;5458:12;5420:52;5508:9;5495:23;5541:18;5533:6;5530:30;5527:50;;;5573:1;5570;5563:12;5527:50;5612:70;5674:7;5665:6;5654:9;5650:22;5612:70;:::i;:::-;5701:8;;5586:96;;-1:-1:-1;5305:437:11;-1:-1:-1;;;;5305:437:11:o;5747:349::-;5831:12;;-1:-1:-1;;;;;5827:38:11;5815:51;;5919:4;5908:16;;;5902:23;5927:18;5898:48;5882:14;;;5875:72;6010:4;5999:16;;;5993:23;5986:31;5979:39;5963:14;;;5956:63;6072:4;6061:16;;;6055:23;6080:8;6051:38;6035:14;;6028:62;5747:349::o;6101:724::-;6336:2;6388:21;;;6458:13;;6361:18;;;6480:22;;;6307:4;;6336:2;6559:15;;;;6533:2;6518:18;;;6307:4;6602:197;6616:6;6613:1;6610:13;6602:197;;;6665:52;6713:3;6704:6;6698:13;6665:52;:::i;:::-;6774:15;;;;6746:4;6737:14;;;;;6638:1;6631:9;6602:197;;6830:946;6914:6;6945:2;6988;6976:9;6967:7;6963:23;6959:32;6956:52;;;7004:1;7001;6994:12;6956:52;7044:9;7031:23;7073:18;7114:2;7106:6;7103:14;7100:34;;;7130:1;7127;7120:12;7100:34;7168:6;7157:9;7153:22;7143:32;;7213:7;7206:4;7202:2;7198:13;7194:27;7184:55;;7235:1;7232;7225:12;7184:55;7271:2;7258:16;7293:2;7289;7286:10;7283:36;;;7299:18;;:::i;:::-;7345:2;7342:1;7338:10;7328:20;;7368:28;7392:2;7388;7384:11;7368:28;:::i;:::-;7430:15;;;7500:11;;;7496:20;;;7461:12;;;;7528:19;;;7525:39;;;7560:1;7557;7550:12;7525:39;7584:11;;;;7604:142;7620:6;7615:3;7612:15;7604:142;;;7686:17;;7674:30;;7637:12;;;;7724;;;;7604:142;;;7765:5;6830:946;-1:-1:-1;;;;;;;;6830:946:11:o;7966:632::-;8137:2;8189:21;;;8259:13;;8162:18;;;8281:22;;;8108:4;;8137:2;8360:15;;;;8334:2;8319:18;;;8108:4;8403:169;8417:6;8414:1;8411:13;8403:169;;;8478:13;;8466:26;;8547:15;;;;8512:12;;;;8439:1;8432:9;8403:169;;8603:322;8680:6;8688;8696;8749:2;8737:9;8728:7;8724:23;8720:32;8717:52;;;8765:1;8762;8755:12;8717:52;8788:29;8807:9;8788:29;:::i;:::-;8778:39;8864:2;8849:18;;8836:32;;-1:-1:-1;8915:2:11;8900:18;;;8887:32;;8603:322;-1:-1:-1;;;8603:322:11:o;8930:315::-;8995:6;9003;9056:2;9044:9;9035:7;9031:23;9027:32;9024:52;;;9072:1;9069;9062:12;9024:52;9095:29;9114:9;9095:29;:::i;:::-;9085:39;;9174:2;9163:9;9159:18;9146:32;9187:28;9209:5;9187:28;:::i;:::-;9234:5;9224:15;;;8930:315;;;;;:::o;9250:667::-;9345:6;9353;9361;9369;9422:3;9410:9;9401:7;9397:23;9393:33;9390:53;;;9439:1;9436;9429:12;9390:53;9462:29;9481:9;9462:29;:::i;:::-;9452:39;;9510:38;9544:2;9533:9;9529:18;9510:38;:::i;:::-;9500:48;;9595:2;9584:9;9580:18;9567:32;9557:42;;9650:2;9639:9;9635:18;9622:32;9677:18;9669:6;9666:30;9663:50;;;9709:1;9706;9699:12;9663:50;9732:22;;9785:4;9777:13;;9773:27;-1:-1:-1;9763:55:11;;9814:1;9811;9804:12;9763:55;9837:74;9903:7;9898:2;9885:16;9880:2;9876;9872:11;9837:74;:::i;:::-;9827:84;;;9250:667;;;;;;;:::o;9922:268::-;10120:3;10105:19;;10133:51;10109:9;10166:6;10133:51;:::i;10195:505::-;10290:6;10298;10306;10359:2;10347:9;10338:7;10334:23;10330:32;10327:52;;;10375:1;10372;10365:12;10327:52;10411:9;10398:23;10388:33;;10472:2;10461:9;10457:18;10444:32;10499:18;10491:6;10488:30;10485:50;;;10531:1;10528;10521:12;10485:50;10570:70;10632:7;10623:6;10612:9;10608:22;10570:70;:::i;:::-;10195:505;;10659:8;;-1:-1:-1;10544:96:11;;-1:-1:-1;;;;10195:505:11:o;10705:260::-;10773:6;10781;10834:2;10822:9;10813:7;10809:23;10805:32;10802:52;;;10850:1;10847;10840:12;10802:52;10873:29;10892:9;10873:29;:::i;:::-;10863:39;;10921:38;10955:2;10944:9;10940:18;10921:38;:::i;:::-;10911:48;;10705:260;;;;;:::o;10970:254::-;11038:6;11046;11099:2;11087:9;11078:7;11074:23;11070:32;11067:52;;;11115:1;11112;11105:12;11067:52;11151:9;11138:23;11128:33;;11180:38;11214:2;11203:9;11199:18;11180:38;:::i;11229:380::-;11308:1;11304:12;;;;11351;;;11372:61;;11426:4;11418:6;11414:17;11404:27;;11372:61;11479:2;11471:6;11468:14;11448:18;11445:38;11442:161;;;11525:10;11520:3;11516:20;11513:1;11506:31;11560:4;11557:1;11550:15;11588:4;11585:1;11578:15;11442:161;;11229:380;;;:::o;12232:127::-;12293:10;12288:3;12284:20;12281:1;12274:31;12324:4;12321:1;12314:15;12348:4;12345:1;12338:15;12996:245;13063:6;13116:2;13104:9;13095:7;13091:23;13087:32;13084:52;;;13132:1;13129;13122:12;13084:52;13164:9;13158:16;13183:28;13205:5;13183:28;:::i;13246:127::-;13307:10;13302:3;13298:20;13295:1;13288:31;13338:4;13335:1;13328:15;13362:4;13359:1;13352:15;13378:135;13417:3;-1:-1:-1;;13438:17:11;;13435:43;;;13458:18;;:::i;:::-;-1:-1:-1;13505:1:11;13494:13;;13378:135::o;13518:344::-;13720:2;13702:21;;;13759:2;13739:18;;;13732:30;-1:-1:-1;;;13793:2:11;13778:18;;13771:50;13853:2;13838:18;;13518:344::o;13867:128::-;13907:3;13938:1;13934:6;13931:1;13928:13;13925:39;;;13944:18;;:::i;:::-;-1:-1:-1;13980:9:11;;13867:128::o;14000:344::-;14202:2;14184:21;;;14241:2;14221:18;;;14214:30;-1:-1:-1;;;14275:2:11;14260:18;;14253:50;14335:2;14320:18;;14000:344::o;15060:355::-;15262:2;15244:21;;;15301:2;15281:18;;;15274:30;15340:33;15335:2;15320:18;;15313:61;15406:2;15391:18;;15060:355::o;15420:168::-;15460:7;15526:1;15522;15518:6;15514:14;15511:1;15508:21;15503:1;15496:9;15489:17;15485:45;15482:71;;;15533:18;;:::i;:::-;-1:-1:-1;15573:9:11;;15420:168::o;15593:125::-;15633:4;15661:1;15658;15655:8;15652:34;;;15666:18;;:::i;:::-;-1:-1:-1;15703:9:11;;15593:125::o;15723:343::-;15925:2;15907:21;;;15964:2;15944:18;;;15937:30;-1:-1:-1;;;15998:2:11;15983:18;;15976:49;16057:2;16042:18;;15723:343::o;16613:1527::-;16837:3;16875:6;16869:13;16901:4;16914:51;16958:6;16953:3;16948:2;16940:6;16936:15;16914:51;:::i;:::-;17028:13;;16987:16;;;;17050:55;17028:13;16987:16;17072:15;;;17050:55;:::i;:::-;17194:13;;17127:20;;;17167:1;;17254;17276:18;;;;17329;;;;17356:93;;17434:4;17424:8;17420:19;17408:31;;17356:93;17497:2;17487:8;17484:16;17464:18;17461:40;17458:167;;;-1:-1:-1;;;17524:33:11;;17580:4;17577:1;17570:15;17610:4;17531:3;17598:17;17458:167;17641:18;17668:110;;;;17792:1;17787:328;;;;17634:481;;17668:110;-1:-1:-1;;17703:24:11;;17689:39;;17748:20;;;;-1:-1:-1;17668:110:11;;17787:328;16560:1;16553:14;;;16597:4;16584:18;;17882:1;17896:169;17910:8;17907:1;17904:15;17896:169;;;17992:14;;17977:13;;;17970:37;18035:16;;;;17927:10;;17896:169;;;17900:3;;18096:8;18089:5;18085:20;18078:27;;17634:481;-1:-1:-1;18131:3:11;;16613:1527;-1:-1:-1;;;;;;;;;;;16613:1527:11:o;19885:136::-;19924:3;19952:5;19942:39;;19961:18;;:::i;:::-;-1:-1:-1;;;19997:18:11;;19885:136::o;20747:489::-;-1:-1:-1;;;;;21016:15:11;;;20998:34;;21068:15;;21063:2;21048:18;;21041:43;21115:2;21100:18;;21093:34;;;21163:3;21158:2;21143:18;;21136:31;;;20941:4;;21184:46;;21210:19;;21202:6;21184:46;:::i;:::-;21176:54;20747:489;-1:-1:-1;;;;;;20747:489:11:o;21241:249::-;21310:6;21363:2;21351:9;21342:7;21338:23;21334:32;21331:52;;;21379:1;21376;21369:12;21331:52;21411:9;21405:16;21430:30;21454:5;21430:30;:::i

Swarm Source

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