ETH Price: $3,521.31 (-2.14%)
Gas: 7 Gwei

Token

Cupcat Kittens (CCK)
 

Overview

Max Total Supply

8,681 CCK

Holders

2,778

Market

Volume (24H)

N/A

Min Price (24H)

N/A

Max Price (24H)

N/A
Filtered by Token Holder
infohazard.eth
Balance
1 CCK
0x8143aad694567424162a949c1580c91d03437858
Loading...
Loading
Loading...
Loading
Loading...
Loading

OVERVIEW

Cupcat Kittens are a collection made by Cupcats as 2nd season. This collection includes cute kittens that are part of Cupcats ecosystem.

# Exchange Pair Price  24H Volume % Volume

Contract Source Code Verified (Exact Match)

Contract Name:
CupcatKittens

Compiler Version
v0.8.4+commit.c7e474f2

Optimization Enabled:
No with 200 runs

Other Settings:
default evmVersion, None license
File 1 of 16 : CCK.sol
// SPDX-License-Identifier: MIT
pragma solidity ^0.8.4;
import "@openzeppelin/contracts/token/ERC721/extensions/ERC721Enumerable.sol";
import "@openzeppelin/contracts/access/Ownable.sol";
import "@openzeppelin/contracts/token/ERC721/IERC721.sol";
import "@openzeppelin/contracts/security/ReentrancyGuard.sol";
import "@openzeppelin/contracts/utils/cryptography/MerkleProof.sol";
import "@openzeppelin/contracts/utils/math/SafeMath.sol";

interface CupCatInterface is IERC721{
    function walletOfOwner(address _owner) external view returns (uint256[] memory);
}

contract CupcatKittens is ERC721Enumerable, Ownable, ReentrancyGuard  {  
    using SafeMath for uint256;
    uint256 public _tokenIdTrackerReserve;
    uint256 public _tokenIdTrackerSale;
    using Strings for uint256;
    uint256 public constant MAXCLAIMSUPPLY = 5025;
    uint256 public constant MAX_TOTAL_SUPPLY = 10000; 
    uint256 public constant MAXRESERVE = 225;
    uint256 public constant MAXSALE = MAX_TOTAL_SUPPLY - MAXCLAIMSUPPLY - MAXRESERVE;
    string public baseURI;
    string public baseExtension = ".json";
    uint256 public cost = 17500000000000000;
    bool public paused = false;
    bool public claimState = false;
    bool public saleState = false;
    bytes32 public merkleRoot = 0x0000000000000000000000000000000000000000000000000000000000000000;
    mapping(address => uint256) public addressMintedBalance;
    event MerkleRootUpdated(bytes32 new_merkle_root);
    CupCatInterface public cupCats;

constructor(
    ) ERC721("Cupcat Kittens", "CCK") {
    setBaseURI("exampleurl");
    setCupcats(0x8Cd8155e1af6AD31dd9Eec2cEd37e04145aCFCb3);
    }
    // internal
    function _baseURI() internal view virtual override returns (string memory) {
    return baseURI;
    }
    //Modify
    modifier claimIsOpen {
          require(claimState, "Claim is Closed");
          require(!paused, "Contract Paused");
          _;
      }
    modifier saleIsOpen {
          require(saleState, "Sale is Closed");
          require(!paused, "Contract Paused");
          _;
      }
    // public
    function whiteListMint(bytes32[] calldata _merkleProof ) public payable  {
          require(!paused, "the contract is paused");
          require(merkleRoot != 0x0000000000000000000000000000000000000000000000000000000000000000 , "White List Mints Closed");
          require(_tokenIdTrackerSale.add(1) <= MAXSALE, "Sold Out!");
          //Verify Already whiteListMint this Wallet
          require(addressMintedBalance[msg.sender] < 1 , "Already Claimed the whitelisted mint");
          //Merkle
          require(MerkleProof.verify(_merkleProof, merkleRoot,  keccak256(abi.encodePacked(msg.sender))  ), "Invalid proof");
          //verify Cost
          require(msg.value == cost.mul(1),  "Ether value sent is not correct");
          //Mark Claim
          addressMintedBalance[msg.sender]++;
          //Mint --
          _safeMint(_msgSender(), MAXCLAIMSUPPLY +  _tokenIdTrackerSale);
          _tokenIdTrackerSale += 1;
    }
    function mint(uint256 _count) public payable saleIsOpen nonReentrant{
          require(!paused, "the contract is paused");
          require(_tokenIdTrackerSale.add(_count) <= MAXSALE, "Sold Out!");
          require(_count > 0 && _count <= 9, "Can only mint 9 tokens at a time");
          require(msg.value==cost.mul(_count), "Ether value sent is not correct");
          for (uint256 i = 0; i < _count; i++) {
              addressMintedBalance[msg.sender]++;
              _safeMint(_msgSender(), MAXCLAIMSUPPLY  + _tokenIdTrackerSale);
              _tokenIdTrackerSale += 1;
          }
    }
    function claim(uint256[] memory _tokensId) public claimIsOpen {
          //Require claimIsOpen True
          for (uint256 i = 0; i < _tokensId.length; i++) {
          uint256 tokenId = _tokensId[i];
          require(_exists(tokenId) == false, "Already claimed!");
          require(tokenId < MAXCLAIMSUPPLY, "Post-claim cupcat!");
          require(cupCats.ownerOf(tokenId) == _msgSender(), "Bad owner!");
        _safeMint(_msgSender(), tokenId); 
          }
    }
    function reserve(uint256 _count) public onlyOwner {
          require(_tokenIdTrackerReserve + _count <= MAXRESERVE, "Exceeded giveaways.");
            for (uint256 i = 0; i < _count; i++) {
                  _safeMint(_msgSender(), MAXCLAIMSUPPLY + MAXSALE+ _tokenIdTrackerReserve);
                  _tokenIdTrackerReserve += 1;
            }
    }
    function checkClaim(uint256 _tokenId) public view returns(bool) {
        return _exists(_tokenId) == false;
    }
    function walletOfOwner(address _owner)
        public
        view
        returns (uint256[] memory)
        {
        uint256 ownerTokenCount = balanceOf(_owner);
        uint256[] memory tokenIds = new uint256[](ownerTokenCount);
        for (uint256 i; i < ownerTokenCount; i++) {
        tokenIds[i] = tokenOfOwnerByIndex(_owner, i);
        }
      return tokenIds;
    }
    function tokenURI(uint256 tokenId)
        public
        view
        virtual
        override
        returns (string memory)
      {
        require(
          _exists(tokenId),
          "ERC721Metadata: URI query for nonexistent token"
        );
        string memory currentBaseURI = _baseURI();
        return bytes(currentBaseURI).length > 0
            ? string(abi.encodePacked(currentBaseURI, tokenId.toString(), baseExtension))
            : "";
    }
    //only owner
    function setCupcats(address _cupCats) public onlyOwner {
        cupCats = CupCatInterface(_cupCats);
    }
    function setBaseURI(string memory _newBaseURI) public onlyOwner {
        baseURI = _newBaseURI;
    }
    function setBaseExtension(string memory _newBaseExtension) public onlyOwner {
        baseExtension = _newBaseExtension;
    }
    function pause(bool _state) public onlyOwner {
        paused = _state;
    }
    function setSaleState(bool _state) public onlyOwner{
        saleState = _state;
    }
    function setClaimState(bool _state) public onlyOwner {
        claimState = _state;
    }
    function withdraw() public payable onlyOwner {
        (bool os, ) = payable(owner()).call{value: address(this).balance}("");
        require(os);
    }
    // to set the merkle proof
    function updateMerkleRoot(bytes32 newmerkleRoot) external onlyOwner {
        merkleRoot = newmerkleRoot;
        emit MerkleRootUpdated(merkleRoot);
    }
}

File 2 of 16 : ERC721Enumerable.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (token/ERC721/extensions/ERC721Enumerable.sol)

pragma solidity ^0.8.0;

import "../ERC721.sol";
import "./IERC721Enumerable.sol";

/**
 * @dev This implements an optional extension of {ERC721} defined in the EIP that adds
 * enumerability of all the token ids in the contract as well as all token ids owned by each
 * account.
 */
abstract contract ERC721Enumerable is ERC721, IERC721Enumerable {
    // Mapping from owner to list of owned token IDs
    mapping(address => mapping(uint256 => uint256)) private _ownedTokens;

    // Mapping from token ID to index of the owner tokens list
    mapping(uint256 => uint256) private _ownedTokensIndex;

    // Array with all token ids, used for enumeration
    uint256[] private _allTokens;

    // Mapping from token id to position in the allTokens array
    mapping(uint256 => uint256) private _allTokensIndex;

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

    /**
     * @dev See {IERC721Enumerable-tokenOfOwnerByIndex}.
     */
    function tokenOfOwnerByIndex(address owner, uint256 index) public view virtual override returns (uint256) {
        require(index < ERC721.balanceOf(owner), "ERC721Enumerable: owner index out of bounds");
        return _ownedTokens[owner][index];
    }

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

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

    /**
     * @dev Hook that is called before any token transfer. This includes minting
     * and burning.
     *
     * Calling conditions:
     *
     * - When `from` and `to` are both non-zero, ``from``'s `tokenId` will be
     * transferred to `to`.
     * - When `from` is zero, `tokenId` will be minted for `to`.
     * - When `to` is zero, ``from``'s `tokenId` will be burned.
     * - `from` cannot be the zero address.
     * - `to` cannot be the zero address.
     *
     * To learn more about hooks, head to xref:ROOT:extending-contracts.adoc#using-hooks[Using Hooks].
     */
    function _beforeTokenTransfer(
        address from,
        address to,
        uint256 tokenId
    ) internal virtual override {
        super._beforeTokenTransfer(from, to, tokenId);

        if (from == address(0)) {
            _addTokenToAllTokensEnumeration(tokenId);
        } else if (from != to) {
            _removeTokenFromOwnerEnumeration(from, tokenId);
        }
        if (to == address(0)) {
            _removeTokenFromAllTokensEnumeration(tokenId);
        } else if (to != from) {
            _addTokenToOwnerEnumeration(to, tokenId);
        }
    }

    /**
     * @dev Private function to add a token to this extension's ownership-tracking data structures.
     * @param to address representing the new owner of the given token ID
     * @param tokenId uint256 ID of the token to be added to the tokens list of the given address
     */
    function _addTokenToOwnerEnumeration(address to, uint256 tokenId) private {
        uint256 length = ERC721.balanceOf(to);
        _ownedTokens[to][length] = tokenId;
        _ownedTokensIndex[tokenId] = length;
    }

    /**
     * @dev Private function to add a token to this extension's token tracking data structures.
     * @param tokenId uint256 ID of the token to be added to the tokens list
     */
    function _addTokenToAllTokensEnumeration(uint256 tokenId) private {
        _allTokensIndex[tokenId] = _allTokens.length;
        _allTokens.push(tokenId);
    }

    /**
     * @dev Private function to remove a token from this extension's ownership-tracking data structures. Note that
     * while the token is not assigned a new owner, the `_ownedTokensIndex` mapping is _not_ updated: this allows for
     * gas optimizations e.g. when performing a transfer operation (avoiding double writes).
     * This has O(1) time complexity, but alters the order of the _ownedTokens array.
     * @param from address representing the previous owner of the given token ID
     * @param tokenId uint256 ID of the token to be removed from the tokens list of the given address
     */
    function _removeTokenFromOwnerEnumeration(address from, uint256 tokenId) private {
        // To prevent a gap in from's tokens array, we store the last token in the index of the token to delete, and
        // then delete the last slot (swap and pop).

        uint256 lastTokenIndex = ERC721.balanceOf(from) - 1;
        uint256 tokenIndex = _ownedTokensIndex[tokenId];

        // When the token to delete is the last token, the swap operation is unnecessary
        if (tokenIndex != lastTokenIndex) {
            uint256 lastTokenId = _ownedTokens[from][lastTokenIndex];

            _ownedTokens[from][tokenIndex] = lastTokenId; // Move the last token to the slot of the to-delete token
            _ownedTokensIndex[lastTokenId] = tokenIndex; // Update the moved token's index
        }

        // This also deletes the contents at the last position of the array
        delete _ownedTokensIndex[tokenId];
        delete _ownedTokens[from][lastTokenIndex];
    }

    /**
     * @dev Private function to remove a token from this extension's token tracking data structures.
     * This has O(1) time complexity, but alters the order of the _allTokens array.
     * @param tokenId uint256 ID of the token to be removed from the tokens list
     */
    function _removeTokenFromAllTokensEnumeration(uint256 tokenId) private {
        // To prevent a gap in the tokens array, we store the last token in the index of the token to delete, and
        // then delete the last slot (swap and pop).

        uint256 lastTokenIndex = _allTokens.length - 1;
        uint256 tokenIndex = _allTokensIndex[tokenId];

        // When the token to delete is the last token, the swap operation is unnecessary. However, since this occurs so
        // rarely (when the last minted token is burnt) that we still do the swap here to avoid the gas cost of adding
        // an 'if' statement (like in _removeTokenFromOwnerEnumeration)
        uint256 lastTokenId = _allTokens[lastTokenIndex];

        _allTokens[tokenIndex] = lastTokenId; // Move the last token to the slot of the to-delete token
        _allTokensIndex[lastTokenId] = tokenIndex; // Update the moved token's index

        // This also deletes the contents at the last position of the array
        delete _allTokensIndex[tokenId];
        _allTokens.pop();
    }
}

File 3 of 16 : Ownable.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (access/Ownable.sol)

pragma solidity ^0.8.0;

import "../utils/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 4 of 16 : IERC721.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (token/ERC721/IERC721.sol)

pragma solidity ^0.8.0;

import "../../utils/introspection/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 5 of 16 : ReentrancyGuard.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (security/ReentrancyGuard.sol)

pragma solidity ^0.8.0;

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

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

    uint256 private _status;

    constructor() {
        _status = _NOT_ENTERED;
    }

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

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

        _;

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

File 6 of 16 : 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 7 of 16 : SafeMath.sol
// SPDX-License-Identifier: MIT
// OpenZeppelin Contracts v4.4.1 (utils/math/SafeMath.sol)

pragma solidity ^0.8.0;

// CAUTION
// This version of SafeMath should only be used with Solidity 0.8 or later,
// because it relies on the compiler's built in overflow checks.

/**
 * @dev Wrappers over Solidity's arithmetic operations.
 *
 * NOTE: `SafeMath` is generally not needed starting with Solidity 0.8, since the compiler
 * now has built in overflow checking.
 */
library SafeMath {
    /**
     * @dev Returns the addition of two unsigned integers, with an overflow flag.
     *
     * _Available since v3.4._
     */
    function tryAdd(uint256 a, uint256 b) internal pure returns (bool, uint256) {
        unchecked {
            uint256 c = a + b;
            if (c < a) return (false, 0);
            return (true, c);
        }
    }

    /**
     * @dev Returns the substraction of two unsigned integers, with an overflow flag.
     *
     * _Available since v3.4._
     */
    function trySub(uint256 a, uint256 b) internal pure returns (bool, uint256) {
        unchecked {
            if (b > a) return (false, 0);
            return (true, a - b);
        }
    }

    /**
     * @dev Returns the multiplication of two unsigned integers, with an overflow flag.
     *
     * _Available since v3.4._
     */
    function tryMul(uint256 a, uint256 b) internal pure returns (bool, uint256) {
        unchecked {
            // Gas optimization: this is cheaper than requiring 'a' not being zero, but the
            // benefit is lost if 'b' is also tested.
            // See: https://github.com/OpenZeppelin/openzeppelin-contracts/pull/522
            if (a == 0) return (true, 0);
            uint256 c = a * b;
            if (c / a != b) return (false, 0);
            return (true, c);
        }
    }

    /**
     * @dev Returns the division of two unsigned integers, with a division by zero flag.
     *
     * _Available since v3.4._
     */
    function tryDiv(uint256 a, uint256 b) internal pure returns (bool, uint256) {
        unchecked {
            if (b == 0) return (false, 0);
            return (true, a / b);
        }
    }

    /**
     * @dev Returns the remainder of dividing two unsigned integers, with a division by zero flag.
     *
     * _Available since v3.4._
     */
    function tryMod(uint256 a, uint256 b) internal pure returns (bool, uint256) {
        unchecked {
            if (b == 0) return (false, 0);
            return (true, a % b);
        }
    }

    /**
     * @dev Returns the addition of two unsigned integers, reverting on
     * overflow.
     *
     * Counterpart to Solidity's `+` operator.
     *
     * Requirements:
     *
     * - Addition cannot overflow.
     */
    function add(uint256 a, uint256 b) internal pure returns (uint256) {
        return a + b;
    }

    /**
     * @dev Returns the subtraction of two unsigned integers, reverting on
     * overflow (when the result is negative).
     *
     * Counterpart to Solidity's `-` operator.
     *
     * Requirements:
     *
     * - Subtraction cannot overflow.
     */
    function sub(uint256 a, uint256 b) internal pure returns (uint256) {
        return a - b;
    }

    /**
     * @dev Returns the multiplication of two unsigned integers, reverting on
     * overflow.
     *
     * Counterpart to Solidity's `*` operator.
     *
     * Requirements:
     *
     * - Multiplication cannot overflow.
     */
    function mul(uint256 a, uint256 b) internal pure returns (uint256) {
        return a * b;
    }

    /**
     * @dev Returns the integer division of two unsigned integers, reverting on
     * division by zero. The result is rounded towards zero.
     *
     * Counterpart to Solidity's `/` operator.
     *
     * Requirements:
     *
     * - The divisor cannot be zero.
     */
    function div(uint256 a, uint256 b) internal pure returns (uint256) {
        return a / b;
    }

    /**
     * @dev Returns the remainder of dividing two unsigned integers. (unsigned integer modulo),
     * reverting when dividing by zero.
     *
     * Counterpart to Solidity's `%` operator. This function uses a `revert`
     * opcode (which leaves remaining gas untouched) while Solidity uses an
     * invalid opcode to revert (consuming all remaining gas).
     *
     * Requirements:
     *
     * - The divisor cannot be zero.
     */
    function mod(uint256 a, uint256 b) internal pure returns (uint256) {
        return a % b;
    }

    /**
     * @dev Returns the subtraction of two unsigned integers, reverting with custom message on
     * overflow (when the result is negative).
     *
     * CAUTION: This function is deprecated because it requires allocating memory for the error
     * message unnecessarily. For custom revert reasons use {trySub}.
     *
     * Counterpart to Solidity's `-` operator.
     *
     * Requirements:
     *
     * - Subtraction cannot overflow.
     */
    function sub(
        uint256 a,
        uint256 b,
        string memory errorMessage
    ) internal pure returns (uint256) {
        unchecked {
            require(b <= a, errorMessage);
            return a - b;
        }
    }

    /**
     * @dev Returns the integer division of two unsigned integers, reverting with custom message on
     * division by zero. The result is rounded towards zero.
     *
     * Counterpart to Solidity's `/` operator. Note: this function uses a
     * `revert` opcode (which leaves remaining gas untouched) while Solidity
     * uses an invalid opcode to revert (consuming all remaining gas).
     *
     * Requirements:
     *
     * - The divisor cannot be zero.
     */
    function div(
        uint256 a,
        uint256 b,
        string memory errorMessage
    ) internal pure returns (uint256) {
        unchecked {
            require(b > 0, errorMessage);
            return a / b;
        }
    }

    /**
     * @dev Returns the remainder of dividing two unsigned integers. (unsigned integer modulo),
     * reverting with custom message when dividing by zero.
     *
     * CAUTION: This function is deprecated because it requires allocating memory for the error
     * message unnecessarily. For custom revert reasons use {tryMod}.
     *
     * Counterpart to Solidity's `%` operator. This function uses a `revert`
     * opcode (which leaves remaining gas untouched) while Solidity uses an
     * invalid opcode to revert (consuming all remaining gas).
     *
     * Requirements:
     *
     * - The divisor cannot be zero.
     */
    function mod(
        uint256 a,
        uint256 b,
        string memory errorMessage
    ) internal pure returns (uint256) {
        unchecked {
            require(b > 0, errorMessage);
            return a % b;
        }
    }
}

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

pragma solidity ^0.8.0;

import "./IERC721.sol";
import "./IERC721Receiver.sol";
import "./extensions/IERC721Metadata.sol";
import "../../utils/Address.sol";
import "../../utils/Context.sol";
import "../../utils/Strings.sol";
import "../../utils/introspection/ERC165.sol";

/**
 * @dev Implementation of https://eips.ethereum.org/EIPS/eip-721[ERC721] Non-Fungible Token Standard, including
 * the Metadata extension, but not including the Enumerable extension, which is available separately as
 * {ERC721Enumerable}.
 */
