ETH Price: $3,436.32 (-0.63%)
Gas: 20 Gwei

Token

DuckyCity Island (ISLAND)
 

Overview

Max Total Supply

5,000 ISLAND

Holders

1,063

Market

Volume (24H)

N/A

Min Price (24H)

N/A

Max Price (24H)

N/A
Balance
1 ISLAND
0xbed0cbab8c917fefdafb1a9060737f82ce1f1511
Loading...
Loading
Loading...
Loading
Loading...
Loading

OVERVIEW

DuckyCity - Island is a player-owned house and farm in the metaverse. 5,000 unique islands: own fishing lakes, farms, forests, mines... for a lifetime

# Exchange Pair Price  24H Volume % Volume

Contract Source Code Verified (Exact Match)

Contract Name:
DuckyCityIsland

Compiler Version
v0.8.9+commit.e5eed63a

Optimization Enabled:
Yes with 200 runs

Other Settings:
byzantium EvmVersion, None license

Contract Source Code (Solidity Multiple files format)

File 3 of 17: DuckyCityIsland.sol
// SPDX-License-Identifier: AGPL-3.0

pragma solidity ^0.8.9;

import "./Ownable.sol";
import "./PaymentSplitter.sol";
import "./Pausable.sol";
import "./MerkleProof.sol";
import "./ERC721A.sol";

contract DuckyCityIsland is ERC721A, Ownable, Pausable, PaymentSplitter {
  string public _baseTokenURI;

  bytes32 public _merkleRoot;

  uint256 public _price;
  uint256 public _presalePrice;
  uint256 public _maxSupply;
  uint256 public _maxPerAddress;
  uint256 public _presaleMaxPerAddress;
  uint256 public _publicSaleTime;
  uint256 public _preSaleTime;
  uint256 public _maxTxPerAddress;
  mapping(address => uint256) public _purchases;
  mapping(address => uint256) public _presaleMaxPerAddressMap;

  event EarlyPurchase(address indexed addr, uint256 indexed atPrice, uint256 indexed count);
  event Purchase(address indexed addr, uint256 indexed atPrice, uint256 indexed count);

  constructor(
    string memory name,
    string memory symbol,
    string memory baseTokenURI,
    uint256[] memory numericValues,
    bytes32 merkleRoot,
    address[] memory payees,
    uint256[] memory shares
  ) ERC721A(name, symbol, numericValues[2]) PaymentSplitter(payees, shares) {
    _baseTokenURI = baseTokenURI;

    _price = numericValues[0];
    _presalePrice = numericValues[1];
    _maxSupply = numericValues[2];
    _maxPerAddress = numericValues[3];
    _presaleMaxPerAddress = numericValues[4];
    _publicSaleTime = numericValues[5];
    _preSaleTime = numericValues[6];
    _maxTxPerAddress = numericValues[7];

    _merkleRoot = merkleRoot;
  }

  function setPresaleMaxPerAddress(
    address[] memory whitelist,
    uint256[] memory maxPerAddress
  ) external onlyOwner {
    require(whitelist.length == maxPerAddress.length, "whitelist and maxPerAddress length mismatch");
    require(whitelist.length > 0, "No whitelist");

    for (uint256 i = 0; i < whitelist.length; i++) {
      _presaleMaxPerAddressMap[whitelist[i]] = maxPerAddress[i];
    }
  }

  function setSaleInformation(
    uint256 publicSaleTime,
    uint256 preSaleTime,
    uint256 maxPerAddress,
    uint256 presaleMaxPerAddress,
    uint256 price,
    uint256 presalePrice,
    bytes32 merkleRoot,
    uint256 maxTxPerAddress
  ) external onlyOwner {
    _publicSaleTime = publicSaleTime;
    _preSaleTime = preSaleTime;
    _maxPerAddress = maxPerAddress;
    _presaleMaxPerAddress = presaleMaxPerAddress;
    _price = price;
    _presalePrice = presalePrice;
    _merkleRoot = merkleRoot;
    _maxTxPerAddress = maxTxPerAddress;
  }

  function setBaseUri(
    string memory baseUri
  ) external onlyOwner {
    _baseTokenURI = baseUri;
  }

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

  function _baseURI() override internal view virtual returns (string memory) {
    return string(
      abi.encodePacked(
        _baseTokenURI,
        Strings.toHexString(uint256(uint160(address(this))), 20),
        '/'
      )
    );
  }

  function mint(address to, uint256 count) external payable onlyOwner {
    ensureMintConditions(count);

    _safeMint(to, count);
  }

  function purchase(uint256 count) external payable whenNotPaused {
    ensurePublicMintConditions(msg.sender, count, _maxPerAddress);
    require(isPublicSaleActive(), "BASE_COLLECTION/CANNOT_MINT");

    _purchase(count, _price);
    emit Purchase(msg.sender, _price, count);
  }

  function earlyPurchase(uint256 count, bytes32[] calldata merkleProof) external payable whenNotPaused {
    ensurePublicMintConditions(msg.sender, count, _presaleMaxPerAddressMap[msg.sender]);
    require(isPreSaleActive() && onEarlyPurchaseList(msg.sender, merkleProof), "BASE_COLLECTION/CANNOT_MINT_PRESALE");

    _purchase(count, _presalePrice);
    emit EarlyPurchase(msg.sender, _presalePrice, count);
  }

  function _purchase(uint256 count, uint256 price) private {
    require(price * count <= msg.value, 'BASE_COLLECTION/INSUFFICIENT_ETH_AMOUNT');

    _purchases[msg.sender] += count;
    _safeMint(msg.sender, count);
  }

  function ensureMintConditions(uint256 count) internal view {
    require(totalSupply() + count <= _maxSupply, "BASE_COLLECTION/EXCEEDS_MAX_SUPPLY");
  }

  function ensurePublicMintConditions(address to, uint256 count, uint256 maxPerAddress) internal view {
    ensureMintConditions(count);

    require((_maxTxPerAddress != 0) && (count <= _maxTxPerAddress), "BASE_COLLECTION/EXCEEDS_MAX_PER_TRANSACTION");
    uint256 totalMintFromAddress = _purchases[to] + count;
    require ((maxPerAddress != 0) && (totalMintFromAddress <= maxPerAddress), "BASE_COLLECTION/EXCEEDS_INDIVIDUAL_SUPPLY");
  }

  function isPublicSaleActive() public view returns (bool) {
    return (_publicSaleTime != 0 && _publicSaleTime < block.timestamp);
  }

  function isPreSaleActive() public view returns (bool) {
    return (_preSaleTime != 0 && (_preSaleTime < block.timestamp) && (block.timestamp < _publicSaleTime));
  }

  function onEarlyPurchaseList(address addr, bytes32[] calldata merkleProof) public view returns (bool) {
    require(_merkleRoot.length > 0, "BASE_COLLECTION/PRESALE_MINT_LIST_UNSET");

    bytes32 node = keccak256(abi.encodePacked(addr));
    return MerkleProof.verify(merkleProof, _merkleRoot, node);
  }

  function MAX_TOTAL_MINT() public view returns (uint256) {
    return _maxSupply;
  }

  function PRICE() public view returns (uint256) {
    if (isPreSaleActive()) {
      return _presalePrice;
    }

    return _price;
  }

  function MAX_TOTAL_MINT_PER_ADDRESS() public view returns (uint256) {
    if (isPreSaleActive()) {
      return _presaleMaxPerAddress;
    }

    return _maxPerAddress;
  }

  function pause() external onlyOwner {
    _pause();
  }

  function unpause() external onlyOwner {
    _unpause();
  }
}

File 1 of 17: Address.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (utils/Address.sol)

pragma solidity ^0.8.0;

/**
 * @dev Collection of functions related to the address type
 */
library Address {
    /**
     * @dev Returns true if `account` is a contract.
     *
     * [IMPORTANT]
     * ====
     * It is unsafe to assume that an address for which this function returns
     * false is an externally-owned account (EOA) and not a contract.
     *
     * Among others, `isContract` will return false for the following
     * types of addresses:
     *
     *  - an externally-owned account
     *  - a contract in construction
     *  - an address where a contract will be created
     *  - an address where a contract lived, but was destroyed
     * ====
     */
    function isContract(address account) internal view returns (bool) {
        // This method relies on extcodesize, which returns 0 for contracts in
        // construction, since the code is only stored at the end of the
        // constructor execution.

        uint256 size;
        assembly {
            size := extcodesize(account)
        }
        return size > 0;
    }

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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

File 2 of 17: 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 4 of 17: ERC165.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (utils/introspection/ERC165.sol)

pragma solidity ^0.8.0;

import "./IERC165.sol";

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

File 5 of 17: ERC721A.sol
// SPDX-License-Identifier: MIT
// Creators: locationtba.eth, 2pmflow.eth

pragma solidity ^0.8.0;

import "./IERC721.sol";
import "./IERC721Receiver.sol";
import "./IERC721Metadata.sol";
import "./IERC721Enumerable.sol";
import "./Address.sol";
import "./Context.sol";
import "./Strings.sol";
import "./ERC165.sol";

/**
 * @dev Implementation of https://eips.ethereum.org/EIPS/eip-721[ERC721] Non-Fungible Token Standard, including
 * the Metadata and Enumerable extension. Built to optimize for lower gas during batch mints.
 *
 * Assumes serials are sequentially minted starting at 0 (e.g. 0, 1, 2, 3..).
 *
 * Does not support burning tokens to address(0).
 */
contract ERC721A is
  Context,
  ERC165,
  IERC721,
  IERC721Metadata,
  IERC721Enumerable
{
  using Address for address;
  using Strings for uint256;

  struct TokenOwnership {
    address addr;
    uint64 startTimestamp;
  }

  struct AddressData {
    uint128 balance;
    uint128 numberMinted;
  }

  uint256 private currentIndex = 1;

  uint256 internal immutable maxBatchSize;

  // Token name
  string private _name;

  // Token symbol
  string private _symbol;

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

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

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

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

  /**
   * @dev
   * `maxBatchSize` refers to how much a minter can mint at a time.
   */
  constructor(
    string memory name_,
    string memory symbol_,
    uint256 maxBatchSize_
  ) {
    require(maxBatchSize_ > 0, "ERC721A: max batch size must be nonzero");
    _name = name_;
    _symbol = symbol_;
    maxBatchSize = maxBatchSize_;
  }

  /**
   * @dev See {IERC721Enumerable-totalSupply}.
   */
  function totalSupply() public view override returns (uint256) {
    return currentIndex - 1;
  }

  /**
   * @dev See {IERC721Enumerable-tokenByIndex}.
   */
  function tokenByIndex(uint256 index) public view override returns (uint256) {
    require(index < totalSupply(), "ERC721A: global index out of bounds");
    return index;
  }

  /**
   * @dev See {IERC721Enumerable-tokenOfOwnerByIndex}.
   * This read function is O(totalSupply). If calling from a separate contract, be sure to test gas first.
   * It may also degrade with extremely large collection sizes (e.g >> 10000), test for your use case.
   */
  function tokenOfOwnerByIndex(address owner, uint256 index)
    public
    view
    override
    returns (uint256)
  {
    require(index < balanceOf(owner), "ERC721A: owner index out of bounds");
    uint256 numMintedSoFar = totalSupply();
    uint256 tokenIdsIdx = 0;
    address currOwnershipAddr = address(0);
    for (uint256 i = 0; i < numMintedSoFar; i++) {
      TokenOwnership memory ownership = _ownerships[i];
      if (ownership.addr != address(0)) {
        currOwnershipAddr = ownership.addr;
      }
      if (currOwnershipAddr == owner) {
        if (tokenIdsIdx == index) {
          return i;
        }
        tokenIdsIdx++;
      }
    }
    revert("ERC721A: unable to get token of owner by index");
  }

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

  /**
   * @dev See {IERC721-balanceOf}.
   */
  function balanceOf(address owner) public view override returns (uint256) {
    require(owner != address(0), "ERC721A: balance query for the zero address");
    return uint256(_addressData[owner].balance);
  }

  function _numberMinted(address owner) internal view returns (uint256) {
    require(
      owner != address(0),
      "ERC721A: number minted query for the zero address"
    );
    return uint256(_addressData[owner].numberMinted);
  }

  function ownershipOf(uint256 tokenId)
    internal
    view
    returns (TokenOwnership memory)
  {
    require(_exists(tokenId), "ERC721A: owner query for nonexistent token");

    uint256 lowestTokenToCheck;
    if (tokenId >= maxBatchSize) {
      lowestTokenToCheck = tokenId - maxBatchSize + 1;
    }

    for (uint256 curr = tokenId; curr >= lowestTokenToCheck; curr--) {
      TokenOwnership memory ownership = _ownerships[curr];
      if (ownership.addr != address(0)) {
        return ownership;
      }
    }

    revert("ERC721A: unable to determine the owner of token");
  }

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

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

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

  /**
   * @dev See {IERC721Metadata-tokenURI}.
   */
  function tokenURI(uint256 tokenId)
    public
    view
    virtual
    override
    returns (string memory)
  {
    require(
      _exists(tokenId),
      "ERC721Metadata: URI query for nonexistent token"
    );

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

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

  /**
   * @dev See {IERC721-approve}.
   */
  function approve(address to, uint256 tokenId) public override {
    address owner = ERC721A.ownerOf(tokenId);
    require(to != owner, "ERC721A: approval to current owner");

    require(
      _msgSender() == owner || isApprovedForAll(owner, _msgSender()),
      "ERC721A: approve caller is not owner nor approved for all"
    );

    _approve(to, tokenId, owner);
  }

  /**
   * @dev See {IERC721-getApproved}.
   */
  function getApproved(uint256 tokenId) public view override returns (address) {
    require(_exists(tokenId), "ERC721A: approved query for nonexistent token");

    return _tokenApprovals[tokenId];
  }

  /**
   * @dev See {IERC721-setApprovalForAll}.
   */
  function setApprovalForAll(address operator, bool approved) public override {
    require(operator != _msgSender(), "ERC721A: approve to caller");

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

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

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

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

  /**
   * @dev See {IERC721-safeTransferFrom}.
   */
  function safeTransferFrom(
    address from,
    address to,
    uint256 tokenId,
    bytes memory _data
  ) public override {
    _transfer(from, to, tokenId);
    require(
      _checkOnERC721Received(from, to, tokenId, _data),
      "ERC721A: transfer to non ERC721Receiver implementer"
    );
  }

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

  function _safeMint(address to, uint256 quantity) internal {
    _safeMint(to, quantity, "");
  }

  /**
   * @dev Mints `quantity` tokens and transfers them to `to`.
   *
   * Requirements:
   *
   * - `to` cannot be the zero address.
   * - `quantity` cannot be larger than the max batch size.
   *
   * Emits a {Transfer} event.
   */
  function _safeMint(
    address to,
    uint256 quantity,
    bytes memory _data
  ) internal {
    uint256 startTokenId = currentIndex;
    require(to != address(0), "ERC721A: mint to the zero address");
    // We know if the first token in the batch doesn't exist, the other ones don't as well, because of serial ordering.
    require(!_exists(startTokenId), "ERC721A: token already minted");
    require(quantity <= maxBatchSize, "ERC721A: quantity to mint too high");

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

    AddressData memory addressData = _addressData[to];
    _addressData[to] = AddressData(
      addressData.balance + uint128(quantity),
      addressData.numberMinted + uint128(quantity)
    );
    _ownerships[startTokenId] = TokenOwnership(to, uint64(block.timestamp));

    uint256 updatedIndex = startTokenId;

    for (uint256 i = 0; i < quantity; i++) {
      emit Transfer(address(0), to, updatedIndex);
      require(
        _checkOnERC721Received(address(0), to, updatedIndex, _data),
        "ERC721A: transfer to non ERC721Receiver implementer"
      );
      updatedIndex++;
    }

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

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

    bool isApprovedOrOwner = (_msgSender() == prevOwnership.addr ||
      getApproved(tokenId) == _msgSender() ||
      isApprovedForAll(prevOwnership.addr, _msgSender()));

    require(
      isApprovedOrOwner,
      "ERC721A: transfer caller is not owner nor approved"
    );

    require(
      prevOwnership.addr == from,
      "ERC721A: transfer from incorrect owner"
    );
    require(to != address(0), "ERC721A: transfer to the zero address");

    _beforeTokenTransfers(from, to, tokenId, 1);

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

    _addressData[from].balance -= 1;
    _addressData[to].balance += 1;
    _ownerships[tokenId] = TokenOwnership(to, uint64(block.timestamp));

    // If the ownership slot of tokenId+1 is not explicitly set, that means the transfer initiator owns it.
    // Set the slot of tokenId+1 explicitly in storage to maintain correctness for ownerOf(tokenId+1) calls.
    uint256 nextTokenId = tokenId + 1;
    if (_ownerships[nextTokenId].addr == address(0)) {
      if (_exists(nextTokenId)) {
        _ownerships[nextTokenId] = TokenOwnership(
          prevOwnership.addr,
          prevOwnership.startTimestamp
        );
      }
    }

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

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

  uint256 public nextOwnerToExplicitlySet = 0;

  /**
   * @dev Explicitly set `owners` to eliminate loops in future calls of ownerOf().
   */
  function _setOwnersExplicit(uint256 quantity) internal {
    uint256 oldNextOwnerToSet = nextOwnerToExplicitlySet;
    require(quantity > 0, "quantity must be nonzero");
    uint256 endIndex = oldNextOwnerToSet + quantity - 1;
    if (endIndex > currentIndex - 1) {
      endIndex = currentIndex - 1;
    }
    // We know if the last one in the group exists, all in the group exist, due to serial ordering.
    require(_exists(endIndex), "not enough minted yet for this cleanup");
    for (uint256 i = oldNextOwnerToSet; i <= endIndex; i++) {
      if (_ownerships[i].addr == address(0)) {
        TokenOwnership memory ownership = ownershipOf(i);
        _ownerships[i] = TokenOwnership(
          ownership.addr,
          ownership.startTimestamp
        );
      }
    }
    nextOwnerToExplicitlySet = endIndex + 1;
  }

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

  /**
   * @dev Hook that is called before a set of serially-ordered token ids are about to be transferred. This includes minting.
   *
   * 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`.
   */
  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.
   *
   * 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` and `to` are never both zero.
   */
  function _afterTokenTransfers(
    address from,
    address to,
    uint256 startTokenId,
    uint256 quantity
  ) internal virtual {}
}

File 6 of 17: IERC165.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (utils/introspection/IERC165.sol)

pragma solidity ^0.8.0;

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

File 7 of 17: IERC20.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (token/ERC20/IERC20.sol)

pragma solidity ^0.8.0;

/**
 * @dev Interface of the ERC20 standard as defined in the EIP.
 */
interface IERC20 {
    /**
     * @dev Returns the amount of tokens in existence.
     */
    function totalSupply() external view returns (uint256);

    /**
     * @dev Returns the amount of tokens owned by `account`.
     */
    function balanceOf(address account) external view returns (uint256);

    /**
     * @dev Moves `amount` tokens from the caller's account to `recipient`.
     *
     * Returns a boolean value indicating whether the operation succeeded.
     *
     * Emits a {Transfer} event.
     */
    function transfer(address recipient, uint256 amount) external returns (bool);

    /**
     * @dev Returns the remaining number of tokens that `spender` will be
     * allowed to spend on behalf of `owner` through {transferFrom}. This is
     * zero by default.
     *
     * This value changes when {approve} or {transferFrom} are called.
     */
    function allowance(address owner, address spender) external view returns (uint256);

    /**
     * @dev Sets `amount` as the allowance of `spender` over the caller's tokens.
     *
     * Returns a boolean value indicating whether the operation succeeded.
     *
     * IMPORTANT: Beware that changing an allowance with this method brings the risk
     * that someone may use both the old and the new allowance by unfortunate
     * transaction ordering. One possible solution to mitigate this race
     * condition is to first reduce the spender's allowance to 0 and set the
     * desired value afterwards:
     * https://github.com/ethereum/EIPs/issues/20#issuecomment-263524729
     *
     * Emits an {Approval} event.
     */
    function approve(address spender, uint256 amount) external returns (bool);

    /**
     * @dev Moves `amount` tokens from `sender` to `recipient` using the
     * allowance mechanism. `amount` is then deducted from the caller's
     * allowance.
     *
     * Returns a boolean value indicating whether the operation succeeded.
     *
     * Emits a {Transfer} event.
     */
    function transferFrom(
        address sender,
        address recipient,
        uint256 amount
    ) external returns (bool);

    /**
     * @dev Emitted when `value` tokens are moved from one account (`from`) to
     * another (`to`).
     *
     * Note that `value` may be zero.
     */
    event Transfer(address indexed from, address indexed to, uint256 value);

    /**
     * @dev Emitted when the allowance of a `spender` for an `owner` is set by
     * a call to {approve}. `value` is the new allowance.
     */
    event Approval(address indexed owner, address indexed spender, uint256 value);
}

File 8 of 17: IERC721.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (token/ERC721/IERC721.sol)

pragma solidity ^0.8.0;

import "./IERC165.sol";

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

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

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

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

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

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

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

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

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

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

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

File 9 of 17: IERC721Enumerable.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (token/ERC721/extensions/IERC721Enumerable.sol)

pragma solidity ^0.8.0;

import "./IERC721.sol";

/**
 * @title ERC-721 Non-Fungible Token Standard, optional enumeration extension
 * @dev See https://eips.ethereum.org/EIPS/eip-721
 */
interface IERC721Enumerable is IERC721 {
    /**
     * @dev Returns the total amount of tokens stored by the contract.
     */
    function totalSupply() external view returns (uint256);

    /**
     * @dev Returns a token ID owned by `owner` at a given `index` of its token list.
     * Use along with {balanceOf} to enumerate all of ``owner``'s tokens.
     */
    function tokenOfOwnerByIndex(address owner, uint256 index) external view returns (uint256 tokenId);

    /**
     * @dev Returns a token ID at a given `index` of all the tokens stored by the contract.
     * Use along with {totalSupply} to enumerate all tokens.
     */
    function tokenByIndex(uint256 index) external view returns (uint256);
}

File 10 of 17: IERC721Metadata.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (token/ERC721/extensions/IERC721Metadata.sol)

pragma solidity ^0.8.0;

import "./IERC721.sol";

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

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

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

File 11 of 17: IERC721Receiver.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (token/ERC721/IERC721Receiver.sol)

pragma solidity ^0.8.0;

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

File 12 of 17: MerkleProof.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (utils/cryptography/MerkleProof.sol)

pragma solidity ^0.8.0;

/**
 * @dev These functions deal with verification of Merkle Trees proofs.
 *
 * The proofs can be generated using the JavaScript library
 * https://github.com/miguelmota/merkletreejs[merkletreejs].
 * Note: the hashing algorithm should be keccak256 and pair sorting should be enabled.
 *
 * See `test/utils/cryptography/MerkleProof.test.js` for some examples.
 */
library MerkleProof {
    /**
     * @dev Returns true if a `leaf` can be proved to be a part of a Merkle tree
     * defined by `root`. For this, a `proof` must be provided, containing
     * sibling hashes on the branch from the leaf to the root of the tree. Each
     * pair of leaves and each pair of pre-images are assumed to be sorted.
     */
    function verify(
        bytes32[] memory proof,
        bytes32 root,
        bytes32 leaf
    ) internal pure returns (bool) {
        return processProof(proof, leaf) == root;
    }

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

File 13 of 17: Ownable.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (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 Returns the address of the current owner.
     */
    function owner() public view virtual returns (address) {
        return _owner;
    }

    /**
     * @dev Throws if called by any account other than the owner.
     */
    modifier onlyOwner() {
        require(owner() == _msgSender(), "Ownable: caller is not the owner");
        _;
    }

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

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

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

File 14 of 17: Pausable.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (security/Pausable.sol)

pragma solidity ^0.8.0;

import "./Context.sol";

/**
 * @dev Contract module which allows children to implement an emergency stop
 * mechanism that can be triggered by an authorized account.
 *
 * This module is used through inheritance. It will make available the
 * modifiers `whenNotPaused` and `whenPaused`, which can be applied to
 * the functions of your contract. Note that they will not be pausable by
 * simply including this module, only once the modifiers are put in place.
 */
abstract contract Pausable is Context {
    /**
     * @dev Emitted when the pause is triggered by `account`.
     */
    event Paused(address account);

    /**
     * @dev Emitted when the pause is lifted by `account`.
     */
    event Unpaused(address account);

    bool private _paused;

    /**
     * @dev Initializes the contract in unpaused state.
     */
    constructor() {
        _paused = false;
    }

    /**
     * @dev Returns true if the contract is paused, and false otherwise.
     */
    function paused() public view virtual returns (bool) {
        return _paused;
    }

    /**
     * @dev Modifier to make a function callable only when the contract is not paused.
     *
     * Requirements:
     *
     * - The contract must not be paused.
     */
    modifier whenNotPaused() {
        require(!paused(), "Pausable: paused");
        _;
    }

    /**
     * @dev Modifier to make a function callable only when the contract is paused.
     *
     * Requirements:
     *
     * - The contract must be paused.
     */
    modifier whenPaused() {
        require(paused(), "Pausable: not paused");
        _;
    }

    /**
     * @dev Triggers stopped state.
     *
     * Requirements:
     *
     * - The contract must not be paused.
     */
    function _pause() internal virtual whenNotPaused {
        _paused = true;
        emit Paused(_msgSender());
    }

    /**
     * @dev Returns to normal state.
     *
     * Requirements:
     *
     * - The contract must be paused.
     */
    function _unpause() internal virtual whenPaused {
        _paused = false;
        emit Unpaused(_msgSender());
    }
}

File 15 of 17: PaymentSplitter.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (finance/PaymentSplitter.sol)

pragma solidity ^0.8.0;

import "./SafeERC20.sol";
import "./Address.sol";
import "./Context.sol";

/**
 * @title PaymentSplitter
 * @dev This contract allows to split Ether payments among a group of accounts. The sender does not need to be aware
 * that the Ether will be split in this way, since it is handled transparently by the contract.
 *
 * The split can be in equal parts or in any other arbitrary proportion. The way this is specified is by assigning each
 * account to a number of shares. Of all the Ether that this contract receives, each account will then be able to claim
 * an amount proportional to the percentage of total shares they were assigned.
 *
 * `PaymentSplitter` follows a _pull payment_ model. This means that payments are not automatically forwarded to the
 * accounts but kept in this contract, and the actual transfer is triggered as a separate step by calling the {release}
 * function.
 *
 * NOTE: This contract assumes that ERC20 tokens will behave similarly to native tokens (Ether). Rebasing tokens, and
 * tokens that apply fees during transfers, are likely to not be supported as expected. If in doubt, we encourage you
 * to run tests before sending real value to this contract.
 */
contract PaymentSplitter is Context {
    event PayeeAdded(address account, uint256 shares);
    event PaymentReleased(address to, uint256 amount);
    event ERC20PaymentReleased(IERC20 indexed token, address to, uint256 amount);
    event PaymentReceived(address from, uint256 amount);

    uint256 private _totalShares;
    uint256 private _totalReleased;

    mapping(address => uint256) private _shares;
    mapping(address => uint256) private _released;
    address[] private _payees;

    mapping(IERC20 => uint256) private _erc20TotalReleased;
    mapping(IERC20 => mapping(address => uint256)) private _erc20Released;

    /**
     * @dev Creates an instance of `PaymentSplitter` where each account in `payees` is assigned the number of shares at
     * the matching position in the `shares` array.
     *
     * All addresses in `payees` must be non-zero. Both arrays must have the same non-zero length, and there must be no
     * duplicates in `payees`.
     */
    constructor(address[] memory payees, uint256[] memory shares_) payable {
        require(payees.length == shares_.length, "PaymentSplitter: payees and shares length mismatch");
        require(payees.length > 0, "PaymentSplitter: no payees");

        for (uint256 i = 0; i < payees.length; i++) {
            _addPayee(payees[i], shares_[i]);
        }
    }

    /**
     * @dev The Ether received will be logged with {PaymentReceived} events. Note that these events are not fully
     * reliable: it's possible for a contract to receive Ether without triggering this function. This only affects the
     * reliability of the events, and not the actual splitting of Ether.
     *
     * To learn more about this see the Solidity documentation for
     * https://solidity.readthedocs.io/en/latest/contracts.html#fallback-function[fallback
     * functions].
     */
    receive() external payable virtual {
        emit PaymentReceived(_msgSender(), msg.value);
    }

    /**
     * @dev Getter for the total shares held by payees.
     */
    function totalShares() public view returns (uint256) {
        return _totalShares;
    }

    /**
     * @dev Getter for the total amount of Ether already released.
     */
    function totalReleased() public view returns (uint256) {
        return _totalReleased;
    }

    /**
     * @dev Getter for the total amount of `token` already released. `token` should be the address of an IERC20
     * contract.
     */
    function totalReleased(IERC20 token) public view returns (uint256) {
        return _erc20TotalReleased[token];
    }

    /**
     * @dev Getter for the amount of shares held by an account.
     */
    function shares(address account) public view returns (uint256) {
        return _shares[account];
    }

    /**
     * @dev Getter for the amount of Ether already released to a payee.
     */
    function released(address account) public view returns (uint256) {
        return _released[account];
    }

    /**
     * @dev Getter for the amount of `token` tokens already released to a payee. `token` should be the address of an
     * IERC20 contract.
     */
    function released(IERC20 token, address account) public view returns (uint256) {
        return _erc20Released[token][account];
    }

    /**
     * @dev Getter for the address of the payee number `index`.
     */
    function payee(uint256 index) public view returns (address) {
        return _payees[index];
    }

    /**
     * @dev Triggers a transfer to `account` of the amount of Ether they are owed, according to their percentage of the
     * total shares and their previous withdrawals.
     */
    function release(address payable account) public virtual {
        require(_shares[account] > 0, "PaymentSplitter: account has no shares");

        uint256 totalReceived = address(this).balance + totalReleased();
        uint256 payment = _pendingPayment(account, totalReceived, released(account));

        require(payment != 0, "PaymentSplitter: account is not due payment");

        _released[account] += payment;
        _totalReleased += payment;

        Address.sendValue(account, payment);
        emit PaymentReleased(account, payment);
    }

    /**
     * @dev Triggers a transfer to `account` of the amount of `token` tokens they are owed, according to their
     * percentage of the total shares and their previous withdrawals. `token` must be the address of an IERC20
     * contract.
     */
    function release(IERC20 token, address account) public virtual {
        require(_shares[account] > 0, "PaymentSplitter: account has no shares");

        uint256 totalReceived = token.balanceOf(address(this)) + totalReleased(token);
        uint256 payment = _pendingPayment(account, totalReceived, released(token, account));

        require(payment != 0, "PaymentSplitter: account is not due payment");

        _erc20Released[token][account] += payment;
        _erc20TotalReleased[token] += payment;

        SafeERC20.safeTransfer(token, account, payment);
        emit ERC20PaymentReleased(token, account, payment);
    }

    /**
     * @dev internal logic for computing the pending payment of an `account` given the token historical balances and
     * already released amounts.
     */
    function _pendingPayment(
        address account,
        uint256 totalReceived,
        uint256 alreadyReleased
    ) private view returns (uint256) {
        return (totalReceived * _shares[account]) / _totalShares - alreadyReleased;
    }

    /**
     * @dev Add a new payee to the contract.
     * @param account The address of the payee to add.
     * @param shares_ The number of shares owned by the payee.
     */
    function _addPayee(address account, uint256 shares_) private {
        require(account != address(0), "PaymentSplitter: account is the zero address");
        require(shares_ > 0, "PaymentSplitter: shares are 0");
        require(_shares[account] == 0, "PaymentSplitter: account already has shares");

        _payees.push(account);
        _shares[account] = shares_;
        _totalShares = _totalShares + shares_;
        emit PayeeAdded(account, shares_);
    }
}

File 16 of 17: SafeERC20.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (token/ERC20/utils/SafeERC20.sol)

pragma solidity ^0.8.0;

import "./IERC20.sol";
import "./Address.sol";

/**
 * @title SafeERC20
 * @dev Wrappers around ERC20 operations that throw on failure (when the token
 * contract returns false). Tokens that return no value (and instead revert or
 * throw on failure) are also supported, non-reverting calls are assumed to be
 * successful.
 * To use this library you can add a `using SafeERC20 for IERC20;` statement to your contract,
 * which allows you to call the safe operations as `token.safeTransfer(...)`, etc.
 */
library SafeERC20 {
    using Address for address;

    function safeTransfer(
        IERC20 token,
        address to,
        uint256 value
    ) internal {
        _callOptionalReturn(token, abi.encodeWithSelector(token.transfer.selector, to, value));
    }

    function safeTransferFrom(
        IERC20 token,
        address from,
        address to,
        uint256 value
    ) internal {
        _callOptionalReturn(token, abi.encodeWithSelector(token.transferFrom.selector, from, to, value));
    }

    /**
     * @dev Deprecated. This function has issues similar to the ones found in
     * {IERC20-approve}, and its usage is discouraged.
     *
     * Whenever possible, use {safeIncreaseAllowance} and
     * {safeDecreaseAllowance} instead.
     */
    function safeApprove(
        IERC20 token,
        address spender,
        uint256 value
    ) internal {
        // safeApprove should only be called when setting an initial allowance,
        // or when resetting it to zero. To increase and decrease it, use
        // 'safeIncreaseAllowance' and 'safeDecreaseAllowance'
        require(
            (value == 0) || (token.allowance(address(this), spender) == 0),
            "SafeERC20: approve from non-zero to non-zero allowance"
        );
        _callOptionalReturn(token, abi.encodeWithSelector(token.approve.selector, spender, value));
    }

    function safeIncreaseAllowance(
        IERC20 token,
        address spender,
        uint256 value
    ) internal {
        uint256 newAllowance = token.allowance(address(this), spender) + value;
        _callOptionalReturn(token, abi.encodeWithSelector(token.approve.selector, spender, newAllowance));
    }

    function safeDecreaseAllowance(
        IERC20 token,
        address spender,
        uint256 value
    ) internal {
        unchecked {
            uint256 oldAllowance = token.allowance(address(this), spender);
            require(oldAllowance >= value, "SafeERC20: decreased allowance below zero");
            uint256 newAllowance = oldAllowance - value;
            _callOptionalReturn(token, abi.encodeWithSelector(token.approve.selector, spender, newAllowance));
        }
    }

    /**
     * @dev Imitates a Solidity high-level call (i.e. a regular function call to a contract), relaxing the requirement
     * on the return value: the return value is optional (but if data is returned, it must not be false).
     * @param token The token targeted by the call.
     * @param data The call data (encoded using abi.encode or one of its variants).
     */
    function _callOptionalReturn(IERC20 token, bytes memory data) private {
        // We need to perform a low level call here, to bypass Solidity's return data size checking mechanism, since
        // we're implementing it ourselves. We use {Address.functionCall} to perform this call, which verifies that
        // the target address contains contract code and also asserts for success in the low-level call.

        bytes memory returndata = address(token).functionCall(data, "SafeERC20: low-level call failed");
        if (returndata.length > 0) {
            // Return data is optional
            require(abi.decode(returndata, (bool)), "SafeERC20: ERC20 operation did not succeed");
        }
    }
}

File 17 of 17: Strings.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (utils/Strings.sol)

pragma solidity ^0.8.0;

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

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

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

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

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

Contract Security Audit

Contract ABI

[{"inputs":[{"internalType":"string","name":"name","type":"string"},{"internalType":"string","name":"symbol","type":"string"},{"internalType":"string","name":"baseTokenURI","type":"string"},{"internalType":"uint256[]","name":"numericValues","type":"uint256[]"},{"internalType":"bytes32","name":"merkleRoot","type":"bytes32"},{"internalType":"address[]","name":"payees","type":"address[]"},{"internalType":"uint256[]","name":"shares","type":"uint256[]"}],"stateMutability":"nonpayable","type":"constructor"},{"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":"contract IERC20","name":"token","type":"address"},{"indexed":false,"internalType":"address","name":"to","type":"address"},{"indexed":false,"internalType":"uint256","name":"amount","type":"uint256"}],"name":"ERC20PaymentReleased","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"addr","type":"address"},{"indexed":true,"internalType":"uint256","name":"atPrice","type":"uint256"},{"indexed":true,"internalType":"uint256","name":"count","type":"uint256"}],"name":"EarlyPurchase","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":false,"internalType":"address","name":"account","type":"address"}],"name":"Paused","type":"event"},{"anonymous":false,"inputs":[{"indexed":false,"internalType":"address","name":"account","type":"address"},{"indexed":false,"internalType":"uint256","name":"shares","type":"uint256"}],"name":"PayeeAdded","type":"event"},{"anonymous":false,"inputs":[{"indexed":false,"internalType":"address","name":"from","type":"address"},{"indexed":false,"internalType":"uint256","name":"amount","type":"uint256"}],"name":"PaymentReceived","type":"event"},{"anonymous":false,"inputs":[{"indexed":false,"internalType":"address","name":"to","type":"address"},{"indexed":false,"internalType":"uint256","name":"amount","type":"uint256"}],"name":"PaymentReleased","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"addr","type":"address"},{"indexed":true,"internalType":"uint256","name":"atPrice","type":"uint256"},{"indexed":true,"internalType":"uint256","name":"count","type":"uint256"}],"name":"Purchase","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Transfer","type":"event"},{"anonymous":false,"inputs":[{"indexed":false,"internalType":"address","name":"account","type":"address"}],"name":"Unpaused","type":"event"},{"inputs":[],"name":"MAX_TOTAL_MINT","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"MAX_TOTAL_MINT_PER_ADDRESS","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"PRICE","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"_baseTokenURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"_maxPerAddress","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":"_maxTxPerAddress","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"_merkleRoot","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"_preSaleTime","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"_presaleMaxPerAddress","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"_presaleMaxPerAddressMap","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"_presalePrice","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"_price","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"_publicSaleTime","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"_purchases","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"approve","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"}],"name":"balanceOf","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"count","type":"uint256"},{"internalType":"bytes32[]","name":"merkleProof","type":"bytes32[]"}],"name":"earlyPurchase","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"getApproved","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"},{"internalType":"address","name":"operator","type":"address"}],"name":"isApprovedForAll","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"isPreSaleActive","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"isPublicSaleActive","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"count","type":"uint256"}],"name":"mint","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"name","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"nextOwnerToExplicitlySet","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"addr","type":"address"},{"internalType":"bytes32[]","name":"merkleProof","type":"bytes32[]"}],"name":"onEarlyPurchaseList","outputs":[{"internalType":"bool","name":"","type":"bool"}],"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":"pause","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"paused","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"index","type":"uint256"}],"name":"payee","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"count","type":"uint256"}],"name":"purchase","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"address payable","name":"account","type":"address"}],"name":"release","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"contract IERC20","name":"token","type":"address"},{"internalType":"address","name":"account","type":"address"}],"name":"release","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"contract IERC20","name":"token","type":"address"},{"internalType":"address","name":"account","type":"address"}],"name":"released","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"account","type":"address"}],"name":"released","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"},{"internalType":"bytes","name":"_data","type":"bytes"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"operator","type":"address"},{"internalType":"bool","name":"approved","type":"bool"}],"name":"setApprovalForAll","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"baseUri","type":"string"}],"name":"setBaseUri","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"merkleRoot","type":"bytes32"}],"name":"setMerkleRoot","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address[]","name":"whitelist","type":"address[]"},{"internalType":"uint256[]","name":"maxPerAddress","type":"uint256[]"}],"name":"setPresaleMaxPerAddress","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"publicSaleTime","type":"uint256"},{"internalType":"uint256","name":"preSaleTime","type":"uint256"},{"internalType":"uint256","name":"maxPerAddress","type":"uint256"},{"internalType":"uint256","name":"presaleMaxPerAddress","type":"uint256"},{"internalType":"uint256","name":"price","type":"uint256"},{"internalType":"uint256","name":"presalePrice","type":"uint256"},{"internalType":"bytes32","name":"merkleRoot","type":"bytes32"},{"internalType":"uint256","name":"maxTxPerAddress","type":"uint256"}],"name":"setSaleInformation","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"account","type":"address"}],"name":"shares","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","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":"index","type":"uint256"}],"name":"tokenByIndex","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"},{"internalType":"uint256","name":"index","type":"uint256"}],"name":"tokenOfOwnerByIndex","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"tokenURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"contract IERC20","name":"token","type":"address"}],"name":"totalReleased","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"totalReleased","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"totalShares","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":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"newOwner","type":"address"}],"name":"transferOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"unpause","outputs":[],"stateMutability":"nonpayable","type":"function"},{"stateMutability":"payable","type":"receive"}]

60a0604052600160005560006007553480156200001b57600080fd5b5060405162004b6f38038062004b6f8339810160408190526200003e916200097a565b818188888760028151811062000058576200005862000a8c565b602002602001015160008111620000f6576040517f08c379a000000000000000000000000000000000000000000000000000000000815260206004820152602760248201527f455243373231413a206d61782062617463682073697a65206d7573742062652060448201527f6e6f6e7a65726f0000000000000000000000000000000000000000000000000060648201526084015b60405180910390fd5b82516200010b906001906020860190620006d1565b50815162000121906002906020850190620006d1565b50608052506200014e90506200013f6401000000006200041c810204565b64010000000062000420810204565b6008805460a060020a60ff02191690558051825114620001f1576040517f08c379a000000000000000000000000000000000000000000000000000000000815260206004820152603260248201527f5061796d656e7453706c69747465723a2070617965657320616e64207368617260448201527f6573206c656e677468206d69736d6174636800000000000000000000000000006064820152608401620000ed565b60008251116200025e576040517f08c379a000000000000000000000000000000000000000000000000000000000815260206004820152601a60248201527f5061796d656e7453706c69747465723a206e6f207061796565730000000000006044820152606401620000ed565b60005b8251811015620002d357620002be83828151811062000284576200028462000a8c565b6020026020010151838381518110620002a157620002a162000a8c565b602002602001015162000472640100000000026401000000009004565b80620002ca8162000aea565b91505062000261565b50508551620002eb91506010906020880190620006d1565b508360008151811062000302576200030262000a8c565b60200260200101516012819055508360018151811062000326576200032662000a8c565b6020026020010151601381905550836002815181106200034a576200034a62000a8c565b6020026020010151601481905550836003815181106200036e576200036e62000a8c565b60200260200101516015819055508360048151811062000392576200039262000a8c565b602002602001015160168190555083600581518110620003b657620003b662000a8c565b602002602001015160178190555083600681518110620003da57620003da62000a8c565b602002602001015160188190555083600781518110620003fe57620003fe62000a8c565b602090810291909101015160195550506011555062000b7992505050565b3390565b60088054600160a060020a03838116600160a060020a0319831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b600160a060020a0382166200050a576040517f08c379a000000000000000000000000000000000000000000000000000000000815260206004820152602c60248201527f5061796d656e7453706c69747465723a206163636f756e74206973207468652060448201527f7a65726f206164647265737300000000000000000000000000000000000000006064820152608401620000ed565b6000811162000576576040517f08c379a000000000000000000000000000000000000000000000000000000000815260206004820152601d60248201527f5061796d656e7453706c69747465723a207368617265732061726520300000006044820152606401620000ed565b600160a060020a0382166000908152600b6020526040902054156200061e576040517f08c379a000000000000000000000000000000000000000000000000000000000815260206004820152602b60248201527f5061796d656e7453706c69747465723a206163636f756e7420616c726561647960448201527f20686173207368617265730000000000000000000000000000000000000000006064820152608401620000ed565b600d8054600181019091557fd7b6990105719101dabeb77144f2a3385c8033acd3af97e9423a695e81ad1eb5018054600160a060020a031916600160a060020a0384169081179091556000908152600b602052604090208190556009546200068890829062000b08565b60095560408051600160a060020a0384168152602081018390527f40c340f65e17194d14ddddb073d3c9f888e3cb52b5aae0c6c7706b4fbc905fac910160405180910390a15050565b828054620006df9062000b23565b90600052602060002090601f0160209004810192826200070357600085556200074e565b82601f106200071e57805160ff19168380011785556200074e565b828001600101855582156200074e579182015b828111156200074e57825182559160200191906001019062000731565b506200075c92915062000760565b5090565b5b808211156200075c576000815560010162000761565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b604051601f8201601f191681016001604060020a0381118282101715620007d157620007d162000777565b604052919050565b600082601f830112620007eb57600080fd5b81516001604060020a0381111562000807576200080762000777565b60206200081d601f8301601f19168201620007a6565b82815285828487010111156200083257600080fd5b60005b838110156200085257858101830151828201840152820162000835565b83811115620008645760008385840101525b5095945050505050565b60006001604060020a038211156200088a576200088a62000777565b5060209081020190565b600082601f830112620008a657600080fd5b81516020620008bf620008b9836200086e565b620007a6565b82815291810284018101918181019086841115620008dc57600080fd5b8286015b84811015620008f95780518352918301918301620008e0565b509695505050505050565b600082601f8301126200091657600080fd5b8151602062000929620008b9836200086e565b828152918102840181019181810190868411156200094657600080fd5b8286015b84811015620008f9578051600160a060020a03811681146200096c5760008081fd5b83529183019183016200094a565b600080600080600080600060e0888a0312156200099657600080fd5b87516001604060020a0380821115620009ae57600080fd5b620009bc8b838c01620007d9565b985060208a0151915080821115620009d357600080fd5b620009e18b838c01620007d9565b975060408a0151915080821115620009f857600080fd5b62000a068b838c01620007d9565b965060608a015191508082111562000a1d57600080fd5b62000a2b8b838c0162000894565b955060808a0151945060a08a015191508082111562000a4957600080fd5b62000a578b838c0162000904565b935060c08a015191508082111562000a6e57600080fd5b5062000a7d8a828b0162000894565b91505092959891949750929550565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b600060001982141562000b015762000b0162000abb565b5060010190565b6000821982111562000b1e5762000b1e62000abb565b500190565b60028104600182168062000b3857607f821691505b6020821081141562000b73577f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b50919050565b608051613fcc62000ba3600039600081816125fb015281816126250152612d9c0152613fcc6000f3fe608060405260043610610397576000357c01000000000000000000000000000000000000000000000000000000009004806374721235116101ee578063b88d4fde1161011f578063d79779b2116100bd578063e985e9c51161008c578063e985e9c514610a40578063efef39a114610a89578063f2fde38b14610a9c578063fa156f9a14610abc57600080fd5b8063d79779b2146109cc578063e2ab10ce14610a02578063e2d5ee2d14610a15578063e33b7de314610a2b57600080fd5b8063ce7c2ac2116100f9578063ce7c2ac214610956578063cf9e8e691461098c578063cfc86f7b146109a1578063d7224ba0146109b657600080fd5b8063b88d4fde146108e9578063c4ec2c1614610909578063c87b56dd1461093657600080fd5b8063904be6da1161018c5780639d044ed3116101665780639d044ed31461087e578063a0bcfc7f14610893578063a22cb465146108b3578063b85ef036146108d357600080fd5b8063904be6da1461081d57806395d89b41146108335780639852595c1461084857600080fd5b80638456cb59116101c85780638456cb59146107b55780638b83209b146107ca5780638d859f3e146107ea5780638da5cb5b146107ff57600080fd5b806374721235146107555780637b96a3b2146107755780637cb647591461079557600080fd5b80633a98ef39116102c85780635c975abb1161026657806366cfb1f31161024057806366cfb1f3146106f5578063696fa41e1461070a57806370a0823114610720578063715018a61461074057600080fd5b80635c975abb146106a05780635f0d246a146106bf5780636352211e146106d557600080fd5b806340c10f19116102a257806340c10f191461062d57806342842e0e1461064057806348b75044146106605780634f6ccce71461068057600080fd5b80633a98ef39146105bd5780633f4ba83a146105d2578063406072a9146105e757600080fd5b80631916558711610335578063235b6ea11161030f578063235b6ea11461055157806323b872dd146105675780632f745c59146105875780632fc37ab2146105a757600080fd5b806319165587146105065780631e84c4131461052657806322f4596f1461053b57600080fd5b8063095ea7b311610371578063095ea7b3146104745780630d5fbb72146104965780631687edb5146104d157806318160ddd146104f157600080fd5b806301ffc9a7146103e557806306fdde031461041a578063081812fc1461043c57600080fd5b366103e0577f6ef95f06320e7a25a04a175ca677b7052bdd97131872c2192525a629f51be7703360408051600160a060020a0390921682523460208301520160405180910390a1005b600080fd5b3480156103f157600080fd5b50610405610400366004613542565b610ad2565b60405190151581526020015b60405180910390f35b34801561042657600080fd5b5061042f610ba3565b60405161041191906135b7565b34801561044857600080fd5b5061045c6104573660046135ca565b610c35565b604051600160a060020a039091168152602001610411565b34801561048057600080fd5b5061049461048f3660046135f8565b610cd8565b005b3480156104a257600080fd5b506104c36104b1366004613624565b601a6020526000908152604090205481565b604051908152602001610411565b3480156104dd57600080fd5b506104946104ec366004613717565b610e11565b3480156104fd57600080fd5b506104c3610f87565b34801561051257600080fd5b50610494610521366004613624565b610f9d565b34801561053257600080fd5b506104056110d2565b34801561054757600080fd5b506104c360145481565b34801561055d57600080fd5b506104c360125481565b34801561057357600080fd5b506104946105823660046137d6565b6110ec565b34801561059357600080fd5b506104c36105a23660046135f8565b6110f7565b3480156105b357600080fd5b506104c360115481565b3480156105c957600080fd5b506009546104c3565b3480156105de57600080fd5b5061049461129f565b3480156105f357600080fd5b506104c3610602366004613817565b600160a060020a039182166000908152600f6020908152604080832093909416825291909152205490565b61049461063b3660046135f8565b6112d6565b34801561064c57600080fd5b5061049461065b3660046137d6565b61131a565b34801561066c57600080fd5b5061049461067b366004613817565b611335565b34801561068c57600080fd5b506104c361069b3660046135ca565b61153c565b3480156106ac57600080fd5b5060085460a060020a900460ff16610405565b3480156106cb57600080fd5b506104c360135481565b3480156106e157600080fd5b5061045c6106f03660046135ca565b6115c1565b34801561070157600080fd5b506104c36115d3565b34801561071657600080fd5b506104c360195481565b34801561072c57600080fd5b506104c361073b366004613624565b6115f0565b34801561074c57600080fd5b50610494611696565b34801561076157600080fd5b50610494610770366004613850565b6116cd565b34801561078157600080fd5b506104056107903660046138f0565b611720565b3480156107a157600080fd5b506104946107b03660046135ca565b6117ad565b3480156107c157600080fd5b506104946117df565b3480156107d657600080fd5b5061045c6107e53660046135ca565b611814565b3480156107f657600080fd5b506104c3611844565b34801561080b57600080fd5b50600854600160a060020a031661045c565b34801561082957600080fd5b506104c360165481565b34801561083f57600080fd5b5061042f611861565b34801561085457600080fd5b506104c3610863366004613624565b600160a060020a03166000908152600c602052604090205490565b34801561088a57600080fd5b50610405611870565b34801561089f57600080fd5b506104946108ae36600461399d565b611896565b3480156108bf57600080fd5b506104946108ce3660046139f4565b6118d6565b3480156108df57600080fd5b506104c360175481565b3480156108f557600080fd5b50610494610904366004613a22565b61199e565b34801561091557600080fd5b506104c3610924366004613624565b601b6020526000908152604090205481565b34801561094257600080fd5b5061042f6109513660046135ca565b6119da565b34801561096257600080fd5b506104c3610971366004613624565b600160a060020a03166000908152600b602052604090205490565b34801561099857600080fd5b506014546104c3565b3480156109ad57600080fd5b5061042f611ab7565b3480156109c257600080fd5b506104c360075481565b3480156109d857600080fd5b506104c36109e7366004613624565b600160a060020a03166000908152600e602052604090205490565b610494610a10366004613aa2565b611b45565b348015610a2157600080fd5b506104c360155481565b348015610a3757600080fd5b50600a546104c3565b348015610a4c57600080fd5b50610405610a5b366004613817565b600160a060020a03918216600090815260066020908152604080832093909416825291909152205460ff1690565b610494610a973660046135ca565b611c5f565b348015610aa857600080fd5b50610494610ab7366004613624565b611d30565b348015610ac857600080fd5b506104c360185481565b6000600160e060020a031982167f80ac58cd000000000000000000000000000000000000000000000000000000001480610b355750600160e060020a031982167f5b5e139f00000000000000000000000000000000000000000000000000000000145b80610b695750600160e060020a031982167f780e9d6300000000000000000000000000000000000000000000000000000000145b80610b9d57507f01ffc9a700000000000000000000000000000000000000000000000000000000600160e060020a03198316145b92915050565b606060018054610bb290613ad5565b80601f0160208091040260200160405190810160405280929190818152602001828054610bde90613ad5565b8015610c2b5780601f10610c0057610100808354040283529160200191610c2b565b820191906000526020600020905b815481529060010190602001808311610c0e57829003601f168201915b5050505050905090565b6000610c42826000541190565b610cbc5760405160e560020a62461bcd02815260206004820152602d60248201527f455243373231413a20617070726f76656420717565727920666f72206e6f6e6560448201527f78697374656e7420746f6b656e0000000000000000000000000000000000000060648201526084015b60405180910390fd5b50600090815260056020526040902054600160a060020a031690565b6000610ce3826115c1565b905080600160a060020a031683600160a060020a03161415610d705760405160e560020a62461bcd02815260206004820152602260248201527f455243373231413a20617070726f76616c20746f2063757272656e74206f776e60448201527f65720000000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b33600160a060020a0382161480610d8c5750610d8c8133610a5b565b610e015760405160e560020a62461bcd02815260206004820152603960248201527f455243373231413a20617070726f76652063616c6c6572206973206e6f74206f60448201527f776e6572206e6f7220617070726f76656420666f7220616c6c000000000000006064820152608401610cb3565b610e0c838383611de8565b505050565b600854600160a060020a03163314610e3e5760405160e560020a62461bcd028152600401610cb390613b13565b8051825114610eb85760405160e560020a62461bcd02815260206004820152602b60248201527f77686974656c69737420616e64206d617850657241646472657373206c656e6760448201527f7468206d69736d617463680000000000000000000000000000000000000000006064820152608401610cb3565b6000825111610f0c5760405160e560020a62461bcd02815260206004820152600c60248201527f4e6f2077686974656c69737400000000000000000000000000000000000000006044820152606401610cb3565b60005b8251811015610e0c57818181518110610f2a57610f2a613b48565b6020026020010151601b6000858481518110610f4857610f48613b48565b6020026020010151600160a060020a0316600160a060020a03168152602001908152602001600020819055508080610f7f90613b7a565b915050610f0f565b60006001600054610f989190613b95565b905090565b600160a060020a0381166000908152600b6020526040902054610fd55760405160e560020a62461bcd028152600401610cb390613bac565b6000610fe0600a5490565b610feb903031613c09565b90506000611018838361101386600160a060020a03166000908152600c602052604090205490565b611e51565b90508061103a5760405160e560020a62461bcd028152600401610cb390613c21565b600160a060020a0383166000908152600c602052604081208054839290611062908490613c09565b9250508190555080600a600082825461107b9190613c09565b9091555061108b90508382611e97565b60408051600160a060020a0385168152602081018390527fdf20fd1e76bc69d672e4814fafb2c449bba3a5369d8359adf9e05e6fde87b056910160405180910390a1505050565b6000601754600014158015610f9857504260175410905090565b610e0c838383611fb7565b6000611102836115f0565b82106111795760405160e560020a62461bcd02815260206004820152602260248201527f455243373231413a206f776e657220696e646578206f7574206f6620626f756e60448201527f64730000000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b6000611183610f87565b905060008060005b8381101561122d57600081815260036020908152604091829020825180840190935254600160a060020a03811680845260a060020a90910467ffffffffffffffff1691830191909152156111de57805192505b87600160a060020a031683600160a060020a0316141561121a578684141561120c57509350610b9d92505050565b8361121681613b7a565b9450505b508061122581613b7a565b91505061118b565b5060405160e560020a62461bcd02815260206004820152602e60248201527f455243373231413a20756e61626c6520746f2067657420746f6b656e206f662060448201527f6f776e657220627920696e6465780000000000000000000000000000000000006064820152608401610cb3565b600854600160a060020a031633146112cc5760405160e560020a62461bcd028152600401610cb390613b13565b6112d4612382565b565b600854600160a060020a031633146113035760405160e560020a62461bcd028152600401610cb390613b13565b61130c8161243c565b61131682826124c9565b5050565b610e0c8383836040518060200160405280600081525061199e565b600160a060020a0381166000908152600b602052604090205461136d5760405160e560020a62461bcd028152600401610cb390613bac565b600160a060020a0382166000908152600e60205260408120546040517f70a08231000000000000000000000000000000000000000000000000000000008152306004820152600160a060020a038516906370a082319060240160206040518083038186803b1580156113de57600080fd5b505afa1580156113f2573d6000803e3d6000fd5b505050506040513d601f19601f820116820180604052508101906114169190613c7e565b6114209190613c09565b9050600061145983836110138787600160a060020a039182166000908152600f6020908152604080832093909416825291909152205490565b90508061147b5760405160e560020a62461bcd028152600401610cb390613c21565b600160a060020a038085166000908152600f60209081526040808320938716835292905290812080548392906114b2908490613c09565b9091555050600160a060020a0384166000908152600e6020526040812080548392906114df908490613c09565b909155506114f090508484836124e3565b60408051600160a060020a038581168252602082018490528616917f3be5b7a71e84ed12875d241991c70855ac5817d847039e17a9d895c1ceb0f18a910160405180910390a250505050565b6000611546610f87565b82106115bd5760405160e560020a62461bcd02815260206004820152602360248201527f455243373231413a20676c6f62616c20696e646578206f7574206f6620626f7560448201527f6e647300000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b5090565b60006115cc82612563565b5192915050565b60006115dd611870565b156115e9575060165490565b5060155490565b6000600160a060020a0382166116715760405160e560020a62461bcd02815260206004820152602b60248201527f455243373231413a2062616c616e636520717565727920666f7220746865207a60448201527f65726f20616464726573730000000000000000000000000000000000000000006064820152608401610cb3565b50600160a060020a03166000908152600460205260409020546001608060020a031690565b600854600160a060020a031633146116c35760405160e560020a62461bcd028152600401610cb390613b13565b6112d46000612734565b600854600160a060020a031633146116fa5760405160e560020a62461bcd028152600401610cb390613b13565b601797909755601895909555601593909355601691909155601255601355601155601955565b60006040516c01000000000000000000000000600160a060020a0386160260208201526000906034016040516020818303038152906040528051906020012090506117a2848480806020026020016040519081016040528093929190818152602001838360200280828437600092019190915250506011549150849050612793565b9150505b9392505050565b600854600160a060020a031633146117da5760405160e560020a62461bcd028152600401610cb390613b13565b601155565b600854600160a060020a0316331461180c5760405160e560020a62461bcd028152600401610cb390613b13565b6112d46127a9565b6000600d828154811061182957611829613b48565b600091825260209091200154600160a060020a031692915050565b600061184e611870565b1561185a575060135490565b5060125490565b606060028054610bb290613ad5565b6000601854600014158015611886575042601854105b8015610f98575050601754421090565b600854600160a060020a031633146118c35760405160e560020a62461bcd028152600401610cb390613b13565b805161131690601090602084019061349c565b600160a060020a0382163314156119325760405160e560020a62461bcd02815260206004820152601a60248201527f455243373231413a20617070726f766520746f2063616c6c65720000000000006044820152606401610cb3565b336000818152600660209081526040808320600160a060020a03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b6119a9848484611fb7565b6119b584848484612822565b6119d45760405160e560020a62461bcd028152600401610cb390613c97565b50505050565b60606119e7826000541190565b611a5c5760405160e560020a62461bcd02815260206004820152602f60248201527f4552433732314d657461646174613a2055524920717565727920666f72206e6f60448201527f6e6578697374656e7420746f6b656e00000000000000000000000000000000006064820152608401610cb3565b6000611a66612964565b90506000815111611a8657604051806020016040528060008152506117a6565b80611a9084612998565b604051602001611aa1929190613d10565b6040516020818303038152906040529392505050565b60108054611ac490613ad5565b80601f0160208091040260200160405190810160405280929190818152602001828054611af090613ad5565b8015611b3d5780601f10611b1257610100808354040283529160200191611b3d565b820191906000526020600020905b815481529060010190602001808311611b2057829003601f168201915b505050505081565b60085460a060020a900460ff1615611b725760405160e560020a62461bcd028152600401610cb390613d3f565b336000818152601b6020526040902054611b8e91908590612ad1565b611b96611870565b8015611ba85750611ba8338383611720565b611c1d5760405160e560020a62461bcd02815260206004820152602360248201527f424153455f434f4c4c454354494f4e2f43414e4e4f545f4d494e545f5052455360448201527f414c4500000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b611c2983601354612c0c565b60135460405184919033907f38bd02858ca92987ff585a4c06998aea8187e96864df1eaf349dec3cfddc0fbb90600090a4505050565b60085460a060020a900460ff1615611c8c5760405160e560020a62461bcd028152600401610cb390613d3f565b611c993382601554612ad1565b611ca16110d2565b611cf05760405160e560020a62461bcd02815260206004820152601b60248201527f424153455f434f4c4c454354494f4e2f43414e4e4f545f4d494e5400000000006044820152606401610cb3565b611cfc81601254612c0c565b60125460405182919033907f12cb4648cf3058b17ceeb33e579f8b0bc269fe0843f3900b8e24b6c54871703c90600090a450565b600854600160a060020a03163314611d5d5760405160e560020a62461bcd028152600401610cb390613b13565b600160a060020a038116611ddc5760405160e560020a62461bcd02815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201527f64647265737300000000000000000000000000000000000000000000000000006064820152608401610cb3565b611de581612734565b50565b600082815260056020526040808220805473ffffffffffffffffffffffffffffffffffffffff1916600160a060020a0387811691821790925591518593918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a4505050565b600954600160a060020a0384166000908152600b602052604081205490918391611e7b9086613d76565b611e859190613dae565b611e8f9190613b95565b949350505050565b3031811115611eeb5760405160e560020a62461bcd02815260206004820152601d60248201527f416464726573733a20696e73756666696369656e742062616c616e63650000006044820152606401610cb3565b600082600160a060020a03168260405160006040518083038185875af1925050503d8060008114611f38576040519150601f19603f3d011682016040523d82523d6000602084013e611f3d565b606091505b5050905080610e0c5760405160e560020a62461bcd02815260206004820152603a60248201527f416464726573733a20756e61626c6520746f2073656e642076616c75652c207260448201527f6563697069656e74206d617920686176652072657665727465640000000000006064820152608401610cb3565b6000611fc282612563565b8051909150600090600160a060020a031633600160a060020a03161480611ff9575033611fee84610c35565b600160a060020a0316145b8061200b5750815161200b9033610a5b565b9050806120835760405160e560020a62461bcd02815260206004820152603260248201527f455243373231413a207472616e736665722063616c6c6572206973206e6f742060448201527f6f776e6572206e6f7220617070726f76656400000000000000000000000000006064820152608401610cb3565b84600160a060020a03168260000151600160a060020a0316146121115760405160e560020a62461bcd02815260206004820152602660248201527f455243373231413a207472616e736665722066726f6d20696e636f727265637460448201527f206f776e657200000000000000000000000000000000000000000000000000006064820152608401610cb3565b600160a060020a0384166121905760405160e560020a62461bcd02815260206004820152602560248201527f455243373231413a207472616e7366657220746f20746865207a65726f20616460448201527f64726573730000000000000000000000000000000000000000000000000000006064820152608401610cb3565b6121a06000848460000151611de8565b600160a060020a03851660009081526004602052604081208054600192906121d29084906001608060020a0316613dc2565b82546101009290920a6001608060020a03818102199093169183160217909155600160a060020a0386166000908152600460205260408120805460019450909261221e91859116613dea565b82546001608060020a039182166101009390930a928302919092021990911617905550604080518082018252600160a060020a03808716825267ffffffffffffffff42811660208085019182526000898152600390915294852093518454915190921660a060020a02600160e060020a031990911691909216171790556122a6846001613c09565b600081815260036020526040902054909150600160a060020a0316612338576122d0816000541190565b15612338576040805180820182528451600160a060020a03908116825260208087015167ffffffffffffffff908116828501908152600087815260039093529490912092518354945190911660a060020a02600160e060020a03199094169116179190911790555b8385600160a060020a031687600160a060020a03167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a45b505050505050565b60085460a060020a900460ff166123de5760405160e560020a62461bcd02815260206004820152601460248201527f5061757361626c653a206e6f74207061757365640000000000000000000000006044820152606401610cb3565b6008805474ff0000000000000000000000000000000000000000191690557f5db9ee0a495bf2e6ff9c91a7834c1ba4fdd244a5e8aa4e537bd38aeae4b073aa335b604051600160a060020a03909116815260200160405180910390a1565b60145481612448610f87565b6124529190613c09565b1115611de55760405160e560020a62461bcd02815260206004820152602260248201527f424153455f434f4c4c454354494f4e2f455843454544535f4d41585f5355505060448201527f4c590000000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b611316828260405180602001604052806000815250612cbd565b60408051600160a060020a038416602482015260448082018490528251808303909101815260649091019091526020810180517bffffffffffffffffffffffffffffffffffffffffffffffffffffffff167fa9059cbb00000000000000000000000000000000000000000000000000000000179052610e0c908490612ff5565b6040805180820190915260008082526020820152612582826000541190565b6125f75760405160e560020a62461bcd02815260206004820152602a60248201527f455243373231413a206f776e657220717565727920666f72206e6f6e6578697360448201527f74656e7420746f6b656e000000000000000000000000000000000000000000006064820152608401610cb3565b60007f000000000000000000000000000000000000000000000000000000000000000083106126585761264a7f000000000000000000000000000000000000000000000000000000000000000084613b95565b612655906001613c09565b90505b825b8181106126c257600081815260036020908152604091829020825180840190935254600160a060020a03811680845260a060020a90910467ffffffffffffffff1691830191909152156126af57949350505050565b50806126ba81613e0c565b91505061265a565b5060405160e560020a62461bcd02815260206004820152602f60248201527f455243373231413a20756e61626c6520746f2064657465726d696e652074686560448201527f206f776e6572206f6620746f6b656e00000000000000000000000000000000006064820152608401610cb3565b60088054600160a060020a0383811673ffffffffffffffffffffffffffffffffffffffff19831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b6000826127a085846130dd565b14949350505050565b60085460a060020a900460ff16156127d65760405160e560020a62461bcd028152600401610cb390613d3f565b6008805474ff0000000000000000000000000000000000000000191660a060020a1790557f62e78cea01bee320cd4e420270b5ea74000d11b0c9f74754ebdbfc544b05a25861241f3390565b6000600160a060020a0384163b15612959576040517f150b7a02000000000000000000000000000000000000000000000000000000008152600160a060020a0385169063150b7a029061287f903390899088908890600401613e23565b602060405180830381600087803b15801561289957600080fd5b505af19250505080156128c9575060408051601f3d908101601f191682019092526128c691810190613e5f565b60015b612926573d8080156128f7576040519150601f19603f3d011682016040523d82523d6000602084013e6128fc565b606091505b50805161291e5760405160e560020a62461bcd028152600401610cb390613c97565b805181602001fd5b600160e060020a0319167f150b7a0200000000000000000000000000000000000000000000000000000000149050611e8f565b506001949350505050565b60606010612973306014613189565b604051602001612984929190613e7c565b604051602081830303815290604052905090565b6060816129d857505060408051808201909152600181527f3000000000000000000000000000000000000000000000000000000000000000602082015290565b8160005b8115612a0257806129ec81613b7a565b91506129fb9050600a83613dae565b91506129dc565b60008167ffffffffffffffff811115612a1d57612a1d613641565b6040519080825280601f01601f191660200182016040528015612a47576020820181803683370190505b5090505b8415611e8f57612a5c600183613b95565b9150612a69600a86613f49565b612a74906030613c09565b7f010000000000000000000000000000000000000000000000000000000000000002818381518110612aa857612aa8613b48565b6020010190600160f860020a031916908160001a905350612aca600a86613dae565b9450612a4b565b612ada8261243c565b60195415801590612aed57506019548211155b612b625760405160e560020a62461bcd02815260206004820152602b60248201527f424153455f434f4c4c454354494f4e2f455843454544535f4d41585f5045525f60448201527f5452414e53414354494f4e0000000000000000000000000000000000000000006064820152608401610cb3565b600160a060020a0383166000908152601a6020526040812054612b86908490613c09565b90508115801590612b975750818111155b6119d45760405160e560020a62461bcd02815260206004820152602960248201527f424153455f434f4c4c454354494f4e2f455843454544535f494e44495649445560448201527f414c5f535550504c5900000000000000000000000000000000000000000000006064820152608401610cb3565b34612c178383613d76565b1115612c8e5760405160e560020a62461bcd02815260206004820152602760248201527f424153455f434f4c4c454354494f4e2f494e53554646494349454e545f45544860448201527f5f414d4f554e54000000000000000000000000000000000000000000000000006064820152608401610cb3565b336000908152601a602052604081208054849290612cad908490613c09565b90915550611316905033836124c9565b600054600160a060020a038416612d3f5760405160e560020a62461bcd02815260206004820152602160248201527f455243373231413a206d696e7420746f20746865207a65726f2061646472657360448201527f73000000000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b612d4a816000541190565b15612d9a5760405160e560020a62461bcd02815260206004820152601d60248201527f455243373231413a20746f6b656e20616c7265616479206d696e7465640000006044820152606401610cb3565b7f0000000000000000000000000000000000000000000000000000000000000000831115612e335760405160e560020a62461bcd02815260206004820152602260248201527f455243373231413a207175616e7469747920746f206d696e7420746f6f20686960448201527f67680000000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b600160a060020a0384166000908152600460209081526040918290208251808401845290546001608060020a0380821683527001000000000000000000000000000000009091041691810191909152815180830190925280519091908190612e9c908790613dea565b6001608060020a03168152602001858360200151612eba9190613dea565b6001608060020a03908116909152600160a060020a03808816600081815260046020908152604080832087519783015187167001000000000000000000000000000000000297909616969096179094558451808601865291825267ffffffffffffffff428116838601908152888352600390955294812091518254945190951660a060020a02600160e060020a031990941694909216939093179190911790915582905b85811015612fea576040518290600160a060020a038916906000907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef908290a4612fab6000888488612822565b612fca5760405160e560020a62461bcd028152600401610cb390613c97565b81612fd481613b7a565b9250508080612fe290613b7a565b915050612f5e565b50600081905561237a565b600061304a826040518060400160405280602081526020017f5361666545524332303a206c6f772d6c6576656c2063616c6c206661696c656481525085600160a060020a031661338b9092919063ffffffff16565b805190915015610e0c57808060200190518101906130689190613f5d565b610e0c5760405160e560020a62461bcd02815260206004820152602a60248201527f5361666545524332303a204552433230206f7065726174696f6e20646964206e60448201527f6f742073756363656564000000000000000000000000000000000000000000006064820152608401610cb3565b600081815b84518110156131815760008582815181106130ff576130ff613b48565b6020026020010151905080831161314157604080516020810185905290810182905260600160405160208183030381529060405280519060200120925061316e565b60408051602081018390529081018490526060016040516020818303038152906040528051906020012092505b508061317981613b7a565b9150506130e2565b509392505050565b60606000613198836002613d76565b6131a3906002613c09565b67ffffffffffffffff8111156131bb576131bb613641565b6040519080825280601f01601f1916602001820160405280156131e5576020820181803683370190505b5090507f30000000000000000000000000000000000000000000000000000000000000008160008151811061321c5761321c613b48565b6020010190600160f860020a031916908160001a9053507f78000000000000000000000000000000000000000000000000000000000000008160018151811061326757613267613b48565b6020010190600160f860020a031916908160001a905350600061328b846002613d76565b613296906001613c09565b90505b6001811115613339577f303132333435363738396162636465660000000000000000000000000000000085600f16601081106132d7576132d7613b48565b1a7f01000000000000000000000000000000000000000000000000000000000000000282828151811061330c5761330c613b48565b6020010190600160f860020a031916908160001a90535060109094049361333281613e0c565b9050613299565b5083156117a65760405160e560020a62461bcd02815260206004820181905260248201527f537472696e67733a20686578206c656e67746820696e73756666696369656e746044820152606401610cb3565b6060611e8f848460008585843b6133e75760405160e560020a62461bcd02815260206004820152601d60248201527f416464726573733a2063616c6c20746f206e6f6e2d636f6e74726163740000006044820152606401610cb3565b60008086600160a060020a031685876040516134039190613f7a565b60006040518083038185875af1925050503d8060008114613440576040519150601f19603f3d011682016040523d82523d6000602084013e613445565b606091505b5091509150613455828286613460565b979650505050505050565b6060831561346f5750816117a6565b82511561347f5782518084602001fd5b8160405160e560020a62461bcd028152600401610cb391906135b7565b8280546134a890613ad5565b90600052602060002090601f0160209004810192826134ca5760008555613510565b82601f106134e357805160ff1916838001178555613510565b82800160010185558215613510579182015b828111156135105782518255916020019190600101906134f5565b506115bd9291505b808211156115bd5760008155600101613518565b600160e060020a031981168114611de557600080fd5b60006020828403121561355457600080fd5b81356117a68161352c565b60005b8381101561357a578181015183820152602001613562565b838111156119d45750506000910152565b600081518084526135a381602086016020860161355f565b601f01601f19169290920160200192915050565b6020815260006117a6602083018461358b565b6000602082840312156135dc57600080fd5b5035919050565b600160a060020a0381168114611de557600080fd5b6000806040838503121561360b57600080fd5b8235613616816135e3565b946020939093013593505050565b60006020828403121561363657600080fd5b81356117a6816135e3565b60e060020a634e487b7102600052604160045260246000fd5b604051601f8201601f1916810167ffffffffffffffff8111828210171561368357613683613641565b604052919050565b600067ffffffffffffffff8211156136a5576136a5613641565b5060209081020190565b600082601f8301126136c057600080fd5b813560206136d56136d08361368b565b61365a565b828152918102840181019181810190868411156136f157600080fd5b8286015b8481101561370c57803583529183019183016136f5565b509695505050505050565b6000806040838503121561372a57600080fd5b823567ffffffffffffffff8082111561374257600080fd5b818501915085601f83011261375657600080fd5b813560206137666136d08361368b565b8281529181028401810191818101908984111561378257600080fd5b948201945b838610156137a957853561379a816135e3565b82529482019490820190613787565b965050860135925050808211156137bf57600080fd5b506137cc858286016136af565b9150509250929050565b6000806000606084860312156137eb57600080fd5b83356137f6816135e3565b92506020840135613806816135e3565b929592945050506040919091013590565b6000806040838503121561382a57600080fd5b8235613835816135e3565b91506020830135613845816135e3565b809150509250929050565b600080600080600080600080610100898b03121561386d57600080fd5b505086359860208801359850604088013597606081013597506080810135965060a0810135955060c0810135945060e0013592509050565b60008083601f8401126138b757600080fd5b50813567ffffffffffffffff8111156138cf57600080fd5b60208301915083602080830285010111156138e957600080fd5b9250929050565b60008060006040848603121561390557600080fd5b8335613910816135e3565b9250602084013567ffffffffffffffff81111561392c57600080fd5b613938868287016138a5565b9497909650939450505050565b600067ffffffffffffffff83111561395f5761395f613641565b613972601f8401601f191660200161365a565b905082815283838301111561398657600080fd5b828260208301376000602084830101529392505050565b6000602082840312156139af57600080fd5b813567ffffffffffffffff8111156139c657600080fd5b8201601f810184136139d757600080fd5b611e8f84823560208401613945565b8015158114611de557600080fd5b60008060408385031215613a0757600080fd5b8235613a12816135e3565b91506020830135613845816139e6565b60008060008060808587031215613a3857600080fd5b8435613a43816135e3565b93506020850135613a53816135e3565b925060408501359150606085013567ffffffffffffffff811115613a7657600080fd5b8501601f81018713613a8757600080fd5b613a9687823560208401613945565b91505092959194509250565b600080600060408486031215613ab757600080fd5b83359250602084013567ffffffffffffffff81111561392c57600080fd5b600281046001821680613ae957607f821691505b60208210811415613b0d5760e060020a634e487b7102600052602260045260246000fd5b50919050565b6020808252818101527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572604082015260600190565b60e060020a634e487b7102600052603260045260246000fd5b60e060020a634e487b7102600052601160045260246000fd5b6000600019821415613b8e57613b8e613b61565b5060010190565b600082821015613ba757613ba7613b61565b500390565b60208082526026908201527f5061796d656e7453706c69747465723a206163636f756e7420686173206e6f2060408201527f7368617265730000000000000000000000000000000000000000000000000000606082015260800190565b60008219821115613c1c57613c1c613b61565b500190565b6020808252602b908201527f5061796d656e7453706c69747465723a206163636f756e74206973206e6f742060408201527f647565207061796d656e74000000000000000000000000000000000000000000606082015260800190565b600060208284031215613c9057600080fd5b5051919050565b60208082526033908201527f455243373231413a207472616e7366657220746f206e6f6e204552433732315260408201527f6563656976657220696d706c656d656e74657200000000000000000000000000606082015260800190565b60008151613d0681856020860161355f565b9290920192915050565b60008351613d2281846020880161355f565b835190830190613d3681836020880161355f565b01949350505050565b60208082526010908201527f5061757361626c653a2070617573656400000000000000000000000000000000604082015260600190565b6000816000190483118215151615613d9057613d90613b61565b500290565b60e060020a634e487b7102600052601260045260246000fd5b600082613dbd57613dbd613d95565b500490565b60006001608060020a0383811690831681811015613de257613de2613b61565b039392505050565b60006001608060020a03808316818516808303821115613d3657613d36613b61565b600081613e1b57613e1b613b61565b506000190190565b6000600160a060020a03808716835280861660208401525083604083015260806060830152613e55608083018461358b565b9695505050505050565b600060208284031215613e7157600080fd5b81516117a68161352c565b8254600090819060028104600180831680613e9857607f831692505b6020808410821415613ebb5760e060020a634e487b710286526022600452602486fd5b818015613ecf5760018114613ee057613f0d565b60ff19861689528489019650613f0d565b60008b81526020902060005b86811015613f055781548b820152908501908301613eec565b505084890196505b5050505050506117a2613f208286613cf4565b7f2f00000000000000000000000000000000000000000000000000000000000000815260010190565b600082613f5857613f58613d95565b500690565b600060208284031215613f6f57600080fd5b81516117a6816139e6565b60008251613f8c81846020870161355f565b919091019291505056fea264697066735822122038ac16b6d745c2fcbb74ddb282bb60ea5aad5fe860a99b3ab917cd44eaacd2e064736f6c6343000809003300000000000000000000000000000000000000000000000000000000000000e00000000000000000000000000000000000000000000000000000000000000120000000000000000000000000000000000000000000000000000000000000016000000000000000000000000000000000000000000000000000000000000001c07a610e10c860ba28cc8a082a8d850a658b8c9368f163237fe7c0545c6299fadb00000000000000000000000000000000000000000000000000000000000002e0000000000000000000000000000000000000000000000000000000000000032000000000000000000000000000000000000000000000000000000000000000104475636b79436974792049736c616e6400000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000649534c414e440000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000002368747470733a2f2f6e66742e6475636b79636974792e696f2f636f6e7472616374732f00000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000008000000000000000000000000000000000000000000000000008e1bc9bf040000000000000000000000000000000000000000000000000000007fe5cf2bea00000000000000000000000000000000000000000000000000000000000000001388000000000000000000000000000000000000000000000000000000000000000a000000000000000000000000000000000000000000000000000000000000000a0000000000000000000000000000000000000000000000000000000065b2f6000000000000000000000000000000000000000000000000000000000065b24d40000000000000000000000000000000000000000000000000000000000000000a00000000000000000000000000000000000000000000000000000000000000010000000000000000000000004927af9dd5a1257f565d063b85e4d45e3faebffe00000000000000000000000000000000000000000000000000000000000000010000000000000000000000000000000000000000000000000000000000000001

Deployed Bytecode

0x608060405260043610610397576000357c01000000000000000000000000000000000000000000000000000000009004806374721235116101ee578063b88d4fde1161011f578063d79779b2116100bd578063e985e9c51161008c578063e985e9c514610a40578063efef39a114610a89578063f2fde38b14610a9c578063fa156f9a14610abc57600080fd5b8063d79779b2146109cc578063e2ab10ce14610a02578063e2d5ee2d14610a15578063e33b7de314610a2b57600080fd5b8063ce7c2ac2116100f9578063ce7c2ac214610956578063cf9e8e691461098c578063cfc86f7b146109a1578063d7224ba0146109b657600080fd5b8063b88d4fde146108e9578063c4ec2c1614610909578063c87b56dd1461093657600080fd5b8063904be6da1161018c5780639d044ed3116101665780639d044ed31461087e578063a0bcfc7f14610893578063a22cb465146108b3578063b85ef036146108d357600080fd5b8063904be6da1461081d57806395d89b41146108335780639852595c1461084857600080fd5b80638456cb59116101c85780638456cb59146107b55780638b83209b146107ca5780638d859f3e146107ea5780638da5cb5b146107ff57600080fd5b806374721235146107555780637b96a3b2146107755780637cb647591461079557600080fd5b80633a98ef39116102c85780635c975abb1161026657806366cfb1f31161024057806366cfb1f3146106f5578063696fa41e1461070a57806370a0823114610720578063715018a61461074057600080fd5b80635c975abb146106a05780635f0d246a146106bf5780636352211e146106d557600080fd5b806340c10f19116102a257806340c10f191461062d57806342842e0e1461064057806348b75044146106605780634f6ccce71461068057600080fd5b80633a98ef39146105bd5780633f4ba83a146105d2578063406072a9146105e757600080fd5b80631916558711610335578063235b6ea11161030f578063235b6ea11461055157806323b872dd146105675780632f745c59146105875780632fc37ab2146105a757600080fd5b806319165587146105065780631e84c4131461052657806322f4596f1461053b57600080fd5b8063095ea7b311610371578063095ea7b3146104745780630d5fbb72146104965780631687edb5146104d157806318160ddd146104f157600080fd5b806301ffc9a7146103e557806306fdde031461041a578063081812fc1461043c57600080fd5b366103e0577f6ef95f06320e7a25a04a175ca677b7052bdd97131872c2192525a629f51be7703360408051600160a060020a0390921682523460208301520160405180910390a1005b600080fd5b3480156103f157600080fd5b50610405610400366004613542565b610ad2565b60405190151581526020015b60405180910390f35b34801561042657600080fd5b5061042f610ba3565b60405161041191906135b7565b34801561044857600080fd5b5061045c6104573660046135ca565b610c35565b604051600160a060020a039091168152602001610411565b34801561048057600080fd5b5061049461048f3660046135f8565b610cd8565b005b3480156104a257600080fd5b506104c36104b1366004613624565b601a6020526000908152604090205481565b604051908152602001610411565b3480156104dd57600080fd5b506104946104ec366004613717565b610e11565b3480156104fd57600080fd5b506104c3610f87565b34801561051257600080fd5b50610494610521366004613624565b610f9d565b34801561053257600080fd5b506104056110d2565b34801561054757600080fd5b506104c360145481565b34801561055d57600080fd5b506104c360125481565b34801561057357600080fd5b506104946105823660046137d6565b6110ec565b34801561059357600080fd5b506104c36105a23660046135f8565b6110f7565b3480156105b357600080fd5b506104c360115481565b3480156105c957600080fd5b506009546104c3565b3480156105de57600080fd5b5061049461129f565b3480156105f357600080fd5b506104c3610602366004613817565b600160a060020a039182166000908152600f6020908152604080832093909416825291909152205490565b61049461063b3660046135f8565b6112d6565b34801561064c57600080fd5b5061049461065b3660046137d6565b61131a565b34801561066c57600080fd5b5061049461067b366004613817565b611335565b34801561068c57600080fd5b506104c361069b3660046135ca565b61153c565b3480156106ac57600080fd5b5060085460a060020a900460ff16610405565b3480156106cb57600080fd5b506104c360135481565b3480156106e157600080fd5b5061045c6106f03660046135ca565b6115c1565b34801561070157600080fd5b506104c36115d3565b34801561071657600080fd5b506104c360195481565b34801561072c57600080fd5b506104c361073b366004613624565b6115f0565b34801561074c57600080fd5b50610494611696565b34801561076157600080fd5b50610494610770366004613850565b6116cd565b34801561078157600080fd5b506104056107903660046138f0565b611720565b3480156107a157600080fd5b506104946107b03660046135ca565b6117ad565b3480156107c157600080fd5b506104946117df565b3480156107d657600080fd5b5061045c6107e53660046135ca565b611814565b3480156107f657600080fd5b506104c3611844565b34801561080b57600080fd5b50600854600160a060020a031661045c565b34801561082957600080fd5b506104c360165481565b34801561083f57600080fd5b5061042f611861565b34801561085457600080fd5b506104c3610863366004613624565b600160a060020a03166000908152600c602052604090205490565b34801561088a57600080fd5b50610405611870565b34801561089f57600080fd5b506104946108ae36600461399d565b611896565b3480156108bf57600080fd5b506104946108ce3660046139f4565b6118d6565b3480156108df57600080fd5b506104c360175481565b3480156108f557600080fd5b50610494610904366004613a22565b61199e565b34801561091557600080fd5b506104c3610924366004613624565b601b6020526000908152604090205481565b34801561094257600080fd5b5061042f6109513660046135ca565b6119da565b34801561096257600080fd5b506104c3610971366004613624565b600160a060020a03166000908152600b602052604090205490565b34801561099857600080fd5b506014546104c3565b3480156109ad57600080fd5b5061042f611ab7565b3480156109c257600080fd5b506104c360075481565b3480156109d857600080fd5b506104c36109e7366004613624565b600160a060020a03166000908152600e602052604090205490565b610494610a10366004613aa2565b611b45565b348015610a2157600080fd5b506104c360155481565b348015610a3757600080fd5b50600a546104c3565b348015610a4c57600080fd5b50610405610a5b366004613817565b600160a060020a03918216600090815260066020908152604080832093909416825291909152205460ff1690565b610494610a973660046135ca565b611c5f565b348015610aa857600080fd5b50610494610ab7366004613624565b611d30565b348015610ac857600080fd5b506104c360185481565b6000600160e060020a031982167f80ac58cd000000000000000000000000000000000000000000000000000000001480610b355750600160e060020a031982167f5b5e139f00000000000000000000000000000000000000000000000000000000145b80610b695750600160e060020a031982167f780e9d6300000000000000000000000000000000000000000000000000000000145b80610b9d57507f01ffc9a700000000000000000000000000000000000000000000000000000000600160e060020a03198316145b92915050565b606060018054610bb290613ad5565b80601f0160208091040260200160405190810160405280929190818152602001828054610bde90613ad5565b8015610c2b5780601f10610c0057610100808354040283529160200191610c2b565b820191906000526020600020905b815481529060010190602001808311610c0e57829003601f168201915b5050505050905090565b6000610c42826000541190565b610cbc5760405160e560020a62461bcd02815260206004820152602d60248201527f455243373231413a20617070726f76656420717565727920666f72206e6f6e6560448201527f78697374656e7420746f6b656e0000000000000000000000000000000000000060648201526084015b60405180910390fd5b50600090815260056020526040902054600160a060020a031690565b6000610ce3826115c1565b905080600160a060020a031683600160a060020a03161415610d705760405160e560020a62461bcd02815260206004820152602260248201527f455243373231413a20617070726f76616c20746f2063757272656e74206f776e60448201527f65720000000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b33600160a060020a0382161480610d8c5750610d8c8133610a5b565b610e015760405160e560020a62461bcd02815260206004820152603960248201527f455243373231413a20617070726f76652063616c6c6572206973206e6f74206f60448201527f776e6572206e6f7220617070726f76656420666f7220616c6c000000000000006064820152608401610cb3565b610e0c838383611de8565b505050565b600854600160a060020a03163314610e3e5760405160e560020a62461bcd028152600401610cb390613b13565b8051825114610eb85760405160e560020a62461bcd02815260206004820152602b60248201527f77686974656c69737420616e64206d617850657241646472657373206c656e6760448201527f7468206d69736d617463680000000000000000000000000000000000000000006064820152608401610cb3565b6000825111610f0c5760405160e560020a62461bcd02815260206004820152600c60248201527f4e6f2077686974656c69737400000000000000000000000000000000000000006044820152606401610cb3565b60005b8251811015610e0c57818181518110610f2a57610f2a613b48565b6020026020010151601b6000858481518110610f4857610f48613b48565b6020026020010151600160a060020a0316600160a060020a03168152602001908152602001600020819055508080610f7f90613b7a565b915050610f0f565b60006001600054610f989190613b95565b905090565b600160a060020a0381166000908152600b6020526040902054610fd55760405160e560020a62461bcd028152600401610cb390613bac565b6000610fe0600a5490565b610feb903031613c09565b90506000611018838361101386600160a060020a03166000908152600c602052604090205490565b611e51565b90508061103a5760405160e560020a62461bcd028152600401610cb390613c21565b600160a060020a0383166000908152600c602052604081208054839290611062908490613c09565b9250508190555080600a600082825461107b9190613c09565b9091555061108b90508382611e97565b60408051600160a060020a0385168152602081018390527fdf20fd1e76bc69d672e4814fafb2c449bba3a5369d8359adf9e05e6fde87b056910160405180910390a1505050565b6000601754600014158015610f9857504260175410905090565b610e0c838383611fb7565b6000611102836115f0565b82106111795760405160e560020a62461bcd02815260206004820152602260248201527f455243373231413a206f776e657220696e646578206f7574206f6620626f756e60448201527f64730000000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b6000611183610f87565b905060008060005b8381101561122d57600081815260036020908152604091829020825180840190935254600160a060020a03811680845260a060020a90910467ffffffffffffffff1691830191909152156111de57805192505b87600160a060020a031683600160a060020a0316141561121a578684141561120c57509350610b9d92505050565b8361121681613b7a565b9450505b508061122581613b7a565b91505061118b565b5060405160e560020a62461bcd02815260206004820152602e60248201527f455243373231413a20756e61626c6520746f2067657420746f6b656e206f662060448201527f6f776e657220627920696e6465780000000000000000000000000000000000006064820152608401610cb3565b600854600160a060020a031633146112cc5760405160e560020a62461bcd028152600401610cb390613b13565b6112d4612382565b565b600854600160a060020a031633146113035760405160e560020a62461bcd028152600401610cb390613b13565b61130c8161243c565b61131682826124c9565b5050565b610e0c8383836040518060200160405280600081525061199e565b600160a060020a0381166000908152600b602052604090205461136d5760405160e560020a62461bcd028152600401610cb390613bac565b600160a060020a0382166000908152600e60205260408120546040517f70a08231000000000000000000000000000000000000000000000000000000008152306004820152600160a060020a038516906370a082319060240160206040518083038186803b1580156113de57600080fd5b505afa1580156113f2573d6000803e3d6000fd5b505050506040513d601f19601f820116820180604052508101906114169190613c7e565b6114209190613c09565b9050600061145983836110138787600160a060020a039182166000908152600f6020908152604080832093909416825291909152205490565b90508061147b5760405160e560020a62461bcd028152600401610cb390613c21565b600160a060020a038085166000908152600f60209081526040808320938716835292905290812080548392906114b2908490613c09565b9091555050600160a060020a0384166000908152600e6020526040812080548392906114df908490613c09565b909155506114f090508484836124e3565b60408051600160a060020a038581168252602082018490528616917f3be5b7a71e84ed12875d241991c70855ac5817d847039e17a9d895c1ceb0f18a910160405180910390a250505050565b6000611546610f87565b82106115bd5760405160e560020a62461bcd02815260206004820152602360248201527f455243373231413a20676c6f62616c20696e646578206f7574206f6620626f7560448201527f6e647300000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b5090565b60006115cc82612563565b5192915050565b60006115dd611870565b156115e9575060165490565b5060155490565b6000600160a060020a0382166116715760405160e560020a62461bcd02815260206004820152602b60248201527f455243373231413a2062616c616e636520717565727920666f7220746865207a60448201527f65726f20616464726573730000000000000000000000000000000000000000006064820152608401610cb3565b50600160a060020a03166000908152600460205260409020546001608060020a031690565b600854600160a060020a031633146116c35760405160e560020a62461bcd028152600401610cb390613b13565b6112d46000612734565b600854600160a060020a031633146116fa5760405160e560020a62461bcd028152600401610cb390613b13565b601797909755601895909555601593909355601691909155601255601355601155601955565b60006040516c01000000000000000000000000600160a060020a0386160260208201526000906034016040516020818303038152906040528051906020012090506117a2848480806020026020016040519081016040528093929190818152602001838360200280828437600092019190915250506011549150849050612793565b9150505b9392505050565b600854600160a060020a031633146117da5760405160e560020a62461bcd028152600401610cb390613b13565b601155565b600854600160a060020a0316331461180c5760405160e560020a62461bcd028152600401610cb390613b13565b6112d46127a9565b6000600d828154811061182957611829613b48565b600091825260209091200154600160a060020a031692915050565b600061184e611870565b1561185a575060135490565b5060125490565b606060028054610bb290613ad5565b6000601854600014158015611886575042601854105b8015610f98575050601754421090565b600854600160a060020a031633146118c35760405160e560020a62461bcd028152600401610cb390613b13565b805161131690601090602084019061349c565b600160a060020a0382163314156119325760405160e560020a62461bcd02815260206004820152601a60248201527f455243373231413a20617070726f766520746f2063616c6c65720000000000006044820152606401610cb3565b336000818152600660209081526040808320600160a060020a03871680855290835292819020805460ff191686151590811790915590519081529192917f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31910160405180910390a35050565b6119a9848484611fb7565b6119b584848484612822565b6119d45760405160e560020a62461bcd028152600401610cb390613c97565b50505050565b60606119e7826000541190565b611a5c5760405160e560020a62461bcd02815260206004820152602f60248201527f4552433732314d657461646174613a2055524920717565727920666f72206e6f60448201527f6e6578697374656e7420746f6b656e00000000000000000000000000000000006064820152608401610cb3565b6000611a66612964565b90506000815111611a8657604051806020016040528060008152506117a6565b80611a9084612998565b604051602001611aa1929190613d10565b6040516020818303038152906040529392505050565b60108054611ac490613ad5565b80601f0160208091040260200160405190810160405280929190818152602001828054611af090613ad5565b8015611b3d5780601f10611b1257610100808354040283529160200191611b3d565b820191906000526020600020905b815481529060010190602001808311611b2057829003601f168201915b505050505081565b60085460a060020a900460ff1615611b725760405160e560020a62461bcd028152600401610cb390613d3f565b336000818152601b6020526040902054611b8e91908590612ad1565b611b96611870565b8015611ba85750611ba8338383611720565b611c1d5760405160e560020a62461bcd02815260206004820152602360248201527f424153455f434f4c4c454354494f4e2f43414e4e4f545f4d494e545f5052455360448201527f414c4500000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b611c2983601354612c0c565b60135460405184919033907f38bd02858ca92987ff585a4c06998aea8187e96864df1eaf349dec3cfddc0fbb90600090a4505050565b60085460a060020a900460ff1615611c8c5760405160e560020a62461bcd028152600401610cb390613d3f565b611c993382601554612ad1565b611ca16110d2565b611cf05760405160e560020a62461bcd02815260206004820152601b60248201527f424153455f434f4c4c454354494f4e2f43414e4e4f545f4d494e5400000000006044820152606401610cb3565b611cfc81601254612c0c565b60125460405182919033907f12cb4648cf3058b17ceeb33e579f8b0bc269fe0843f3900b8e24b6c54871703c90600090a450565b600854600160a060020a03163314611d5d5760405160e560020a62461bcd028152600401610cb390613b13565b600160a060020a038116611ddc5760405160e560020a62461bcd02815260206004820152602660248201527f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160448201527f64647265737300000000000000000000000000000000000000000000000000006064820152608401610cb3565b611de581612734565b50565b600082815260056020526040808220805473ffffffffffffffffffffffffffffffffffffffff1916600160a060020a0387811691821790925591518593918516917f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92591a4505050565b600954600160a060020a0384166000908152600b602052604081205490918391611e7b9086613d76565b611e859190613dae565b611e8f9190613b95565b949350505050565b3031811115611eeb5760405160e560020a62461bcd02815260206004820152601d60248201527f416464726573733a20696e73756666696369656e742062616c616e63650000006044820152606401610cb3565b600082600160a060020a03168260405160006040518083038185875af1925050503d8060008114611f38576040519150601f19603f3d011682016040523d82523d6000602084013e611f3d565b606091505b5050905080610e0c5760405160e560020a62461bcd02815260206004820152603a60248201527f416464726573733a20756e61626c6520746f2073656e642076616c75652c207260448201527f6563697069656e74206d617920686176652072657665727465640000000000006064820152608401610cb3565b6000611fc282612563565b8051909150600090600160a060020a031633600160a060020a03161480611ff9575033611fee84610c35565b600160a060020a0316145b8061200b5750815161200b9033610a5b565b9050806120835760405160e560020a62461bcd02815260206004820152603260248201527f455243373231413a207472616e736665722063616c6c6572206973206e6f742060448201527f6f776e6572206e6f7220617070726f76656400000000000000000000000000006064820152608401610cb3565b84600160a060020a03168260000151600160a060020a0316146121115760405160e560020a62461bcd02815260206004820152602660248201527f455243373231413a207472616e736665722066726f6d20696e636f727265637460448201527f206f776e657200000000000000000000000000000000000000000000000000006064820152608401610cb3565b600160a060020a0384166121905760405160e560020a62461bcd02815260206004820152602560248201527f455243373231413a207472616e7366657220746f20746865207a65726f20616460448201527f64726573730000000000000000000000000000000000000000000000000000006064820152608401610cb3565b6121a06000848460000151611de8565b600160a060020a03851660009081526004602052604081208054600192906121d29084906001608060020a0316613dc2565b82546101009290920a6001608060020a03818102199093169183160217909155600160a060020a0386166000908152600460205260408120805460019450909261221e91859116613dea565b82546001608060020a039182166101009390930a928302919092021990911617905550604080518082018252600160a060020a03808716825267ffffffffffffffff42811660208085019182526000898152600390915294852093518454915190921660a060020a02600160e060020a031990911691909216171790556122a6846001613c09565b600081815260036020526040902054909150600160a060020a0316612338576122d0816000541190565b15612338576040805180820182528451600160a060020a03908116825260208087015167ffffffffffffffff908116828501908152600087815260039093529490912092518354945190911660a060020a02600160e060020a03199094169116179190911790555b8385600160a060020a031687600160a060020a03167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a45b505050505050565b60085460a060020a900460ff166123de5760405160e560020a62461bcd02815260206004820152601460248201527f5061757361626c653a206e6f74207061757365640000000000000000000000006044820152606401610cb3565b6008805474ff0000000000000000000000000000000000000000191690557f5db9ee0a495bf2e6ff9c91a7834c1ba4fdd244a5e8aa4e537bd38aeae4b073aa335b604051600160a060020a03909116815260200160405180910390a1565b60145481612448610f87565b6124529190613c09565b1115611de55760405160e560020a62461bcd02815260206004820152602260248201527f424153455f434f4c4c454354494f4e2f455843454544535f4d41585f5355505060448201527f4c590000000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b611316828260405180602001604052806000815250612cbd565b60408051600160a060020a038416602482015260448082018490528251808303909101815260649091019091526020810180517bffffffffffffffffffffffffffffffffffffffffffffffffffffffff167fa9059cbb00000000000000000000000000000000000000000000000000000000179052610e0c908490612ff5565b6040805180820190915260008082526020820152612582826000541190565b6125f75760405160e560020a62461bcd02815260206004820152602a60248201527f455243373231413a206f776e657220717565727920666f72206e6f6e6578697360448201527f74656e7420746f6b656e000000000000000000000000000000000000000000006064820152608401610cb3565b60007f000000000000000000000000000000000000000000000000000000000000138883106126585761264a7f000000000000000000000000000000000000000000000000000000000000138884613b95565b612655906001613c09565b90505b825b8181106126c257600081815260036020908152604091829020825180840190935254600160a060020a03811680845260a060020a90910467ffffffffffffffff1691830191909152156126af57949350505050565b50806126ba81613e0c565b91505061265a565b5060405160e560020a62461bcd02815260206004820152602f60248201527f455243373231413a20756e61626c6520746f2064657465726d696e652074686560448201527f206f776e6572206f6620746f6b656e00000000000000000000000000000000006064820152608401610cb3565b60088054600160a060020a0383811673ffffffffffffffffffffffffffffffffffffffff19831681179093556040519116919082907f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e090600090a35050565b6000826127a085846130dd565b14949350505050565b60085460a060020a900460ff16156127d65760405160e560020a62461bcd028152600401610cb390613d3f565b6008805474ff0000000000000000000000000000000000000000191660a060020a1790557f62e78cea01bee320cd4e420270b5ea74000d11b0c9f74754ebdbfc544b05a25861241f3390565b6000600160a060020a0384163b15612959576040517f150b7a02000000000000000000000000000000000000000000000000000000008152600160a060020a0385169063150b7a029061287f903390899088908890600401613e23565b602060405180830381600087803b15801561289957600080fd5b505af19250505080156128c9575060408051601f3d908101601f191682019092526128c691810190613e5f565b60015b612926573d8080156128f7576040519150601f19603f3d011682016040523d82523d6000602084013e6128fc565b606091505b50805161291e5760405160e560020a62461bcd028152600401610cb390613c97565b805181602001fd5b600160e060020a0319167f150b7a0200000000000000000000000000000000000000000000000000000000149050611e8f565b506001949350505050565b60606010612973306014613189565b604051602001612984929190613e7c565b604051602081830303815290604052905090565b6060816129d857505060408051808201909152600181527f3000000000000000000000000000000000000000000000000000000000000000602082015290565b8160005b8115612a0257806129ec81613b7a565b91506129fb9050600a83613dae565b91506129dc565b60008167ffffffffffffffff811115612a1d57612a1d613641565b6040519080825280601f01601f191660200182016040528015612a47576020820181803683370190505b5090505b8415611e8f57612a5c600183613b95565b9150612a69600a86613f49565b612a74906030613c09565b7f010000000000000000000000000000000000000000000000000000000000000002818381518110612aa857612aa8613b48565b6020010190600160f860020a031916908160001a905350612aca600a86613dae565b9450612a4b565b612ada8261243c565b60195415801590612aed57506019548211155b612b625760405160e560020a62461bcd02815260206004820152602b60248201527f424153455f434f4c4c454354494f4e2f455843454544535f4d41585f5045525f60448201527f5452414e53414354494f4e0000000000000000000000000000000000000000006064820152608401610cb3565b600160a060020a0383166000908152601a6020526040812054612b86908490613c09565b90508115801590612b975750818111155b6119d45760405160e560020a62461bcd02815260206004820152602960248201527f424153455f434f4c4c454354494f4e2f455843454544535f494e44495649445560448201527f414c5f535550504c5900000000000000000000000000000000000000000000006064820152608401610cb3565b34612c178383613d76565b1115612c8e5760405160e560020a62461bcd02815260206004820152602760248201527f424153455f434f4c4c454354494f4e2f494e53554646494349454e545f45544860448201527f5f414d4f554e54000000000000000000000000000000000000000000000000006064820152608401610cb3565b336000908152601a602052604081208054849290612cad908490613c09565b90915550611316905033836124c9565b600054600160a060020a038416612d3f5760405160e560020a62461bcd02815260206004820152602160248201527f455243373231413a206d696e7420746f20746865207a65726f2061646472657360448201527f73000000000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b612d4a816000541190565b15612d9a5760405160e560020a62461bcd02815260206004820152601d60248201527f455243373231413a20746f6b656e20616c7265616479206d696e7465640000006044820152606401610cb3565b7f0000000000000000000000000000000000000000000000000000000000001388831115612e335760405160e560020a62461bcd02815260206004820152602260248201527f455243373231413a207175616e7469747920746f206d696e7420746f6f20686960448201527f67680000000000000000000000000000000000000000000000000000000000006064820152608401610cb3565b600160a060020a0384166000908152600460209081526040918290208251808401845290546001608060020a0380821683527001000000000000000000000000000000009091041691810191909152815180830190925280519091908190612e9c908790613dea565b6001608060020a03168152602001858360200151612eba9190613dea565b6001608060020a03908116909152600160a060020a03808816600081815260046020908152604080832087519783015187167001000000000000000000000000000000000297909616969096179094558451808601865291825267ffffffffffffffff428116838601908152888352600390955294812091518254945190951660a060020a02600160e060020a031990941694909216939093179190911790915582905b85811015612fea576040518290600160a060020a038916906000907fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef908290a4612fab6000888488612822565b612fca5760405160e560020a62461bcd028152600401610cb390613c97565b81612fd481613b7a565b9250508080612fe290613b7a565b915050612f5e565b50600081905561237a565b600061304a826040518060400160405280602081526020017f5361666545524332303a206c6f772d6c6576656c2063616c6c206661696c656481525085600160a060020a031661338b9092919063ffffffff16565b805190915015610e0c57808060200190518101906130689190613f5d565b610e0c5760405160e560020a62461bcd02815260206004820152602a60248201527f5361666545524332303a204552433230206f7065726174696f6e20646964206e60448201527f6f742073756363656564000000000000000000000000000000000000000000006064820152608401610cb3565b600081815b84518110156131815760008582815181106130ff576130ff613b48565b6020026020010151905080831161314157604080516020810185905290810182905260600160405160208183030381529060405280519060200120925061316e565b60408051602081018390529081018490526060016040516020818303038152906040528051906020012092505b508061317981613b7a565b9150506130e2565b509392505050565b60606000613198836002613d76565b6131a3906002613c09565b67ffffffffffffffff8111156131bb576131bb613641565b6040519080825280601f01601f1916602001820160405280156131e5576020820181803683370190505b5090507f30000000000000000000000000000000000000000000000000000000000000008160008151811061321c5761321c613b48565b6020010190600160f860020a031916908160001a9053507f78000000000000000000000000000000000000000000000000000000000000008160018151811061326757613267613b48565b6020010190600160f860020a031916908160001a905350600061328b846002613d76565b613296906001613c09565b90505b6001811115613339577f303132333435363738396162636465660000000000000000000000000000000085600f16601081106132d7576132d7613b48565b1a7f01000000000000000000000000000000000000000000000000000000000000000282828151811061330c5761330c613b48565b6020010190600160f860020a031916908160001a90535060109094049361333281613e0c565b9050613299565b5083156117a65760405160e560020a62461bcd02815260206004820181905260248201527f537472696e67733a20686578206c656e67746820696e73756666696369656e746044820152606401610cb3565b6060611e8f848460008585843b6133e75760405160e560020a62461bcd02815260206004820152601d60248201527f416464726573733a2063616c6c20746f206e6f6e2d636f6e74726163740000006044820152606401610cb3565b60008086600160a060020a031685876040516134039190613f7a565b60006040518083038185875af1925050503d8060008114613440576040519150601f19603f3d011682016040523d82523d6000602084013e613445565b606091505b5091509150613455828286613460565b979650505050505050565b6060831561346f5750816117a6565b82511561347f5782518084602001fd5b8160405160e560020a62461bcd028152600401610cb391906135b7565b8280546134a890613ad5565b90600052602060002090601f0160209004810192826134ca5760008555613510565b82601f106134e357805160ff1916838001178555613510565b82800160010185558215613510579182015b828111156135105782518255916020019190600101906134f5565b506115bd9291505b808211156115bd5760008155600101613518565b600160e060020a031981168114611de557600080fd5b60006020828403121561355457600080fd5b81356117a68161352c565b60005b8381101561357a578181015183820152602001613562565b838111156119d45750506000910152565b600081518084526135a381602086016020860161355f565b601f01601f19169290920160200192915050565b6020815260006117a6602083018461358b565b6000602082840312156135dc57600080fd5b5035919050565b600160a060020a0381168114611de557600080fd5b6000806040838503121561360b57600080fd5b8235613616816135e3565b946020939093013593505050565b60006020828403121561363657600080fd5b81356117a6816135e3565b60e060020a634e487b7102600052604160045260246000fd5b604051601f8201601f1916810167ffffffffffffffff8111828210171561368357613683613641565b604052919050565b600067ffffffffffffffff8211156136a5576136a5613641565b5060209081020190565b600082601f8301126136c057600080fd5b813560206136d56136d08361368b565b61365a565b828152918102840181019181810190868411156136f157600080fd5b8286015b8481101561370c57803583529183019183016136f5565b509695505050505050565b6000806040838503121561372a57600080fd5b823567ffffffffffffffff8082111561374257600080fd5b818501915085601f83011261375657600080fd5b813560206137666136d08361368b565b8281529181028401810191818101908984111561378257600080fd5b948201945b838610156137a957853561379a816135e3565b82529482019490820190613787565b965050860135925050808211156137bf57600080fd5b506137cc858286016136af565b9150509250929050565b6000806000606084860312156137eb57600080fd5b83356137f6816135e3565b92506020840135613806816135e3565b929592945050506040919091013590565b6000806040838503121561382a57600080fd5b8235613835816135e3565b91506020830135613845816135e3565b809150509250929050565b600080600080600080600080610100898b03121561386d57600080fd5b505086359860208801359850604088013597606081013597506080810135965060a0810135955060c0810135945060e0013592509050565b60008083601f8401126138b757600080fd5b50813567ffffffffffffffff8111156138cf57600080fd5b60208301915083602080830285010111156138e957600080fd5b9250929050565b60008060006040848603121561390557600080fd5b8335613910816135e3565b9250602084013567ffffffffffffffff81111561392c57600080fd5b613938868287016138a5565b9497909650939450505050565b600067ffffffffffffffff83111561395f5761395f613641565b613972601f8401601f191660200161365a565b905082815283838301111561398657600080fd5b828260208301376000602084830101529392505050565b6000602082840312156139af57600080fd5b813567ffffffffffffffff8111156139c657600080fd5b8201601f810184136139d757600080fd5b611e8f84823560208401613945565b8015158114611de557600080fd5b60008060408385031215613a0757600080fd5b8235613a12816135e3565b91506020830135613845816139e6565b60008060008060808587031215613a3857600080fd5b8435613a43816135e3565b93506020850135613a53816135e3565b925060408501359150606085013567ffffffffffffffff811115613a7657600080fd5b8501601f81018713613a8757600080fd5b613a9687823560208401613945565b91505092959194509250565b600080600060408486031215613ab757600080fd5b83359250602084013567ffffffffffffffff81111561392c57600080fd5b600281046001821680613ae957607f821691505b60208210811415613b0d5760e060020a634e487b7102600052602260045260246000fd5b50919050565b6020808252818101527f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572604082015260600190565b60e060020a634e487b7102600052603260045260246000fd5b60e060020a634e487b7102600052601160045260246000fd5b6000600019821415613b8e57613b8e613b61565b5060010190565b600082821015613ba757613ba7613b61565b500390565b60208082526026908201527f5061796d656e7453706c69747465723a206163636f756e7420686173206e6f2060408201527f7368617265730000000000000000000000000000000000000000000000000000606082015260800190565b60008219821115613c1c57613c1c613b61565b500190565b6020808252602b908201527f5061796d656e7453706c69747465723a206163636f756e74206973206e6f742060408201527f647565207061796d656e74000000000000000000000000000000000000000000606082015260800190565b600060208284031215613c9057600080fd5b5051919050565b60208082526033908201527f455243373231413a207472616e7366657220746f206e6f6e204552433732315260408201527f6563656976657220696d706c656d656e74657200000000000000000000000000606082015260800190565b60008151613d0681856020860161355f565b9290920192915050565b60008351613d2281846020880161355f565b835190830190613d3681836020880161355f565b01949350505050565b60208082526010908201527f5061757361626c653a2070617573656400000000000000000000000000000000604082015260600190565b6000816000190483118215151615613d9057613d90613b61565b500290565b60e060020a634e487b7102600052601260045260246000fd5b600082613dbd57613dbd613d95565b500490565b60006001608060020a0383811690831681811015613de257613de2613b61565b039392505050565b60006001608060020a03808316818516808303821115613d3657613d36613b61565b600081613e1b57613e1b613b61565b506000190190565b6000600160a060020a03808716835280861660208401525083604083015260806060830152613e55608083018461358b565b9695505050505050565b600060208284031215613e7157600080fd5b81516117a68161352c565b8254600090819060028104600180831680613e9857607f831692505b6020808410821415613ebb5760e060020a634e487b710286526022600452602486fd5b818015613ecf5760018114613ee057613f0d565b60ff19861689528489019650613f0d565b60008b81526020902060005b86811015613f055781548b820152908501908301613eec565b505084890196505b5050505050506117a2613f208286613cf4565b7f2f00000000000000000000000000000000000000000000000000000000000000815260010190565b600082613f5857613f58613d95565b500690565b600060208284031215613f6f57600080fd5b81516117a6816139e6565b60008251613f8c81846020870161355f565b919091019291505056fea264697066735822122038ac16b6d745c2fcbb74ddb282bb60ea5aad5fe860a99b3ab917cd44eaacd2e064736f6c63430008090033

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

00000000000000000000000000000000000000000000000000000000000000e00000000000000000000000000000000000000000000000000000000000000120000000000000000000000000000000000000000000000000000000000000016000000000000000000000000000000000000000000000000000000000000001c07a610e10c860ba28cc8a082a8d850a658b8c9368f163237fe7c0545c6299fadb00000000000000000000000000000000000000000000000000000000000002e0000000000000000000000000000000000000000000000000000000000000032000000000000000000000000000000000000000000000000000000000000000104475636b79436974792049736c616e6400000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000649534c414e440000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000002368747470733a2f2f6e66742e6475636b79636974792e696f2f636f6e7472616374732f00000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000000008000000000000000000000000000000000000000000000000008e1bc9bf040000000000000000000000000000000000000000000000000000007fe5cf2bea00000000000000000000000000000000000000000000000000000000000000001388000000000000000000000000000000000000000000000000000000000000000a000000000000000000000000000000000000000000000000000000000000000a0000000000000000000000000000000000000000000000000000000065b2f6000000000000000000000000000000000000000000000000000000000065b24d40000000000000000000000000000000000000000000000000000000000000000a00000000000000000000000000000000000000000000000000000000000000010000000000000000000000004927af9dd5a1257f565d063b85e4d45e3faebffe00000000000000000000000000000000000000000000000000000000000000010000000000000000000000000000000000000000000000000000000000000001

-----Decoded View---------------
Arg [0] : name (string): DuckyCity Island
Arg [1] : symbol (string): ISLAND
Arg [2] : baseTokenURI (string): https://nft.duckycity.io/contracts/
Arg [3] : numericValues (uint256[]): 40000000000000000,36000000000000000,5000,10,10,1706227200,1706184000,10
Arg [4] : merkleRoot (bytes32): 0x7a610e10c860ba28cc8a082a8d850a658b8c9368f163237fe7c0545c6299fadb
Arg [5] : payees (address[]): 0x4927aF9dD5A1257F565D063b85e4D45E3FaEBfFe
Arg [6] : shares (uint256[]): 1

-----Encoded View---------------
27 Constructor Arguments found :
Arg [0] : 00000000000000000000000000000000000000000000000000000000000000e0
Arg [1] : 0000000000000000000000000000000000000000000000000000000000000120
Arg [2] : 0000000000000000000000000000000000000000000000000000000000000160
Arg [3] : 00000000000000000000000000000000000000000000000000000000000001c0
Arg [4] : 7a610e10c860ba28cc8a082a8d850a658b8c9368f163237fe7c0545c6299fadb
Arg [5] : 00000000000000000000000000000000000000000000000000000000000002e0
Arg [6] : 0000000000000000000000000000000000000000000000000000000000000320
Arg [7] : 0000000000000000000000000000000000000000000000000000000000000010
Arg [8] : 4475636b79436974792049736c616e6400000000000000000000000000000000
Arg [9] : 0000000000000000000000000000000000000000000000000000000000000006
Arg [10] : 49534c414e440000000000000000000000000000000000000000000000000000
Arg [11] : 0000000000000000000000000000000000000000000000000000000000000023
Arg [12] : 68747470733a2f2f6e66742e6475636b79636974792e696f2f636f6e74726163
Arg [13] : 74732f0000000000000000000000000000000000000000000000000000000000
Arg [14] : 0000000000000000000000000000000000000000000000000000000000000008
Arg [15] : 000000000000000000000000000000000000000000000000008e1bc9bf040000
Arg [16] : 000000000000000000000000000000000000000000000000007fe5cf2bea0000
Arg [17] : 0000000000000000000000000000000000000000000000000000000000001388
Arg [18] : 000000000000000000000000000000000000000000000000000000000000000a
Arg [19] : 000000000000000000000000000000000000000000000000000000000000000a
Arg [20] : 0000000000000000000000000000000000000000000000000000000065b2f600
Arg [21] : 0000000000000000000000000000000000000000000000000000000065b24d40
Arg [22] : 000000000000000000000000000000000000000000000000000000000000000a
Arg [23] : 0000000000000000000000000000000000000000000000000000000000000001
Arg [24] : 0000000000000000000000004927af9dd5a1257f565d063b85e4d45e3faebffe
Arg [25] : 0000000000000000000000000000000000000000000000000000000000000001
Arg [26] : 0000000000000000000000000000000000000000000000000000000000000001


Deployed Bytecode Sourcemap

207:5749:2:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;3284:40:14;736:10:1;3284:40:14;;;-1:-1:-1;;;;;206:55:17;;;188:74;;3314:9:14;293:2:17;278:18;;271:34;161:18;3284:40:14;;;;;;;207:5749:2;;;;;3616:370:4;;;;;;;;;;-1:-1:-1;3616:370:4;;;;;:::i;:::-;;:::i;:::-;;;913:14:17;;906:22;888:41;;876:2;861:18;3616:370:4;;;;;;;;5342:94;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;6867:204::-;;;;;;;;;;-1:-1:-1;6867:204:4;;;;;:::i;:::-;;:::i;:::-;;;-1:-1:-1;;;;;2062:55:17;;;2044:74;;2032:2;2017:18;6867:204:4;1898:226:17;6430:379:4;;;;;;;;;;-1:-1:-1;6430:379:4;;;;;:::i;:::-;;:::i;:::-;;618:45:2;;;;;;;;;;-1:-1:-1;618:45:2;;;;;:::i;:::-;;;;;;;;;;;;;;;;;3006:25:17;;;2994:2;2979:18;618:45:2;2860:177:17;1612:417:2;;;;;;;;;;-1:-1:-1;1612:417:2;;;;;:::i;:::-;;:::i;2176:98:4:-;;;;;;;;;;;;;:::i;5070:566:14:-;;;;;;;;;;-1:-1:-1;5070:566:14;;;;;:::i;:::-;;:::i;4774:136:2:-;;;;;;;;;;;;;:::i;410:25::-;;;;;;;;;;;;;;;;351:21;;;;;;;;;;;;;;;;7717:142:4;;;;;;;;;;-1:-1:-1;7717:142:4;;;;;:::i;:::-;;:::i;2808:744::-;;;;;;;;;;-1:-1:-1;2808:744:4;;;;;:::i;:::-;;:::i;318:26:2:-;;;;;;;;;;;;;;;;3415:91:14;;;;;;;;;;-1:-1:-1;3486:12:14;;3415:91;;5892:61:2;;;;;;;;;;;;;:::i;4544:135:14:-;;;;;;;;;;-1:-1:-1;4544:135:14;;;;;:::i;:::-;-1:-1:-1;;;;;4641:21:14;;;4614:7;4641:21;;;:14;:21;;;;;;;;:30;;;;;;;;;;;;;4544:135;3079:137:2;;;;;;:::i;:::-;;:::i;7922:157:4:-;;;;;;;;;;-1:-1:-1;7922:157:4;;;;;:::i;:::-;;:::i;5904:641:14:-;;;;;;;;;;-1:-1:-1;5904:641:14;;;;;:::i;:::-;;:::i;2343:177:4:-;;;;;;;;;;-1:-1:-1;2343:177:4;;;;;:::i;:::-;;:::i;1130:86:13:-;;;;;;;;;;-1:-1:-1;1201:7:13;;-1:-1:-1;;;1201:7:13;;;;1130:86;;377:28:2;;;;;;;;;;;;;;;;5165:118:4;;;;;;;;;;-1:-1:-1;5165:118:4;;;;;:::i;:::-;;:::i;5645:178:2:-;;;;;;;;;;;;;:::i;582:31::-;;;;;;;;;;;;;;;;4042:211:4;;;;;;;;;;-1:-1:-1;4042:211:4;;;;;:::i;:::-;;:::i;1714:103:12:-;;;;;;;;;;;;;:::i;2035:566:2:-;;;;;;;;;;-1:-1:-1;2035:566:2;;;;;:::i;:::-;;:::i;5090:310::-;;;;;;;;;;-1:-1:-1;5090:310:2;;;;;:::i;:::-;;:::i;2721:99::-;;;;;;;;;;-1:-1:-1;2721:99:2;;;;;:::i;:::-;;:::i;5829:57::-;;;;;;;;;;;;;:::i;4770:100:14:-;;;;;;;;;;-1:-1:-1;4770:100:14;;;;;:::i;:::-;;:::i;5498:141:2:-;;;;;;;;;;;;;:::i;1063:87:12:-;;;;;;;;;;-1:-1:-1;1136:6:12;;-1:-1:-1;;;;;1136:6:12;1063:87;;474:36:2;;;;;;;;;;;;;;;;5497:98:4;;;;;;;;;;;;;:::i;4266:109:14:-;;;;;;;;;;-1:-1:-1;4266:109:14;;;;;:::i;:::-;-1:-1:-1;;;;;4349:18:14;4322:7;4349:18;;;:9;:18;;;;;;;4266:109;4916:168:2;;;;;;;;;;;;;:::i;2607:108::-;;;;;;;;;;-1:-1:-1;2607:108:2;;;;;:::i;:::-;;:::i;7135:274:4:-;;;;;;;;;;-1:-1:-1;7135:274:4;;;;;:::i;:::-;;:::i;515:30:2:-;;;;;;;;;;;;;;;;8142:311:4;;;;;;;;;;-1:-1:-1;8142:311:4;;;;;:::i;:::-;;:::i;668:59:2:-;;;;;;;;;;-1:-1:-1;668:59:2;;;;;:::i;:::-;;;;;;;;;;;;;;5658:394:4;;;;;;;;;;-1:-1:-1;5658:394:4;;;;;:::i;:::-;;:::i;4062:105:14:-;;;;;;;;;;-1:-1:-1;4062:105:14;;;;;:::i;:::-;-1:-1:-1;;;;;4143:16:14;4116:7;4143:16;;;:7;:16;;;;;;;4062:105;5406:86:2;;;;;;;;;;-1:-1:-1;5476:10:2;;5406:86;;284:27;;;;;;;;;;;;;:::i;12473:43:4:-;;;;;;;;;;;;;;;;3852:119:14;;;;;;;;;;-1:-1:-1;3852:119:14;;;;;:::i;:::-;-1:-1:-1;;;;;3937:26:14;3910:7;3937:26;;;:19;:26;;;;;;;3852:119;3513:416:2;;;;;;:::i;:::-;;:::i;440:29::-;;;;;;;;;;;;;;;;3600:95:14;;;;;;;;;;-1:-1:-1;3673:14:14;;3600:95;;7472:186:4;;;;;;;;;;-1:-1:-1;7472:186:4;;;;;:::i;:::-;-1:-1:-1;;;;;7617:25:4;;;7594:4;7617:25;;;:18;:25;;;;;;;;:35;;;;;;;;;;;;;;;7472:186;3222:285:2;;;;;;:::i;:::-;;:::i;1972:201:12:-;;;;;;;;;;-1:-1:-1;1972:201:12;;;;;:::i;:::-;;:::i;550:27:2:-;;;;;;;;;;;;;;;;3616:370:4;3743:4;-1:-1:-1;;;;;;3773:40:4;;3788:25;3773:40;;:99;;-1:-1:-1;;;;;;;3824:48:4;;3839:33;3824:48;3773:99;:160;;;-1:-1:-1;;;;;;;3883:50:4;;3898:35;3883:50;3773:160;:207;;;-1:-1:-1;978:25:3;-1:-1:-1;;;;;;963:40:3;;;3944:36:4;3759:221;3616:370;-1:-1:-1;;3616:370:4:o;5342:94::-;5396:13;5425:5;5418:12;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;5342:94;:::o;6867:204::-;6935:7;6959:16;6967:7;8749:4;8779:12;-1:-1:-1;8769:22:4;8692:105;6959:16;6951:74;;;;-1:-1:-1;;;;;6951:74:4;;12697:2:17;6951:74:4;;;12679:21:17;12736:2;12716:18;;;12709:30;12775:34;12755:18;;;12748:62;12846:15;12826:18;;;12819:43;12879:19;;6951:74:4;;;;;;;;;-1:-1:-1;7041:24:4;;;;:15;:24;;;;;;-1:-1:-1;;;;;7041:24:4;;6867:204::o;6430:379::-;6499:13;6515:24;6531:7;6515:15;:24::i;:::-;6499:40;;6560:5;-1:-1:-1;;;;;6554:11:4;:2;-1:-1:-1;;;;;6554:11:4;;;6546:58;;;;-1:-1:-1;;;;;6546:58:4;;13111:2:17;6546:58:4;;;13093:21:17;13150:2;13130:18;;;13123:30;13189:34;13169:18;;;13162:62;13260:4;13240:18;;;13233:32;13282:19;;6546:58:4;12909:398:17;6546:58:4;736:10:1;-1:-1:-1;;;;;6629:21:4;;;;:62;;-1:-1:-1;6654:37:4;6671:5;736:10:1;7472:186:4;:::i;6654:37::-;6613:153;;;;-1:-1:-1;;;;;6613:153:4;;13514:2:17;6613:153:4;;;13496:21:17;13553:2;13533:18;;;13526:30;13592:34;13572:18;;;13565:62;13663:27;13643:18;;;13636:55;13708:19;;6613:153:4;13312:421:17;6613:153:4;6775:28;6784:2;6788:7;6797:5;6775:8;:28::i;:::-;6492:317;6430:379;;:::o;1612:417:2:-;1136:6:12;;-1:-1:-1;;;;;1136:6:12;736:10:1;1283:23:12;1275:68;;;;-1:-1:-1;;;;;1275:68:12;;;;;;;:::i;:::-;1774:13:2::1;:20;1754:9;:16;:40;1746:96;;;::::0;-1:-1:-1;;;;;1746:96:2;;14301:2:17;1746:96:2::1;::::0;::::1;14283:21:17::0;14340:2;14320:18;;;14313:30;14379:34;14359:18;;;14352:62;14450:13;14430:18;;;14423:41;14481:19;;1746:96:2::1;14099:407:17::0;1746:96:2::1;1876:1;1857:9;:16;:20;1849:45;;;::::0;-1:-1:-1;;;;;1849:45:2;;14713:2:17;1849:45:2::1;::::0;::::1;14695:21:17::0;14752:2;14732:18;;;14725:30;14791:14;14771:18;;;14764:42;14823:18;;1849:45:2::1;14511:336:17::0;1849:45:2::1;1908:9;1903:121;1927:9;:16;1923:1;:20;1903:121;;;2000:13;2014:1;2000:16;;;;;;;;:::i;:::-;;;;;;;1959:24;:38;1984:9;1994:1;1984:12;;;;;;;;:::i;:::-;;;;;;;-1:-1:-1::0;;;;;1959:38:2::1;-1:-1:-1::0;;;;;1959:38:2::1;;;;;;;;;;;;:57;;;;1945:3;;;;;:::i;:::-;;;;1903:121;;2176:98:4::0;2229:7;2267:1;2252:12;;:16;;;;:::i;:::-;2245:23;;2176:98;:::o;5070:566:14:-;-1:-1:-1;;;;;5146:16:14;;5165:1;5146:16;;;:7;:16;;;;;;5138:71;;;;-1:-1:-1;;;;;5138:71:14;;;;;;;:::i;:::-;5222:21;5270:15;3673:14;;;3600:95;5270:15;5246:39;;5254:4;5246:21;:39;:::i;:::-;5222:63;;5296:15;5314:58;5330:7;5339:13;5354:17;5363:7;-1:-1:-1;;;;;4349:18:14;4322:7;4349:18;;;:9;:18;;;;;;;4266:109;5354:17;5314:15;:58::i;:::-;5296:76;-1:-1:-1;5393:12:14;5385:68;;;;-1:-1:-1;;;;;5385:68:14;;;;;;;:::i;:::-;-1:-1:-1;;;;;5466:18:14;;;;;;:9;:18;;;;;:29;;5488:7;;5466:18;:29;;5488:7;;5466:29;:::i;:::-;;;;;;;;5524:7;5506:14;;:25;;;;;;;:::i;:::-;;;;-1:-1:-1;5544:35:14;;-1:-1:-1;5562:7:14;5571;5544:17;:35::i;:::-;5595:33;;;-1:-1:-1;;;;;206:55:17;;188:74;;293:2;278:18;;271:34;;;5595:33:14;;161:18:17;5595:33:14;;;;;;;5127:509;;5070:566;:::o;4774:136:2:-;4825:4;4846:15;;4865:1;4846:20;;:57;;;;;4888:15;4870;;:33;4838:66;;4774:136;:::o;7717:142:4:-;7825:28;7835:4;7841:2;7845:7;7825:9;:28::i;2808:744::-;2917:7;2952:16;2962:5;2952:9;:16::i;:::-;2944:5;:24;2936:71;;;;-1:-1:-1;;;;;2936:71:4;;16964:2:17;2936:71:4;;;16946:21:17;17003:2;16983:18;;;16976:30;17042:34;17022:18;;;17015:62;17113:4;17093:18;;;17086:32;17135:19;;2936:71:4;16762:398:17;2936:71:4;3014:22;3039:13;:11;:13::i;:::-;3014:38;;3059:19;3089:25;3139:9;3134:350;3158:14;3154:1;:18;3134:350;;;3188:31;3222:14;;;:11;:14;;;;;;;;;3188:48;;;;;;;;;-1:-1:-1;;;;;3188:48:4;;;;;-1:-1:-1;;;3188:48:4;;;;;;;;;;;;3249:28;3245:89;;3310:14;;;-1:-1:-1;3245:89:4;3367:5;-1:-1:-1;;;;;3346:26:4;:17;-1:-1:-1;;;;;3346:26:4;;3342:135;;;3404:5;3389:11;:20;3385:59;;;-1:-1:-1;3431:1:4;-1:-1:-1;3424:8:4;;-1:-1:-1;;;3424:8:4;3385:59;3454:13;;;;:::i;:::-;;;;3342:135;-1:-1:-1;3174:3:4;;;;:::i;:::-;;;;3134:350;;;-1:-1:-1;3490:56:4;;-1:-1:-1;;;;;3490:56:4;;17367:2:17;3490:56:4;;;17349:21:17;17406:2;17386:18;;;17379:30;17445:34;17425:18;;;17418:62;17516:16;17496:18;;;17489:44;17550:19;;3490:56:4;17165:410:17;5892:61:2;1136:6:12;;-1:-1:-1;;;;;1136:6:12;736:10:1;1283:23:12;1275:68;;;;-1:-1:-1;;;;;1275:68:12;;;;;;;:::i;:::-;5937:10:2::1;:8;:10::i;:::-;5892:61::o:0;3079:137::-;1136:6:12;;-1:-1:-1;;;;;1136:6:12;736:10:1;1283:23:12;1275:68;;;;-1:-1:-1;;;;;1275:68:12;;;;;;;:::i;:::-;3154:27:2::1;3175:5;3154:20;:27::i;:::-;3190:20;3200:2;3204:5;3190:9;:20::i;:::-;3079:137:::0;;:::o;7922:157:4:-;8034:39;8051:4;8057:2;8061:7;8034:39;;;;;;;;;;;;:16;:39::i;5904:641:14:-;-1:-1:-1;;;;;5986:16:14;;6005:1;5986:16;;;:7;:16;;;;;;5978:71;;;;-1:-1:-1;;;;;5978:71:14;;;;;;;:::i;:::-;-1:-1:-1;;;;;3937:26:14;;6062:21;3937:26;;;:19;:26;;;;;;6086:30;;;;;6110:4;6086:30;;;2044:74:17;-1:-1:-1;;;;;6086:15:14;;;;;2017:18:17;;6086:30:14;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;:53;;;;:::i;:::-;6062:77;;6150:15;6168:65;6184:7;6193:13;6208:24;6217:5;6224:7;-1:-1:-1;;;;;4641:21:14;;;4614:7;4641:21;;;:14;:21;;;;;;;;:30;;;;;;;;;;;;;4544:135;6168:65;6150:83;-1:-1:-1;6254:12:14;6246:68;;;;-1:-1:-1;;;;;6246:68:14;;;;;;;:::i;:::-;-1:-1:-1;;;;;6327:21:14;;;;;;;:14;:21;;;;;;;;:30;;;;;;;;;;;:41;;6361:7;;6327:21;:41;;6361:7;;6327:41;:::i;:::-;;;;-1:-1:-1;;;;;;;6379:26:14;;;;;;:19;:26;;;;;:37;;6409:7;;6379:26;:37;;6409:7;;6379:37;:::i;:::-;;;;-1:-1:-1;6429:47:14;;-1:-1:-1;6452:5:14;6459:7;6468;6429:22;:47::i;:::-;6492:45;;;-1:-1:-1;;;;;206:55:17;;;188:74;;293:2;278:18;;271:34;;;6492:45:14;;;;;161:18:17;6492:45:14;;;;;;;5967:578;;5904:641;;:::o;2343:177:4:-;2410:7;2442:13;:11;:13::i;:::-;2434:5;:21;2426:69;;;;-1:-1:-1;;;;;2426:69:4;;17971:2:17;2426:69:4;;;17953:21:17;18010:2;17990:18;;;17983:30;18049:34;18029:18;;;18022:62;18120:5;18100:18;;;18093:33;18143:19;;2426:69:4;17769:399:17;2426:69:4;-1:-1:-1;2509:5:4;2343:177::o;5165:118::-;5229:7;5252:20;5264:7;5252:11;:20::i;:::-;:25;;5165:118;-1:-1:-1;;5165:118:4:o;5645:178:2:-;5704:7;5724:17;:15;:17::i;:::-;5720:68;;;-1:-1:-1;5759:21:2;;;5645:178::o;5720:68::-;-1:-1:-1;5803:14:2;;;5645:178::o;4042:211:4:-;4106:7;-1:-1:-1;;;;;4130:19:4;;4122:75;;;;-1:-1:-1;;;;;4122:75:4;;18375:2:17;4122:75:4;;;18357:21:17;18414:2;18394:18;;;18387:30;18453:34;18433:18;;;18426:62;18524:13;18504:18;;;18497:41;18555:19;;4122:75:4;18173:407:17;4122:75:4;-1:-1:-1;;;;;;4219:19:4;;;;;:12;:19;;;;;:27;-1:-1:-1;;;;;4219:27:4;;4042:211::o;1714:103:12:-;1136:6;;-1:-1:-1;;;;;1136:6:12;736:10:1;1283:23:12;1275:68;;;;-1:-1:-1;;;;;1275:68:12;;;;;;;:::i;:::-;1779:30:::1;1806:1;1779:18;:30::i;2035:566:2:-:0;1136:6:12;;-1:-1:-1;;;;;1136:6:12;736:10:1;1283:23:12;1275:68;;;;-1:-1:-1;;;;;1275:68:12;;;;;;;:::i;:::-;2314:15:2::1;:32:::0;;;;2353:12:::1;:26:::0;;;;2386:14:::1;:30:::0;;;;2423:21:::1;:44:::0;;;;2474:6:::1;:14:::0;2495:13:::1;:28:::0;2530:11:::1;:24:::0;2561:16:::1;:34:::0;2035:566::o;5090:310::-;5186:4;5307:22;;19195:28:17;-1:-1:-1;;;;;19138:55:17;;19134:90;5307:22:2;;;19122:103:17;5282:12:2;;19241::17;;5307:22:2;;;;;;;;;;;;5297:33;;;;;;5282:48;;5344:50;5363:11;;5344:50;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;;5376:11:2;;;-1:-1:-1;5389:4:2;;-1:-1:-1;5344:18:2;:50::i;:::-;5337:57;;;5090:310;;;;;;:::o;2721:99::-;1136:6:12;;-1:-1:-1;;;;;1136:6:12;736:10:1;1283:23:12;1275:68;;;;-1:-1:-1;;;;;1275:68:12;;;;;;;:::i;:::-;2790:11:2::1;:24:::0;2721:99::o;5829:57::-;1136:6:12;;-1:-1:-1;;;;;1136:6:12;736:10:1;1283:23:12;1275:68;;;;-1:-1:-1;;;;;1275:68:12;;;;;;;:::i;:::-;5872:8:2::1;:6;:8::i;4770:100:14:-:0;4821:7;4848;4856:5;4848:14;;;;;;;;:::i;:::-;;;;;;;;;;;-1:-1:-1;;;;;4848:14:14;;4770:100;-1:-1:-1;;4770:100:14:o;5498:141:2:-;5536:7;5556:17;:15;:17::i;:::-;5552:60;;;-1:-1:-1;5591:13:2;;;5498:141::o;5552:60::-;-1:-1:-1;5627:6:2;;;5498:141::o;5497:98:4:-;5553:13;5582:7;5575:14;;;;;:::i;4916:168:2:-;4964:4;4985:12;;5001:1;4985:17;;:53;;;;;5022:15;5007:12;;:30;4985:53;:92;;;;-1:-1:-1;;5061:15:2;;5043;:33;;4916:168::o;2607:108::-;1136:6:12;;-1:-1:-1;;;;;1136:6:12;736:10:1;1283:23:12;1275:68;;;;-1:-1:-1;;;;;1275:68:12;;;;;;;:::i;:::-;2686:23:2;;::::1;::::0;:13:::1;::::0;:23:::1;::::0;::::1;::::0;::::1;:::i;7135:274:4:-:0;-1:-1:-1;;;;;7226:24:4;;736:10:1;7226:24:4;;7218:63;;;;-1:-1:-1;;;;;7218:63:4;;19466:2:17;7218:63:4;;;19448:21:17;19505:2;19485:18;;;19478:30;19544:28;19524:18;;;19517:56;19590:18;;7218:63:4;19264:350:17;7218:63:4;736:10:1;7290:32:4;;;;:18;:32;;;;;;;;-1:-1:-1;;;;;7290:42:4;;;;;;;;;;;;:53;;-1:-1:-1;;7290:53:4;;;;;;;;;;7355:48;;888:41:17;;;7290:42:4;;736:10:1;7355:48:4;;861:18:17;7355:48:4;;;;;;;7135:274;;:::o;8142:311::-;8279:28;8289:4;8295:2;8299:7;8279:9;:28::i;:::-;8330:48;8353:4;8359:2;8363:7;8372:5;8330:22;:48::i;:::-;8314:133;;;;-1:-1:-1;;;;;8314:133:4;;;;;;;:::i;:::-;8142:311;;;;:::o;5658:394::-;5756:13;5797:16;5805:7;8749:4;8779:12;-1:-1:-1;8769:22:4;8692:105;5797:16;5781:97;;;;-1:-1:-1;;;;;5781:97:4;;20241:2:17;5781:97:4;;;20223:21:17;20280:2;20260:18;;;20253:30;20319:34;20299:18;;;20292:62;20390:17;20370:18;;;20363:45;20425:19;;5781:97:4;20039:411:17;5781:97:4;5887:21;5911:10;:8;:10::i;:::-;5887:34;;5966:1;5948:7;5942:21;:25;:104;;;;;;;;;;;;;;;;;6003:7;6012:18;:7;:16;:18::i;:::-;5986:45;;;;;;;;;:::i;:::-;;;;;;;;;;;;;5928:118;5658:394;-1:-1:-1;;;5658:394:4:o;284:27:2:-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;3513:416::-;1201:7:13;;-1:-1:-1;;;1201:7:13;;;;1455:9;1447:38;;;;-1:-1:-1;;;;;1447:38:13;;;;;;;:::i;:::-;3648:10:2::1;3667:36;::::0;;;:24:::1;:36;::::0;;;;;3621:83:::1;::::0;3648:10;3660:5;;3621:26:::1;:83::i;:::-;3719:17;:15;:17::i;:::-;:65;;;;;3740:44;3760:10;3772:11;;3740:19;:44::i;:::-;3711:113;;;::::0;-1:-1:-1;;;;;3711:113:2;;21667:2:17;3711:113:2::1;::::0;::::1;21649:21:17::0;21706:2;21686:18;;;21679:30;21745:34;21725:18;;;21718:62;21816:5;21796:18;;;21789:33;21839:19;;3711:113:2::1;21465:399:17::0;3711:113:2::1;3833:31;3843:5;3850:13;;3833:9;:31::i;:::-;3902:13;::::0;3876:47:::1;::::0;3917:5;;3902:13;3890:10:::1;::::0;3876:47:::1;::::0;;;::::1;3513:416:::0;;;:::o;3222:285::-;1201:7:13;;-1:-1:-1;;;1201:7:13;;;;1455:9;1447:38;;;;-1:-1:-1;;;;;1447:38:13;;;;;;;:::i;:::-;3293:61:2::1;3320:10;3332:5;3339:14;;3293:26;:61::i;:::-;3369:20;:18;:20::i;:::-;3361:60;;;::::0;-1:-1:-1;;;;;3361:60:2;;22071:2:17;3361:60:2::1;::::0;::::1;22053:21:17::0;22110:2;22090:18;;;22083:30;22149:29;22129:18;;;22122:57;22196:18;;3361:60:2::1;21869:351:17::0;3361:60:2::1;3430:24;3440:5;3447:6;;3430:9;:24::i;:::-;3487:6;::::0;3466:35:::1;::::0;3495:5;;3487:6;3475:10:::1;::::0;3466:35:::1;::::0;;;::::1;3222:285:::0;:::o;1972:201:12:-;1136:6;;-1:-1:-1;;;;;1136:6:12;736:10:1;1283:23:12;1275:68;;;;-1:-1:-1;;;;;1275:68:12;;;;;;;:::i;:::-;-1:-1:-1;;;;;2061:22:12;::::1;2053:73;;;::::0;-1:-1:-1;;;;;2053:73:12;;22427:2:17;2053:73:12::1;::::0;::::1;22409:21:17::0;22466:2;22446:18;;;22439:30;22505:34;22485:18;;;22478:62;22576:8;22556:18;;;22549:36;22602:19;;2053:73:12::1;22225:402:17::0;2053:73:12::1;2137:28;2156:8;2137:18;:28::i;:::-;1972:201:::0;:::o;12295:172:4:-;12392:24;;;;:15;:24;;;;;;:29;;-1:-1:-1;;12392:29:4;-1:-1:-1;;;;;12392:29:4;;;;;;;;;12433:28;;12392:24;;12433:28;;;;;;;12295:172;;;:::o;6723:248:14:-;6933:12;;-1:-1:-1;;;;;6913:16:14;;6869:7;6913:16;;;:7;:16;;;;;;6869:7;;6948:15;;6897:32;;:13;:32;:::i;:::-;6896:49;;;;:::i;:::-;:67;;;;:::i;:::-;6889:74;6723:248;-1:-1:-1;;;;6723:248:14:o;2119:317:0:-;2217:4;2209:21;:31;-1:-1:-1;2209:31:0;2201:73;;;;-1:-1:-1;;;;;2201:73:0;;23321:2:17;2201:73:0;;;23303:21:17;23360:2;23340:18;;;23333:30;23399:31;23379:18;;;23372:59;23448:18;;2201:73:0;23119:353:17;2201:73:0;2288:12;2306:9;-1:-1:-1;;;;;2306:14:0;2328:6;2306:33;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;2287:52;;;2358:7;2350:78;;;;-1:-1:-1;;;;;2350:78:0;;23889:2:17;2350:78:0;;;23871:21:17;23928:2;23908:18;;;23901:30;23967:34;23947:18;;;23940:62;24038:28;24018:18;;;24011:56;24084:19;;2350:78:0;23687:422:17;10660:1529:4;10757:35;10795:20;10807:7;10795:11;:20::i;:::-;10866:18;;10757:58;;-1:-1:-1;10824:22:4;;-1:-1:-1;;;;;10850:34:4;736:10:1;-1:-1:-1;;;;;10850:34:4;;:81;;;-1:-1:-1;736:10:1;10895:20:4;10907:7;10895:11;:20::i;:::-;-1:-1:-1;;;;;10895:36:4;;10850:81;:142;;;-1:-1:-1;10959:18:4;;10942:50;;736:10:1;7472:186:4;:::i;10942:50::-;10824:169;;11018:17;11002:101;;;;-1:-1:-1;;;;;11002:101:4;;24316:2:17;11002:101:4;;;24298:21:17;24355:2;24335:18;;;24328:30;24394:34;24374:18;;;24367:62;24465:20;24445:18;;;24438:48;24503:19;;11002:101:4;24114:414:17;11002:101:4;11150:4;-1:-1:-1;;;;;11128:26:4;:13;:18;;;-1:-1:-1;;;;;11128:26:4;;11112:98;;;;-1:-1:-1;;;;;11112:98:4;;24735:2:17;11112:98:4;;;24717:21:17;24774:2;24754:18;;;24747:30;24813:34;24793:18;;;24786:62;24884:8;24864:18;;;24857:36;24910:19;;11112:98:4;24533:402:17;11112:98:4;-1:-1:-1;;;;;11225:16:4;;11217:66;;;;-1:-1:-1;;;;;11217:66:4;;25142:2:17;11217:66:4;;;25124:21:17;25181:2;25161:18;;;25154:30;25220:34;25200:18;;;25193:62;25291:7;25271:18;;;25264:35;25316:19;;11217:66:4;24940:401:17;11217:66:4;11392:49;11409:1;11413:7;11422:13;:18;;;11392:8;:49::i;:::-;-1:-1:-1;;;;;11450:18:4;;;;;;:12;:18;;;;;:31;;11480:1;;11450:18;:31;;11480:1;;-1:-1:-1;;;;;11450:31:4;;:::i;:::-;;;;;;;;-1:-1:-1;;;;;11450:31:4;;;;;;;;;;;;;;;-1:-1:-1;;;;;11488:16:4;;-1:-1:-1;11488:16:4;;;:12;:16;;;;;:29;;-1:-1:-1;;;11488:16:4;;:29;;-1:-1:-1;;11488:29:4;;:::i;:::-;;;-1:-1:-1;;;;;11488:29:4;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;11547:43:4;;;;;;;;-1:-1:-1;;;;;11547:43:4;;;;;;11573:15;11547:43;;;;;;;;;-1:-1:-1;11524:20:4;;;:11;:20;;;;;;:66;;;;;;;;;-1:-1:-1;;;11524:66:4;-1:-1:-1;;;;;;11524:66:4;;;;;;;;;;;11840:11;11536:7;-1:-1:-1;11840:11:4;:::i;:::-;11903:1;11862:24;;;:11;:24;;;;;:29;11818:33;;-1:-1:-1;;;;;;11862:29:4;11858:236;;11920:20;11928:11;8749:4;8779:12;-1:-1:-1;8769:22:4;8692:105;11920:20;11916:171;;;11980:97;;;;;;;;12007:18;;-1:-1:-1;;;;;11980:97:4;;;;;;12038:28;;;;11980:97;;;;;;;;;;-1:-1:-1;11953:24:4;;;:11;:24;;;;;;;:124;;;;;;;;;-1:-1:-1;;;11953:124:4;-1:-1:-1;;;;;;11953:124:4;;;;;;;;;;;;11916:171;12126:7;12122:2;-1:-1:-1;;;;;12107:27:4;12116:4;-1:-1:-1;;;;;12107:27:4;;;;;;;;;;;12141:42;10750:1439;;;10660:1529;;;:::o;2189:120:13:-;1201:7;;-1:-1:-1;;;1201:7:13;;;;1725:41;;;;-1:-1:-1;;;;;1725:41:13;;26057:2:17;1725:41:13;;;26039:21:17;26096:2;26076:18;;;26069:30;26135:22;26115:18;;;26108:50;26175:18;;1725:41:13;25855:344:17;1725:41:13;2248:7:::1;:15:::0;;-1:-1:-1;;2248:15:13::1;::::0;;2279:22:::1;736:10:1::0;2288:12:13::1;2279:22;::::0;-1:-1:-1;;;;;2062:55:17;;;2044:74;;2032:2;2017:18;2279:22:13::1;;;;;;;2189:120::o:0;4164:154:2:-;4263:10;;4254:5;4238:13;:11;:13::i;:::-;:21;;;;:::i;:::-;:35;;4230:82;;;;-1:-1:-1;;;;;4230:82:2;;26406:2:17;4230:82:2;;;26388:21:17;26445:2;26425:18;;;26418:30;26484:34;26464:18;;;26457:62;26555:4;26535:18;;;26528:32;26577:19;;4230:82:2;26204:398:17;8803:98:4;8868:27;8878:2;8882:8;8868:27;;;;;;;;;;;;:9;:27::i;707:211:15:-;851:58;;;-1:-1:-1;;;;;206:55:17;;851:58:15;;;188:74:17;278:18;;;;271:34;;;851:58:15;;;;;;;;;;161:18:17;;;;851:58:15;;;;;;;;;;874:23;851:58;;;824:86;;844:5;;824:19;:86::i;4505:606:4:-;-1:-1:-1;;;;;;;;;;;;;;;;;4622:16:4;4630:7;8749:4;8779:12;-1:-1:-1;8769:22:4;8692:105;4622:16;4614:71;;;;-1:-1:-1;;;;;4614:71:4;;26809:2:17;4614:71:4;;;26791:21:17;26848:2;26828:18;;;26821:30;26887:34;26867:18;;;26860:62;26958:12;26938:18;;;26931:40;26988:19;;4614:71:4;26607:406:17;4614:71:4;4694:26;4742:12;4731:7;:23;4727:93;;4786:22;4796:12;4786:7;:22;:::i;:::-;:26;;4811:1;4786:26;:::i;:::-;4765:47;;4727:93;4848:7;4828:212;4865:18;4857:4;:26;4828:212;;4902:31;4936:17;;;:11;:17;;;;;;;;;4902:51;;;;;;;;;-1:-1:-1;;;;;4902:51:4;;;;;-1:-1:-1;;;4902:51:4;;;;;;;;;;;;4966:28;4962:71;;5014:9;4505:606;-1:-1:-1;;;;4505:606:4:o;4962:71::-;-1:-1:-1;4885:6:4;;;;:::i;:::-;;;;4828:212;;;-1:-1:-1;5048:57:4;;-1:-1:-1;;;;;5048:57:4;;27361:2:17;5048:57:4;;;27343:21:17;27400:2;27380:18;;;27373:30;27439:34;27419:18;;;27412:62;27510:17;27490:18;;;27483:45;27545:19;;5048:57:4;27159:411:17;2333:191:12;2426:6;;;-1:-1:-1;;;;;2443:17:12;;;-1:-1:-1;;2443:17:12;;;;;;;2476:40;;2426:6;;;2443:17;2426:6;;2476:40;;2407:16;;2476:40;2396:128;2333:191;:::o;868:190:11:-;993:4;1046;1017:25;1030:5;1037:4;1017:12;:25::i;:::-;:33;;868:190;-1:-1:-1;;;;868:190:11:o;1930:118:13:-;1201:7;;-1:-1:-1;;;1201:7:13;;;;1455:9;1447:38;;;;-1:-1:-1;;;;;1447:38:13;;;;;;;:::i;:::-;1990:7:::1;:14:::0;;-1:-1:-1;;1990:14:13::1;-1:-1:-1::0;;;1990:14:13::1;::::0;;2020:20:::1;2027:12;736:10:1::0;;656:98;14006:690:4;14143:4;-1:-1:-1;;;;;14160:13:4;;1120:20:0;1168:8;14156:535:4;;14199:72;;;;;-1:-1:-1;;;;;14199:36:4;;;;;:72;;736:10:1;;14250:4:4;;14256:7;;14265:5;;14199:72;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;14199:72:4;;;;;;;;-1:-1:-1;;14199:72:4;;;;;;;;;;;;:::i;:::-;;;14186:464;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;14430:13:4;;14426:215;;14463:61;;-1:-1:-1;;;;;14463:61:4;;;;;;;:::i;14426:215::-;14609:6;14603:13;14594:6;14590:2;14586:15;14579:38;14186:464;-1:-1:-1;;;;;;14321:55:4;14331:45;14321:55;;-1:-1:-1;14314:62:4;;14156:535;-1:-1:-1;14679:4:4;14006:690;;;;;;:::o;2826:247:2:-;2886:13;2957;2981:56;3025:4;3034:2;2981:19;:56::i;:::-;2930:130;;;;;;;;;:::i;:::-;;;;;;;;;;;;;2908:159;;2826:247;:::o;342:723:16:-;398:13;619:10;615:53;;-1:-1:-1;;646:10:16;;;;;;;;;;;;;;;;;;342:723::o;615:53::-;693:5;678:12;734:78;741:9;;734:78;;767:8;;;;:::i;:::-;;-1:-1:-1;790:10:16;;-1:-1:-1;798:2:16;790:10;;:::i;:::-;;;734:78;;;822:19;854:6;844:17;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;844:17:16;;822:39;;872:154;879:10;;872:154;;906:11;916:1;906:11;;:::i;:::-;;-1:-1:-1;975:10:16;983:2;975:5;:10;:::i;:::-;962:24;;:2;:24;:::i;:::-;949:39;;932:6;939;932:14;;;;;;;;:::i;:::-;;;;:56;-1:-1:-1;;;;;932:56:16;;;;;;;;-1:-1:-1;1003:11:16;1012:2;1003:11;;:::i;:::-;;;872:154;;4324:444:2;4431:27;4452:5;4431:20;:27::i;:::-;4476:16;;:21;;;;4475:54;;;4512:16;;4503:5;:25;;4475:54;4467:110;;;;-1:-1:-1;;;;;4467:110:2;;30288:2:17;4467:110:2;;;30270:21:17;30327:2;30307:18;;;30300:30;30366:34;30346:18;;;30339:62;30437:13;30417:18;;;30410:41;30468:19;;4467:110:2;30086:407:17;4467:110:2;-1:-1:-1;;;;;4615:14:2;;4584:28;4615:14;;;:10;:14;;;;;;:22;;4632:5;;4615:22;:::i;:::-;4584:53;-1:-1:-1;4654:18:2;;;;;4653:63;;;4702:13;4678:20;:37;;4653:63;4644:118;;;;-1:-1:-1;;;;;4644:118:2;;30700:2:17;4644:118:2;;;30682:21:17;30739:2;30719:18;;;30712:30;30778:34;30758:18;;;30751:62;30849:11;30829:18;;;30822:39;30878:19;;4644:118:2;30498:405:17;3935:223:2;4024:9;4007:13;4015:5;4007;:13;:::i;:::-;:26;;3999:78;;;;-1:-1:-1;;;;;3999:78:2;;31110:2:17;3999:78:2;;;31092:21:17;31149:2;31129:18;;;31122:30;31188:34;31168:18;;;31161:62;31259:9;31239:18;;;31232:37;31286:19;;3999:78:2;30908:403:17;3999:78:2;4097:10;4086:22;;;;:10;:22;;;;;:31;;4112:5;;4086:22;:31;;4112:5;;4086:31;:::i;:::-;;;;-1:-1:-1;4124:28:2;;-1:-1:-1;4134:10:2;4146:5;4124:9;:28::i;9156:1272:4:-;9261:20;9284:12;-1:-1:-1;;;;;9311:16:4;;9303:62;;;;-1:-1:-1;;;;;9303:62:4;;31518:2:17;9303:62:4;;;31500:21:17;31557:2;31537:18;;;31530:30;31596:34;31576:18;;;31569:62;31667:3;31647:18;;;31640:31;31688:19;;9303:62:4;31316:397:17;9303:62:4;9502:21;9510:12;8749:4;8779:12;-1:-1:-1;8769:22:4;8692:105;9502:21;9501:22;9493:64;;;;-1:-1:-1;;;;;9493:64:4;;31920:2:17;9493:64:4;;;31902:21:17;31959:2;31939:18;;;31932:30;31998:31;31978:18;;;31971:59;32047:18;;9493:64:4;31718:353:17;9493:64:4;9584:12;9572:8;:24;;9564:71;;;;-1:-1:-1;;;;;9564:71:4;;32278:2:17;9564:71:4;;;32260:21:17;32317:2;32297:18;;;32290:30;32356:34;32336:18;;;32329:62;32427:4;32407:18;;;32400:32;32449:19;;9564:71:4;32076:398:17;9564:71:4;-1:-1:-1;;;;;9747:16:4;;9714:30;9747:16;;;:12;:16;;;;;;;;;9714:49;;;;;;;;;-1:-1:-1;;;;;9714:49:4;;;;;;;;;;;;;;;;;9789:119;;;;;;;;9809:19;;9714:49;;9789:119;;;9809:39;;9839:8;;9809:39;:::i;:::-;-1:-1:-1;;;;;9789:119:4;;;;;9892:8;9857:11;:24;;;:44;;;;:::i;:::-;-1:-1:-1;;;;;9789:119:4;;;;;;-1:-1:-1;;;;;9770:16:4;;;;;;;:12;:16;;;;;;;;:138;;;;;;;;;;;;;;;;;;;;;9943:43;;;;;;;;;;;9969:15;9943:43;;;;;;;;9915:25;;;:11;:25;;;;;;:71;;;;;;;;;-1:-1:-1;;;9915:71:4;-1:-1:-1;;;;;;9915:71:4;;;;;;;;;;;;;;;;;;9927:12;;10039:281;10063:8;10059:1;:12;10039:281;;;10092:38;;10117:12;;-1:-1:-1;;;;;10092:38:4;;;10109:1;;10092:38;;10109:1;;10092:38;10157:59;10188:1;10192:2;10196:12;10210:5;10157:22;:59::i;:::-;10139:150;;;;-1:-1:-1;;;;;10139:150:4;;;;;;;:::i;:::-;10298:14;;;;:::i;:::-;;;;10073:3;;;;;:::i;:::-;;;;10039:281;;;-1:-1:-1;10328:12:4;:27;;;10362:60;8142:311;3280:716:15;3704:23;3730:69;3758:4;3730:69;;;;;;;;;;;;;;;;;3738:5;-1:-1:-1;;;;;3730:27:15;;;:69;;;;;:::i;:::-;3814:17;;3704:95;;-1:-1:-1;3814:21:15;3810:179;;3911:10;3900:30;;;;;;;;;;;;:::i;:::-;3892:85;;;;-1:-1:-1;;;;;3892:85:15;;32931:2:17;3892:85:15;;;32913:21:17;32970:2;32950:18;;;32943:30;33009:34;32989:18;;;32982:62;33080:12;33060:18;;;33053:40;33110:19;;3892:85:15;32729:406:17;1420:701:11;1503:7;1546:4;1503:7;1561:523;1585:5;:12;1581:1;:16;1561:523;;;1619:20;1642:5;1648:1;1642:8;;;;;;;;:::i;:::-;;;;;;;1619:31;;1685:12;1669;:28;1665:408;;1822:44;;;;;;33297:19:17;;;33332:12;;;33325:28;;;33369:12;;1822:44:11;;;;;;;;;;;;1812:55;;;;;;1797:70;;1665:408;;;2012:44;;;;;;33297:19:17;;;33332:12;;;33325:28;;;33369:12;;2012:44:11;;;;;;;;;;;;2002:55;;;;;;1987:70;;1665:408;-1:-1:-1;1599:3:11;;;;:::i;:::-;;;;1561:523;;;-1:-1:-1;2101:12:11;1420:701;-1:-1:-1;;;1420:701:11:o;1643:451:16:-;1718:13;1744:19;1776:10;1780:6;1776:1;:10;:::i;:::-;:14;;1789:1;1776:14;:::i;:::-;1766:25;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;-1:-1:-1;1766:25:16;;1744:47;;1802:15;:6;1809:1;1802:9;;;;;;;;:::i;:::-;;;;:15;-1:-1:-1;;;;;1802:15:16;;;;;;;;;1828;:6;1835:1;1828:9;;;;;;;;:::i;:::-;;;;:15;-1:-1:-1;;;;;1828:15:16;;;;;;;;-1:-1:-1;1859:9:16;1871:10;1875:6;1871:1;:10;:::i;:::-;:14;;1884:1;1871:14;:::i;:::-;1859:26;;1854:135;1891:1;1887;:5;1854:135;;;1926:12;1939:5;1947:3;1939:11;1926:25;;;;;;;:::i;:::-;;;;1914:6;1921:1;1914:9;;;;;;;;:::i;:::-;;;;:37;-1:-1:-1;;;;;1914:37:16;;;;;;;;-1:-1:-1;1966:11:16;;;;;1894:3;;;:::i;:::-;;;1854:135;;;-1:-1:-1;2007:10:16;;1999:55;;;;-1:-1:-1;;;;;1999:55:16;;33594:2:17;1999:55:16;;;33576:21:17;;;33613:18;;;33606:30;33672:34;33652:18;;;33645:62;33724:18;;1999:55:16;33392:356:17;3603:229:0;3740:12;3772:52;3794:6;3802:4;3808:1;3811:12;3740;1120:20;;5010:60;;;;-1:-1:-1;;;;;5010:60:0;;34362:2:17;5010:60:0;;;34344:21:17;34401:2;34381:18;;;34374:30;34440:31;34420:18;;;34413:59;34489:18;;5010:60:0;34160:353:17;5010:60:0;5084:12;5098:23;5125:6;-1:-1:-1;;;;;5125:11:0;5144:5;5151:4;5125:31;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;5083:73;;;;5174:51;5191:7;5200:10;5212:12;5174:16;:51::i;:::-;5167:58;4723:510;-1:-1:-1;;;;;;;4723:510:0:o;7409:712::-;7559:12;7588:7;7584:530;;;-1:-1:-1;7619:10:0;7612:17;;7584:530;7733:17;;:21;7729:374;;7931:10;7925:17;7992:15;7979:10;7975:2;7971:19;7964:44;7729:374;8074:12;8067:20;;-1:-1:-1;;;;;8067:20:0;;;;;;;;:::i;-1:-1:-1:-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;316:177:17;-1:-1:-1;;;;;;394:5:17;390:78;383:5;380:89;370:117;;483:1;480;473:12;498:245;556:6;609:2;597:9;588:7;584:23;580:32;577:52;;;625:1;622;615:12;577:52;664:9;651:23;683:30;707:5;683:30;:::i;940:258::-;1012:1;1022:113;1036:6;1033:1;1030:13;1022:113;;;1112:11;;;1106:18;1093:11;;;1086:39;1058:2;1051:10;1022:113;;;1153:6;1150:1;1147:13;1144:48;;;-1:-1:-1;;1188:1:17;1170:16;;1163:27;940:258::o;1203:269::-;1256:3;1294:5;1288:12;1321:6;1316:3;1309:19;1337:63;1393:6;1386:4;1381:3;1377:14;1370:4;1363:5;1359:16;1337:63;:::i;:::-;1454:2;1433:15;-1:-1:-1;;1429:29:17;1420:39;;;;1461:4;1416:50;;1203:269;-1:-1:-1;;1203:269:17:o;1477:231::-;1626:2;1615:9;1608:21;1589:4;1646:56;1698:2;1687:9;1683:18;1675:6;1646:56;:::i;1713:180::-;1772:6;1825:2;1813:9;1804:7;1800:23;1796:32;1793:52;;;1841:1;1838;1831:12;1793:52;-1:-1:-1;1864:23:17;;1713:180;-1:-1:-1;1713:180:17:o;2129:154::-;-1:-1:-1;;;;;2208:5:17;2204:54;2197:5;2194:65;2184:93;;2273:1;2270;2263:12;2288:315;2356:6;2364;2417:2;2405:9;2396:7;2392:23;2388:32;2385:52;;;2433:1;2430;2423:12;2385:52;2472:9;2459:23;2491:31;2516:5;2491:31;:::i;:::-;2541:5;2593:2;2578:18;;;;2565:32;;-1:-1:-1;;;2288:315:17:o;2608:247::-;2667:6;2720:2;2708:9;2699:7;2695:23;2691:32;2688:52;;;2736:1;2733;2726:12;2688:52;2775:9;2762:23;2794:31;2819:5;2794:31;:::i;3042:184::-;-1:-1:-1;;;;;3091:1:17;3084:88;3191:4;3188:1;3181:15;3215:4;3212:1;3205:15;3231:275;3302:2;3296:9;3367:2;3348:13;;-1:-1:-1;;3344:27:17;3332:40;;3402:18;3387:34;;3423:22;;;3384:62;3381:88;;;3449:18;;:::i;:::-;3485:2;3478:22;3231:275;;-1:-1:-1;3231:275:17:o;3511:186::-;3571:4;3604:18;3596:6;3593:30;3590:56;;;3626:18;;:::i;:::-;-1:-1:-1;3686:4:17;3667:17;;;3663:28;;3511:186::o;3702:663::-;3756:5;3809:3;3802:4;3794:6;3790:17;3786:27;3776:55;;3827:1;3824;3817:12;3776:55;3863:6;3850:20;3889:4;3913:60;3929:43;3969:2;3929:43;:::i;:::-;3913:60;:::i;:::-;4007:15;;;4089:11;;;4077:24;;4073:33;;;4038:12;;;;4118:15;;;4115:35;;;4146:1;4143;4136:12;4115:35;4182:2;4174:6;4170:15;4194:142;4210:6;4205:3;4202:15;4194:142;;;4276:17;;4264:30;;4314:12;;;;4227;;4194:142;;;-1:-1:-1;4354:5:17;3702:663;-1:-1:-1;;;;;;3702:663:17:o;4370:1216::-;4488:6;4496;4549:2;4537:9;4528:7;4524:23;4520:32;4517:52;;;4565:1;4562;4555:12;4517:52;4605:9;4592:23;4634:18;4675:2;4667:6;4664:14;4661:34;;;4691:1;4688;4681:12;4661:34;4729:6;4718:9;4714:22;4704:32;;4774:7;4767:4;4763:2;4759:13;4755:27;4745:55;;4796:1;4793;4786:12;4745:55;4832:2;4819:16;4854:4;4878:60;4894:43;4934:2;4894:43;:::i;4878:60::-;4972:15;;;5050:11;;;5042:20;;5038:29;;;5003:12;;;;5079:19;;;5076:39;;;5111:1;5108;5101:12;5076:39;5135:11;;;;5155:217;5171:6;5166:3;5163:15;5155:217;;;5251:3;5238:17;5268:31;5293:5;5268:31;:::i;:::-;5312:18;;5188:12;;;;5350;;;;5155:217;;;5391:5;-1:-1:-1;;5434:18:17;;5421:32;;-1:-1:-1;;5465:16:17;;;5462:36;;;5494:1;5491;5484:12;5462:36;;5517:63;5572:7;5561:8;5550:9;5546:24;5517:63;:::i;:::-;5507:73;;;4370:1216;;;;;:::o;5851:456::-;5928:6;5936;5944;5997:2;5985:9;5976:7;5972:23;5968:32;5965:52;;;6013:1;6010;6003:12;5965:52;6052:9;6039:23;6071:31;6096:5;6071:31;:::i;:::-;6121:5;-1:-1:-1;6178:2:17;6163:18;;6150:32;6191:33;6150:32;6191:33;:::i;:::-;5851:456;;6243:7;;-1:-1:-1;;;6297:2:17;6282:18;;;;6269:32;;5851:456::o;6494:403::-;6577:6;6585;6638:2;6626:9;6617:7;6613:23;6609:32;6606:52;;;6654:1;6651;6644:12;6606:52;6693:9;6680:23;6712:31;6737:5;6712:31;:::i;:::-;6762:5;-1:-1:-1;6819:2:17;6804:18;;6791:32;6832:33;6791:32;6832:33;:::i;:::-;6884:7;6874:17;;;6494:403;;;;;:::o;6902:661::-;7024:6;7032;7040;7048;7056;7064;7072;7080;7133:3;7121:9;7112:7;7108:23;7104:33;7101:53;;;7150:1;7147;7140:12;7101:53;-1:-1:-1;;7173:23:17;;;7243:2;7228:18;;7215:32;;-1:-1:-1;7294:2:17;7279:18;;7266:32;;7345:2;7330:18;;7317:32;;-1:-1:-1;7396:3:17;7381:19;;7368:33;;-1:-1:-1;7448:3:17;7433:19;;7420:33;;-1:-1:-1;7500:3:17;7485:19;;7472:33;;-1:-1:-1;7552:3:17;7537:19;7524:33;;-1:-1:-1;6902:661:17;-1:-1:-1;6902:661:17:o;7568:370::-;7631:8;7641:6;7695:3;7688:4;7680:6;7676:17;7672:27;7662:55;;7713:1;7710;7703:12;7662:55;-1:-1:-1;7736:20:17;;7779:18;7768:30;;7765:50;;;7811:1;7808;7801:12;7765:50;7848:4;7840:6;7836:17;7824:29;;7911:3;7904:4;7896;7888:6;7884:17;7876:6;7872:30;7868:41;7865:50;7862:70;;;7928:1;7925;7918:12;7862:70;7568:370;;;;;:::o;7943:572::-;8038:6;8046;8054;8107:2;8095:9;8086:7;8082:23;8078:32;8075:52;;;8123:1;8120;8113:12;8075:52;8162:9;8149:23;8181:31;8206:5;8181:31;:::i;:::-;8231:5;-1:-1:-1;8287:2:17;8272:18;;8259:32;8314:18;8303:30;;8300:50;;;8346:1;8343;8336:12;8300:50;8385:70;8447:7;8438:6;8427:9;8423:22;8385:70;:::i;:::-;7943:572;;8474:8;;-1:-1:-1;8359:96:17;;-1:-1:-1;;;;7943:572:17:o;8705:407::-;8770:5;8804:18;8796:6;8793:30;8790:56;;;8826:18;;:::i;:::-;8864:57;8909:2;8888:15;;-1:-1:-1;;8884:29:17;8915:4;8880:40;8864:57;:::i;:::-;8855:66;;8944:6;8937:5;8930:21;8984:3;8975:6;8970:3;8966:16;8963:25;8960:45;;;9001:1;8998;8991:12;8960:45;9050:6;9045:3;9038:4;9031:5;9027:16;9014:43;9104:1;9097:4;9088:6;9081:5;9077:18;9073:29;9066:40;8705:407;;;;;:::o;9117:451::-;9186:6;9239:2;9227:9;9218:7;9214:23;9210:32;9207:52;;;9255:1;9252;9245:12;9207:52;9295:9;9282:23;9328:18;9320:6;9317:30;9314:50;;;9360:1;9357;9350:12;9314:50;9383:22;;9436:4;9428:13;;9424:27;-1:-1:-1;9414:55:17;;9465:1;9462;9455:12;9414:55;9488:74;9554:7;9549:2;9536:16;9531:2;9527;9523:11;9488:74;:::i;9573:118::-;9659:5;9652:13;9645:21;9638:5;9635:32;9625:60;;9681:1;9678;9671:12;9696:382;9761:6;9769;9822:2;9810:9;9801:7;9797:23;9793:32;9790:52;;;9838:1;9835;9828:12;9790:52;9877:9;9864:23;9896:31;9921:5;9896:31;:::i;:::-;9946:5;-1:-1:-1;10003:2:17;9988:18;;9975:32;10016:30;9975:32;10016:30;:::i;10083:795::-;10178:6;10186;10194;10202;10255:3;10243:9;10234:7;10230:23;10226:33;10223:53;;;10272:1;10269;10262:12;10223:53;10311:9;10298:23;10330:31;10355:5;10330:31;:::i;:::-;10380:5;-1:-1:-1;10437:2:17;10422:18;;10409:32;10450:33;10409:32;10450:33;:::i;:::-;10502:7;-1:-1:-1;10556:2:17;10541:18;;10528:32;;-1:-1:-1;10611:2:17;10596:18;;10583:32;10638:18;10627:30;;10624:50;;;10670:1;10667;10660:12;10624:50;10693:22;;10746:4;10738:13;;10734:27;-1:-1:-1;10724:55:17;;10775:1;10772;10765:12;10724:55;10798:74;10864:7;10859:2;10846:16;10841:2;10837;10833:11;10798:74;:::i;:::-;10788:84;;;10083:795;;;;;;;:::o;11150:505::-;11245:6;11253;11261;11314:2;11302:9;11293:7;11289:23;11285:32;11282:52;;;11330:1;11327;11320:12;11282:52;11366:9;11353:23;11343:33;;11427:2;11416:9;11412:18;11399:32;11454:18;11446:6;11443:30;11440:50;;;11486:1;11483;11476:12;12053:437;12138:1;12128:12;;12185:1;12175:12;;;12196:61;;12250:4;12242:6;12238:17;12228:27;;12196:61;12303:2;12295:6;12292:14;12272:18;12269:38;12266:218;;;-1:-1:-1;;;;;12337:1:17;12330:88;12441:4;12438:1;12431:15;12469:4;12466:1;12459:15;12266:218;;12053:437;;;:::o;13738:356::-;13940:2;13922:21;;;13959:18;;;13952:30;14018:34;14013:2;13998:18;;13991:62;14085:2;14070:18;;13738:356::o;14852:184::-;-1:-1:-1;;;;;14901:1:17;14894:88;15001:4;14998:1;14991:15;15025:4;15022:1;15015:15;15041:184;-1:-1:-1;;;;;15090:1:17;15083:88;15190:4;15187:1;15180:15;15214:4;15211:1;15204:15;15230:135;15269:3;-1:-1:-1;;15290:17:17;;15287:43;;;15310:18;;:::i;:::-;-1:-1:-1;15357:1:17;15346:13;;15230:135::o;15370:125::-;15410:4;15438:1;15435;15432:8;15429:34;;;15443:18;;:::i;:::-;-1:-1:-1;15480:9:17;;15370:125::o;15500:402::-;15702:2;15684:21;;;15741:2;15721:18;;;15714:30;15780:34;15775:2;15760:18;;15753:62;15851:8;15846:2;15831:18;;15824:36;15892:3;15877:19;;15500:402::o;15907:128::-;15947:3;15978:1;15974:6;15971:1;15968:13;15965:39;;;15984:18;;:::i;:::-;-1:-1:-1;16020:9:17;;15907:128::o;16040:407::-;16242:2;16224:21;;;16281:2;16261:18;;;16254:30;16320:34;16315:2;16300:18;;16293:62;16391:13;16386:2;16371:18;;16364:41;16437:3;16422:19;;16040:407::o;17580:184::-;17650:6;17703:2;17691:9;17682:7;17678:23;17674:32;17671:52;;;17719:1;17716;17709:12;17671:52;-1:-1:-1;17742:16:17;;17580:184;-1:-1:-1;17580:184:17:o;19619:415::-;19821:2;19803:21;;;19860:2;19840:18;;;19833:30;19899:34;19894:2;19879:18;;19872:62;19970:21;19965:2;19950:18;;19943:49;20024:3;20009:19;;19619:415::o;20455:185::-;20497:3;20535:5;20529:12;20550:52;20595:6;20590:3;20583:4;20576:5;20572:16;20550:52;:::i;:::-;20618:16;;;;;20455:185;-1:-1:-1;;20455:185:17:o;20645:470::-;20824:3;20862:6;20856:13;20878:53;20924:6;20919:3;20912:4;20904:6;20900:17;20878:53;:::i;:::-;20994:13;;20953:16;;;;21016:57;20994:13;20953:16;21050:4;21038:17;;21016:57;:::i;:::-;21089:20;;20645:470;-1:-1:-1;;;;20645:470:17:o;21120:340::-;21322:2;21304:21;;;21361:2;21341:18;;;21334:30;21400:18;21395:2;21380:18;;21373:46;21451:2;21436:18;;21120:340::o;22632:168::-;22672:7;22738:1;22734;22730:6;22726:14;22723:1;22720:21;22715:1;22708:9;22701:17;22697:45;22694:71;;;22745:18;;:::i;:::-;-1:-1:-1;22785:9:17;;22632:168::o;22805:184::-;-1:-1:-1;;;;;22854:1:17;22847:88;22954:4;22951:1;22944:15;22978:4;22975:1;22968:15;22994:120;23034:1;23060;23050:35;;23065:18;;:::i;:::-;-1:-1:-1;23099:9:17;;22994:120::o;25346:246::-;25386:4;-1:-1:-1;;;;;25499:10:17;;;;25469;;25521:12;;;25518:38;;;25536:18;;:::i;:::-;25573:13;;25346:246;-1:-1:-1;;;25346:246:17:o;25597:253::-;25637:3;-1:-1:-1;;;;;25726:2:17;25723:1;25719:10;25756:2;25753:1;25749:10;25787:3;25783:2;25779:12;25774:3;25771:21;25768:47;;;25795:18;;:::i;27018:136::-;27057:3;27085:5;27075:39;;27094:18;;:::i;:::-;-1:-1:-1;;;27130:18:17;;27018:136::o;27575:523::-;27769:4;-1:-1:-1;;;;;27879:2:17;27871:6;27867:15;27856:9;27849:34;27931:2;27923:6;27919:15;27914:2;27903:9;27899:18;27892:43;;27971:6;27966:2;27955:9;27951:18;27944:34;28014:3;28009:2;27998:9;27994:18;27987:31;28035:57;28087:3;28076:9;28072:19;28064:6;28035:57;:::i;:::-;28027:65;27575:523;-1:-1:-1;;;;;;27575:523:17:o;28103:249::-;28172:6;28225:2;28213:9;28204:7;28200:23;28196:32;28193:52;;;28241:1;28238;28231:12;28193:52;28273:9;28267:16;28292:30;28316:5;28292:30;:::i;28602:1362::-;28935:13;;28879:3;;;;29008:1;28993:17;;29029:1;29065:18;;;;29092:61;;29146:4;29138:6;29134:17;29124:27;;29092:61;29172:2;29220;29212:6;29209:14;29189:18;29186:38;29183:222;;;-1:-1:-1;;;;;29254:3:17;29247:90;29360:4;29357:1;29350:15;29390:4;29385:3;29378:17;29183:222;29421:18;29448:104;;;;29566:1;29561:320;;;;29414:467;;29448:104;-1:-1:-1;;29481:24:17;;29469:37;;29526:16;;;;-1:-1:-1;29448:104:17;;29561:320;28430:1;28423:14;;;28467:4;28454:18;;29656:1;29670:165;29684:6;29681:1;29678:13;29670:165;;;29762:14;;29749:11;;;29742:35;29805:16;;;;29699:10;;29670:165;;;29674:3;;29864:6;29859:3;29855:16;29848:23;;29414:467;;;;;;;29897:61;29927:30;29953:3;29945:6;29927:30;:::i;:::-;28560:3;28548:16;;28589:1;28580:11;;28483:114;29969:112;30001:1;30027;30017:35;;30032:18;;:::i;:::-;-1:-1:-1;30066:9:17;;29969:112::o;32479:245::-;32546:6;32599:2;32587:9;32578:7;32574:23;32570:32;32567:52;;;32615:1;32612;32605:12;32567:52;32647:9;32641:16;32666:28;32688:5;32666:28;:::i;34518:274::-;34647:3;34685:6;34679:13;34701:53;34747:6;34742:3;34735:4;34727:6;34723:17;34701:53;:::i;:::-;34770:16;;;;;34518:274;-1:-1:-1;;34518:274:17:o

Swarm Source

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