contract ERC721 is Context, ERC165, IERC721, IERC721Metadata {
    using Address for address;
    using Strings for uint256;

    // Token name
    string private _name;

    // Token symbol
    string private _symbol;

    // Mapping from token ID to owner address
    mapping(uint256 => address) private _owners;

    // Mapping owner address to token count
    mapping(address => uint256) private _balances;

    // 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 Initializes the contract by setting a `name` and a `symbol` to the token collection.
     */
    constructor(string memory name_, string memory symbol_) {
        _name = name_;
        _symbol = symbol_;
    }

    /**
     * @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 ||
            super.supportsInterface(interfaceId);
    }

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

    /**
     * @dev See {IERC721-ownerOf}.
     */
    function ownerOf(uint256 tokenId) public view virtual override returns (address) {
        address owner = _owners[tokenId];
        require(owner != address(0), "ERC721: owner query for nonexistent token");
        return owner;
    }

    /**
     * @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 virtual override {
        address owner = ERC721.ownerOf(tokenId);
        require(to != owner, "ERC721: approval to current owner");

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

        _approve(to, tokenId);
    }

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

        return _tokenApprovals[tokenId];
    }

    /**
     * @dev See {IERC721-setApprovalForAll}.
     */
    function setApprovalForAll(address operator, bool approved) public virtual override {
        _setApprovalForAll(_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 virtual override {
        //solhint-disable-next-line max-line-length
        require(_isApprovedOrOwner(_msgSender(), tokenId), "ERC721: transfer caller is not owner nor approved");

        _transfer(from, to, tokenId);
    }

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

    /**
     * @dev See {IERC721-safeTransferFrom}.
     */
    function safeTransferFrom(
        address from,
        address to,
        uint256 tokenId,
        bytes memory _data
    ) public virtual override {
        require(_isApprovedOrOwner(_msgSender(), tokenId), "ERC721: transfer caller is not owner nor approved");
        _safeTransfer(from, to, tokenId, _data);
    }

    /**
     * @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.
     *
     * `_data` is additional data, it has no specified format and it is sent in call to `to`.
     *
     * This internal function is equivalent to {safeTransferFrom}, and can be used to e.g.
     * implement alternative mechanisms to perform token transfer, such as signature-based.
     *
     * Requirements:
     *
     * - `from` cannot be the zero address.
     * - `to` cannot be the zero address.
     * - `tokenId` token must exist and be owned by `from`.
     * - If `to` refers to a smart contract, it must implement {IERC721Receiver-onERC721Received}, which is called upon a safe transfer.
     *
     * Emits a {Transfer} event.
     */
    function _safeTransfer(
        address from,
        address to,
        uint256 tokenId,
        bytes memory _data
    ) internal virtual {
        _transfer(from, to, tokenId);
        require(_checkOnERC721Received(from, to, tokenId, _data), "ERC721: 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`),
     * and stop existing when they are burned (`_burn`).
     */
    function _exists(uint256 tokenId) internal view virtual returns (bool) {
        return _owners[tokenId] != address(0);
    }

    /**
     * @dev Returns whether `spender` is allowed to manage `tokenId`.
     *
     * Requirements:
     *
     * - `tokenId` must exist.
     */
    function _isApprovedOrOwner(address spender, uint256 tokenId) internal view virtual returns (bool) {
        require(_exists(tokenId), "ERC721: operator query for nonexistent token");
        address owner = ERC721.ownerOf(tokenId);
        return (spender == owner || getApproved(tokenId) == spender || isApprovedForAll(owner, spender));
    }

    /**
     * @dev Safely mints `tokenId` and transfers it to `to`.
     *
     * Requirements:
     *
     * - `tokenId` must not exist.
     * - If `to` refers to a smart contract, it must implement {IERC721Receiver-onERC721Received}, which is called upon a safe transfer.
     *
     * Emits a {Transfer} event.
     */
    function _safeMint(address to, uint256 tokenId) internal virtual {
        _safeMint(to, tokenId, "");
    }

    /**
     * @dev Same as {xref-ERC721-_safeMint-address-uint256-}[`_safeMint`], with an additional `data` parameter which is
     * forwarded in {IERC721Receiver-onERC721Received} to contract recipients.
     */
    function _safeMint(
        address to,
        uint256 tokenId,
        bytes memory _data
    ) internal virtual {
        _mint(to, tokenId);
        require(
            _checkOnERC721Received(address(0), to, tokenId, _data),
            "ERC721: transfer to non ERC721Receiver implementer"
        );
    }

    /**
     * @dev Mints `tokenId` and transfers it to `to`.
     *
     * WARNING: Usage of this method is discouraged, use {_safeMint} whenever possible
     *
     * Requirements:
     *
     * - `tokenId` must not exist.
     * - `to` cannot be the zero address.
     *
     * Emits a {Transfer} event.
     */
    function _mint(address to, uint256 tokenId) internal virtual {
        require(to != address(0), "ERC721: mint to the zero address");
        require(!_exists(tokenId), "ERC721: token already minted");

        _beforeTokenTransfer(address(0), to, tokenId);

        _balances[to] += 1;
        _owners[tokenId] = to;

        emit Transfer(address(0), to, tokenId);
    }

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

        _beforeTokenTransfer(owner, address(0), tokenId);

        // Clear approvals
        _approve(address(0), tokenId);

        _balances[owner] -= 1;
        delete _owners[tokenId];

        emit Transfer(owner, address(0), tokenId);
    }

    /**
     * @dev Transfers `tokenId` from `from` to `to`.
     *  As opposed to {transferFrom}, this imposes no restrictions on msg.sender.
     *
     * 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
    ) internal virtual {
        require(ERC721.ownerOf(tokenId) == from, "ERC721: transfer of token that is not own");
        require(to != address(0), "ERC721: transfer to the zero address");

        _beforeTokenTransfer(from, to, tokenId);

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

        _balances[from] -= 1;
        _balances[to] += 1;
        _owners[tokenId] = to;

        emit Transfer(from, to, tokenId);
    }

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

    /**
     * @dev Approve `operator` to operate on all of `owner` tokens
     *
     * Emits a {ApprovalForAll} event.
     */
    function _setApprovalForAll(
        address owner,
        address operator,
        bool approved
    ) internal virtual {
        require(owner != operator, "ERC721: approve to caller");
        _operatorApprovals[owner][operator] = approved;
        emit ApprovalForAll(owner, operator, approved);
    }

    /**
     * @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.onERC721Received.selector;
            } catch (bytes memory reason) {
                if (reason.length == 0) {
                    revert("ERC721: transfer to non ERC721Receiver implementer");
                } else {
                    assembly {
                        revert(add(32, reason), mload(reason))
                    }
                }
            }
        } else {
            return true;
        }
    }

    /**
     * @dev Hook that is called before any token transfer. This includes minting
     * and burning.
     *
     * Calling conditions:
     *
     * - When `from` and `to` are both non-zero, ``from``'s `tokenId` will be
     * transferred to `to`.
     * - When `from` is zero, `tokenId` will be minted for `to`.
     * - When `to` is zero, ``from``'s `tokenId` will be burned.
     * - `from` and `to` are never both zero.
     *
     * To learn more about hooks, head to xref:ROOT:extending-contracts.adoc#using-hooks[Using Hooks].
     */
    function _beforeTokenTransfer(
        address from,
        address to,
        uint256 tokenId
    ) internal virtual {}
}

File 9 of 16 : 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 16 : 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 11 of 16 : 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 12 of 16 : 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 13 of 16 : 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 14 of 16 : 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);
    }
}

File 15 of 16 : 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 16 of 16 : 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);
}

Settings
{
  "optimizer": {
    "enabled": false,
    "runs": 200
  },
  "outputSelection": {
    "*": {
      "*": [
        "evm.bytecode",
        "evm.deployedBytecode",
        "abi"
      ]
    }
  }
}

Contract Security Audit

Contract ABI

[{"inputs":[],"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":false,"internalType":"bytes32","name":"new_merkle_root","type":"bytes32"}],"name":"MerkleRootUpdated","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"previousOwner","type":"address"},{"indexed":true,"internalType":"address","name":"newOwner","type":"address"}],"name":"OwnershipTransferred","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Transfer","type":"event"},{"inputs":[],"name":"MAXCLAIMSUPPLY","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"MAXRESERVE","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"MAXSALE","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"MAX_TOTAL_SUPPLY","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"_tokenIdTrackerReserve","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"_tokenIdTrackerSale","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"addressMintedBalance","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":[],"name":"baseExtension","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"baseURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"_tokenId","type":"uint256"}],"name":"checkClaim","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256[]","name":"_tokensId","type":"uint256[]"}],"name":"claim","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"claimState","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"cost","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"cupCats","outputs":[{"internalType":"contract CupCatInterface","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"getApproved","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"},{"internalType":"address","name":"operator","type":"address"}],"name":"isApprovedForAll","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"merkleRoot","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[{"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":"owner","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"ownerOf","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"bool","name":"_state","type":"bool"}],"name":"pause","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"paused","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_count","type":"uint256"}],"name":"reserve","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":[],"name":"saleState","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","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":"_newBaseExtension","type":"string"}],"name":"setBaseExtension","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"_newBaseURI","type":"string"}],"name":"setBaseURI","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bool","name":"_state","type":"bool"}],"name":"setClaimState","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"_cupCats","type":"address"}],"name":"setCupcats","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bool","name":"_state","type":"bool"}],"name":"setSaleState","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes4","name":"interfaceId","type":"bytes4"}],"name":"supportsInterface","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"symbol","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"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":[],"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":[{"internalType":"bytes32","name":"newmerkleRoot","type":"bytes32"}],"name":"updateMerkleRoot","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"_owner","type":"address"}],"name":"walletOfOwner","outputs":[{"internalType":"uint256[]","name":"","type":"uint256[]"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"bytes32[]","name":"_merkleProof","type":"bytes32[]"}],"name":"whiteListMint","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[],"name":"withdraw","outputs":[],"stateMutability":"payable","type":"function"}]

60806040526040518060400160405280600581526020017f2e6a736f6e000000000000000000000000000000000000000000000000000000815250600f90805190602001906200005192919062000472565b50663e2c284391c0006010556000601160006101000a81548160ff0219169083151502179055506000601160016101000a81548160ff0219169083151502179055506000601160026101000a81548160ff0219169083151502179055506000801b601255348015620000c257600080fd5b506040518060400160405280600e81526020017f437570636174204b697474656e730000000000000000000000000000000000008152506040518060400160405280600381526020017f43434b000000000000000000000000000000000000000000000000000000000081525081600090805190602001906200014792919062000472565b5080600190805190602001906200016092919062000472565b5050506200018362000177620001fc60201b60201c565b6200020460201b60201c565b6001600b81905550620001d16040518060400160405280600a81526020017f6578616d706c6575726c00000000000000000000000000000000000000000000815250620002ca60201b60201c565b620001f6738cd8155e1af6ad31dd9eec2ced37e04145acfcb36200037560201b60201c565b6200060a565b600033905090565b6000600a60009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600a60006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b620002da620001fc60201b60201c565b73ffffffffffffffffffffffffffffffffffffffff16620003006200044860201b60201c565b73ffffffffffffffffffffffffffffffffffffffff161462000359576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401620003509062000549565b60405180910390fd5b80600e90805190602001906200037192919062000472565b5050565b62000385620001fc60201b60201c565b73ffffffffffffffffffffffffffffffffffffffff16620003ab6200044860201b60201c565b73ffffffffffffffffffffffffffffffffffffffff161462000404576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401620003fb9062000549565b60405180910390fd5b80601460006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555050565b6000600a60009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b82805462000480906200057c565b90600052602060002090601f016020900481019282620004a45760008555620004f0565b82601f10620004bf57805160ff1916838001178555620004f0565b82800160010185558215620004f0579182015b82811115620004ef578251825591602001919060010190620004d2565b5b509050620004ff919062000503565b5090565b5b808211156200051e57600081600090555060010162000504565b5090565b6000620005316020836200056b565b91506200053e82620005e1565b602082019050919050565b60006020820190508181036000830152620005648162000522565b9050919050565b600082825260208201905092915050565b600060028204905060018216806200059557607f821691505b60208210811415620005ac57620005ab620005b2565b5b50919050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b615bcb806200061a6000396000f3fe6080604052600436106102935760003560e01c80636ba4c1381161015a578063b88d4fde116100c1578063da3ef23f1161007a578063da3ef23f146109ed578063dc559fce14610a16578063e985e9c514610a41578063f1c51b3914610a7e578063f2fde38b14610aa9578063f94a279b14610ad257610293565b8063b88d4fde146108df578063b90ae3ed14610908578063c4e3709514610933578063c66828621461095c578063c87b56dd14610987578063d1be66ba146109c457610293565b806395d89b411161011357806395d89b41146107fd57806397254e55146108285780639a72580914610844578063a0712d681461086f578063a22cb4651461088b578063aaa25f4e146108b457610293565b80636ba4c138146107015780636c0360eb1461072a57806370a0823114610755578063715018a614610792578063819b25ba146107a95780638da5cb5b146107d257610293565b80632f745c59116101fe5780634b014e28116101b75780634b014e28146105df5780634f6ccce71461060857806355f804b3146106455780635c975abb1461066e578063603f4d52146106995780636352211e146106c457610293565b80632f745c59146104de57806333039d3d1461051b5780633ccfd60b1461054657806342842e0e14610550578063438b6300146105795780634783f0ef146105b657610293565b806313faede61161025057806313faede6146103ba5780631681d158146103e557806318160ddd1461042257806318cae2691461044d57806323b872dd1461048a5780632eb4a7ab146104b357610293565b806301e05ba41461029857806301ffc9a7146102c357806302329a291461030057806306fdde0314610329578063081812fc14610354578063095ea7b314610391575b600080fd5b3480156102a457600080fd5b506102ad610afd565b6040516102ba9190614e54565b60405180910390f35b3480156102cf57600080fd5b506102ea60048036038101906102e59190614129565b610b03565b6040516102f791906149c1565b60405180910390f35b34801561030c57600080fd5b50610327600480360381019061032291906140d7565b610b7d565b005b34801561033557600080fd5b5061033e610c16565b60405161034b9190614a12565b60405180910390f35b34801561036057600080fd5b5061037b600480360381019061037691906141bc565b610ca8565b6040516103889190614938565b60405180910390f35b34801561039d57600080fd5b506103b860048036038101906103b39190614015565b610d2d565b005b3480156103c657600080fd5b506103cf610e45565b6040516103dc9190614e54565b60405180910390f35b3480156103f157600080fd5b5061040c600480360381019061040791906141bc565b610e4b565b60405161041991906149c1565b60405180910390f35b34801561042e57600080fd5b50610437610e63565b6040516104449190614e54565b60405180910390f35b34801561045957600080fd5b50610474600480360381019061046f9190613e81565b610e70565b6040516104819190614e54565b60405180910390f35b34801561049657600080fd5b506104b160048036038101906104ac9190613f0f565b610e88565b005b3480156104bf57600080fd5b506104c8610ee8565b6040516104d591906149dc565b60405180910390f35b3480156104ea57600080fd5b5061050560048036038101906105009190614015565b610eee565b6040516105129190614e54565b60405180910390f35b34801561052757600080fd5b50610530610f93565b60405161053d9190614e54565b60405180910390f35b61054e610f99565b005b34801561055c57600080fd5b5061057760048036038101906105729190613f0f565b611095565b005b34801561058557600080fd5b506105a0600480360381019061059b9190613e81565b6110b5565b6040516105ad919061499f565b60405180910390f35b3480156105c257600080fd5b506105dd60048036038101906105d89190614100565b6111af565b005b3480156105eb57600080fd5b50610606600480360381019061060191906140d7565b61126e565b005b34801561061457600080fd5b5061062f600480360381019061062a91906141bc565b611307565b60405161063c9190614e54565b60405180910390f35b34801561065157600080fd5b5061066c6004803603810190610667919061417b565b61139e565b005b34801561067a57600080fd5b50610683611434565b60405161069091906149c1565b60405180910390f35b3480156106a557600080fd5b506106ae611447565b6040516106bb91906149c1565b60405180910390f35b3480156106d057600080fd5b506106eb60048036038101906106e691906141bc565b61145a565b6040516106f89190614938565b60405180910390f35b34801561070d57600080fd5b5061072860048036038101906107239190614096565b61150c565b005b34801561073657600080fd5b5061073f6117d7565b60405161074c9190614a12565b60405180910390f35b34801561076157600080fd5b5061077c60048036038101906107779190613e81565b611865565b6040516107899190614e54565b60405180910390f35b34801561079e57600080fd5b506107a761191d565b005b3480156107b557600080fd5b506107d060048036038101906107cb91906141bc565b6119a5565b005b3480156107de57600080fd5b506107e7611af4565b6040516107f49190614938565b60405180910390f35b34801561080957600080fd5b50610812611b1e565b60405161081f9190614a12565b60405180910390f35b610842600480360381019061083d9190614051565b611bb0565b005b34801561085057600080fd5b50610859611eda565b60405161086691906149c1565b60405180910390f35b610889600480360381019061088491906141bc565b611eed565b005b34801561089757600080fd5b506108b260048036038101906108ad9190613fd9565b6121fb565b005b3480156108c057600080fd5b506108c9612211565b6040516108d69190614e54565b60405180910390f35b3480156108eb57600080fd5b5061090660048036038101906109019190613f5e565b612230565b005b34801561091457600080fd5b5061091d612292565b60405161092a91906149f7565b60405180910390f35b34801561093f57600080fd5b5061095a600480360381019061095591906140d7565b6122b8565b005b34801561096857600080fd5b50610971612351565b60405161097e9190614a12565b60405180910390f35b34801561099357600080fd5b506109ae60048036038101906109a991906141bc565b6123df565b6040516109bb9190614a12565b60405180910390f35b3480156109d057600080fd5b506109eb60048036038101906109e69190613e81565b612489565b005b3480156109f957600080fd5b50610a146004803603810190610a0f919061417b565b612549565b005b348015610a2257600080fd5b50610a2b6125df565b604051610a389190614e54565b60405180910390f35b348015610a4d57600080fd5b50610a686004803603810190610a639190613ed3565b6125e5565b604051610a7591906149c1565b60405180910390f35b348015610a8a57600080fd5b50610a93612679565b604051610aa09190614e54565b60405180910390f35b348015610ab557600080fd5b50610ad06004803603810190610acb9190613e81565b61267f565b005b348015610ade57600080fd5b50610ae7612777565b604051610af49190614e54565b60405180910390f35b6113a181565b60007f780e9d63000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff19161480610b765750610b758261277c565b5b9050919050565b610b8561285e565b73ffffffffffffffffffffffffffffffffffffffff16610ba3611af4565b73ffffffffffffffffffffffffffffffffffffffff1614610bf9576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610bf090614c74565b60405180910390fd5b80601160006101000a81548160ff02191690831515021790555050565b606060008054610c25906151b7565b80601f0160208091040260200160405190810160405280929190818152602001828054610c51906151b7565b8015610c9e5780601f10610c7357610100808354040283529160200191610c9e565b820191906000526020600020905b815481529060010190602001808311610c8157829003601f168201915b5050505050905090565b6000610cb382612866565b610cf2576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610ce990614c54565b60405180910390fd5b6004600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff169050919050565b6000610d388261145a565b90508073ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff161415610da9576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610da090614d54565b60405180910390fd5b8073ffffffffffffffffffffffffffffffffffffffff16610dc861285e565b73ffffffffffffffffffffffffffffffffffffffff161480610df75750610df681610df161285e565b6125e5565b5b610e36576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610e2d90614bb4565b60405180910390fd5b610e4083836128d2565b505050565b60105481565b6000801515610e5983612866565b1515149050919050565b6000600880549050905090565b60136020528060005260406000206000915090505481565b610e99610e9361285e565b8261298b565b610ed8576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610ecf90614d94565b60405180910390fd5b610ee3838383612a69565b505050565b60125481565b6000610ef983611865565b8210610f3a576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610f3190614a74565b60405180910390fd5b600660008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600083815260200190815260200160002054905092915050565b61271081565b610fa161285e565b73ffffffffffffffffffffffffffffffffffffffff16610fbf611af4565b73ffffffffffffffffffffffffffffffffffffffff1614611015576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161100c90614c74565b60405180910390fd5b600061101f611af4565b73ffffffffffffffffffffffffffffffffffffffff164760405161104290614923565b60006040518083038185875af1925050503d806000811461107f576040519150601f19603f3d011682016040523d82523d6000602084013e611084565b606091505b505090508061109257600080fd5b50565b6110b083838360405180602001604052806000815250612230565b505050565b606060006110c283611865565b905060008167ffffffffffffffff811115611106577f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b6040519080825280602002602001820160405280156111345781602001602082028036833780820191505090505b50905060005b828110156111a45761114c8582610eee565b828281518110611185577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b602002602001018181525050808061119c9061521a565b91505061113a565b508092505050919050565b6111b761285e565b73ffffffffffffffffffffffffffffffffffffffff166111d5611af4565b73ffffffffffffffffffffffffffffffffffffffff161461122b576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161122290614c74565b60405180910390fd5b806012819055507f90004c04698bc3322499a575ed3752dd4abf33e0a7294c06a787a0fe01bea94160125460405161126391906149dc565b60405180910390a150565b61127661285e565b73ffffffffffffffffffffffffffffffffffffffff16611294611af4565b73ffffffffffffffffffffffffffffffffffffffff16146112ea576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016112e190614c74565b60405180910390fd5b80601160016101000a81548160ff02191690831515021790555050565b6000611311610e63565b8210611352576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161134990614db4565b60405180910390fd5b6008828154811061138c577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b90600052602060002001549050919050565b6113a661285e565b73ffffffffffffffffffffffffffffffffffffffff166113c4611af4565b73ffffffffffffffffffffffffffffffffffffffff161461141a576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161141190614c74565b60405180910390fd5b80600e9080519060200190611430929190613b9b565b5050565b601160009054906101000a900460ff1681565b601160029054906101000a900460ff1681565b6000806002600084815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff169050600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff161415611503576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016114fa90614bf4565b60405180910390fd5b80915050919050565b601160019054906101000a900460ff1661155b576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161155290614c14565b60405180910390fd5b601160009054906101000a900460ff16156115ab576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016115a290614e34565b60405180910390fd5b60005b81518110156117d35760008282815181106115f2577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b602002602001015190506000151561160982612866565b15151461164b576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161164290614a54565b60405180910390fd5b6113a1811061168f576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161168690614cb4565b60405180910390fd5b61169761285e565b73ffffffffffffffffffffffffffffffffffffffff16601460009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16636352211e836040518263ffffffff1660e01b81526004016117089190614e54565b60206040518083038186803b15801561172057600080fd5b505afa158015611734573d6000803e3d6000fd5b505050506040513d601f19601f820116820180604052508101906117589190613eaa565b73ffffffffffffffffffffffffffffffffffffffff16146117ae576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016117a590614b14565b60405180910390fd5b6117bf6117b961285e565b82612cc5565b5080806117cb9061521a565b9150506115ae565b5050565b600e80546117e4906151b7565b80601f0160208091040260200160405190810160405280929190818152602001828054611810906151b7565b801561185d5780601f106118325761010080835404028352916020019161185d565b820191906000526020600020905b81548152906001019060200180831161184057829003601f168201915b505050505081565b60008073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff1614156118d6576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016118cd90614bd4565b60405180910390fd5b600360008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020549050919050565b61192561285e565b73ffffffffffffffffffffffffffffffffffffffff16611943611af4565b73ffffffffffffffffffffffffffffffffffffffff1614611999576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161199090614c74565b60405180910390fd5b6119a36000612ce3565b565b6119ad61285e565b73ffffffffffffffffffffffffffffffffffffffff166119cb611af4565b73ffffffffffffffffffffffffffffffffffffffff1614611a21576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611a1890614c74565b60405180910390fd5b60e181600c54611a319190614fbe565b1115611a72576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611a6990614a34565b60405180910390fd5b60005b81811015611af057611ac3611a8861285e565b600c5460e16113a1612710611a9d919061509f565b611aa7919061509f565b6113a1611ab49190614fbe565b611abe9190614fbe565b612cc5565b6001600c6000828254611ad69190614fbe565b925050819055508080611ae89061521a565b915050611a75565b5050565b6000600a60009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b606060018054611b2d906151b7565b80601f0160208091040260200160405190810160405280929190818152602001828054611b59906151b7565b8015611ba65780601f10611b7b57610100808354040283529160200191611ba6565b820191906000526020600020905b815481529060010190602001808311611b8957829003601f168201915b5050505050905090565b601160009054906101000a900460ff1615611c00576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611bf790614cd4565b60405180910390fd5b6000801b6012541415611c48576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611c3f90614d34565b60405180910390fd5b60e16113a1612710611c5a919061509f565b611c64919061509f565b611c7a6001600d54612da990919063ffffffff16565b1115611cbb576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611cb290614ad4565b60405180910390fd5b6001601360003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000205410611d3d576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611d3490614c94565b60405180910390fd5b611db1828280806020026020016040519081016040528093929190818152602001838360200280828437600081840152601f19601f8201169050808301925050505050505060125433604051602001611d9691906148ab565b60405160208183030381529060405280519060200120612dbf565b611df0576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611de790614dd4565b60405180910390fd5b611e066001601054612dd690919063ffffffff16565b3414611e47576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611e3e90614b74565b60405180910390fd5b601360003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000815480929190611e979061521a565b9190505550611ebc611ea761285e565b600d546113a1611eb79190614fbe565b612cc5565b6001600d6000828254611ecf9190614fbe565b925050819055505050565b601160019054906101000a900460ff1681565b601160029054906101000a900460ff16611f3c576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611f3390614d74565b60405180910390fd5b601160009054906101000a900460ff1615611f8c576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611f8390614e34565b60405180910390fd5b6002600b541415611fd2576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611fc990614e14565b60405180910390fd5b6002600b81905550601160009054906101000a900460ff161561202a576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161202190614cd4565b60405180910390fd5b60e16113a161271061203c919061509f565b612046919061509f565b61205b82600d54612da990919063ffffffff16565b111561209c576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161209390614ad4565b60405180910390fd5b6000811180156120ad575060098111155b6120ec576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016120e390614df4565b60405180910390fd5b61210181601054612dd690919063ffffffff16565b3414612142576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161213990614b74565b60405180910390fd5b60005b818110156121ef57601360003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600081548092919061219d9061521a565b91905055506121c26121ad61285e565b600d546113a16121bd9190614fbe565b612cc5565b6001600d60008282546121d59190614fbe565b9250508190555080806121e79061521a565b915050612145565b506001600b8190555050565b61220d61220661285e565b8383612dec565b5050565b60e16113a1612710612223919061509f565b61222d919061509f565b81565b61224161223b61285e565b8361298b565b612280576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161227790614d94565b60405180910390fd5b61228c84848484612f59565b50505050565b601460009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1681565b6122c061285e565b73ffffffffffffffffffffffffffffffffffffffff166122de611af4565b73ffffffffffffffffffffffffffffffffffffffff1614612334576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161232b90614c74565b60405180910390fd5b80601160026101000a81548160ff02191690831515021790555050565b600f805461235e906151b7565b80601f016020809104026020016040519081016040528092919081815260200182805461238a906151b7565b80156123d75780601f106123ac576101008083540402835291602001916123d7565b820191906000526020600020905b8154815290600101906020018083116123ba57829003601f168201915b505050505081565b60606123ea82612866565b612429576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161242090614d14565b60405180910390fd5b6000612433612fb5565b905060008151116124535760405180602001604052806000815250612481565b8061245d84613047565b600f604051602001612471939291906148f2565b6040516020818303038152906040525b915050919050565b61249161285e565b73ffffffffffffffffffffffffffffffffffffffff166124af611af4565b73ffffffffffffffffffffffffffffffffffffffff1614612505576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016124fc90614c74565b60405180910390fd5b80601460006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555050565b61255161285e565b73ffffffffffffffffffffffffffffffffffffffff1661256f611af4565b73ffffffffffffffffffffffffffffffffffffffff16146125c5576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016125bc90614c74565b60405180910390fd5b80600f90805190602001906125db929190613b9b565b5050565b600d5481565b6000600560008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff16905092915050565b600c5481565b61268761285e565b73ffffffffffffffffffffffffffffffffffffffff166126a5611af4565b73ffffffffffffffffffffffffffffffffffffffff16146126fb576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016126f290614c74565b60405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff16141561276b576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161276290614ab4565b60405180910390fd5b61277481612ce3565b50565b60e181565b60007f80ac58cd000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916148061284757507f5b5e139f000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b806128575750612856826131f4565b5b9050919050565b600033905090565b60008073ffffffffffffffffffffffffffffffffffffffff166002600084815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1614159050919050565b816004600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550808273ffffffffffffffffffffffffffffffffffffffff166129458361145a565b73ffffffffffffffffffffffffffffffffffffffff167f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92560405160405180910390a45050565b600061299682612866565b6129d5576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016129cc90614b94565b60405180910390fd5b60006129e08361145a565b90508073ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff161480612a4f57508373ffffffffffffffffffffffffffffffffffffffff16612a3784610ca8565b73ffffffffffffffffffffffffffffffffffffffff16145b80612a605750612a5f81856125e5565b5b91505092915050565b8273ffffffffffffffffffffffffffffffffffffffff16612a898261145a565b73ffffffffffffffffffffffffffffffffffffffff1614612adf576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612ad690614cf4565b60405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415612b4f576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612b4690614b34565b60405180910390fd5b612b5a83838361325e565b612b656000826128d2565b6001600360008573ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254612bb5919061509f565b925050819055506001600360008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254612c0c9190614fbe565b92505081905550816002600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550808273ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4505050565b612cdf828260405180602001604052806000815250613372565b5050565b6000600a60009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600a60006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b60008183612db79190614fbe565b905092915050565b600082612dcc85846133cd565b1490509392505050565b60008183612de49190615045565b905092915050565b8173ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff161415612e5b576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612e5290614b54565b60405180910390fd5b80600560008573ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060006101000a81548160ff0219169083151502179055508173ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff167f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c3183604051612f4c91906149c1565b60405180910390a3505050565b612f64848484612a69565b612f70848484846134a6565b612faf576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612fa690614a94565b60405180910390fd5b50505050565b6060600e8054612fc4906151b7565b80601f0160208091040260200160405190810160405280929190818152602001828054612ff0906151b7565b801561303d5780601f106130125761010080835404028352916020019161303d565b820191906000526020600020905b81548152906001019060200180831161302057829003601f168201915b5050505050905090565b6060600082141561308f576040518060400160405280600181526020017f300000000000000000000000000000000000000000000000000000000000000081525090506131ef565b600082905060005b600082146130c15780806130aa9061521a565b915050600a826130ba9190615014565b9150613097565b60008167ffffffffffffffff811115613103577f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b6040519080825280601f01601f1916602001820160405280156131355781602001600182028036833780820191505090505b5090505b600085146131e85760018261314e919061509f565b9150600a8561315d9190615291565b60306131699190614fbe565b60f81b8183815181106131a5577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b60200101907effffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916908160001a905350600a856131e19190615014565b9450613139565b8093505050505b919050565b60007f01ffc9a7000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916149050919050565b61326983838361363d565b600073ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff1614156132ac576132a781613642565b6132eb565b8173ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff16146132ea576132e9838261368b565b5b5b600073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff16141561332e57613329816137f8565b61336d565b8273ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161461336c5761336b828261393b565b5b5b505050565b61337c83836139ba565b61338960008484846134a6565b6133c8576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016133bf90614a94565b60405180910390fd5b505050565b60008082905060005b845181101561349b57600085828151811061341a577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b6020026020010151905080831161345b57828160405160200161343e9291906148c6565b604051602081830303815290604052805190602001209250613487565b808360405160200161346e9291906148c6565b6040516020818303038152906040528051906020012092505b5080806134939061521a565b9150506133d6565b508091505092915050565b60006134c78473ffffffffffffffffffffffffffffffffffffffff16613b88565b15613630578373ffffffffffffffffffffffffffffffffffffffff1663150b7a026134f061285e565b8786866040518563ffffffff1660e01b81526004016135129493929190614953565b602060405180830381600087803b15801561352c57600080fd5b505af192505050801561355d57506040513d601f19601f8201168201806040525081019061355a9190614152565b60015b6135e0573d806000811461358d576040519150601f19603f3d011682016040523d82523d6000602084013e613592565b606091505b506000815114156135d8576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016135cf90614a94565b60405180910390fd5b805181602001fd5b63150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916817bffffffffffffffffffffffffffffffffffffffffffffffffffffffff191614915050613635565b600190505b949350505050565b505050565b6008805490506009600083815260200190815260200160002081905550600881908060018154018082558091505060019003906000526020600020016000909190919091505550565b6000600161369884611865565b6136a2919061509f565b9050600060076000848152602001908152602001600020549050818114613787576000600660008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600084815260200190815260200160002054905080600660008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600084815260200190815260200160002081905550816007600083815260200190815260200160002081905550505b6007600084815260200190815260200160002060009055600660008573ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008381526020019081526020016000206000905550505050565b6000600160088054905061380c919061509f565b9050600060096000848152602001908152602001600020549050600060088381548110613862577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b9060005260206000200154905080600883815481106138aa577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b90600052602060002001819055508160096000838152602001908152602001600020819055506009600085815260200190815260200160002060009055600880548061391f577f4e487b7100000000000000000000000000000000000000000000000000000000600052603160045260246000fd5b6001900381819060005260206000200160009055905550505050565b600061394683611865565b905081600660008573ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600083815260200190815260200160002081905550806007600084815260200190815260200160002081905550505050565b600073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415613a2a576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401613a2190614c34565b60405180910390fd5b613a3381612866565b15613a73576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401613a6a90614af4565b60405180910390fd5b613a7f6000838361325e565b6001600360008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254613acf9190614fbe565b92505081905550816002600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550808273ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a45050565b600080823b905060008111915050919050565b828054613ba7906151b7565b90600052602060002090601f016020900481019282613bc95760008555613c10565b82601f10613be257805160ff1916838001178555613c10565b82800160010185558215613c10579182015b82811115613c0f578251825591602001919060010190613bf4565b5b509050613c1d9190613c21565b5090565b5b80821115613c3a576000816000905550600101613c22565b5090565b6000613c51613c4c84614e94565b614e6f565b90508083825260208201905082856020860282011115613c7057600080fd5b60005b85811015613ca05781613c868882613e6c565b845260208401935060208301925050600181019050613c73565b5050509392505050565b6000613cbd613cb884614ec0565b614e6f565b905082815260208101848484011115613cd557600080fd5b613ce0848285615175565b509392505050565b6000613cfb613cf684614ef1565b614e6f565b905082815260208101848484011115613d1357600080fd5b613d1e848285615175565b509392505050565b600081359050613d3581615b22565b92915050565b600081519050613d4a81615b22565b92915050565b60008083601f840112613d6257600080fd5b8235905067ffffffffffffffff811115613d7b57600080fd5b602083019150836020820283011115613d9357600080fd5b9250929050565b600082601f830112613dab57600080fd5b8135613dbb848260208601613c3e565b91505092915050565b600081359050613dd381615b39565b92915050565b600081359050613de881615b50565b92915050565b600081359050613dfd81615b67565b92915050565b600081519050613e1281615b67565b92915050565b600082601f830112613e2957600080fd5b8135613e39848260208601613caa565b91505092915050565b600082601f830112613e5357600080fd5b8135613e63848260208601613ce8565b91505092915050565b600081359050613e7b81615b7e565b92915050565b600060208284031215613e9357600080fd5b6000613ea184828501613d26565b91505092915050565b600060208284031215613ebc57600080fd5b6000613eca84828501613d3b565b91505092915050565b60008060408385031215613ee657600080fd5b6000613ef485828601613d26565b9250506020613f0585828601613d26565b9150509250929050565b600080600060608486031215613f2457600080fd5b6000613f3286828701613d26565b9350506020613f4386828701613d26565b9250506040613f5486828701613e6c565b9150509250925092565b60008060008060808587031215613f7457600080fd5b6000613f8287828801613d26565b9450506020613f9387828801613d26565b9350506040613fa487828801613e6c565b925050606085013567ffffffffffffffff811115613fc157600080fd5b613fcd87828801613e18565b91505092959194509250565b60008060408385031215613fec57600080fd5b6000613ffa85828601613d26565b925050602061400b85828601613dc4565b9150509250929050565b6000806040838503121561402857600080fd5b600061403685828601613d26565b925050602061404785828601613e6c565b9150509250929050565b6000806020838503121561406457600080fd5b600083013567ffffffffffffffff81111561407e57600080fd5b61408a85828601613d50565b92509250509250929050565b6000602082840312156140a857600080fd5b600082013567ffffffffffffffff8111156140c257600080fd5b6140ce84828501613d9a565b91505092915050565b6000602082840312156140e957600080fd5b60006140f784828501613dc4565b91505092915050565b60006020828403121561411257600080fd5b600061412084828501613dd9565b91505092915050565b60006020828403121561413b57600080fd5b600061414984828501613dee565b91505092915050565b60006020828403121561416457600080fd5b600061417284828501613e03565b91505092915050565b60006020828403121561418d57600080fd5b600082013567ffffffffffffffff8111156141a757600080fd5b6141b384828501613e42565b91505092915050565b6000602082840312156141ce57600080fd5b60006141dc84828501613e6c565b91505092915050565b60006141f1838361488d565b60208301905092915050565b614206816150d3565b82525050565b61421d614218826150d3565b615263565b82525050565b600061422e82614f47565b6142388185614f75565b935061424383614f22565b8060005b8381101561427457815161425b88826141e5565b975061426683614f68565b925050600181019050614247565b5085935050505092915050565b61428a816150e5565b82525050565b614299816150f1565b82525050565b6142b06142ab826150f1565b615275565b82525050565b60006142c182614f52565b6142cb8185614f86565b93506142db818560208601615184565b6142e48161537e565b840191505092915050565b6142f881615151565b82525050565b600061430982614f5d565b6143138185614fa2565b9350614323818560208601615184565b61432c8161537e565b840191505092915050565b600061434282614f5d565b61434c8185614fb3565b935061435c818560208601615184565b80840191505092915050565b60008154614375816151b7565b61437f8186614fb3565b9450600182166000811461439a57600181146143ab576143de565b60ff198316865281860193506143de565b6143b485614f32565b60005b838110156143d6578154818901526001820191506020810190506143b7565b838801955050505b50505092915050565b60006143f4601383614fa2565b91506143ff8261539c565b602082019050919050565b6000614417601083614fa2565b9150614422826153c5565b602082019050919050565b600061443a602b83614fa2565b9150614445826153ee565b604082019050919050565b600061445d603283614fa2565b91506144688261543d565b604082019050919050565b6000614480602683614fa2565b915061448b8261548c565b604082019050919050565b60006144a3600983614fa2565b91506144ae826154db565b602082019050919050565b60006144c6601c83614fa2565b91506144d182615504565b602082019050919050565b60006144e9600a83614fa2565b91506144f48261552d565b602082019050919050565b600061450c602483614fa2565b915061451782615556565b604082019050919050565b600061452f601983614fa2565b915061453a826155a5565b602082019050919050565b6000614552601f83614fa2565b915061455d826155ce565b602082019050919050565b6000614575602c83614fa2565b9150614580826155f7565b604082019050919050565b6000614598603883614fa2565b91506145a382615646565b604082019050919050565b60006145bb602a83614fa2565b91506145c682615695565b604082019050919050565b60006145de602983614fa2565b91506145e9826156e4565b604082019050919050565b6000614601600f83614fa2565b915061460c82615733565b602082019050919050565b6000614624602083614fa2565b915061462f8261575c565b602082019050919050565b6000614647602c83614fa2565b915061465282615785565b604082019050919050565b600061466a602083614fa2565b9150614675826157d4565b602082019050919050565b600061468d602483614fa2565b9150614698826157fd565b604082019050919050565b60006146b0601283614fa2565b91506146bb8261584c565b602082019050919050565b60006146d3601683614fa2565b91506146de82615875565b602082019050919050565b60006146f6602983614fa2565b91506147018261589e565b604082019050919050565b6000614719602f83614fa2565b9150614724826158ed565b604082019050919050565b600061473c601783614fa2565b91506147478261593c565b602082019050919050565b600061475f602183614fa2565b915061476a82615965565b604082019050919050565b6000614782600e83614fa2565b915061478d826159b4565b602082019050919050565b60006147a5600083614f97565b91506147b0826159dd565b600082019050919050565b60006147c8603183614fa2565b91506147d3826159e0565b604082019050919050565b60006147eb602c83614fa2565b91506147f682615a2f565b604082019050919050565b600061480e600d83614fa2565b915061481982615a7e565b602082019050919050565b6000614831602083614fa2565b915061483c82615aa7565b602082019050919050565b6000614854601f83614fa2565b915061485f82615ad0565b602082019050919050565b6000614877600f83614fa2565b915061488282615af9565b602082019050919050565b61489681615147565b82525050565b6148a581615147565b82525050565b60006148b7828461420c565b60148201915081905092915050565b60006148d2828561429f565b6020820191506148e2828461429f565b6020820191508190509392505050565b60006148fe8286614337565b915061490a8285614337565b91506149168284614368565b9150819050949350505050565b600061492e82614798565b9150819050919050565b600060208201905061494d60008301846141fd565b92915050565b600060808201905061496860008301876141fd565b61497560208301866141fd565b614982604083018561489c565b818103606083015261499481846142b6565b905095945050505050565b600060208201905081810360008301526149b98184614223565b905092915050565b60006020820190506149d66000830184614281565b92915050565b60006020820190506149f16000830184614290565b92915050565b6000602082019050614a0c60008301846142ef565b92915050565b60006020820190508181036000830152614a2c81846142fe565b905092915050565b60006020820190508181036000830152614a4d816143e7565b9050919050565b60006020820190508181036000830152614a6d8161440a565b9050919050565b60006020820190508181036000830152614a8d8161442d565b9050919050565b60006020820190508181036000830152614aad81614450565b9050919050565b60006020820190508181036000830152614acd81614473565b9050919050565b60006020820190508181036000830152614aed81614496565b9050919050565b60006020820190508181036000830152614b0d816144b9565b9050919050565b60006020820190508181036000830152614b2d816144dc565b9050919050565b60006020820190508181036000830152614b4d816144ff565b9050919050565b60006020820190508181036000830152614b6d81614522565b9050919050565b60006020820190508181036000830152614b8d81614545565b9050919050565b60006020820190508181036000830152614bad81614568565b9050919050565b60006020820190508181036000830152614bcd8161458b565b9050919050565b60006020820190508181036000830152614bed816145ae565b9050919050565b60006020820190508181036000830152614c0d816145d1565b9050919050565b60006020820190508181036000830152614c2d816145f4565b9050919050565b60006020820190508181036000830152614c4d81614617565b9050919050565b60006020820190508181036000830152614c6d8161463a565b9050919050565b60006020820190508181036000830152614c8d8161465d565b9050919050565b60006020820190508181036000830152614cad81614680565b9050919050565b60006020820190508181036000830152614ccd816146a3565b9050919050565b60006020820190508181036000830152614ced816146c6565b9050919050565b60006020820190508181036000830152614d0d816146e9565b9050919050565b60006020820190508181036000830152614d2d8161470c565b9050919050565b60006020820190508181036000830152614d4d8161472f565b9050919050565b60006020820190508181036000830152614d6d81614752565b9050919050565b60006020820190508181036000830152614d8d81614775565b9050919050565b60006020820190508181036000830152614dad816147bb565b9050919050565b60006020820190508181036000830152614dcd816147de565b9050919050565b60006020820190508181036000830152614ded81614801565b9050919050565b60006020820190508181036000830152614e0d81614824565b9050919050565b60006020820190508181036000830152614e2d81614847565b9050919050565b60006020820190508181036000830152614e4d8161486a565b9050919050565b6000602082019050614e69600083018461489c565b92915050565b6000614e79614e8a565b9050614e8582826151e9565b919050565b6000604051905090565b600067ffffffffffffffff821115614eaf57614eae61534f565b5b602082029050602081019050919050565b600067ffffffffffffffff821115614edb57614eda61534f565b5b614ee48261537e565b9050602081019050919050565b600067ffffffffffffffff821115614f0c57614f0b61534f565b5b614f158261537e565b9050602081019050919050565b6000819050602082019050919050565b60008190508160005260206000209050919050565b600081519050919050565b600081519050919050565b600081519050919050565b6000602082019050919050565b600082825260208201905092915050565b600082825260208201905092915050565b600081905092915050565b600082825260208201905092915050565b600081905092915050565b6000614fc982615147565b9150614fd483615147565b9250827fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff03821115615009576150086152c2565b5b828201905092915050565b600061501f82615147565b915061502a83615147565b92508261503a576150396152f1565b5b828204905092915050565b600061505082615147565b915061505b83615147565b9250817fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff0483118215151615615094576150936152c2565b5b828202905092915050565b60006150aa82615147565b91506150b583615147565b9250828210156150c8576150c76152c2565b5b828203905092915050565b60006150de82615127565b9050919050565b60008115159050919050565b6000819050919050565b60007fffffffff0000000000000000000000000000000000000000000000000000000082169050919050565b600073ffffffffffffffffffffffffffffffffffffffff82169050919050565b6000819050919050565b600061515c82615163565b9050919050565b600061516e82615127565b9050919050565b82818337600083830152505050565b60005b838110156151a2578082015181840152602081019050615187565b838111156151b1576000848401525b50505050565b600060028204905060018216806151cf57607f821691505b602082108114156151e3576151e2615320565b5b50919050565b6151f28261537e565b810181811067ffffffffffffffff821117156152115761521061534f565b5b80604052505050565b600061522582615147565b91507fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff821415615258576152576152c2565b5b600182019050919050565b600061526e8261527f565b9050919050565b6000819050919050565b600061528a8261538f565b9050919050565b600061529c82615147565b91506152a783615147565b9250826152b7576152b66152f1565b5b828206905092915050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b6000601f19601f8301169050919050565b60008160601b9050919050565b7f4578636565646564206769766561776179732e00000000000000000000000000600082015250565b7f416c726561647920636c61696d65642100000000000000000000000000000000600082015250565b7f455243373231456e756d657261626c653a206f776e657220696e646578206f7560008201527f74206f6620626f756e6473000000000000000000000000000000000000000000602082015250565b7f4552433732313a207472616e7366657220746f206e6f6e20455243373231526560008201527f63656976657220696d706c656d656e7465720000000000000000000000000000602082015250565b7f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160008201527f6464726573730000000000000000000000000000000000000000000000000000602082015250565b7f536f6c64204f7574210000000000000000000000000000000000000000000000600082015250565b7f4552433732313a20746f6b656e20616c7265616479206d696e74656400000000600082015250565b7f426164206f776e65722100000000000000000000000000000000000000000000600082015250565b7f4552433732313a207472616e7366657220746f20746865207a65726f2061646460008201527f7265737300000000000000000000000000000000000000000000000000000000602082015250565b7f4552433732313a20617070726f766520746f2063616c6c657200000000000000600082015250565b7f45746865722076616c75652073656e74206973206e6f7420636f727265637400600082015250565b7f4552433732313a206f70657261746f7220717565727920666f72206e6f6e657860008201527f697374656e7420746f6b656e0000000000000000000000000000000000000000602082015250565b7f4552433732313a20617070726f76652063616c6c6572206973206e6f74206f7760008201527f6e6572206e6f7220617070726f76656420666f7220616c6c0000000000000000602082015250565b7f4552433732313a2062616c616e636520717565727920666f7220746865207a6560008201527f726f206164647265737300000000000000000000000000000000000000000000602082015250565b7f4552433732313a206f776e657220717565727920666f72206e6f6e657869737460008201527f656e7420746f6b656e0000000000000000000000000000000000000000000000602082015250565b7f436c61696d20697320436c6f7365640000000000000000000000000000000000600082015250565b7f4552433732313a206d696e7420746f20746865207a65726f2061646472657373600082015250565b7f4552433732313a20617070726f76656420717565727920666f72206e6f6e657860008201527f697374656e7420746f6b656e0000000000000000000000000000000000000000602082015250565b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b7f416c726561647920436c61696d6564207468652077686974656c69737465642060008201527f6d696e7400000000000000000000000000000000000000000000000000000000602082015250565b7f506f73742d636c61696d20637570636174210000000000000000000000000000600082015250565b7f74686520636f6e74726163742069732070617573656400000000000000000000600082015250565b7f4552433732313a207472616e73666572206f6620746f6b656e2074686174206960008201527f73206e6f74206f776e0000000000000000000000000000000000000000000000602082015250565b7f4552433732314d657461646174613a2055524920717565727920666f72206e6f60008201527f6e6578697374656e7420746f6b656e0000000000000000000000000000000000602082015250565b7f5768697465204c697374204d696e747320436c6f736564000000000000000000600082015250565b7f4552433732313a20617070726f76616c20746f2063757272656e74206f776e6560008201527f7200000000000000000000000000000000000000000000000000000000000000602082015250565b7f53616c6520697320436c6f736564000000000000000000000000000000000000600082015250565b50565b7f4552433732313a207472616e736665722063616c6c6572206973206e6f74206f60008201527f776e6572206e6f7220617070726f766564000000000000000000000000000000602082015250565b7f455243373231456e756d657261626c653a20676c6f62616c20696e646578206f60008201527f7574206f6620626f756e64730000000000000000000000000000000000000000602082015250565b7f496e76616c69642070726f6f6600000000000000000000000000000000000000600082015250565b7f43616e206f6e6c79206d696e74203920746f6b656e7320617420612074696d65600082015250565b7f5265656e7472616e637947756172643a207265656e7472616e742063616c6c00600082015250565b7f436f6e7472616374205061757365640000000000000000000000000000000000600082015250565b615b2b816150d3565b8114615b3657600080fd5b50565b615b42816150e5565b8114615b4d57600080fd5b50565b615b59816150f1565b8114615b6457600080fd5b50565b615b70816150fb565b8114615b7b57600080fd5b50565b615b8781615147565b8114615b9257600080fd5b5056fea2646970667358221220b611edcdeb8e3e4c5d4bb98b38a73e6e8c44a3f807ab441ac72d53a4b224c81464736f6c63430008040033

Deployed Bytecode

0x6080604052600436106102935760003560e01c80636ba4c1381161015a578063b88d4fde116100c1578063da3ef23f1161007a578063da3ef23f146109ed578063dc559fce14610a16578063e985e9c514610a41578063f1c51b3914610a7e578063f2fde38b14610aa9578063f94a279b14610ad257610293565b8063b88d4fde146108df578063b90ae3ed14610908578063c4e3709514610933578063c66828621461095c578063c87b56dd14610987578063d1be66ba146109c457610293565b806395d89b411161011357806395d89b41146107fd57806397254e55146108285780639a72580914610844578063a0712d681461086f578063a22cb4651461088b578063aaa25f4e146108b457610293565b80636ba4c138146107015780636c0360eb1461072a57806370a0823114610755578063715018a614610792578063819b25ba146107a95780638da5cb5b146107d257610293565b80632f745c59116101fe5780634b014e28116101b75780634b014e28146105df5780634f6ccce71461060857806355f804b3146106455780635c975abb1461066e578063603f4d52146106995780636352211e146106c457610293565b80632f745c59146104de57806333039d3d1461051b5780633ccfd60b1461054657806342842e0e14610550578063438b6300146105795780634783f0ef146105b657610293565b806313faede61161025057806313faede6146103ba5780631681d158146103e557806318160ddd1461042257806318cae2691461044d57806323b872dd1461048a5780632eb4a7ab146104b357610293565b806301e05ba41461029857806301ffc9a7146102c357806302329a291461030057806306fdde0314610329578063081812fc14610354578063095ea7b314610391575b600080fd5b3480156102a457600080fd5b506102ad610afd565b6040516102ba9190614e54565b60405180910390f35b3480156102cf57600080fd5b506102ea60048036038101906102e59190614129565b610b03565b6040516102f791906149c1565b60405180910390f35b34801561030c57600080fd5b50610327600480360381019061032291906140d7565b610b7d565b005b34801561033557600080fd5b5061033e610c16565b60405161034b9190614a12565b60405180910390f35b34801561036057600080fd5b5061037b600480360381019061037691906141bc565b610ca8565b6040516103889190614938565b60405180910390f35b34801561039d57600080fd5b506103b860048036038101906103b39190614015565b610d2d565b005b3480156103c657600080fd5b506103cf610e45565b6040516103dc9190614e54565b60405180910390f35b3480156103f157600080fd5b5061040c600480360381019061040791906141bc565b610e4b565b60405161041991906149c1565b60405180910390f35b34801561042e57600080fd5b50610437610e63565b6040516104449190614e54565b60405180910390f35b34801561045957600080fd5b50610474600480360381019061046f9190613e81565b610e70565b6040516104819190614e54565b60405180910390f35b34801561049657600080fd5b506104b160048036038101906104ac9190613f0f565b610e88565b005b3480156104bf57600080fd5b506104c8610ee8565b6040516104d591906149dc565b60405180910390f35b3480156104ea57600080fd5b5061050560048036038101906105009190614015565b610eee565b6040516105129190614e54565b60405180910390f35b34801561052757600080fd5b50610530610f93565b60405161053d9190614e54565b60405180910390f35b61054e610f99565b005b34801561055c57600080fd5b5061057760048036038101906105729190613f0f565b611095565b005b34801561058557600080fd5b506105a0600480360381019061059b9190613e81565b6110b5565b6040516105ad919061499f565b60405180910390f35b3480156105c257600080fd5b506105dd60048036038101906105d89190614100565b6111af565b005b3480156105eb57600080fd5b50610606600480360381019061060191906140d7565b61126e565b005b34801561061457600080fd5b5061062f600480360381019061062a91906141bc565b611307565b60405161063c9190614e54565b60405180910390f35b34801561065157600080fd5b5061066c6004803603810190610667919061417b565b61139e565b005b34801561067a57600080fd5b50610683611434565b60405161069091906149c1565b60405180910390f35b3480156106a557600080fd5b506106ae611447565b6040516106bb91906149c1565b60405180910390f35b3480156106d057600080fd5b506106eb60048036038101906106e691906141bc565b61145a565b6040516106f89190614938565b60405180910390f35b34801561070d57600080fd5b5061072860048036038101906107239190614096565b61150c565b005b34801561073657600080fd5b5061073f6117d7565b60405161074c9190614a12565b60405180910390f35b34801561076157600080fd5b5061077c60048036038101906107779190613e81565b611865565b6040516107899190614e54565b60405180910390f35b34801561079e57600080fd5b506107a761191d565b005b3480156107b557600080fd5b506107d060048036038101906107cb91906141bc565b6119a5565b005b3480156107de57600080fd5b506107e7611af4565b6040516107f49190614938565b60405180910390f35b34801561080957600080fd5b50610812611b1e565b60405161081f9190614a12565b60405180910390f35b610842600480360381019061083d9190614051565b611bb0565b005b34801561085057600080fd5b50610859611eda565b60405161086691906149c1565b60405180910390f35b610889600480360381019061088491906141bc565b611eed565b005b34801561089757600080fd5b506108b260048036038101906108ad9190613fd9565b6121fb565b005b3480156108c057600080fd5b506108c9612211565b6040516108d69190614e54565b60405180910390f35b3480156108eb57600080fd5b5061090660048036038101906109019190613f5e565b612230565b005b34801561091457600080fd5b5061091d612292565b60405161092a91906149f7565b60405180910390f35b34801561093f57600080fd5b5061095a600480360381019061095591906140d7565b6122b8565b005b34801561096857600080fd5b50610971612351565b60405161097e9190614a12565b60405180910390f35b34801561099357600080fd5b506109ae60048036038101906109a991906141bc565b6123df565b6040516109bb9190614a12565b60405180910390f35b3480156109d057600080fd5b506109eb60048036038101906109e69190613e81565b612489565b005b3480156109f957600080fd5b50610a146004803603810190610a0f919061417b565b612549565b005b348015610a2257600080fd5b50610a2b6125df565b604051610a389190614e54565b60405180910390f35b348015610a4d57600080fd5b50610a686004803603810190610a639190613ed3565b6125e5565b604051610a7591906149c1565b60405180910390f35b348015610a8a57600080fd5b50610a93612679565b604051610aa09190614e54565b60405180910390f35b348015610ab557600080fd5b50610ad06004803603810190610acb9190613e81565b61267f565b005b348015610ade57600080fd5b50610ae7612777565b604051610af49190614e54565b60405180910390f35b6113a181565b60007f780e9d63000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff19161480610b765750610b758261277c565b5b9050919050565b610b8561285e565b73ffffffffffffffffffffffffffffffffffffffff16610ba3611af4565b73ffffffffffffffffffffffffffffffffffffffff1614610bf9576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610bf090614c74565b60405180910390fd5b80601160006101000a81548160ff02191690831515021790555050565b606060008054610c25906151b7565b80601f0160208091040260200160405190810160405280929190818152602001828054610c51906151b7565b8015610c9e5780601f10610c7357610100808354040283529160200191610c9e565b820191906000526020600020905b815481529060010190602001808311610c8157829003601f168201915b5050505050905090565b6000610cb382612866565b610cf2576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610ce990614c54565b60405180910390fd5b6004600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff169050919050565b6000610d388261145a565b90508073ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff161415610da9576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610da090614d54565b60405180910390fd5b8073ffffffffffffffffffffffffffffffffffffffff16610dc861285e565b73ffffffffffffffffffffffffffffffffffffffff161480610df75750610df681610df161285e565b6125e5565b5b610e36576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610e2d90614bb4565b60405180910390fd5b610e4083836128d2565b505050565b60105481565b6000801515610e5983612866565b1515149050919050565b6000600880549050905090565b60136020528060005260406000206000915090505481565b610e99610e9361285e565b8261298b565b610ed8576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610ecf90614d94565b60405180910390fd5b610ee3838383612a69565b505050565b60125481565b6000610ef983611865565b8210610f3a576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610f3190614a74565b60405180910390fd5b600660008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600083815260200190815260200160002054905092915050565b61271081565b610fa161285e565b73ffffffffffffffffffffffffffffffffffffffff16610fbf611af4565b73ffffffffffffffffffffffffffffffffffffffff1614611015576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161100c90614c74565b60405180910390fd5b600061101f611af4565b73ffffffffffffffffffffffffffffffffffffffff164760405161104290614923565b60006040518083038185875af1925050503d806000811461107f576040519150601f19603f3d011682016040523d82523d6000602084013e611084565b606091505b505090508061109257600080fd5b50565b6110b083838360405180602001604052806000815250612230565b505050565b606060006110c283611865565b905060008167ffffffffffffffff811115611106577f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b6040519080825280602002602001820160405280156111345781602001602082028036833780820191505090505b50905060005b828110156111a45761114c8582610eee565b828281518110611185577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b602002602001018181525050808061119c9061521a565b91505061113a565b508092505050919050565b6111b761285e565b73ffffffffffffffffffffffffffffffffffffffff166111d5611af4565b73ffffffffffffffffffffffffffffffffffffffff161461122b576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161122290614c74565b60405180910390fd5b806012819055507f90004c04698bc3322499a575ed3752dd4abf33e0a7294c06a787a0fe01bea94160125460405161126391906149dc565b60405180910390a150565b61127661285e565b73ffffffffffffffffffffffffffffffffffffffff16611294611af4565b73ffffffffffffffffffffffffffffffffffffffff16146112ea576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016112e190614c74565b60405180910390fd5b80601160016101000a81548160ff02191690831515021790555050565b6000611311610e63565b8210611352576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161134990614db4565b60405180910390fd5b6008828154811061138c577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b90600052602060002001549050919050565b6113a661285e565b73ffffffffffffffffffffffffffffffffffffffff166113c4611af4565b73ffffffffffffffffffffffffffffffffffffffff161461141a576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161141190614c74565b60405180910390fd5b80600e9080519060200190611430929190613b9b565b5050565b601160009054906101000a900460ff1681565b601160029054906101000a900460ff1681565b6000806002600084815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff169050600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff161415611503576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016114fa90614bf4565b60405180910390fd5b80915050919050565b601160019054906101000a900460ff1661155b576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161155290614c14565b60405180910390fd5b601160009054906101000a900460ff16156115ab576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016115a290614e34565b60405180910390fd5b60005b81518110156117d35760008282815181106115f2577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b602002602001015190506000151561160982612866565b15151461164b576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161164290614a54565b60405180910390fd5b6113a1811061168f576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161168690614cb4565b60405180910390fd5b61169761285e565b73ffffffffffffffffffffffffffffffffffffffff16601460009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16636352211e836040518263ffffffff1660e01b81526004016117089190614e54565b60206040518083038186803b15801561172057600080fd5b505afa158015611734573d6000803e3d6000fd5b505050506040513d601f19601f820116820180604052508101906117589190613eaa565b73ffffffffffffffffffffffffffffffffffffffff16146117ae576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016117a590614b14565b60405180910390fd5b6117bf6117b961285e565b82612cc5565b5080806117cb9061521a565b9150506115ae565b5050565b600e80546117e4906151b7565b80601f0160208091040260200160405190810160405280929190818152602001828054611810906151b7565b801561185d5780601f106118325761010080835404028352916020019161185d565b820191906000526020600020905b81548152906001019060200180831161184057829003601f168201915b505050505081565b60008073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff1614156118d6576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016118cd90614bd4565b60405180910390fd5b600360008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020549050919050565b61192561285e565b73ffffffffffffffffffffffffffffffffffffffff16611943611af4565b73ffffffffffffffffffffffffffffffffffffffff1614611999576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161199090614c74565b60405180910390fd5b6119a36000612ce3565b565b6119ad61285e565b73ffffffffffffffffffffffffffffffffffffffff166119cb611af4565b73ffffffffffffffffffffffffffffffffffffffff1614611a21576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611a1890614c74565b60405180910390fd5b60e181600c54611a319190614fbe565b1115611a72576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611a6990614a34565b60405180910390fd5b60005b81811015611af057611ac3611a8861285e565b600c5460e16113a1612710611a9d919061509f565b611aa7919061509f565b6113a1611ab49190614fbe565b611abe9190614fbe565b612cc5565b6001600c6000828254611ad69190614fbe565b925050819055508080611ae89061521a565b915050611a75565b5050565b6000600a60009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b606060018054611b2d906151b7565b80601f0160208091040260200160405190810160405280929190818152602001828054611b59906151b7565b8015611ba65780601f10611b7b57610100808354040283529160200191611ba6565b820191906000526020600020905b815481529060010190602001808311611b8957829003601f168201915b5050505050905090565b601160009054906101000a900460ff1615611c00576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611bf790614cd4565b60405180910390fd5b6000801b6012541415611c48576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611c3f90614d34565b60405180910390fd5b60e16113a1612710611c5a919061509f565b611c64919061509f565b611c7a6001600d54612da990919063ffffffff16565b1115611cbb576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611cb290614ad4565b60405180910390fd5b6001601360003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000205410611d3d576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611d3490614c94565b60405180910390fd5b611db1828280806020026020016040519081016040528093929190818152602001838360200280828437600081840152601f19601f8201169050808301925050505050505060125433604051602001611d9691906148ab565b60405160208183030381529060405280519060200120612dbf565b611df0576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611de790614dd4565b60405180910390fd5b611e066001601054612dd690919063ffffffff16565b3414611e47576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611e3e90614b74565b60405180910390fd5b601360003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000815480929190611e979061521a565b9190505550611ebc611ea761285e565b600d546113a1611eb79190614fbe565b612cc5565b6001600d6000828254611ecf9190614fbe565b925050819055505050565b601160019054906101000a900460ff1681565b601160029054906101000a900460ff16611f3c576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611f3390614d74565b60405180910390fd5b601160009054906101000a900460ff1615611f8c576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611f8390614e34565b60405180910390fd5b6002600b541415611fd2576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611fc990614e14565b60405180910390fd5b6002600b81905550601160009054906101000a900460ff161561202a576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161202190614cd4565b60405180910390fd5b60e16113a161271061203c919061509f565b612046919061509f565b61205b82600d54612da990919063ffffffff16565b111561209c576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161209390614ad4565b60405180910390fd5b6000811180156120ad575060098111155b6120ec576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016120e390614df4565b60405180910390fd5b61210181601054612dd690919063ffffffff16565b3414612142576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161213990614b74565b60405180910390fd5b60005b818110156121ef57601360003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600081548092919061219d9061521a565b91905055506121c26121ad61285e565b600d546113a16121bd9190614fbe565b612cc5565b6001600d60008282546121d59190614fbe565b9250508190555080806121e79061521a565b915050612145565b506001600b8190555050565b61220d61220661285e565b8383612dec565b5050565b60e16113a1612710612223919061509f565b61222d919061509f565b81565b61224161223b61285e565b8361298b565b612280576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161227790614d94565b60405180910390fd5b61228c84848484612f59565b50505050565b601460009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1681565b6122c061285e565b73ffffffffffffffffffffffffffffffffffffffff166122de611af4565b73ffffffffffffffffffffffffffffffffffffffff1614612334576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161232b90614c74565b60405180910390fd5b80601160026101000a81548160ff02191690831515021790555050565b600f805461235e906151b7565b80601f016020809104026020016040519081016040528092919081815260200182805461238a906151b7565b80156123d75780601f106123ac576101008083540402835291602001916123d7565b820191906000526020600020905b8154815290600101906020018083116123ba57829003601f168201915b505050505081565b60606123ea82612866565b612429576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161242090614d14565b60405180910390fd5b6000612433612fb5565b905060008151116124535760405180602001604052806000815250612481565b8061245d84613047565b600f604051602001612471939291906148f2565b6040516020818303038152906040525b915050919050565b61249161285e565b73ffffffffffffffffffffffffffffffffffffffff166124af611af4565b73ffffffffffffffffffffffffffffffffffffffff1614612505576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016124fc90614c74565b60405180910390fd5b80601460006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555050565b61255161285e565b73ffffffffffffffffffffffffffffffffffffffff1661256f611af4565b73ffffffffffffffffffffffffffffffffffffffff16146125c5576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016125bc90614c74565b60405180910390fd5b80600f90805190602001906125db929190613b9b565b5050565b600d5481565b6000600560008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff16905092915050565b600c5481565b61268761285e565b73ffffffffffffffffffffffffffffffffffffffff166126a5611af4565b73ffffffffffffffffffffffffffffffffffffffff16146126fb576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016126f290614c74565b60405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff16141561276b576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161276290614ab4565b60405180910390fd5b61277481612ce3565b50565b60e181565b60007f80ac58cd000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916148061284757507f5b5e139f000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b806128575750612856826131f4565b5b9050919050565b600033905090565b60008073ffffffffffffffffffffffffffffffffffffffff166002600084815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1614159050919050565b816004600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550808273ffffffffffffffffffffffffffffffffffffffff166129458361145a565b73ffffffffffffffffffffffffffffffffffffffff167f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92560405160405180910390a45050565b600061299682612866565b6129d5576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016129cc90614b94565b60405180910390fd5b60006129e08361145a565b90508073ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff161480612a4f57508373ffffffffffffffffffffffffffffffffffffffff16612a3784610ca8565b73ffffffffffffffffffffffffffffffffffffffff16145b80612a605750612a5f81856125e5565b5b91505092915050565b8273ffffffffffffffffffffffffffffffffffffffff16612a898261145a565b73ffffffffffffffffffffffffffffffffffffffff1614612adf576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612ad690614cf4565b60405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415612b4f576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612b4690614b34565b60405180910390fd5b612b5a83838361325e565b612b656000826128d2565b6001600360008573ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254612bb5919061509f565b925050819055506001600360008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254612c0c9190614fbe565b92505081905550816002600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550808273ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4505050565b612cdf828260405180602001604052806000815250613372565b5050565b6000600a60009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600a60006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b60008183612db79190614fbe565b905092915050565b600082612dcc85846133cd565b1490509392505050565b60008183612de49190615045565b905092915050565b8173ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff161415612e5b576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612e5290614b54565b60405180910390fd5b80600560008573ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060006101000a81548160ff0219169083151502179055508173ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff167f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c3183604051612f4c91906149c1565b60405180910390a3505050565b612f64848484612a69565b612f70848484846134a6565b612faf576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612fa690614a94565b60405180910390fd5b50505050565b6060600e8054612fc4906151b7565b80601f0160208091040260200160405190810160405280929190818152602001828054612ff0906151b7565b801561303d5780601f106130125761010080835404028352916020019161303d565b820191906000526020600020905b81548152906001019060200180831161302057829003601f168201915b5050505050905090565b6060600082141561308f576040518060400160405280600181526020017f300000000000000000000000000000000000000000000000000000000000000081525090506131ef565b600082905060005b600082146130c15780806130aa9061521a565b915050600a826130ba9190615014565b9150613097565b60008167ffffffffffffffff811115613103577f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b6040519080825280601f01601f1916602001820160405280156131355781602001600182028036833780820191505090505b5090505b600085146131e85760018261314e919061509f565b9150600a8561315d9190615291565b60306131699190614fbe565b60f81b8183815181106131a5577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b60200101907effffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916908160001a905350600a856131e19190615014565b9450613139565b8093505050505b919050565b60007f01ffc9a7000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916149050919050565b61326983838361363d565b600073ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff1614156132ac576132a781613642565b6132eb565b8173ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff16146132ea576132e9838261368b565b5b5b600073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff16141561332e57613329816137f8565b61336d565b8273ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161461336c5761336b828261393b565b5b5b505050565b61337c83836139ba565b61338960008484846134a6565b6133c8576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016133bf90614a94565b60405180910390fd5b505050565b60008082905060005b845181101561349b57600085828151811061341a577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b6020026020010151905080831161345b57828160405160200161343e9291906148c6565b604051602081830303815290604052805190602001209250613487565b808360405160200161346e9291906148c6565b6040516020818303038152906040528051906020012092505b5080806134939061521a565b9150506133d6565b508091505092915050565b60006134c78473ffffffffffffffffffffffffffffffffffffffff16613b88565b15613630578373ffffffffffffffffffffffffffffffffffffffff1663150b7a026134f061285e565b8786866040518563ffffffff1660e01b81526004016135129493929190614953565b602060405180830381600087803b15801561352c57600080fd5b505af192505050801561355d57506040513d601f19601f8201168201806040525081019061355a9190614152565b60015b6135e0573d806000811461358d576040519150601f19603f3d011682016040523d82523d6000602084013e613592565b606091505b506000815114156135d8576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016135cf90614a94565b60405180910390fd5b805181602001fd5b63150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916817bffffffffffffffffffffffffffffffffffffffffffffffffffffffff191614915050613635565b600190505b949350505050565b505050565b6008805490506009600083815260200190815260200160002081905550600881908060018154018082558091505060019003906000526020600020016000909190919091505550565b6000600161369884611865565b6136a2919061509f565b9050600060076000848152602001908152602001600020549050818114613787576000600660008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600084815260200190815260200160002054905080600660008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600084815260200190815260200160002081905550816007600083815260200190815260200160002081905550505b6007600084815260200190815260200160002060009055600660008573ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008381526020019081526020016000206000905550505050565b6000600160088054905061380c919061509f565b9050600060096000848152602001908152602001600020549050600060088381548110613862577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b9060005260206000200154905080600883815481106138aa577f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b90600052602060002001819055508160096000838152602001908152602001600020819055506009600085815260200190815260200160002060009055600880548061391f577f4e487b7100000000000000000000000000000000000000000000000000000000600052603160045260246000fd5b6001900381819060005260206000200160009055905550505050565b600061394683611865565b905081600660008573ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600083815260200190815260200160002081905550806007600084815260200190815260200160002081905550505050565b600073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415613a2a576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401613a2190614c34565b60405180910390fd5b613a3381612866565b15613a73576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401613a6a90614af4565b60405180910390fd5b613a7f6000838361325e565b6001600360008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254613acf9190614fbe565b92505081905550816002600083815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550808273ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a45050565b600080823b905060008111915050919050565b828054613ba7906151b7565b90600052602060002090601f016020900481019282613bc95760008555613c10565b82601f10613be257805160ff1916838001178555613c10565b82800160010185558215613c10579182015b82811115613c0f578251825591602001919060010190613bf4565b5b509050613c1d9190613c21565b5090565b5b80821115613c3a576000816000905550600101613c22565b5090565b6000613c51613c4c84614e94565b614e6f565b90508083825260208201905082856020860282011115613c7057600080fd5b60005b85811015613ca05781613c868882613e6c565b845260208401935060208301925050600181019050613c73565b5050509392505050565b6000613cbd613cb884614ec0565b614e6f565b905082815260208101848484011115613cd557600080fd5b613ce0848285615175565b509392505050565b6000613cfb613cf684614ef1565b614e6f565b905082815260208101848484011115613d1357600080fd5b613d1e848285615175565b509392505050565b600081359050613d3581615b22565b92915050565b600081519050613d4a81615b22565b92915050565b60008083601f840112613d6257600080fd5b8235905067ffffffffffffffff811115613d7b57600080fd5b602083019150836020820283011115613d9357600080fd5b9250929050565b600082601f830112613dab57600080fd5b8135613dbb848260208601613c3e565b91505092915050565b600081359050613dd381615b39565b92915050565b600081359050613de881615b50565b92915050565b600081359050613dfd81615b67565b92915050565b600081519050613e1281615b67565b92915050565b600082601f830112613e2957600080fd5b8135613e39848260208601613caa565b91505092915050565b600082601f830112613e5357600080fd5b8135613e63848260208601613ce8565b91505092915050565b600081359050613e7b81615b7e565b92915050565b600060208284031215613e9357600080fd5b6000613ea184828501613d26565b91505092915050565b600060208284031215613ebc57600080fd5b6000613eca84828501613d3b565b91505092915050565b60008060408385031215613ee657600080fd5b6000613ef485828601613d26565b9250506020613f0585828601613d26565b9150509250929050565b600080600060608486031215613f2457600080fd5b6000613f3286828701613d26565b9350506020613f4386828701613d26565b9250506040613f5486828701613e6c565b9150509250925092565b60008060008060808587031215613f7457600080fd5b6000613f8287828801613d26565b9450506020613f9387828801613d26565b9350506040613fa487828801613e6c565b925050606085013567ffffffffffffffff811115613fc157600080fd5b613fcd87828801613e18565b91505092959194509250565b60008060408385031215613fec57600080fd5b6000613ffa85828601613d26565b925050602061400b85828601613dc4565b9150509250929050565b6000806040838503121561402857600080fd5b600061403685828601613d26565b925050602061404785828601613e6c565b9150509250929050565b6000806020838503121561406457600080fd5b600083013567ffffffffffffffff81111561407e57600080fd5b61408a85828601613d50565b92509250509250929050565b6000602082840312156140a857600080fd5b600082013567ffffffffffffffff8111156140c257600080fd5b6140ce84828501613d9a565b91505092915050565b6000602082840312156140e957600080fd5b60006140f784828501613dc4565b91505092915050565b60006020828403121561411257600080fd5b600061412084828501613dd9565b91505092915050565b60006020828403121561413b57600080fd5b600061414984828501613dee565b91505092915050565b60006020828403121561416457600080fd5b600061417284828501613e03565b91505092915050565b60006020828403121561418d57600080fd5b600082013567ffffffffffffffff8111156141a757600080fd5b6141b384828501613e42565b91505092915050565b6000602082840312156141ce57600080fd5b60006141dc84828501613e6c565b91505092915050565b60006141f1838361488d565b60208301905092915050565b614206816150d3565b82525050565b61421d614218826150d3565b615263565b82525050565b600061422e82614f47565b6142388185614f75565b935061424383614f22565b8060005b8381101561427457815161425b88826141e5565b975061426683614f68565b925050600181019050614247565b5085935050505092915050565b61428a816150e5565b82525050565b614299816150f1565b82525050565b6142b06142ab826150f1565b615275565b82525050565b60006142c182614f52565b6142cb8185614f86565b93506142db818560208601615184565b6142e48161537e565b840191505092915050565b6142f881615151565b82525050565b600061430982614f5d565b6143138185614fa2565b9350614323818560208601615184565b61432c8161537e565b840191505092915050565b600061434282614f5d565b61434c8185614fb3565b935061435c818560208601615184565b80840191505092915050565b60008154614375816151b7565b61437f8186614fb3565b9450600182166000811461439a57600181146143ab576143de565b60ff198316865281860193506143de565b6143b485614f32565b60005b838110156143d6578154818901526001820191506020810190506143b7565b838801955050505b50505092915050565b60006143f4601383614fa2565b91506143ff8261539c565b602082019050919050565b6000614417601083614fa2565b9150614422826153c5565b602082019050919050565b600061443a602b83614fa2565b9150614445826153ee565b604082019050919050565b600061445d603283614fa2565b91506144688261543d565b604082019050919050565b6000614480602683614fa2565b915061448b8261548c565b604082019050919050565b60006144a3600983614fa2565b91506144ae826154db565b602082019050919050565b60006144c6601c83614fa2565b91506144d182615504565b602082019050919050565b60006144e9600a83614fa2565b91506144f48261552d565b602082019050919050565b600061450c602483614fa2565b915061451782615556565b604082019050919050565b600061452f601983614fa2565b915061453a826155a5565b602082019050919050565b6000614552601f83614fa2565b915061455d826155ce565b602082019050919050565b6000614575602c83614fa2565b9150614580826155f7565b604082019050919050565b6000614598603883614fa2565b91506145a382615646565b604082019050919050565b60006145bb602a83614fa2565b91506145c682615695565b604082019050919050565b60006145de602983614fa2565b91506145e9826156e4565b604082019050919050565b6000614601600f83614fa2565b915061460c82615733565b602082019050919050565b6000614624602083614fa2565b915061462f8261575c565b602082019050919050565b6000614647602c83614fa2565b915061465282615785565b604082019050919050565b600061466a602083614fa2565b9150614675826157d4565b602082019050919050565b600061468d602483614fa2565b9150614698826157fd565b604082019050919050565b60006146b0601283614fa2565b91506146bb8261584c565b602082019050919050565b60006146d3601683614fa2565b91506146de82615875565b602082019050919050565b60006146f6602983614fa2565b91506147018261589e565b604082019050919050565b6000614719602f83614fa2565b9150614724826158ed565b604082019050919050565b600061473c601783614fa2565b91506147478261593c565b602082019050919050565b600061475f602183614fa2565b915061476a82615965565b604082019050919050565b6000614782600e83614fa2565b915061478d826159b4565b602082019050919050565b60006147a5600083614f97565b91506147b0826159dd565b600082019050919050565b60006147c8603183614fa2565b91506147d3826159e0565b604082019050919050565b60006147eb602c83614fa2565b91506147f682615a2f565b604082019050919050565b600061480e600d83614fa2565b915061481982615a7e565b602082019050919050565b6000614831602083614fa2565b915061483c82615aa7565b602082019050919050565b6000614854601f83614fa2565b915061485f82615ad0565b602082019050919050565b6000614877600f83614fa2565b915061488282615af9565b602082019050919050565b61489681615147565b82525050565b6148a581615147565b82525050565b60006148b7828461420c565b60148201915081905092915050565b60006148d2828561429f565b6020820191506148e2828461429f565b6020820191508190509392505050565b60006148fe8286614337565b915061490a8285614337565b91506149168284614368565b9150819050949350505050565b600061492e82614798565b9150819050919050565b600060208201905061494d60008301846141fd565b92915050565b600060808201905061496860008301876141fd565b61497560208301866141fd565b614982604083018561489c565b818103606083015261499481846142b6565b905095945050505050565b600060208201905081810360008301526149b98184614223565b905092915050565b60006020820190506149d66000830184614281565b92915050565b60006020820190506149f16000830184614290565b92915050565b6000602082019050614a0c60008301846142ef565b92915050565b60006020820190508181036000830152614a2c81846142fe565b905092915050565b60006020820190508181036000830152614a4d816143e7565b9050919050565b60006020820190508181036000830152614a6d8161440a565b9050919050565b60006020820190508181036000830152614a8d8161442d565b9050919050565b60006020820190508181036000830152614aad81614450565b9050919050565b60006020820190508181036000830152614acd81614473565b9050919050565b60006020820190508181036000830152614aed81614496565b9050919050565b60006020820190508181036000830152614b0d816144b9565b9050919050565b60006020820190508181036000830152614b2d816144dc565b9050919050565b60006020820190508181036000830152614b4d816144ff565b9050919050565b60006020820190508181036000830152614b6d81614522565b9050919050565b60006020820190508181036000830152614b8d81614545565b9050919050565b60006020820190508181036000830152614bad81614568565b9050919050565b60006020820190508181036000830152614bcd8161458b565b9050919050565b60006020820190508181036000830152614bed816145ae565b9050919050565b60006020820190508181036000830152614c0d816145d1565b9050919050565b60006020820190508181036000830152614c2d816145f4565b9050919050565b60006020820190508181036000830152614c4d81614617565b9050919050565b60006020820190508181036000830152614c6d8161463a565b9050919050565b60006020820190508181036000830152614c8d8161465d565b9050919050565b60006020820190508181036000830152614cad81614680565b9050919050565b60006020820190508181036000830152614ccd816146a3565b9050919050565b60006020820190508181036000830152614ced816146c6565b9050919050565b60006020820190508181036000830152614d0d816146e9565b9050919050565b60006020820190508181036000830152614d2d8161470c565b9050919050565b60006020820190508181036000830152614d4d8161472f565b9050919050565b60006020820190508181036000830152614d6d81614752565b9050919050565b60006020820190508181036000830152614d8d81614775565b9050919050565b60006020820190508181036000830152614dad816147bb565b9050919050565b60006020820190508181036000830152614dcd816147de565b9050919050565b60006020820190508181036000830152614ded81614801565b9050919050565b60006020820190508181036000830152614e0d81614824565b9050919050565b60006020820190508181036000830152614e2d81614847565b9050919050565b60006020820190508181036000830152614e4d8161486a565b9050919050565b6000602082019050614e69600083018461489c565b92915050565b6000614e79614e8a565b9050614e8582826151e9565b919050565b6000604051905090565b600067ffffffffffffffff821115614eaf57614eae61534f565b5b602082029050602081019050919050565b600067ffffffffffffffff821115614edb57614eda61534f565b5b614ee48261537e565b9050602081019050919050565b600067ffffffffffffffff821115614f0c57614f0b61534f565b5b614f158261537e565b9050602081019050919050565b6000819050602082019050919050565b60008190508160005260206000209050919050565b600081519050919050565b600081519050919050565b600081519050919050565b6000602082019050919050565b600082825260208201905092915050565b600082825260208201905092915050565b600081905092915050565b600082825260208201905092915050565b600081905092915050565b6000614fc982615147565b9150614fd483615147565b9250827fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff03821115615009576150086152c2565b5b828201905092915050565b600061501f82615147565b915061502a83615147565b92508261503a576150396152f1565b5b828204905092915050565b600061505082615147565b915061505b83615147565b9250817fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff0483118215151615615094576150936152c2565b5b828202905092915050565b60006150aa82615147565b91506150b583615147565b9250828210156150c8576150c76152c2565b5b828203905092915050565b60006150de82615127565b9050919050565b60008115159050919050565b6000819050919050565b60007fffffffff0000000000000000000000000000000000000000000000000000000082169050919050565b600073ffffffffffffffffffffffffffffffffffffffff82169050919050565b6000819050919050565b600061515c82615163565b9050919050565b600061516e82615127565b9050919050565b82818337600083830152505050565b60005b838110156151a2578082015181840152602081019050615187565b838111156151b1576000848401525b50505050565b600060028204905060018216806151cf57607f821691505b602082108114156151e3576151e2615320565b5b50919050565b6151f28261537e565b810181811067ffffffffffffffff821117156152115761521061534f565b5b80604052505050565b600061522582615147565b91507fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff821415615258576152576152c2565b5b600182019050919050565b600061526e8261527f565b9050919050565b6000819050919050565b600061528a8261538f565b9050919050565b600061529c82615147565b91506152a783615147565b9250826152b7576152b66152f1565b5b828206905092915050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b6000601f19601f8301169050919050565b60008160601b9050919050565b7f4578636565646564206769766561776179732e00000000000000000000000000600082015250565b7f416c726561647920636c61696d65642100000000000000000000000000000000600082015250565b7f455243373231456e756d657261626c653a206f776e657220696e646578206f7560008201527f74206f6620626f756e6473000000000000000000000000000000000000000000602082015250565b7f4552433732313a207472616e7366657220746f206e6f6e20455243373231526560008201527f63656976657220696d706c656d656e7465720000000000000000000000000000602082015250565b7f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160008201527f6464726573730000000000000000000000000000000000000000000000000000602082015250565b7f536f6c64204f7574210000000000000000000000000000000000000000000000600082015250565b7f4552433732313a20746f6b656e20616c7265616479206d696e74656400000000600082015250565b7f426164206f776e65722100000000000000000000000000000000000000000000600082015250565b7f4552433732313a207472616e7366657220746f20746865207a65726f2061646460008201527f7265737300000000000000000000000000000000000000000000000000000000602082015250565b7f4552433732313a20617070726f766520746f2063616c6c657200000000000000600082015250565b7f45746865722076616c75652073656e74206973206e6f7420636f727265637400600082015250565b7f4552433732313a206f70657261746f7220717565727920666f72206e6f6e657860008201527f697374656e7420746f6b656e0000000000000000000000000000000000000000602082015250565b7f4552433732313a20617070726f76652063616c6c6572206973206e6f74206f7760008201527f6e6572206e6f7220617070726f76656420666f7220616c6c0000000000000000602082015250565b7f4552433732313a2062616c616e636520717565727920666f7220746865207a6560008201527f726f206164647265737300000000000000000000000000000000000000000000602082015250565b7f4552433732313a206f776e657220717565727920666f72206e6f6e657869737460008201527f656e7420746f6b656e0000000000000000000000000000000000000000000000602082015250565b7f436c61696d20697320436c6f7365640000000000000000000000000000000000600082015250565b7f4552433732313a206d696e7420746f20746865207a65726f2061646472657373600082015250565b7f4552433732313a20617070726f76656420717565727920666f72206e6f6e657860008201527f697374656e7420746f6b656e0000000000000000000000000000000000000000602082015250565b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b7f416c726561647920436c61696d6564207468652077686974656c69737465642060008201527f6d696e7400000000000000000000000000000000000000000000000000000000602082015250565b7f506f73742d636c61696d20637570636174210000000000000000000000000000600082015250565b7f74686520636f6e74726163742069732070617573656400000000000000000000600082015250565b7f4552433732313a207472616e73666572206f6620746f6b656e2074686174206960008201527f73206e6f74206f776e0000000000000000000000000000000000000000000000602082015250565b7f4552433732314d657461646174613a2055524920717565727920666f72206e6f60008201527f6e6578697374656e7420746f6b656e0000000000000000000000000000000000602082015250565b7f5768697465204c697374204d696e747320436c6f736564000000000000000000600082015250565b7f4552433732313a20617070726f76616c20746f2063757272656e74206f776e6560008201527f7200000000000000000000000000000000000000000000000000000000000000602082015250565b7f53616c6520697320436c6f736564000000000000000000000000000000000000600082015250565b50565b7f4552433732313a207472616e736665722063616c6c6572206973206e6f74206f60008201527f776e6572206e6f7220617070726f766564000000000000000000000000000000602082015250565b7f455243373231456e756d657261626c653a20676c6f62616c20696e646578206f60008201527f7574206f6620626f756e64730000000000000000000000000000000000000000602082015250565b7f496e76616c69642070726f6f6600000000000000000000000000000000000000600082015250565b7f43616e206f6e6c79206d696e74203920746f6b656e7320617420612074696d65600082015250565b7f5265656e7472616e637947756172643a207265656e7472616e742063616c6c00600082015250565b7f436f6e7472616374205061757365640000000000000000000000000000000000600082015250565b615b2b816150d3565b8114615b3657600080fd5b50565b615b42816150e5565b8114615b4d57600080fd5b50565b615b59816150f1565b8114615b6457600080fd5b50565b615b70816150fb565b8114615b7b57600080fd5b50565b615b8781615147565b8114615b9257600080fd5b5056fea2646970667358221220b611edcdeb8e3e4c5d4bb98b38a73e6e8c44a3f807ab441ac72d53a4b224c81464736f6c63430008040033

Deployed Bytecode Sourcemap

564:5841:15:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;788:45;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;990:222:5;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;5793:77:15;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;2473:98:2;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;3984:217;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;3522:401;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;1096:39:15;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;4456:114;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;1615:111:5;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;1344:55:15;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;4711:330:2;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;1244:94:15;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;1291:253:5;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;839:48:15;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;6060:152;;;:::i;:::-;;5107:179:2;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;4575:377:15;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;6248:155;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;5966:89;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;1798:230:5;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;5555:102:15;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;1141:26;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;1209:29;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;2176:235:2;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;3625:470:15;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;1026:21;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;1914:205:2;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;1668:101:0;;;;;;;;;;;;;:::i;:::-;;4100:351:15;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;1036:85:0;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;2635:102:2;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;2082:934:15;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;1173:30;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;3021:599;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;4268:153:2;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;940:80:15;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;5352:320:2;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;1459:30:15;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;5875:86;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;1053:37;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;4957:464;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;5443:107;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;5662:126;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;717:34;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;4487:162:2;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;674:37:15;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;1918:198:0;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;894:40:15;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;788:45;829:4;788:45;:::o;990:222:5:-;1092:4;1130:35;1115:50;;;:11;:50;;;;:90;;;;1169:36;1193:11;1169:23;:36::i;:::-;1115:90;1108:97;;990:222;;;:::o;5793:77:15:-;1259:12:0;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;5857:6:15::1;5848;;:15;;;;;;;;;;;;;;;;;;5793:77:::0;:::o;2473:98:2:-;2527:13;2559:5;2552:12;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;2473:98;:::o;3984:217::-;4060:7;4087:16;4095:7;4087;:16::i;:::-;4079:73;;;;;;;;;;;;:::i;:::-;;;;;;;;;4170:15;:24;4186:7;4170:24;;;;;;;;;;;;;;;;;;;;;4163:31;;3984:217;;;:::o;3522:401::-;3602:13;3618:23;3633:7;3618:14;:23::i;:::-;3602:39;;3665:5;3659:11;;:2;:11;;;;3651:57;;;;;;;;;;;;:::i;:::-;;;;;;;;;3756:5;3740:21;;:12;:10;:12::i;:::-;:21;;;:62;;;;3765:37;3782:5;3789:12;:10;:12::i;:::-;3765:16;:37::i;:::-;3740:62;3719:165;;;;;;;;;;;;:::i;:::-;;;;;;;;;3895:21;3904:2;3908:7;3895:8;:21::i;:::-;3522:401;;;:::o;1096:39:15:-;;;;:::o;4456:114::-;4514:4;4558:5;4537:26;;:17;4545:8;4537:7;:17::i;:::-;:26;;;4530:33;;4456:114;;;:::o;1615:111:5:-;1676:7;1702:10;:17;;;;1695:24;;1615:111;:::o;1344:55:15:-;;;;;;;;;;;;;;;;;:::o;4711:330:2:-;4900:41;4919:12;:10;:12::i;:::-;4933:7;4900:18;:41::i;:::-;4892:103;;;;;;;;;;;;:::i;:::-;;;;;;;;;5006:28;5016:4;5022:2;5026:7;5006:9;:28::i;:::-;4711:330;;;:::o;1244:94:15:-;;;;:::o;1291:253:5:-;1388:7;1423:23;1440:5;1423:16;:23::i;:::-;1415:5;:31;1407:87;;;;;;;;;;;;:::i;:::-;;;;;;;;;1511:12;:19;1524:5;1511:19;;;;;;;;;;;;;;;:26;1531:5;1511:26;;;;;;;;;;;;1504:33;;1291:253;;;;:::o;839:48:15:-;882:5;839:48;:::o;6060:152::-;1259:12:0;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;6116:7:15::1;6137;:5;:7::i;:::-;6129:21;;6158;6129:55;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;6115:69;;;6202:2;6194:11;;;::::0;::::1;;1318:1:0;6060:152:15:o:0;5107:179:2:-;5240:39;5257:4;5263:2;5267:7;5240:39;;;;;;;;;;;;:16;:39::i;:::-;5107:179;;;:::o;4575:377:15:-;4659:16;4695:23;4721:17;4731:6;4721:9;:17::i;:::-;4695:43;;4748:25;4790:15;4776:30;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;4748:58;;4821:9;4816:107;4836:15;4832:1;:19;4816:107;;;4882:30;4902:6;4910:1;4882:19;:30::i;:::-;4868:8;4877:1;4868:11;;;;;;;;;;;;;;;;;;;;;:44;;;;;4853:3;;;;;:::i;:::-;;;;4816:107;;;;4937:8;4930:15;;;;4575:377;;;:::o;6248:155::-;1259:12:0;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;6339:13:15::1;6326:10;:26;;;;6367:29;6385:10;;6367:29;;;;;;:::i;:::-;;;;;;;;6248:155:::0;:::o;5966:89::-;1259:12:0;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;6042:6:15::1;6029:10;;:19;;;;;;;;;;;;;;;;;;5966:89:::0;:::o;1798:230:5:-;1873:7;1908:30;:28;:30::i;:::-;1900:5;:38;1892:95;;;;;;;;;;;;:::i;:::-;;;;;;;;;2004:10;2015:5;2004:17;;;;;;;;;;;;;;;;;;;;;;;;1997:24;;1798:230;;;:::o;5555:102:15:-;1259:12:0;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;5639:11:15::1;5629:7;:21;;;;;;;;;;;;:::i;:::-;;5555:102:::0;:::o;1141:26::-;;;;;;;;;;;;;:::o;1209:29::-;;;;;;;;;;;;;:::o;2176:235:2:-;2248:7;2267:13;2283:7;:16;2291:7;2283:16;;;;;;;;;;;;;;;;;;;;;2267:32;;2334:1;2317:19;;:5;:19;;;;2309:73;;;;;;;;;;;;:::i;:::-;;;;;;;;;2399:5;2392:12;;;2176:235;;;:::o;3625:470:15:-;1822:10;;;;;;;;;;;1814:38;;;;;;;;;;;;:::i;:::-;;;;;;;;;1873:6;;;;;;;;;;;1872:7;1864:35;;;;;;;;;;;;:::i;:::-;;;;;;;;;3741:9:::1;3736:353;3760:9;:16;3756:1;:20;3736:353;;;3795:15;3813:9;3823:1;3813:12;;;;;;;;;;;;;;;;;;;;;;3795:30;;3865:5;3845:25;;:16;3853:7;3845;:16::i;:::-;:25;;;3837:54;;;;;;;;;;;;:::i;:::-;;;;;;;;;829:4;3911:7;:24;3903:55;;;;;;;;;;;;:::i;:::-;;;;;;;;;4006:12;:10;:12::i;:::-;3978:40;;:7;;;;;;;;;;;:15;;;3994:7;3978:24;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;::::0;::::1;;;;;;;;;;;;::::0;::::1;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;:40;;;3970:63;;;;;;;;;;;;:::i;:::-;;;;;;;;;4043:32;4053:12;:10;:12::i;:::-;4067:7;4043:9;:32::i;:::-;3736:353;3778:3;;;;;:::i;:::-;;;;3736:353;;;;3625:470:::0;:::o;1026:21::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;1914:205:2:-;1986:7;2030:1;2013:19;;:5;:19;;;;2005:74;;;;;;;;;;;;:::i;:::-;;;;;;;;;2096:9;:16;2106:5;2096:16;;;;;;;;;;;;;;;;2089:23;;1914:205;;;:::o;1668:101:0:-;1259:12;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;1732:30:::1;1759:1;1732:18;:30::i;:::-;1668:101::o:0;4100:351:15:-;1259:12:0;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;931:3:15::1;4195:6;4170:22;;:31;;;;:::i;:::-;:45;;4162:77;;;;;;;;;;;;:::i;:::-;;;;;;;;;4258:9;4253:192;4277:6;4273:1;:10;4253:192;;;4310:73;4320:12;:10;:12::i;:::-;4360:22;;931:3;829:4;882:5;974:33;;;;:::i;:::-;:46;;;;:::i;:::-;829:4;4334:24;;;;:::i;:::-;:48;;;;:::i;:::-;4310:9;:73::i;:::-;4429:1;4403:22;;:27;;;;;;;:::i;:::-;;;;;;;;4285:3;;;;;:::i;:::-;;;;4253:192;;;;4100:351:::0;:::o;1036:85:0:-;1082:7;1108:6;;;;;;;;;;;1101:13;;1036:85;:::o;2635:102:2:-;2691:13;2723:7;2716:14;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;2635:102;:::o;2082:934:15:-;2176:6;;;;;;;;;;;2175:7;2167:42;;;;;;;;;;;;:::i;:::-;;;;;;;;;2243:66;2229:80;;:10;;:80;;2221:117;;;;;;;;;;;;:::i;:::-;;;;;;;;;931:3;829:4;882:5;974:33;;;;:::i;:::-;:46;;;;:::i;:::-;2358:26;2382:1;2358:19;;:23;;:26;;;;:::i;:::-;:37;;2350:59;;;;;;;;;;;;:::i;:::-;;;;;;;;;2517:1;2482:20;:32;2503:10;2482:32;;;;;;;;;;;;;;;;:36;2474:86;;;;;;;;;;;;:::i;:::-;;;;;;;;;2599:88;2618:12;;2599:88;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;2632:10;;2672;2655:28;;;;;;;;:::i;:::-;;;;;;;;;;;;;2645:39;;;;;;2599:18;:88::i;:::-;2591:114;;;;;;;;;;;;:::i;:::-;;;;;;;;;2762:11;2771:1;2762:4;;:8;;:11;;;;:::i;:::-;2749:9;:24;2741:69;;;;;;;;;;;;:::i;:::-;;;;;;;;;2845:20;:32;2866:10;2845:32;;;;;;;;;;;;;;;;:34;;;;;;;;;:::i;:::-;;;;;;2911:62;2921:12;:10;:12::i;:::-;2953:19;;829:4;2935:37;;;;:::i;:::-;2911:9;:62::i;:::-;3008:1;2985:19;;:24;;;;;;;:::i;:::-;;;;;;;;2082:934;;:::o;1173:30::-;;;;;;;;;;;;;:::o;3021:599::-;1966:9;;;;;;;;;;;1958:36;;;;;;;;;;;;:::i;:::-;;;;;;;;;2015:6;;;;;;;;;;;2014:7;2006:35;;;;;;;;;;;;:::i;:::-;;;;;;;;;1744:1:1::1;2325:7;;:19;;2317:63;;;;;;;;;;;;:::i;:::-;;;;;;;;;1744:1;2455:7;:18;;;;3110:6:15::2;;;;;;;;;;;3109:7;3101:42;;;;;;;;;;;;:::i;:::-;;;;;;;;;931:3;829:4;882:5;974:33;;;;:::i;:::-;:46;;;;:::i;:::-;3163:31;3187:6;3163:19;;:23;;:31;;;;:::i;:::-;:42;;3155:64;;;;;;;;;;;;:::i;:::-;;;;;;;;;3248:1;3239:6;:10;:25;;;;;3263:1;3253:6;:11;;3239:25;3231:70;;;;;;;;;;;;:::i;:::-;;;;;;;;;3332:16;3341:6;3332:4;;:8;;:16;;;;:::i;:::-;3321:9;:27;3313:71;;;;;;;;;;;;:::i;:::-;;;;;;;;;3401:9;3396:218;3420:6;3416:1;:10;3396:218;;;3449:20;:32;3470:10;3449:32;;;;;;;;;;;;;;;;:34;;;;;;;;;:::i;:::-;;;;;;3499:62;3509:12;:10;:12::i;:::-;3541:19;;829:4;3523:37;;;;:::i;:::-;3499:9;:62::i;:::-;3600:1;3577:19;;:24;;;;;;;:::i;:::-;;;;;;;;3428:3;;;;;:::i;:::-;;;;3396:218;;;;1701:1:1::1;2628:7;:22;;;;3021:599:15::0;:::o;4268:153:2:-;4362:52;4381:12;:10;:12::i;:::-;4395:8;4405;4362:18;:52::i;:::-;4268:153;;:::o;940:80:15:-;931:3;829:4;882:5;974:33;;;;:::i;:::-;:46;;;;:::i;:::-;940:80;:::o;5352:320:2:-;5521:41;5540:12;:10;:12::i;:::-;5554:7;5521:18;:41::i;:::-;5513:103;;;;;;;;;;;;:::i;:::-;;;;;;;;;5626:39;5640:4;5646:2;5650:7;5659:5;5626:13;:39::i;:::-;5352:320;;;;:::o;1459:30:15:-;;;;;;;;;;;;;:::o;5875:86::-;1259:12:0;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;5948:6:15::1;5936:9;;:18;;;;;;;;;;;;;;;;;;5875:86:::0;:::o;1053:37::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;4957:464::-;5070:13;5120:16;5128:7;5120;:16::i;:::-;5101:106;;;;;;;;;;;;:::i;:::-;;;;;;;;;5217:28;5248:10;:8;:10::i;:::-;5217:41;;5306:1;5281:14;5275:28;:32;:139;;;;;;;;;;;;;;;;;5346:14;5362:18;:7;:16;:18::i;:::-;5382:13;5329:67;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;5275:139;5268:146;;;4957:464;;;:::o;5443:107::-;1259:12:0;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;5534:8:15::1;5508:7;;:35;;;;;;;;;;;;;;;;;;5443:107:::0;:::o;5662:126::-;1259:12:0;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;5764:17:15::1;5748:13;:33;;;;;;;;;;;;:::i;:::-;;5662:126:::0;:::o;717:34::-;;;;:::o;4487:162:2:-;4584:4;4607:18;:25;4626:5;4607:25;;;;;;;;;;;;;;;:35;4633:8;4607:35;;;;;;;;;;;;;;;;;;;;;;;;;4600:42;;4487:162;;;;:::o;674:37:15:-;;;;:::o;1918:198:0:-;1259:12;:10;:12::i;:::-;1248:23;;:7;:5;:7::i;:::-;:23;;;1240:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;2026:1:::1;2006:22;;:8;:22;;;;1998:73;;;;;;;;;;;;:::i;:::-;;;;;;;;;2081:28;2100:8;2081:18;:28::i;:::-;1918:198:::0;:::o;894:40:15:-;931:3;894:40;:::o;1555:300:2:-;1657:4;1707:25;1692:40;;;:11;:40;;;;:104;;;;1763:33;1748:48;;;:11;:48;;;;1692:104;:156;;;;1812:36;1836:11;1812:23;:36::i;:::-;1692:156;1673:175;;1555:300;;;:::o;640:96:9:-;693:7;719:10;712:17;;640:96;:::o;7144:125:2:-;7209:4;7260:1;7232:30;;:7;:16;7240:7;7232:16;;;;;;;;;;;;;;;;;;;;;:30;;;;7225:37;;7144:125;;;:::o;10995:171::-;11096:2;11069:15;:24;11085:7;11069:24;;;;;;;;;;;;:29;;;;;;;;;;;;;;;;;;11151:7;11147:2;11113:46;;11122:23;11137:7;11122:14;:23::i;:::-;11113:46;;;;;;;;;;;;10995:171;;:::o;7427:344::-;7520:4;7544:16;7552:7;7544;:16::i;:::-;7536:73;;;;;;;;;;;;:::i;:::-;;;;;;;;;7619:13;7635:23;7650:7;7635:14;:23::i;:::-;7619:39;;7687:5;7676:16;;:7;:16;;;:51;;;;7720:7;7696:31;;:20;7708:7;7696:11;:20::i;:::-;:31;;;7676:51;:87;;;;7731:32;7748:5;7755:7;7731:16;:32::i;:::-;7676:87;7668:96;;;7427:344;;;;:::o;10324:560::-;10478:4;10451:31;;:23;10466:7;10451:14;:23::i;:::-;:31;;;10443:85;;;;;;;;;;;;:::i;:::-;;;;;;;;;10560:1;10546:16;;:2;:16;;;;10538:65;;;;;;;;;;;;:::i;:::-;;;;;;;;;10614:39;10635:4;10641:2;10645:7;10614:20;:39::i;:::-;10715:29;10732:1;10736:7;10715:8;:29::i;:::-;10774:1;10755:9;:15;10765:4;10755:15;;;;;;;;;;;;;;;;:20;;;;;;;:::i;:::-;;;;;;;;10802:1;10785:9;:13;10795:2;10785:13;;;;;;;;;;;;;;;;:18;;;;;;;:::i;:::-;;;;;;;;10832:2;10813:7;:16;10821:7;10813:16;;;;;;;;;;;;:21;;;;;;;;;;;;;;;;;;10869:7;10865:2;10850:27;;10859:4;10850:27;;;;;;;;;;;;10324:560;;;:::o;8101:108::-;8176:26;8186:2;8190:7;8176:26;;;;;;;;;;;;:9;:26::i;:::-;8101:108;;:::o;2270:187:0:-;2343:16;2362:6;;;;;;;;;;;2343:25;;2387:8;2378:6;;:17;;;;;;;;;;;;;;;;;;2441:8;2410:40;;2431:8;2410:40;;;;;;;;;;;;2270:187;;:::o;2741:96:14:-;2799:7;2829:1;2825;:5;;;;:::i;:::-;2818:12;;2741:96;;;;:::o;847:184:11:-;968:4;1020;991:25;1004:5;1011:4;991:12;:25::i;:::-;:33;984:40;;847:184;;;;;:::o;3451:96:14:-;3509:7;3539:1;3535;:5;;;;:::i;:::-;3528:12;;3451:96;;;;:::o;11301:307:2:-;11451:8;11442:17;;:5;:17;;;;11434:55;;;;;;;;;;;;:::i;:::-;;;;;;;;;11537:8;11499:18;:25;11518:5;11499:25;;;;;;;;;;;;;;;:35;11525:8;11499:35;;;;;;;;;;;;;;;;:46;;;;;;;;;;;;;;;;;;11582:8;11560:41;;11575:5;11560:41;;;11592:8;11560:41;;;;;;:::i;:::-;;;;;;;;11301:307;;;:::o;6534:::-;6685:28;6695:4;6701:2;6705:7;6685:9;:28::i;:::-;6731:48;6754:4;6760:2;6764:7;6773:5;6731:22;:48::i;:::-;6723:111;;;;;;;;;;;;:::i;:::-;;;;;;;;;6534:307;;;;:::o;1661:102:15:-;1721:13;1749:7;1742:14;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;1661:102;:::o;328:703:10:-;384:13;610:1;601:5;:10;597:51;;;627:10;;;;;;;;;;;;;;;;;;;;;597:51;657:12;672:5;657:20;;687:14;711:75;726:1;718:4;:9;711:75;;743:8;;;;;:::i;:::-;;;;773:2;765:10;;;;;:::i;:::-;;;711:75;;;795:19;827:6;817:17;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;795:39;;844:150;860:1;851:5;:10;844:150;;887:1;877:11;;;;;:::i;:::-;;;953:2;945:5;:10;;;;:::i;:::-;932:2;:24;;;;:::i;:::-;919:39;;902:6;909;902:14;;;;;;;;;;;;;;;;;;;:56;;;;;;;;;;;981:2;972:11;;;;;:::i;:::-;;;844:150;;;1017:6;1003:21;;;;;328:703;;;;:::o;829:155:12:-;914:4;952:25;937:40;;;:11;:40;;;;930:47;;829:155;;;:::o;2624:572:5:-;2763:45;2790:4;2796:2;2800:7;2763:26;:45::i;:::-;2839:1;2823:18;;:4;:18;;;2819:183;;;2857:40;2889:7;2857:31;:40::i;:::-;2819:183;;;2926:2;2918:10;;:4;:10;;;2914:88;;2944:47;2977:4;2983:7;2944:32;:47::i;:::-;2914:88;2819:183;3029:1;3015:16;;:2;:16;;;3011:179;;;3047:45;3084:7;3047:36;:45::i;:::-;3011:179;;;3119:4;3113:10;;:2;:10;;;3109:81;;3139:40;3167:2;3171:7;3139:27;:40::i;:::-;3109:81;3011:179;2624:572;;;:::o;8430:311:2:-;8555:18;8561:2;8565:7;8555:5;:18::i;:::-;8604:54;8635:1;8639:2;8643:7;8652:5;8604:22;:54::i;:::-;8583:151;;;;;;;;;;;;:::i;:::-;;;;;;;;;8430:311;;;:::o;1383:688:11:-;1466:7;1485:20;1508:4;1485:27;;1527:9;1522:514;1546:5;:12;1542:1;:16;1522:514;;;1579:20;1602:5;1608:1;1602:8;;;;;;;;;;;;;;;;;;;;;;1579:31;;1644:12;1628;:28;1624:402;;1796:12;1810;1779:44;;;;;;;;;:::i;:::-;;;;;;;;;;;;;1769:55;;;;;;1754:70;;1624:402;;;1983:12;1997;1966:44;;;;;;;;;:::i;:::-;;;;;;;;;;;;;1956:55;;;;;;1941:70;;1624:402;1522:514;1560:3;;;;;:::i;:::-;;;;1522:514;;;;2052:12;2045:19;;;1383:688;;;;:::o;12161:778:2:-;12311:4;12331:15;:2;:13;;;:15::i;:::-;12327:606;;;12382:2;12366:36;;;12403:12;:10;:12::i;:::-;12417:4;12423:7;12432:5;12366:72;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;12362:519;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;12622:1;12605:6;:13;:18;12601:266;;;12647:60;;;;;;;;;;:::i;:::-;;;;;;;;12601:266;12819:6;12813:13;12804:6;12800:2;12796:15;12789:38;12362:519;12498:41;;;12488:51;;;:6;:51;;;;12481:58;;;;;12327:606;12918:4;12911:11;;12161:778;;;;;;;:::o;13495:122::-;;;;:::o;3902:161:5:-;4005:10;:17;;;;3978:15;:24;3994:7;3978:24;;;;;;;;;;;:44;;;;4032:10;4048:7;4032:24;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;3902:161;:::o;4680:970::-;4942:22;4992:1;4967:22;4984:4;4967:16;:22::i;:::-;:26;;;;:::i;:::-;4942:51;;5003:18;5024:17;:26;5042:7;5024:26;;;;;;;;;;;;5003:47;;5168:14;5154:10;:28;5150:323;;5198:19;5220:12;:18;5233:4;5220:18;;;;;;;;;;;;;;;:34;5239:14;5220:34;;;;;;;;;;;;5198:56;;5302:11;5269:12;:18;5282:4;5269:18;;;;;;;;;;;;;;;:30;5288:10;5269:30;;;;;;;;;;;:44;;;;5418:10;5385:17;:30;5403:11;5385:30;;;;;;;;;;;:43;;;;5150:323;;5566:17;:26;5584:7;5566:26;;;;;;;;;;;5559:33;;;5609:12;:18;5622:4;5609:18;;;;;;;;;;;;;;;:34;5628:14;5609:34;;;;;;;;;;;5602:41;;;4680:970;;;;:::o;5938:1061::-;6187:22;6232:1;6212:10;:17;;;;:21;;;;:::i;:::-;6187:46;;6243:18;6264:15;:24;6280:7;6264:24;;;;;;;;;;;;6243:45;;6610:19;6632:10;6643:14;6632:26;;;;;;;;;;;;;;;;;;;;;;;;6610:48;;6694:11;6669:10;6680;6669:22;;;;;;;;;;;;;;;;;;;;;;;:36;;;;6804:10;6773:15;:28;6789:11;6773:28;;;;;;;;;;;:41;;;;6942:15;:24;6958:7;6942:24;;;;;;;;;;;6935:31;;;6976:10;:16;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;5938:1061;;;;:::o;3490:217::-;3574:14;3591:20;3608:2;3591:16;:20::i;:::-;3574:37;;3648:7;3621:12;:16;3634:2;3621:16;;;;;;;;;;;;;;;:24;3638:6;3621:24;;;;;;;;;;;:34;;;;3694:6;3665:17;:26;3683:7;3665:26;;;;;;;;;;;:35;;;;3490:217;;;:::o;9063:372:2:-;9156:1;9142:16;;:2;:16;;;;9134:61;;;;;;;;;;;;:::i;:::-;;;;;;;;;9214:16;9222:7;9214;:16::i;:::-;9213:17;9205:58;;;;;;;;;;;;:::i;:::-;;;;;;;;;9274:45;9303:1;9307:2;9311:7;9274:20;:45::i;:::-;9347:1;9330:9;:13;9340:2;9330:13;;;;;;;;;;;;;;;;:18;;;;;;;:::i;:::-;;;;;;;;9377:2;9358:7;:16;9366:7;9358:16;;;;;;;;;;;;:21;;;;;;;;;;;;;;;;;;9420:7;9416:2;9395:33;;9412:1;9395:33;;;;;;;;;;;;9063:372;;:::o;771:377:8:-;831:4;1034:12;1099:7;1087:20;1079:28;;1140:1;1133:4;:8;1126:15;;;771:377;;;:::o;-1:-1:-1:-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;:::o;:::-;;;;;;;;;;;;;;;;;;;;;:::o;24:655:16:-;120:5;145:81;161:64;218:6;161:64;:::i;:::-;145:81;:::i;:::-;136:90;;246:5;275:6;268:5;261:21;309:4;302:5;298:16;291:23;;335:6;385:3;377:4;369:6;365:17;360:3;356:27;353:36;350:2;;;414:1;411;404:12;350:2;450:1;435:238;460:6;457:1;454:13;435:238;;;528:3;557:37;590:3;578:10;557:37;:::i;:::-;552:3;545:50;624:4;619:3;615:14;608:21;;658:4;653:3;649:14;642:21;;495:178;482:1;479;475:9;470:14;;435:238;;;439:14;126:553;;;;;;;:::o;685:343::-;762:5;787:65;803:48;844:6;803:48;:::i;:::-;787:65;:::i;:::-;778:74;;875:6;868:5;861:21;913:4;906:5;902:16;951:3;942:6;937:3;933:16;930:25;927:2;;;968:1;965;958:12;927:2;981:41;1015:6;1010:3;1005;981:41;:::i;:::-;768:260;;;;;;:::o;1034:345::-;1112:5;1137:66;1153:49;1195:6;1153:49;:::i;:::-;1137:66;:::i;:::-;1128:75;;1226:6;1219:5;1212:21;1264:4;1257:5;1253:16;1302:3;1293:6;1288:3;1284:16;1281:25;1278:2;;;1319:1;1316;1309:12;1278:2;1332:41;1366:6;1361:3;1356;1332:41;:::i;:::-;1118:261;;;;;;:::o;1385:139::-;1431:5;1469:6;1456:20;1447:29;;1485:33;1512:5;1485:33;:::i;:::-;1437:87;;;;:::o;1530:143::-;1587:5;1618:6;1612:13;1603:22;;1634:33;1661:5;1634:33;:::i;:::-;1593:80;;;;:::o;1696:367::-;1769:8;1779:6;1829:3;1822:4;1814:6;1810:17;1806:27;1796:2;;1847:1;1844;1837:12;1796:2;1883:6;1870:20;1860:30;;1913:18;1905:6;1902:30;1899:2;;;1945:1;1942;1935:12;1899:2;1982:4;1974:6;1970:17;1958:29;;2036:3;2028:4;2020:6;2016:17;2006:8;2002:32;1999:41;1996:2;;;2053:1;2050;2043:12;1996:2;1786:277;;;;;:::o;2086:303::-;2157:5;2206:3;2199:4;2191:6;2187:17;2183:27;2173:2;;2224:1;2221;2214:12;2173:2;2264:6;2251:20;2289:94;2379:3;2371:6;2364:4;2356:6;2352:17;2289:94;:::i;:::-;2280:103;;2163:226;;;;;:::o;2395:133::-;2438:5;2476:6;2463:20;2454:29;;2492:30;2516:5;2492:30;:::i;:::-;2444:84;;;;:::o;2534:139::-;2580:5;2618:6;2605:20;2596:29;;2634:33;2661:5;2634:33;:::i;:::-;2586:87;;;;:::o;2679:137::-;2724:5;2762:6;2749:20;2740:29;;2778:32;2804:5;2778:32;:::i;:::-;2730:86;;;;:::o;2822:141::-;2878:5;2909:6;2903:13;2894:22;;2925:32;2951:5;2925:32;:::i;:::-;2884:79;;;;:::o;2982:271::-;3037:5;3086:3;3079:4;3071:6;3067:17;3063:27;3053:2;;3104:1;3101;3094:12;3053:2;3144:6;3131:20;3169:78;3243:3;3235:6;3228:4;3220:6;3216:17;3169:78;:::i;:::-;3160:87;;3043:210;;;;;:::o;3273:273::-;3329:5;3378:3;3371:4;3363:6;3359:17;3355:27;3345:2;;3396:1;3393;3386:12;3345:2;3436:6;3423:20;3461:79;3536:3;3528:6;3521:4;3513:6;3509:17;3461:79;:::i;:::-;3452:88;;3335:211;;;;;:::o;3552:139::-;3598:5;3636:6;3623:20;3614:29;;3652:33;3679:5;3652:33;:::i;:::-;3604:87;;;;:::o;3697:262::-;3756:6;3805:2;3793:9;3784:7;3780:23;3776:32;3773:2;;;3821:1;3818;3811:12;3773:2;3864:1;3889:53;3934:7;3925:6;3914:9;3910:22;3889:53;:::i;:::-;3879:63;;3835:117;3763:196;;;;:::o;3965:284::-;4035:6;4084:2;4072:9;4063:7;4059:23;4055:32;4052:2;;;4100:1;4097;4090:12;4052:2;4143:1;4168:64;4224:7;4215:6;4204:9;4200:22;4168:64;:::i;:::-;4158:74;;4114:128;4042:207;;;;:::o;4255:407::-;4323:6;4331;4380:2;4368:9;4359:7;4355:23;4351:32;4348:2;;;4396:1;4393;4386:12;4348:2;4439:1;4464:53;4509:7;4500:6;4489:9;4485:22;4464:53;:::i;:::-;4454:63;;4410:117;4566:2;4592:53;4637:7;4628:6;4617:9;4613:22;4592:53;:::i;:::-;4582:63;;4537:118;4338:324;;;;;:::o;4668:552::-;4745:6;4753;4761;4810:2;4798:9;4789:7;4785:23;4781:32;4778:2;;;4826:1;4823;4816:12;4778:2;4869:1;4894:53;4939:7;4930:6;4919:9;4915:22;4894:53;:::i;:::-;4884:63;;4840:117;4996:2;5022:53;5067:7;5058:6;5047:9;5043:22;5022:53;:::i;:::-;5012:63;;4967:118;5124:2;5150:53;5195:7;5186:6;5175:9;5171:22;5150:53;:::i;:::-;5140:63;;5095:118;4768:452;;;;;:::o;5226:809::-;5321:6;5329;5337;5345;5394:3;5382:9;5373:7;5369:23;5365:33;5362:2;;;5411:1;5408;5401:12;5362:2;5454:1;5479:53;5524:7;5515:6;5504:9;5500:22;5479:53;:::i;:::-;5469:63;;5425:117;5581:2;5607:53;5652:7;5643:6;5632:9;5628:22;5607:53;:::i;:::-;5597:63;;5552:118;5709:2;5735:53;5780:7;5771:6;5760:9;5756:22;5735:53;:::i;:::-;5725:63;;5680:118;5865:2;5854:9;5850:18;5837:32;5896:18;5888:6;5885:30;5882:2;;;5928:1;5925;5918:12;5882:2;5956:62;6010:7;6001:6;5990:9;5986:22;5956:62;:::i;:::-;5946:72;;5808:220;5352:683;;;;;;;:::o;6041:401::-;6106:6;6114;6163:2;6151:9;6142:7;6138:23;6134:32;6131:2;;;6179:1;6176;6169:12;6131:2;6222:1;6247:53;6292:7;6283:6;6272:9;6268:22;6247:53;:::i;:::-;6237:63;;6193:117;6349:2;6375:50;6417:7;6408:6;6397:9;6393:22;6375:50;:::i;:::-;6365:60;;6320:115;6121:321;;;;;:::o;6448:407::-;6516:6;6524;6573:2;6561:9;6552:7;6548:23;6544:32;6541:2;;;6589:1;6586;6579:12;6541:2;6632:1;6657:53;6702:7;6693:6;6682:9;6678:22;6657:53;:::i;:::-;6647:63;;6603:117;6759:2;6785:53;6830:7;6821:6;6810:9;6806:22;6785:53;:::i;:::-;6775:63;;6730:118;6531:324;;;;;:::o;6861:425::-;6947:6;6955;7004:2;6992:9;6983:7;6979:23;6975:32;6972:2;;;7020:1;7017;7010:12;6972:2;7091:1;7080:9;7076:17;7063:31;7121:18;7113:6;7110:30;7107:2;;;7153:1;7150;7143:12;7107:2;7189:80;7261:7;7252:6;7241:9;7237:22;7189:80;:::i;:::-;7171:98;;;;7034:245;6962:324;;;;;:::o;7292:405::-;7376:6;7425:2;7413:9;7404:7;7400:23;7396:32;7393:2;;;7441:1;7438;7431:12;7393:2;7512:1;7501:9;7497:17;7484:31;7542:18;7534:6;7531:30;7528:2;;;7574:1;7571;7564:12;7528:2;7602:78;7672:7;7663:6;7652:9;7648:22;7602:78;:::i;:::-;7592:88;;7455:235;7383:314;;;;:::o;7703:256::-;7759:6;7808:2;7796:9;7787:7;7783:23;7779:32;7776:2;;;7824:1;7821;7814:12;7776:2;7867:1;7892:50;7934:7;7925:6;7914:9;7910:22;7892:50;:::i;:::-;7882:60;;7838:114;7766:193;;;;:::o;7965:262::-;8024:6;8073:2;8061:9;8052:7;8048:23;8044:32;8041:2;;;8089:1;8086;8079:12;8041:2;8132:1;8157:53;8202:7;8193:6;8182:9;8178:22;8157:53;:::i;:::-;8147:63;;8103:117;8031:196;;;;:::o;8233:260::-;8291:6;8340:2;8328:9;8319:7;8315:23;8311:32;8308:2;;;8356:1;8353;8346:12;8308:2;8399:1;8424:52;8468:7;8459:6;8448:9;8444:22;8424:52;:::i;:::-;8414:62;;8370:116;8298:195;;;;:::o;8499:282::-;8568:6;8617:2;8605:9;8596:7;8592:23;8588:32;8585:2;;;8633:1;8630;8623:12;8585:2;8676:1;8701:63;8756:7;8747:6;8736:9;8732:22;8701:63;:::i;:::-;8691:73;;8647:127;8575:206;;;;:::o;8787:375::-;8856:6;8905:2;8893:9;8884:7;8880:23;8876:32;8873:2;;;8921:1;8918;8911:12;8873:2;8992:1;8981:9;8977:17;8964:31;9022:18;9014:6;9011:30;9008:2;;;9054:1;9051;9044:12;9008:2;9082:63;9137:7;9128:6;9117:9;9113:22;9082:63;:::i;:::-;9072:73;;8935:220;8863:299;;;;:::o;9168:262::-;9227:6;9276:2;9264:9;9255:7;9251:23;9247:32;9244:2;;;9292:1;9289;9282:12;9244:2;9335:1;9360:53;9405:7;9396:6;9385:9;9381:22;9360:53;:::i;:::-;9350:63;;9306:117;9234:196;;;;:::o;9436:179::-;9505:10;9526:46;9568:3;9560:6;9526:46;:::i;:::-;9604:4;9599:3;9595:14;9581:28;;9516:99;;;;:::o;9621:118::-;9708:24;9726:5;9708:24;:::i;:::-;9703:3;9696:37;9686:53;;:::o;9745:157::-;9850:45;9870:24;9888:5;9870:24;:::i;:::-;9850:45;:::i;:::-;9845:3;9838:58;9828:74;;:::o;9938:732::-;10057:3;10086:54;10134:5;10086:54;:::i;:::-;10156:86;10235:6;10230:3;10156:86;:::i;:::-;10149:93;;10266:56;10316:5;10266:56;:::i;:::-;10345:7;10376:1;10361:284;10386:6;10383:1;10380:13;10361:284;;;10462:6;10456:13;10489:63;10548:3;10533:13;10489:63;:::i;:::-;10482:70;;10575:60;10628:6;10575:60;:::i;:::-;10565:70;;10421:224;10408:1;10405;10401:9;10396:14;;10361:284;;;10365:14;10661:3;10654:10;;10062:608;;;;;;;:::o;10676:109::-;10757:21;10772:5;10757:21;:::i;:::-;10752:3;10745:34;10735:50;;:::o;10791:118::-;10878:24;10896:5;10878:24;:::i;:::-;10873:3;10866:37;10856:53;;:::o;10915:157::-;11020:45;11040:24;11058:5;11040:24;:::i;:::-;11020:45;:::i;:::-;11015:3;11008:58;10998:74;;:::o;11078:360::-;11164:3;11192:38;11224:5;11192:38;:::i;:::-;11246:70;11309:6;11304:3;11246:70;:::i;:::-;11239:77;;11325:52;11370:6;11365:3;11358:4;11351:5;11347:16;11325:52;:::i;:::-;11402:29;11424:6;11402:29;:::i;:::-;11397:3;11393:39;11386:46;;11168:270;;;;;:::o;11444:179::-;11555:61;11610:5;11555:61;:::i;:::-;11550:3;11543:74;11533:90;;:::o;11629:364::-;11717:3;11745:39;11778:5;11745:39;:::i;:::-;11800:71;11864:6;11859:3;11800:71;:::i;:::-;11793:78;;11880:52;11925:6;11920:3;11913:4;11906:5;11902:16;11880:52;:::i;:::-;11957:29;11979:6;11957:29;:::i;:::-;11952:3;11948:39;11941:46;;11721:272;;;;;:::o;11999:377::-;12105:3;12133:39;12166:5;12133:39;:::i;:::-;12188:89;12270:6;12265:3;12188:89;:::i;:::-;12181:96;;12286:52;12331:6;12326:3;12319:4;12312:5;12308:16;12286:52;:::i;:::-;12363:6;12358:3;12354:16;12347:23;;12109:267;;;;;:::o;12406:845::-;12509:3;12546:5;12540:12;12575:36;12601:9;12575:36;:::i;:::-;12627:89;12709:6;12704:3;12627:89;:::i;:::-;12620:96;;12747:1;12736:9;12732:17;12763:1;12758:137;;;;12909:1;12904:341;;;;12725:520;;12758:137;12842:4;12838:9;12827;12823:25;12818:3;12811:38;12878:6;12873:3;12869:16;12862:23;;12758:137;;12904:341;12971:38;13003:5;12971:38;:::i;:::-;13031:1;13045:154;13059:6;13056:1;13053:13;13045:154;;;13133:7;13127:14;13123:1;13118:3;13114:11;13107:35;13183:1;13174:7;13170:15;13159:26;;13081:4;13078:1;13074:12;13069:17;;13045:154;;;13228:6;13223:3;13219:16;13212:23;;12911:334;;12725:520;;12513:738;;;;;;:::o;13257:366::-;13399:3;13420:67;13484:2;13479:3;13420:67;:::i;:::-;13413:74;;13496:93;13585:3;13496:93;:::i;:::-;13614:2;13609:3;13605:12;13598:19;;13403:220;;;:::o;13629:366::-;13771:3;13792:67;13856:2;13851:3;13792:67;:::i;:::-;13785:74;;13868:93;13957:3;13868:93;:::i;:::-;13986:2;13981:3;13977:12;13970:19;;13775:220;;;:::o;14001:366::-;14143:3;14164:67;14228:2;14223:3;14164:67;:::i;:::-;14157:74;;14240:93;14329:3;14240:93;:::i;:::-;14358:2;14353:3;14349:12;14342:19;;14147:220;;;:::o;14373:366::-;14515:3;14536:67;14600:2;14595:3;14536:67;:::i;:::-;14529:74;;14612:93;14701:3;14612:93;:::i;:::-;14730:2;14725:3;14721:12;14714:19;;14519:220;;;:::o;14745:366::-;14887:3;14908:67;14972:2;14967:3;14908:67;:::i;:::-;14901:74;;14984:93;15073:3;14984:93;:::i;:::-;15102:2;15097:3;15093:12;15086:19;;14891:220;;;:::o;15117:365::-;15259:3;15280:66;15344:1;15339:3;15280:66;:::i;:::-;15273:73;;15355:93;15444:3;15355:93;:::i;:::-;15473:2;15468:3;15464:12;15457:19;;15263:219;;;:::o;15488:366::-;15630:3;15651:67;15715:2;15710:3;15651:67;:::i;:::-;15644:74;;15727:93;15816:3;15727:93;:::i;:::-;15845:2;15840:3;15836:12;15829:19;;15634:220;;;:::o;15860:366::-;16002:3;16023:67;16087:2;16082:3;16023:67;:::i;:::-;16016:74;;16099:93;16188:3;16099:93;:::i;:::-;16217:2;16212:3;16208:12;16201:19;;16006:220;;;:::o;16232:366::-;16374:3;16395:67;16459:2;16454:3;16395:67;:::i;:::-;16388:74;;16471:93;16560:3;16471:93;:::i;:::-;16589:2;16584:3;16580:12;16573:19;;16378:220;;;:::o;16604:366::-;16746:3;16767:67;16831:2;16826:3;16767:67;:::i;:::-;16760:74;;16843:93;16932:3;16843:93;:::i;:::-;16961:2;16956:3;16952:12;16945:19;;16750:220;;;:::o;16976:366::-;17118:3;17139:67;17203:2;17198:3;17139:67;:::i;:::-;17132:74;;17215:93;17304:3;17215:93;:::i;:::-;17333:2;17328:3;17324:12;17317:19;;17122:220;;;:::o;17348:366::-;17490:3;17511:67;17575:2;17570:3;17511:67;:::i;:::-;17504:74;;17587:93;17676:3;17587:93;:::i;:::-;17705:2;17700:3;17696:12;17689:19;;17494:220;;;:::o;17720:366::-;17862:3;17883:67;17947:2;17942:3;17883:67;:::i;:::-;17876:74;;17959:93;18048:3;17959:93;:::i;:::-;18077:2;18072:3;18068:12;18061:19;;17866:220;;;:::o;18092:366::-;18234:3;18255:67;18319:2;18314:3;18255:67;:::i;:::-;18248:74;;18331:93;18420:3;18331:93;:::i;:::-;18449:2;18444:3;18440:12;18433:19;;18238:220;;;:::o;18464:366::-;18606:3;18627:67;18691:2;18686:3;18627:67;:::i;:::-;18620:74;;18703:93;18792:3;18703:93;:::i;:::-;18821:2;18816:3;18812:12;18805:19;;18610:220;;;:::o;18836:366::-;18978:3;18999:67;19063:2;19058:3;18999:67;:::i;:::-;18992:74;;19075:93;19164:3;19075:93;:::i;:::-;19193:2;19188:3;19184:12;19177:19;;18982:220;;;:::o;19208:366::-;19350:3;19371:67;19435:2;19430:3;19371:67;:::i;:::-;19364:74;;19447:93;19536:3;19447:93;:::i;:::-;19565:2;19560:3;19556:12;19549:19;;19354:220;;;:::o;19580:366::-;19722:3;19743:67;19807:2;19802:3;19743:67;:::i;:::-;19736:74;;19819:93;19908:3;19819:93;:::i;:::-;19937:2;19932:3;19928:12;19921:19;;19726:220;;;:::o;19952:366::-;20094:3;20115:67;20179:2;20174:3;20115:67;:::i;:::-;20108:74;;20191:93;20280:3;20191:93;:::i;:::-;20309:2;20304:3;20300:12;20293:19;;20098:220;;;:::o;20324:366::-;20466:3;20487:67;20551:2;20546:3;20487:67;:::i;:::-;20480:74;;20563:93;20652:3;20563:93;:::i;:::-;20681:2;20676:3;20672:12;20665:19;;20470:220;;;:::o;20696:366::-;20838:3;20859:67;20923:2;20918:3;20859:67;:::i;:::-;20852:74;;20935:93;21024:3;20935:93;:::i;:::-;21053:2;21048:3;21044:12;21037:19;;20842:220;;;:::o;21068:366::-;21210:3;21231:67;21295:2;21290:3;21231:67;:::i;:::-;21224:74;;21307:93;21396:3;21307:93;:::i;:::-;21425:2;21420:3;21416:12;21409:19;;21214:220;;;:::o;21440:366::-;21582:3;21603:67;21667:2;21662:3;21603:67;:::i;:::-;21596:74;;21679:93;21768:3;21679:93;:::i;:::-;21797:2;21792:3;21788:12;21781:19;;21586:220;;;:::o;21812:366::-;21954:3;21975:67;22039:2;22034:3;21975:67;:::i;:::-;21968:74;;22051:93;22140:3;22051:93;:::i;:::-;22169:2;22164:3;22160:12;22153:19;;21958:220;;;:::o;22184:366::-;22326:3;22347:67;22411:2;22406:3;22347:67;:::i;:::-;22340:74;;22423:93;22512:3;22423:93;:::i;:::-;22541:2;22536:3;22532:12;22525:19;;22330:220;;;:::o;22556:366::-;22698:3;22719:67;22783:2;22778:3;22719:67;:::i;:::-;22712:74;;22795:93;22884:3;22795:93;:::i;:::-;22913:2;22908:3;22904:12;22897:19;;22702:220;;;:::o;22928:366::-;23070:3;23091:67;23155:2;23150:3;23091:67;:::i;:::-;23084:74;;23167:93;23256:3;23167:93;:::i;:::-;23285:2;23280:3;23276:12;23269:19;;23074:220;;;:::o;23300:398::-;23459:3;23480:83;23561:1;23556:3;23480:83;:::i;:::-;23473:90;;23572:93;23661:3;23572:93;:::i;:::-;23690:1;23685:3;23681:11;23674:18;;23463:235;;;:::o;23704:366::-;23846:3;23867:67;23931:2;23926:3;23867:67;:::i;:::-;23860:74;;23943:93;24032:3;23943:93;:::i;:::-;24061:2;24056:3;24052:12;24045:19;;23850:220;;;:::o;24076:366::-;24218:3;24239:67;24303:2;24298:3;24239:67;:::i;:::-;24232:74;;24315:93;24404:3;24315:93;:::i;:::-;24433:2;24428:3;24424:12;24417:19;;24222:220;;;:::o;24448:366::-;24590:3;24611:67;24675:2;24670:3;24611:67;:::i;:::-;24604:74;;24687:93;24776:3;24687:93;:::i;:::-;24805:2;24800:3;24796:12;24789:19;;24594:220;;;:::o;24820:366::-;24962:3;24983:67;25047:2;25042:3;24983:67;:::i;:::-;24976:74;;25059:93;25148:3;25059:93;:::i;:::-;25177:2;25172:3;25168:12;25161:19;;24966:220;;;:::o;25192:366::-;25334:3;25355:67;25419:2;25414:3;25355:67;:::i;:::-;25348:74;;25431:93;25520:3;25431:93;:::i;:::-;25549:2;25544:3;25540:12;25533:19;;25338:220;;;:::o;25564:366::-;25706:3;25727:67;25791:2;25786:3;25727:67;:::i;:::-;25720:74;;25803:93;25892:3;25803:93;:::i;:::-;25921:2;25916:3;25912:12;25905:19;;25710:220;;;:::o;25936:108::-;26013:24;26031:5;26013:24;:::i;:::-;26008:3;26001:37;25991:53;;:::o;26050:118::-;26137:24;26155:5;26137:24;:::i;:::-;26132:3;26125:37;26115:53;;:::o;26174:256::-;26286:3;26301:75;26372:3;26363:6;26301:75;:::i;:::-;26401:2;26396:3;26392:12;26385:19;;26421:3;26414:10;;26290:140;;;;:::o;26436:397::-;26576:3;26591:75;26662:3;26653:6;26591:75;:::i;:::-;26691:2;26686:3;26682:12;26675:19;;26704:75;26775:3;26766:6;26704:75;:::i;:::-;26804:2;26799:3;26795:12;26788:19;;26824:3;26817:10;;26580:253;;;;;:::o;26839:589::-;27064:3;27086:95;27177:3;27168:6;27086:95;:::i;:::-;27079:102;;27198:95;27289:3;27280:6;27198:95;:::i;:::-;27191:102;;27310:92;27398:3;27389:6;27310:92;:::i;:::-;27303:99;;27419:3;27412:10;;27068:360;;;;;;:::o;27434:379::-;27618:3;27640:147;27783:3;27640:147;:::i;:::-;27633:154;;27804:3;27797:10;;27622:191;;;:::o;27819:222::-;27912:4;27950:2;27939:9;27935:18;27927:26;;27963:71;28031:1;28020:9;28016:17;28007:6;27963:71;:::i;:::-;27917:124;;;;:::o;28047:640::-;28242:4;28280:3;28269:9;28265:19;28257:27;;28294:71;28362:1;28351:9;28347:17;28338:6;28294:71;:::i;:::-;28375:72;28443:2;28432:9;28428:18;28419:6;28375:72;:::i;:::-;28457;28525:2;28514:9;28510:18;28501:6;28457:72;:::i;:::-;28576:9;28570:4;28566:20;28561:2;28550:9;28546:18;28539:48;28604:76;28675:4;28666:6;28604:76;:::i;:::-;28596:84;;28247:440;;;;;;;:::o;28693:373::-;28836:4;28874:2;28863:9;28859:18;28851:26;;28923:9;28917:4;28913:20;28909:1;28898:9;28894:17;28887:47;28951:108;29054:4;29045:6;28951:108;:::i;:::-;28943:116;;28841:225;;;;:::o;29072:210::-;29159:4;29197:2;29186:9;29182:18;29174:26;;29210:65;29272:1;29261:9;29257:17;29248:6;29210:65;:::i;:::-;29164:118;;;;:::o;29288:222::-;29381:4;29419:2;29408:9;29404:18;29396:26;;29432:71;29500:1;29489:9;29485:17;29476:6;29432:71;:::i;:::-;29386:124;;;;:::o;29516:270::-;29633:4;29671:2;29660:9;29656:18;29648:26;;29684:95;29776:1;29765:9;29761:17;29752:6;29684:95;:::i;:::-;29638:148;;;;:::o;29792:313::-;29905:4;29943:2;29932:9;29928:18;29920:26;;29992:9;29986:4;29982:20;29978:1;29967:9;29963:17;29956:47;30020:78;30093:4;30084:6;30020:78;:::i;:::-;30012:86;;29910:195;;;;:::o;30111:419::-;30277:4;30315:2;30304:9;30300:18;30292:26;;30364:9;30358:4;30354:20;30350:1;30339:9;30335:17;30328:47;30392:131;30518:4;30392:131;:::i;:::-;30384:139;;30282:248;;;:::o;30536:419::-;30702:4;30740:2;30729:9;30725:18;30717:26;;30789:9;30783:4;30779:20;30775:1;30764:9;30760:17;30753:47;30817:131;30943:4;30817:131;:::i;:::-;30809:139;;30707:248;;;:::o;30961:419::-;31127:4;31165:2;31154:9;31150:18;31142:26;;31214:9;31208:4;31204:20;31200:1;31189:9;31185:17;31178:47;31242:131;31368:4;31242:131;:::i;:::-;31234:139;;31132:248;;;:::o;31386:419::-;31552:4;31590:2;31579:9;31575:18;31567:26;;31639:9;31633:4;31629:20;31625:1;31614:9;31610:17;31603:47;31667:131;31793:4;31667:131;:::i;:::-;31659:139;;31557:248;;;:::o;31811:419::-;31977:4;32015:2;32004:9;32000:18;31992:26;;32064:9;32058:4;32054:20;32050:1;32039:9;32035:17;32028:47;32092:131;32218:4;32092:131;:::i;:::-;32084:139;;31982:248;;;:::o;32236:419::-;32402:4;32440:2;32429:9;32425:18;32417:26;;32489:9;32483:4;32479:20;32475:1;32464:9;32460:17;32453:47;32517:131;32643:4;32517:131;:::i;:::-;32509:139;;32407:248;;;:::o;32661:419::-;32827:4;32865:2;32854:9;32850:18;32842:26;;32914:9;32908:4;32904:20;32900:1;32889:9;32885:17;32878:47;32942:131;33068:4;32942:131;:::i;:::-;32934:139;;32832:248;;;:::o;33086:419::-;33252:4;33290:2;33279:9;33275:18;33267:26;;33339:9;33333:4;33329:20;33325:1;33314:9;33310:17;33303:47;33367:131;33493:4;33367:131;:::i;:::-;33359:139;;33257:248;;;:::o;33511:419::-;33677:4;33715:2;33704:9;33700:18;33692:26;;33764:9;33758:4;33754:20;33750:1;33739:9;33735:17;33728:47;33792:131;33918:4;33792:131;:::i;:::-;33784:139;;33682:248;;;:::o;33936:419::-;34102:4;34140:2;34129:9;34125:18;34117:26;;34189:9;34183:4;34179:20;34175:1;34164:9;34160:17;34153:47;34217:131;34343:4;34217:131;:::i;:::-;34209:139;;34107:248;;;:::o;34361:419::-;34527:4;34565:2;34554:9;34550:18;34542:26;;34614:9;34608:4;34604:20;34600:1;34589:9;34585:17;34578:47;34642:131;34768:4;34642:131;:::i;:::-;34634:139;;34532:248;;;:::o;34786:419::-;34952:4;34990:2;34979:9;34975:18;34967:26;;35039:9;35033:4;35029:20;35025:1;35014:9;35010:17;35003:47;35067:131;35193:4;35067:131;:::i;:::-;35059:139;;34957:248;;;:::o;35211:419::-;35377:4;35415:2;35404:9;35400:18;35392:26;;35464:9;35458:4;35454:20;35450:1;35439:9;35435:17;35428:47;35492:131;35618:4;35492:131;:::i;:::-;35484:139;;35382:248;;;:::o;35636:419::-;35802:4;35840:2;35829:9;35825:18;35817:26;;35889:9;35883:4;35879:20;35875:1;35864:9;35860:17;35853:47;35917:131;36043:4;35917:131;:::i;:::-;35909:139;;35807:248;;;:::o;36061:419::-;36227:4;36265:2;36254:9;36250:18;36242:26;;36314:9;36308:4;36304:20;36300:1;36289:9;36285:17;36278:47;36342:131;36468:4;36342:131;:::i;:::-;36334:139;;36232:248;;;:::o;36486:419::-;36652:4;36690:2;36679:9;36675:18;36667:26;;36739:9;36733:4;36729:20;36725:1;36714:9;36710:17;36703:47;36767:131;36893:4;36767:131;:::i;:::-;36759:139;;36657:248;;;:::o;36911:419::-;37077:4;37115:2;37104:9;37100:18;37092:26;;37164:9;37158:4;37154:20;37150:1;37139:9;37135:17;37128:47;37192:131;37318:4;37192:131;:::i;:::-;37184:139;;37082:248;;;:::o;37336:419::-;37502:4;37540:2;37529:9;37525:18;37517:26;;37589:9;37583:4;37579:20;37575:1;37564:9;37560:17;37553:47;37617:131;37743:4;37617:131;:::i;:::-;37609:139;;37507:248;;;:::o;37761:419::-;37927:4;37965:2;37954:9;37950:18;37942:26;;38014:9;38008:4;38004:20;38000:1;37989:9;37985:17;37978:47;38042:131;38168:4;38042:131;:::i;:::-;38034:139;;37932:248;;;:::o;38186:419::-;38352:4;38390:2;38379:9;38375:18;38367:26;;38439:9;38433:4;38429:20;38425:1;38414:9;38410:17;38403:47;38467:131;38593:4;38467:131;:::i;:::-;38459:139;;38357:248;;;:::o;38611:419::-;38777:4;38815:2;38804:9;38800:18;38792:26;;38864:9;38858:4;38854:20;38850:1;38839:9;38835:17;38828:47;38892:131;39018:4;38892:131;:::i;:::-;38884:139;;38782:248;;;:::o;39036:419::-;39202:4;39240:2;39229:9;39225:18;39217:26;;39289:9;39283:4;39279:20;39275:1;39264:9;39260:17;39253:47;39317:131;39443:4;39317:131;:::i;:::-;39309:139;;39207:248;;;:::o;39461:419::-;39627:4;39665:2;39654:9;39650:18;39642:26;;39714:9;39708:4;39704:20;39700:1;39689:9;39685:17;39678:47;39742:131;39868:4;39742:131;:::i;:::-;39734:139;;39632:248;;;:::o;39886:419::-;40052:4;40090:2;40079:9;40075:18;40067:26;;40139:9;40133:4;40129:20;40125:1;40114:9;40110:17;40103:47;40167:131;40293:4;40167:131;:::i;:::-;40159:139;;40057:248;;;:::o;40311:419::-;40477:4;40515:2;40504:9;40500:18;40492:26;;40564:9;40558:4;40554:20;40550:1;40539:9;40535:17;40528:47;40592:131;40718:4;40592:131;:::i;:::-;40584:139;;40482:248;;;:::o;40736:419::-;40902:4;40940:2;40929:9;40925:18;40917:26;;40989:9;40983:4;40979:20;40975:1;40964:9;40960:17;40953:47;41017:131;41143:4;41017:131;:::i;:::-;41009:139;;40907:248;;;:::o;41161:419::-;41327:4;41365:2;41354:9;41350:18;41342:26;;41414:9;41408:4;41404:20;41400:1;41389:9;41385:17;41378:47;41442:131;41568:4;41442:131;:::i;:::-;41434:139;;41332:248;;;:::o;41586:419::-;41752:4;41790:2;41779:9;41775:18;41767:26;;41839:9;41833:4;41829:20;41825:1;41814:9;41810:17;41803:47;41867:131;41993:4;41867:131;:::i;:::-;41859:139;;41757:248;;;:::o;42011:419::-;42177:4;42215:2;42204:9;42200:18;42192:26;;42264:9;42258:4;42254:20;42250:1;42239:9;42235:17;42228:47;42292:131;42418:4;42292:131;:::i;:::-;42284:139;;42182:248;;;:::o;42436:419::-;42602:4;42640:2;42629:9;42625:18;42617:26;;42689:9;42683:4;42679:20;42675:1;42664:9;42660:17;42653:47;42717:131;42843:4;42717:131;:::i;:::-;42709:139;;42607:248;;;:::o;42861:419::-;43027:4;43065:2;43054:9;43050:18;43042:26;;43114:9;43108:4;43104:20;43100:1;43089:9;43085:17;43078:47;43142:131;43268:4;43142:131;:::i;:::-;43134:139;;43032:248;;;:::o;43286:419::-;43452:4;43490:2;43479:9;43475:18;43467:26;;43539:9;43533:4;43529:20;43525:1;43514:9;43510:17;43503:47;43567:131;43693:4;43567:131;:::i;:::-;43559:139;;43457:248;;;:::o;43711:419::-;43877:4;43915:2;43904:9;43900:18;43892:26;;43964:9;43958:4;43954:20;43950:1;43939:9;43935:17;43928:47;43992:131;44118:4;43992:131;:::i;:::-;43984:139;;43882:248;;;:::o;44136:222::-;44229:4;44267:2;44256:9;44252:18;44244:26;;44280:71;44348:1;44337:9;44333:17;44324:6;44280:71;:::i;:::-;44234:124;;;;:::o;44364:129::-;44398:6;44425:20;;:::i;:::-;44415:30;;44454:33;44482:4;44474:6;44454:33;:::i;:::-;44405:88;;;:::o;44499:75::-;44532:6;44565:2;44559:9;44549:19;;44539:35;:::o;44580:311::-;44657:4;44747:18;44739:6;44736:30;44733:2;;;44769:18;;:::i;:::-;44733:2;44819:4;44811:6;44807:17;44799:25;;44879:4;44873;44869:15;44861:23;;44662:229;;;:::o;44897:307::-;44958:4;45048:18;45040:6;45037:30;45034:2;;;45070:18;;:::i;:::-;45034:2;45108:29;45130:6;45108:29;:::i;:::-;45100:37;;45192:4;45186;45182:15;45174:23;;44963:241;;;:::o;45210:308::-;45272:4;45362:18;45354:6;45351:30;45348:2;;;45384:18;;:::i;:::-;45348:2;45422:29;45444:6;45422:29;:::i;:::-;45414:37;;45506:4;45500;45496:15;45488:23;;45277:241;;;:::o;45524:132::-;45591:4;45614:3;45606:11;;45644:4;45639:3;45635:14;45627:22;;45596:60;;;:::o;45662:141::-;45711:4;45734:3;45726:11;;45757:3;45754:1;45747:14;45791:4;45788:1;45778:18;45770:26;;45716:87;;;:::o;45809:114::-;45876:6;45910:5;45904:12;45894:22;;45883:40;;;:::o;45929:98::-;45980:6;46014:5;46008:12;45998:22;;45987:40;;;:::o;46033:99::-;46085:6;46119:5;46113:12;46103:22;;46092:40;;;:::o;46138:113::-;46208:4;46240;46235:3;46231:14;46223:22;;46213:38;;;:::o;46257:184::-;46356:11;46390:6;46385:3;46378:19;46430:4;46425:3;46421:14;46406:29;;46368:73;;;;:::o;46447:168::-;46530:11;46564:6;46559:3;46552:19;46604:4;46599:3;46595:14;46580:29;;46542:73;;;;:::o;46621:147::-;46722:11;46759:3;46744:18;;46734:34;;;;:::o;46774:169::-;46858:11;46892:6;46887:3;46880:19;46932:4;46927:3;46923:14;46908:29;;46870:73;;;;:::o;46949:148::-;47051:11;47088:3;47073:18;;47063:34;;;;:::o;47103:305::-;47143:3;47162:20;47180:1;47162:20;:::i;:::-;47157:25;;47196:20;47214:1;47196:20;:::i;:::-;47191:25;;47350:1;47282:66;47278:74;47275:1;47272:81;47269:2;;;47356:18;;:::i;:::-;47269:2;47400:1;47397;47393:9;47386:16;;47147:261;;;;:::o;47414:185::-;47454:1;47471:20;47489:1;47471:20;:::i;:::-;47466:25;;47505:20;47523:1;47505:20;:::i;:::-;47500:25;;47544:1;47534:2;;47549:18;;:::i;:::-;47534:2;47591:1;47588;47584:9;47579:14;;47456:143;;;;:::o;47605:348::-;47645:7;47668:20;47686:1;47668:20;:::i;:::-;47663:25;;47702:20;47720:1;47702:20;:::i;:::-;47697:25;;47890:1;47822:66;47818:74;47815:1;47812:81;47807:1;47800:9;47793:17;47789:105;47786:2;;;47897:18;;:::i;:::-;47786:2;47945:1;47942;47938:9;47927:20;;47653:300;;;;:::o;47959:191::-;47999:4;48019:20;48037:1;48019:20;:::i;:::-;48014:25;;48053:20;48071:1;48053:20;:::i;:::-;48048:25;;48092:1;48089;48086:8;48083:2;;;48097:18;;:::i;:::-;48083:2;48142:1;48139;48135:9;48127:17;;48004:146;;;;:::o;48156:96::-;48193:7;48222:24;48240:5;48222:24;:::i;:::-;48211:35;;48201:51;;;:::o;48258:90::-;48292:7;48335:5;48328:13;48321:21;48310:32;;48300:48;;;:::o;48354:77::-;48391:7;48420:5;48409:16;;48399:32;;;:::o;48437:149::-;48473:7;48513:66;48506:5;48502:78;48491:89;;48481:105;;;:::o;48592:126::-;48629:7;48669:42;48662:5;48658:54;48647:65;;48637:81;;;:::o;48724:77::-;48761:7;48790:5;48779:16;;48769:32;;;:::o;48807:174::-;48881:9;48914:61;48969:5;48914:61;:::i;:::-;48901:74;;48891:90;;;:::o;48987:137::-;49061:9;49094:24;49112:5;49094:24;:::i;:::-;49081:37;;49071:53;;;:::o;49130:154::-;49214:6;49209:3;49204;49191:30;49276:1;49267:6;49262:3;49258:16;49251:27;49181:103;;;:::o;49290:307::-;49358:1;49368:113;49382:6;49379:1;49376:13;49368:113;;;49467:1;49462:3;49458:11;49452:18;49448:1;49443:3;49439:11;49432:39;49404:2;49401:1;49397:10;49392:15;;49368:113;;;49499:6;49496:1;49493:13;49490:2;;;49579:1;49570:6;49565:3;49561:16;49554:27;49490:2;49339:258;;;;:::o;49603:320::-;49647:6;49684:1;49678:4;49674:12;49664:22;;49731:1;49725:4;49721:12;49752:18;49742:2;;49808:4;49800:6;49796:17;49786:27;;49742:2;49870;49862:6;49859:14;49839:18;49836:38;49833:2;;;49889:18;;:::i;:::-;49833:2;49654:269;;;;:::o;49929:281::-;50012:27;50034:4;50012:27;:::i;:::-;50004:6;50000:40;50142:6;50130:10;50127:22;50106:18;50094:10;50091:34;50088:62;50085:2;;;50153:18;;:::i;:::-;50085:2;50193:10;50189:2;50182:22;49972:238;;;:::o;50216:233::-;50255:3;50278:24;50296:5;50278:24;:::i;:::-;50269:33;;50324:66;50317:5;50314:77;50311:2;;;50394:18;;:::i;:::-;50311:2;50441:1;50434:5;50430:13;50423:20;;50259:190;;;:::o;50455:100::-;50494:7;50523:26;50543:5;50523:26;:::i;:::-;50512:37;;50502:53;;;:::o;50561:79::-;50600:7;50629:5;50618:16;;50608:32;;;:::o;50646:94::-;50685:7;50714:20;50728:5;50714:20;:::i;:::-;50703:31;;50693:47;;;:::o;50746:176::-;50778:1;50795:20;50813:1;50795:20;:::i;:::-;50790:25;;50829:20;50847:1;50829:20;:::i;:::-;50824:25;;50868:1;50858:2;;50873:18;;:::i;:::-;50858:2;50914:1;50911;50907:9;50902:14;;50780:142;;;;:::o;50928:180::-;50976:77;50973:1;50966:88;51073:4;51070:1;51063:15;51097:4;51094:1;51087:15;51114:180;51162:77;51159:1;51152:88;51259:4;51256:1;51249:15;51283:4;51280:1;51273:15;51300:180;51348:77;51345:1;51338:88;51445:4;51442:1;51435:15;51469:4;51466:1;51459:15;51486:180;51534:77;51531:1;51524:88;51631:4;51628:1;51621:15;51655:4;51652:1;51645:15;51672:102;51713:6;51764:2;51760:7;51755:2;51748:5;51744:14;51740:28;51730:38;;51720:54;;;:::o;51780:94::-;51813:8;51861:5;51857:2;51853:14;51832:35;;51822:52;;;:::o;51880:169::-;52020:21;52016:1;52008:6;52004:14;51997:45;51986:63;:::o;52055:166::-;52195:18;52191:1;52183:6;52179:14;52172:42;52161:60;:::o;52227:230::-;52367:34;52363:1;52355:6;52351:14;52344:58;52436:13;52431:2;52423:6;52419:15;52412:38;52333:124;:::o;52463:237::-;52603:34;52599:1;52591:6;52587:14;52580:58;52672:20;52667:2;52659:6;52655:15;52648:45;52569:131;:::o;52706:225::-;52846:34;52842:1;52834:6;52830:14;52823:58;52915:8;52910:2;52902:6;52898:15;52891:33;52812:119;:::o;52937:159::-;53077:11;53073:1;53065:6;53061:14;53054:35;53043:53;:::o;53102:178::-;53242:30;53238:1;53230:6;53226:14;53219:54;53208:72;:::o;53286:160::-;53426:12;53422:1;53414:6;53410:14;53403:36;53392:54;:::o;53452:223::-;53592:34;53588:1;53580:6;53576:14;53569:58;53661:6;53656:2;53648:6;53644:15;53637:31;53558:117;:::o;53681:175::-;53821:27;53817:1;53809:6;53805:14;53798:51;53787:69;:::o;53862:181::-;54002:33;53998:1;53990:6;53986:14;53979:57;53968:75;:::o;54049:231::-;54189:34;54185:1;54177:6;54173:14;54166:58;54258:14;54253:2;54245:6;54241:15;54234:39;54155:125;:::o;54286:243::-;54426:34;54422:1;54414:6;54410:14;54403:58;54495:26;54490:2;54482:6;54478:15;54471:51;54392:137;:::o;54535:229::-;54675:34;54671:1;54663:6;54659:14;54652:58;54744:12;54739:2;54731:6;54727:15;54720:37;54641:123;:::o;54770:228::-;54910:34;54906:1;54898:6;54894:14;54887:58;54979:11;54974:2;54966:6;54962:15;54955:36;54876:122;:::o;55004:165::-;55144:17;55140:1;55132:6;55128:14;55121:41;55110:59;:::o;55175:182::-;55315:34;55311:1;55303:6;55299:14;55292:58;55281:76;:::o;55363:231::-;55503:34;55499:1;55491:6;55487:14;55480:58;55572:14;55567:2;55559:6;55555:15;55548:39;55469:125;:::o;55600:182::-;55740:34;55736:1;55728:6;55724:14;55717:58;55706:76;:::o;55788:223::-;55928:34;55924:1;55916:6;55912:14;55905:58;55997:6;55992:2;55984:6;55980:15;55973:31;55894:117;:::o;56017:168::-;56157:20;56153:1;56145:6;56141:14;56134:44;56123:62;:::o;56191:172::-;56331:24;56327:1;56319:6;56315:14;56308:48;56297:66;:::o;56369:228::-;56509:34;56505:1;56497:6;56493:14;56486:58;56578:11;56573:2;56565:6;56561:15;56554:36;56475:122;:::o;56603:234::-;56743:34;56739:1;56731:6;56727:14;56720:58;56812:17;56807:2;56799:6;56795:15;56788:42;56709:128;:::o;56843:173::-;56983:25;56979:1;56971:6;56967:14;56960:49;56949:67;:::o;57022:220::-;57162:34;57158:1;57150:6;57146:14;57139:58;57231:3;57226:2;57218:6;57214:15;57207:28;57128:114;:::o;57248:164::-;57388:16;57384:1;57376:6;57372:14;57365:40;57354:58;:::o;57418:114::-;57524:8;:::o;57538:236::-;57678:34;57674:1;57666:6;57662:14;57655:58;57747:19;57742:2;57734:6;57730:15;57723:44;57644:130;:::o;57780:231::-;57920:34;57916:1;57908:6;57904:14;57897:58;57989:14;57984:2;57976:6;57972:15;57965:39;57886:125;:::o;58017:163::-;58157:15;58153:1;58145:6;58141:14;58134:39;58123:57;:::o;58186:182::-;58326:34;58322:1;58314:6;58310:14;58303:58;58292:76;:::o;58374:181::-;58514:33;58510:1;58502:6;58498:14;58491:57;58480:75;:::o;58561:165::-;58701:17;58697:1;58689:6;58685:14;58678:41;58667:59;:::o;58732:122::-;58805:24;58823:5;58805:24;:::i;:::-;58798:5;58795:35;58785:2;;58844:1;58841;58834:12;58785:2;58775:79;:::o;58860:116::-;58930:21;58945:5;58930:21;:::i;:::-;58923:5;58920:32;58910:2;;58966:1;58963;58956:12;58910:2;58900:76;:::o;58982:122::-;59055:24;59073:5;59055:24;:::i;:::-;59048:5;59045:35;59035:2;;59094:1;59091;59084:12;59035:2;59025:79;:::o;59110:120::-;59182:23;59199:5;59182:23;:::i;:::-;59175:5;59172:34;59162:2;;59220:1;59217;59210:12;59162:2;59152:78;:::o;59236:122::-;59309:24;59327:5;59309:24;:::i;:::-;59302:5;59299:35;59289:2;;59348:1;59345;59338:12;59289:2;59279:79;:::o

Swarm Source

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