ETH Price: $3,489.83 (+0.05%)
Gas: 2 Gwei

Token

OshareNFT (OSHARE)
 

Overview

Max Total Supply

100 OSHARE

Holders

61

Market

Volume (24H)

N/A

Min Price (24H)

N/A

Max Price (24H)

N/A
Balance
2 OSHARE
0xc8467e8e6cf6380d99c644d3c9e183a537e90dc1
Loading...
Loading
Loading...
Loading
Loading...
Loading

Click here to update the token information / general information
# Exchange Pair Price  24H Volume % Volume

Contract Source Code Verified (Exact Match)

Contract Name:
OshareNFT

Compiler Version
v0.8.7+commit.e28d00a7

Optimization Enabled:
No with 200 runs

Other Settings:
default evmVersion, MIT license

Contract Source Code (Solidity)

/**
 *Submitted for verification at Etherscan.io on 2022-03-12
*/

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


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

pragma solidity ^0.8.0;

/**
 * @dev These functions deal with verification of Merkle Trees proofs.
 *
 * The proofs can be generated using the JavaScript library
 * https://github.com/miguelmota/merkletreejs[merkletreejs].
 * Note: the hashing algorithm should be keccak256 and pair sorting should be enabled.
 *
 * See `test/utils/cryptography/MerkleProof.test.js` for some examples.
 */
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 = _efficientHash(computedHash, proofElement);
            } else {
                // Hash(current element of the proof + current computed hash)
                computedHash = _efficientHash(proofElement, computedHash);
            }
        }
        return computedHash;
    }

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

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


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

pragma solidity ^0.8.0;

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

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

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

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

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

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


// OpenZeppelin Contracts (last updated v4.5.0) (utils/cryptography/ECDSA.sol)

pragma solidity ^0.8.0;


/**
 * @dev Elliptic Curve Digital Signature Algorithm (ECDSA) operations.
 *
 * These functions can be used to verify that a message was signed by the holder
 * of the private keys of a given address.
 */
library ECDSA {
    enum RecoverError {
        NoError,
        InvalidSignature,
        InvalidSignatureLength,
        InvalidSignatureS,
        InvalidSignatureV
    }

    function _throwError(RecoverError error) private pure {
        if (error == RecoverError.NoError) {
            return; // no error: do nothing
        } else if (error == RecoverError.InvalidSignature) {
            revert("ECDSA: invalid signature");
        } else if (error == RecoverError.InvalidSignatureLength) {
            revert("ECDSA: invalid signature length");
        } else if (error == RecoverError.InvalidSignatureS) {
            revert("ECDSA: invalid signature 's' value");
        } else if (error == RecoverError.InvalidSignatureV) {
            revert("ECDSA: invalid signature 'v' value");
        }
    }

    /**
     * @dev Returns the address that signed a hashed message (`hash`) with
     * `signature` or error string. This address can then be used for verification purposes.
     *
     * The `ecrecover` EVM opcode allows for malleable (non-unique) signatures:
     * this function rejects them by requiring the `s` value to be in the lower
     * half order, and the `v` value to be either 27 or 28.
     *
     * IMPORTANT: `hash` _must_ be the result of a hash operation for the
     * verification to be secure: it is possible to craft signatures that
     * recover to arbitrary addresses for non-hashed data. A safe way to ensure
     * this is by receiving a hash of the original message (which may otherwise
     * be too long), and then calling {toEthSignedMessageHash} on it.
     *
     * Documentation for signature generation:
     * - with https://web3js.readthedocs.io/en/v1.3.4/web3-eth-accounts.html#sign[Web3.js]
     * - with https://docs.ethers.io/v5/api/signer/#Signer-signMessage[ethers]
     *
     * _Available since v4.3._
     */
    function tryRecover(bytes32 hash, bytes memory signature) internal pure returns (address, RecoverError) {
        // Check the signature length
        // - case 65: r,s,v signature (standard)
        // - case 64: r,vs signature (cf https://eips.ethereum.org/EIPS/eip-2098) _Available since v4.1._
        if (signature.length == 65) {
            bytes32 r;
            bytes32 s;
            uint8 v;
            // ecrecover takes the signature parameters, and the only way to get them
            // currently is to use assembly.
            assembly {
                r := mload(add(signature, 0x20))
                s := mload(add(signature, 0x40))
                v := byte(0, mload(add(signature, 0x60)))
            }
            return tryRecover(hash, v, r, s);
        } else if (signature.length == 64) {
            bytes32 r;
            bytes32 vs;
            // ecrecover takes the signature parameters, and the only way to get them
            // currently is to use assembly.
            assembly {
                r := mload(add(signature, 0x20))
                vs := mload(add(signature, 0x40))
            }
            return tryRecover(hash, r, vs);
        } else {
            return (address(0), RecoverError.InvalidSignatureLength);
        }
    }

    /**
     * @dev Returns the address that signed a hashed message (`hash`) with
     * `signature`. This address can then be used for verification purposes.
     *
     * The `ecrecover` EVM opcode allows for malleable (non-unique) signatures:
     * this function rejects them by requiring the `s` value to be in the lower
     * half order, and the `v` value to be either 27 or 28.
     *
     * IMPORTANT: `hash` _must_ be the result of a hash operation for the
     * verification to be secure: it is possible to craft signatures that
     * recover to arbitrary addresses for non-hashed data. A safe way to ensure
     * this is by receiving a hash of the original message (which may otherwise
     * be too long), and then calling {toEthSignedMessageHash} on it.
     */
    function recover(bytes32 hash, bytes memory signature) internal pure returns (address) {
        (address recovered, RecoverError error) = tryRecover(hash, signature);
        _throwError(error);
        return recovered;
    }

    /**
     * @dev Overload of {ECDSA-tryRecover} that receives the `r` and `vs` short-signature fields separately.
     *
     * See https://eips.ethereum.org/EIPS/eip-2098[EIP-2098 short signatures]
     *
     * _Available since v4.3._
     */
    function tryRecover(
        bytes32 hash,
        bytes32 r,
        bytes32 vs
    ) internal pure returns (address, RecoverError) {
        bytes32 s = vs & bytes32(0x7fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff);
        uint8 v = uint8((uint256(vs) >> 255) + 27);
        return tryRecover(hash, v, r, s);
    }

    /**
     * @dev Overload of {ECDSA-recover} that receives the `r and `vs` short-signature fields separately.
     *
     * _Available since v4.2._
     */
    function recover(
        bytes32 hash,
        bytes32 r,
        bytes32 vs
    ) internal pure returns (address) {
        (address recovered, RecoverError error) = tryRecover(hash, r, vs);
        _throwError(error);
        return recovered;
    }

    /**
     * @dev Overload of {ECDSA-tryRecover} that receives the `v`,
     * `r` and `s` signature fields separately.
     *
     * _Available since v4.3._
     */
    function tryRecover(
        bytes32 hash,
        uint8 v,
        bytes32 r,
        bytes32 s
    ) internal pure returns (address, RecoverError) {
        // EIP-2 still allows signature malleability for ecrecover(). Remove this possibility and make the signature
        // unique. Appendix F in the Ethereum Yellow paper (https://ethereum.github.io/yellowpaper/paper.pdf), defines
        // the valid range for s in (301): 0 < s < secp256k1n ÷ 2 + 1, and for v in (302): v ∈ {27, 28}. Most
        // signatures from current libraries generate a unique signature with an s-value in the lower half order.
        //
        // If your library generates malleable signatures, such as s-values in the upper range, calculate a new s-value
        // with 0xFFFFFFFFFFFFFFFFFFFFFFFFFFFFFFFEBAAEDCE6AF48A03BBFD25E8CD0364141 - s1 and flip v from 27 to 28 or
        // vice versa. If your library also generates signatures with 0/1 for v instead 27/28, add 27 to v to accept
        // these malleable signatures as well.
        if (uint256(s) > 0x7FFFFFFFFFFFFFFFFFFFFFFFFFFFFFFF5D576E7357A4501DDFE92F46681B20A0) {
            return (address(0), RecoverError.InvalidSignatureS);
        }
        if (v != 27 && v != 28) {
            return (address(0), RecoverError.InvalidSignatureV);
        }

        // If the signature is valid (and not malleable), return the signer address
        address signer = ecrecover(hash, v, r, s);
        if (signer == address(0)) {
            return (address(0), RecoverError.InvalidSignature);
        }

        return (signer, RecoverError.NoError);
    }

    /**
     * @dev Overload of {ECDSA-recover} that receives the `v`,
     * `r` and `s` signature fields separately.
     */
    function recover(
        bytes32 hash,
        uint8 v,
        bytes32 r,
        bytes32 s
    ) internal pure returns (address) {
        (address recovered, RecoverError error) = tryRecover(hash, v, r, s);
        _throwError(error);
        return recovered;
    }

    /**
     * @dev Returns an Ethereum Signed Message, created from a `hash`. This
     * produces hash corresponding to the one signed with the
     * https://eth.wiki/json-rpc/API#eth_sign[`eth_sign`]
     * JSON-RPC method as part of EIP-191.
     *
     * See {recover}.
     */
    function toEthSignedMessageHash(bytes32 hash) internal pure returns (bytes32) {
        // 32 is the length in bytes of hash,
        // enforced by the type signature above
        return keccak256(abi.encodePacked("\x19Ethereum Signed Message:\n32", hash));
    }

    /**
     * @dev Returns an Ethereum Signed Message, created from `s`. This
     * produces hash corresponding to the one signed with the
     * https://eth.wiki/json-rpc/API#eth_sign[`eth_sign`]
     * JSON-RPC method as part of EIP-191.
     *
     * See {recover}.
     */
    function toEthSignedMessageHash(bytes memory s) internal pure returns (bytes32) {
        return keccak256(abi.encodePacked("\x19Ethereum Signed Message:\n", Strings.toString(s.length), s));
    }

    /**
     * @dev Returns an Ethereum Signed Typed Data, created from a
     * `domainSeparator` and a `structHash`. This produces hash corresponding
     * to the one signed with the
     * https://eips.ethereum.org/EIPS/eip-712[`eth_signTypedData`]
     * JSON-RPC method as part of EIP-712.
     *
     * See {recover}.
     */
    function toTypedDataHash(bytes32 domainSeparator, bytes32 structHash) internal pure returns (bytes32) {
        return keccak256(abi.encodePacked("\x19\x01", domainSeparator, structHash));
    }
}

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


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

pragma solidity ^0.8.0;

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

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

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


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

pragma solidity ^0.8.0;


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

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

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

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

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

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

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

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

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


// OpenZeppelin Contracts (last updated v4.5.0) (utils/Address.sol)

pragma solidity ^0.8.1;

/**
 * @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
     * ====
     *
     * [IMPORTANT]
     * ====
     * You shouldn't rely on `isContract` to protect against flash loan attacks!
     *
     * Preventing calls from contracts is highly discouraged. It breaks composability, breaks support for smart wallets
     * like Gnosis Safe, and does not provide security since it can be circumvented by calling from a contract
     * constructor.
     * ====
     */
    function isContract(address account) internal view returns (bool) {
        // This method relies on extcodesize/address.code.length, which returns 0
        // for contracts in construction, since the code is only stored at the end
        // of the constructor execution.

        return account.code.length > 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: @openzeppelin/contracts/token/ERC721/IERC721Receiver.sol


// 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: @openzeppelin/contracts/utils/introspection/IERC165.sol


// OpenZeppelin Contracts v4.4.1 (utils/introspection/IERC165.sol)

pragma solidity ^0.8.0;

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

// File: @openzeppelin/contracts/utils/introspection/ERC165.sol


// OpenZeppelin Contracts v4.4.1 (utils/introspection/ERC165.sol)

pragma solidity ^0.8.0;


/**
 * @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: @openzeppelin/contracts/token/ERC721/IERC721.sol


// OpenZeppelin Contracts v4.4.1 (token/ERC721/IERC721.sol)

pragma solidity ^0.8.0;


/**
 * @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: @openzeppelin/contracts/token/ERC721/extensions/IERC721Enumerable.sol


// OpenZeppelin Contracts (last updated v4.5.0) (token/ERC721/extensions/IERC721Enumerable.sol)

pragma solidity ^0.8.0;


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

    /**
     * @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: @openzeppelin/contracts/token/ERC721/extensions/IERC721Metadata.sol


// OpenZeppelin Contracts v4.4.1 (token/ERC721/extensions/IERC721Metadata.sol)

pragma solidity ^0.8.0;


/**
 * @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: @openzeppelin/contracts/token/ERC721/ERC721.sol


// OpenZeppelin Contracts (last updated v4.5.0) (token/ERC721/ERC721.sol)

pragma solidity ^0.8.0;








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

        _afterTokenTransfer(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);

        _afterTokenTransfer(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 from incorrect owner");
        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);

        _afterTokenTransfer(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 {}

    /**
     * @dev Hook that is called after any transfer of tokens. This includes
     * minting and burning.
     *
     * Calling conditions:
     *
     * - when `from` and `to` are both non-zero.
     * - `from` and `to` are never both zero.
     *
     * To learn more about hooks, head to xref:ROOT:extending-contracts.adoc#using-hooks[Using Hooks].
     */
    function _afterTokenTransfer(
        address from,
        address to,
        uint256 tokenId
    ) internal virtual {}
}

// File: @openzeppelin/contracts/token/ERC721/extensions/ERC721Enumerable.sol


// OpenZeppelin Contracts v4.4.1 (token/ERC721/extensions/ERC721Enumerable.sol)

pragma solidity ^0.8.0;



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


// Creator: Chiru Labs

pragma solidity ^0.8.4;









error ApprovalCallerNotOwnerNorApproved();
error ApprovalQueryForNonexistentToken();
error ApproveToCaller();
error ApprovalToCurrentOwner();
error BalanceQueryForZeroAddress();
error MintedQueryForZeroAddress();
error BurnedQueryForZeroAddress();
error AuxQueryForZeroAddress();
error MintToZeroAddress();
error MintZeroQuantity();
error OwnerIndexOutOfBounds();
error OwnerQueryForNonexistentToken();
error TokenIndexOutOfBounds();
error TransferCallerNotOwnerNorApproved();
error TransferFromIncorrectOwner();
error TransferToNonERC721ReceiverImplementer();
error TransferToZeroAddress();
error URIQueryForNonexistentToken();

/**
 * @dev Implementation of https://eips.ethereum.org/EIPS/eip-721[ERC721] Non-Fungible Token Standard, including
 * the Metadata extension. Built to optimize for lower gas during batch mints.
 *
 * Assumes serials are sequentially minted starting at _startTokenId() (defaults to 0, e.g. 0, 1, 2, 3..).
 *
 * Assumes that an owner cannot have more than 2**64 - 1 (max value of uint64) of supply.
 *
 * Assumes that the maximum token id cannot exceed 2**256 - 1 (max value of uint256).
 */
contract ERC721A is Context, ERC165, IERC721, IERC721Metadata {
    using Address for address;
    using Strings for uint256;

    // Compiler will pack this into a single 256bit word.
    struct TokenOwnership {
        // The address of the owner.
        address addr;
        // Keeps track of the start time of ownership with minimal overhead for tokenomics.
        uint64 startTimestamp;
        // Whether the token has been burned.
        bool burned;
    }

    // Compiler will pack this into a single 256bit word.
    struct AddressData {
        // Realistically, 2**64-1 is more than enough.
        uint64 balance;
        // Keeps track of mint count with minimal overhead for tokenomics.
        uint64 numberMinted;
        // Keeps track of burn count with minimal overhead for tokenomics.
        uint64 numberBurned;
        // For miscellaneous variable(s) pertaining to the address
        // (e.g. number of whitelist mint slots used).
        // If there are multiple variables, please pack them into a uint64.
        uint64 aux;
    }

    // The tokenId of the next token to be minted.
    uint256 internal _currentIndex;

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

    // Token name
    string private _name;

    // Token symbol
    string private _symbol;

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

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

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

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

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

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

    /**
     * @dev See {IERC721Enumerable-totalSupply}.
     * @dev Burned tokens are calculated here, use _totalMinted() if you want to count just minted tokens.
     */
    function totalSupply() public view returns (uint256) {
        // Counter underflow is impossible as _burnCounter cannot be incremented
        // more than _currentIndex - _startTokenId() times
        unchecked {
            return _currentIndex - _burnCounter - _startTokenId();
        }
    }

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

    /**
     * @dev 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 override returns (uint256) {
        if (owner == address(0)) revert BalanceQueryForZeroAddress();
        return uint256(_addressData[owner].balance);
    }

    /**
     * Returns the number of tokens minted by `owner`.
     */
    function _numberMinted(address owner) internal view returns (uint256) {
        if (owner == address(0)) revert MintedQueryForZeroAddress();
        return uint256(_addressData[owner].numberMinted);
    }

    /**
     * Returns the number of tokens burned by or on behalf of `owner`.
     */
    function _numberBurned(address owner) internal view returns (uint256) {
        if (owner == address(0)) revert BurnedQueryForZeroAddress();
        return uint256(_addressData[owner].numberBurned);
    }

    /**
     * Returns the auxillary data for `owner`. (e.g. number of whitelist mint slots used).
     */
    function _getAux(address owner) internal view returns (uint64) {
        if (owner == address(0)) revert AuxQueryForZeroAddress();
        return _addressData[owner].aux;
    }

    /**
     * Sets the auxillary data for `owner`. (e.g. number of whitelist mint slots used).
     * If there are multiple variables, please pack them into a uint64.
     */
    function _setAux(address owner, uint64 aux) internal {
        if (owner == address(0)) revert AuxQueryForZeroAddress();
        _addressData[owner].aux = aux;
    }

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

        unchecked {
            if (_startTokenId() <= curr && curr < _currentIndex) {
                TokenOwnership memory ownership = _ownerships[curr];
                if (!ownership.burned) {
                    if (ownership.addr != address(0)) {
                        return ownership;
                    }
                    // Invariant:
                    // There will always be an ownership that has an address and is not burned
                    // before an ownership that does not have an address and is not burned.
                    // Hence, curr will not underflow.
                    while (true) {
                        curr--;
                        ownership = _ownerships[curr];
                        if (ownership.addr != address(0)) {
                            return ownership;
                        }
                    }
                }
            }
        }
        revert OwnerQueryForNonexistentToken();
    }

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

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

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

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

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

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

    /**
     * @dev See {IERC721-approve}.
     */
    function approve(address to, uint256 tokenId) public override {
        address owner = ERC721A.ownerOf(tokenId);
        if (to == owner) revert ApprovalToCurrentOwner();

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

        _approve(to, tokenId, owner);
    }

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

        return _tokenApprovals[tokenId];
    }

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

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

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

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

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

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

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

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

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

    /**
     * @dev Mints `quantity` tokens and transfers them to `to`.
     *
     * Requirements:
     *
     * - `to` cannot be the zero address.
     * - `quantity` must be greater than 0.
     *
     * Emits a {Transfer} event.
     */
    function _mint(
        address to,
        uint256 quantity,
        bytes memory _data,
        bool safe
    ) internal {
        uint256 startTokenId = _currentIndex;
        if (to == address(0)) revert MintToZeroAddress();
        if (quantity == 0) revert MintZeroQuantity();

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

        // Overflows are incredibly unrealistic.
        // balance or numberMinted overflow if current value of either + quantity > 1.8e19 (2**64) - 1
        // updatedIndex overflows if _currentIndex + quantity > 1.2e77 (2**256) - 1
        unchecked {
            _addressData[to].balance += uint64(quantity);
            _addressData[to].numberMinted += uint64(quantity);

            _ownerships[startTokenId].addr = to;
            _ownerships[startTokenId].startTimestamp = uint64(block.timestamp);

            uint256 updatedIndex = startTokenId;
            uint256 end = updatedIndex + quantity;

            if (safe && to.isContract()) {
                do {
                    emit Transfer(address(0), to, updatedIndex);
                    if (!_checkContractOnERC721Received(address(0), to, updatedIndex++, _data)) {
                        revert TransferToNonERC721ReceiverImplementer();
                    }
                } while (updatedIndex != end);
                // Reentrancy protection
                if (_currentIndex != startTokenId) revert();
            } else {
                do {
                    emit Transfer(address(0), to, updatedIndex++);
                } while (updatedIndex != end);
            }
            _currentIndex = updatedIndex;
        }
        _afterTokenTransfers(address(0), to, startTokenId, quantity);
    }

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

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

        if (!isApprovedOrOwner) revert TransferCallerNotOwnerNorApproved();
        if (prevOwnership.addr != from) revert TransferFromIncorrectOwner();
        if (to == address(0)) revert TransferToZeroAddress();

        _beforeTokenTransfers(from, to, tokenId, 1);

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

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

            _ownerships[tokenId].addr = to;
            _ownerships[tokenId].startTimestamp = uint64(block.timestamp);

            // If the ownership slot of tokenId+1 is not explicitly set, that means the transfer initiator owns it.
            // Set the slot of tokenId+1 explicitly in storage to maintain correctness for ownerOf(tokenId+1) calls.
            uint256 nextTokenId = tokenId + 1;
            if (_ownerships[nextTokenId].addr == address(0)) {
                // This will suffice for checking _exists(nextTokenId),
                // as a burned slot cannot contain the zero address.
                if (nextTokenId < _currentIndex) {
                    _ownerships[nextTokenId].addr = prevOwnership.addr;
                    _ownerships[nextTokenId].startTimestamp = prevOwnership.startTimestamp;
                }
            }
        }

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

    /**
     * @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 {
        TokenOwnership memory prevOwnership = ownershipOf(tokenId);

        _beforeTokenTransfers(prevOwnership.addr, address(0), tokenId, 1);

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

        // Underflow of the sender's balance is impossible because we check for
        // ownership above and the recipient's balance can't realistically overflow.
        // Counter overflow is incredibly unrealistic as tokenId would have to be 2**256.
        unchecked {
            _addressData[prevOwnership.addr].balance -= 1;
            _addressData[prevOwnership.addr].numberBurned += 1;

            // Keep track of who burned the token, and the timestamp of burning.
            _ownerships[tokenId].addr = prevOwnership.addr;
            _ownerships[tokenId].startTimestamp = uint64(block.timestamp);
            _ownerships[tokenId].burned = true;

            // If the ownership slot of tokenId+1 is not explicitly set, that means the burn initiator owns it.
            // Set the slot of tokenId+1 explicitly in storage to maintain correctness for ownerOf(tokenId+1) calls.
            uint256 nextTokenId = tokenId + 1;
            if (_ownerships[nextTokenId].addr == address(0)) {
                // This will suffice for checking _exists(nextTokenId),
                // as a burned slot cannot contain the zero address.
                if (nextTokenId < _currentIndex) {
                    _ownerships[nextTokenId].addr = prevOwnership.addr;
                    _ownerships[nextTokenId].startTimestamp = prevOwnership.startTimestamp;
                }
            }
        }

        emit Transfer(prevOwnership.addr, address(0), tokenId);
        _afterTokenTransfers(prevOwnership.addr, address(0), tokenId, 1);

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

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

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

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

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

// File: contracts/danasch.sol



pragma solidity ^0.8.4;






contract OshareNFT is ERC721A, Ownable {
    using Strings for uint256;


    uint256 public maxTokensPerWhitelistedFirstAddress = 2;
    uint256 public maxTokensPerWhitelistedSecondAddress = 2;
    uint256 public maxTokensPerMint = 1;

    uint256 public tokenPricePresaleFirst = 0.06 ether;
    uint256 public tokenPricePresaleSecond = 0.09 ether; 
    uint256 public tokenPricePublicSale = 0.09 ether;

    string public tokenBaseURI = "";
    string public unrevealedURI = "";
    string public URIExtension = ".json";

    bool public hasPresaleStarted = false;
    bool public hasPublicSaleStarted = false;

    uint256 public constant BUY_MINT_START = 1;
    uint256 public constant BUY_TOTAL_AMOUNT = 6000;
    uint256 public boughtAmount = 0;

    bytes32 public whitelistRootFirst=0xc06ec807c2f6a93e9b8ba7f83191025eb1dcd9f530a813541a769518fefd9bfe;
    bytes32 public whitelistRootSecond=0x14d15c29b384f640304629354ca55f4e328b0e3b110cebff1ab28b70492b3668;
    mapping(address => uint256) public presaleWhitelistPurchased;

    constructor() ERC721A("OshareNFT", "OSHARE") {
    }

    function setWhitelistRootFirst(bytes32 _whitelistRoot) public onlyOwner {
        whitelistRootFirst = _whitelistRoot;
    }

    function setWhitelistRootSecond(bytes32 _whitelistRoot) public onlyOwner {
        whitelistRootSecond = _whitelistRoot;
    }

    function setTokenPricePresaleFirst(uint256 val) external onlyOwner {
        tokenPricePresaleFirst = val;
    }

    function setTokenPricePresaleSecond(uint256 val) external onlyOwner {
        tokenPricePresaleSecond = val;
    }
    
    function setTokenPricePublicSale(uint256 val) external onlyOwner {
        tokenPricePublicSale = val;
    }

    function setMaxTokensPerWhitelistedFirstAddress(uint256 val) external onlyOwner {
        maxTokensPerWhitelistedFirstAddress = val;
    }

    function setMaxTokensPerWhitelistedSecondAddress(uint256 val) external onlyOwner {
        maxTokensPerWhitelistedSecondAddress = val;
    }

    function verify(address account, bytes32[] memory proof) public view returns (bool)
    {
        bytes32 leaf = keccak256(abi.encodePacked(account));
        return MerkleProof.verify(proof, whitelistRootFirst, leaf) || MerkleProof.verify(proof, whitelistRootSecond, leaf);
    }

    function tokenPrice(address target, bytes32[] memory proof) public view returns (uint256) {
        bytes32 leaf = keccak256(abi.encodePacked(target));
        if (hasPublicSaleStarted) {
            return tokenPricePublicSale;
        }else if(MerkleProof.verify(proof, whitelistRootFirst, leaf)) {
            return tokenPricePresaleFirst;
        }else if (MerkleProof.verify(proof, whitelistRootSecond, leaf)) {
            return tokenPricePresaleSecond;
        }
        return 0;
    }

    function getMaxTokensPerMint(address target, bytes32[] memory proof) public view returns (uint256) {
        bytes32 leaf = keccak256(abi.encodePacked(target));
        if (hasPublicSaleStarted) {
            return maxTokensPerMint;
        }else if(MerkleProof.verify(proof, whitelistRootFirst, leaf)) {
            return maxTokensPerWhitelistedFirstAddress;
        }else if (MerkleProof.verify(proof, whitelistRootSecond, leaf)) {
            return maxTokensPerWhitelistedSecondAddress;
        }
        return 0;
    }

    function setMaxTokensPerMint(uint256 val) external onlyOwner {
        maxTokensPerMint = val;
    }

    function setPresale(bool val) external onlyOwner {
        hasPresaleStarted = val;
    }

    function setPublicSale(bool val) external onlyOwner {
        hasPublicSaleStarted = val;
    }

    function mint(uint256 amount, bytes32[] memory proof) external payable {
        require(msg.value >= tokenPrice(msg.sender, proof) * amount, "Incorrect ETH");
        require(hasPresaleStarted, "Cannot mint before presale");
        require(hasPublicSaleStarted || verify(msg.sender, proof), "Buyer not whitelisted for presale");
        require(amount <= getMaxTokensPerMint(msg.sender, proof), "Cannot mint more than the max tokens per mint");
        require(boughtAmount + amount <= BUY_TOTAL_AMOUNT, "No tokens left for minting");
        require(hasPublicSaleStarted || (presaleWhitelistPurchased[msg.sender] + amount <= getMaxTokensPerMint(msg.sender, proof)),
          "Cannot mint more than the max tokens per whitelisted address");

         _safeMint(msg.sender, amount);

        if (!hasPublicSaleStarted) {
            presaleWhitelistPurchased[msg.sender] += amount;
        }

        boughtAmount += amount;
    }

    function _baseURI() internal view override(ERC721A) returns (string memory) {
        return tokenBaseURI;
    }

    function tokenURI(uint256 tokenId) public view override(ERC721A) 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(), URIExtension)) : unrevealedURI;
    }
   
    function setBaseURI(string calldata URI) external onlyOwner {
        tokenBaseURI = URI;
    }

    function setUnrevealedURI(string calldata URI) external onlyOwner {
        unrevealedURI = URI;
    }

    function setURIExtension(string calldata URI) external onlyOwner {
        URIExtension = URI;
    }

    function _startTokenId() internal pure override(ERC721A) returns (uint256) {
        return 1;
    }

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

}

Contract Security Audit

Contract ABI

[{"inputs":[],"stateMutability":"nonpayable","type":"constructor"},{"inputs":[],"name":"ApprovalCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"ApprovalQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"ApprovalToCurrentOwner","type":"error"},{"inputs":[],"name":"ApproveToCaller","type":"error"},{"inputs":[],"name":"BalanceQueryForZeroAddress","type":"error"},{"inputs":[],"name":"MintToZeroAddress","type":"error"},{"inputs":[],"name":"MintZeroQuantity","type":"error"},{"inputs":[],"name":"OwnerQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"TransferCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"TransferFromIncorrectOwner","type":"error"},{"inputs":[],"name":"TransferToNonERC721ReceiverImplementer","type":"error"},{"inputs":[],"name":"TransferToZeroAddress","type":"error"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"approved","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Approval","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"operator","type":"address"},{"indexed":false,"internalType":"bool","name":"approved","type":"bool"}],"name":"ApprovalForAll","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"previousOwner","type":"address"},{"indexed":true,"internalType":"address","name":"newOwner","type":"address"}],"name":"OwnershipTransferred","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Transfer","type":"event"},{"inputs":[],"name":"BUY_MINT_START","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"BUY_TOTAL_AMOUNT","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"URIExtension","outputs":[{"internalType":"string","name":"","type":"string"}],"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":"boughtAmount","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"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":"target","type":"address"},{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"}],"name":"getMaxTokensPerMint","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"hasPresaleStarted","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"hasPublicSaleStarted","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"},{"internalType":"address","name":"operator","type":"address"}],"name":"isApprovedForAll","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxTokensPerMint","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxTokensPerWhitelistedFirstAddress","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxTokensPerWhitelistedSecondAddress","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"amount","type":"uint256"},{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"}],"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":"address","name":"","type":"address"}],"name":"presaleWhitelistPurchased","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"},{"internalType":"bytes","name":"_data","type":"bytes"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"operator","type":"address"},{"internalType":"bool","name":"approved","type":"bool"}],"name":"setApprovalForAll","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"URI","type":"string"}],"name":"setBaseURI","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"val","type":"uint256"}],"name":"setMaxTokensPerMint","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"val","type":"uint256"}],"name":"setMaxTokensPerWhitelistedFirstAddress","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"val","type":"uint256"}],"name":"setMaxTokensPerWhitelistedSecondAddress","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bool","name":"val","type":"bool"}],"name":"setPresale","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bool","name":"val","type":"bool"}],"name":"setPublicSale","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"val","type":"uint256"}],"name":"setTokenPricePresaleFirst","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"val","type":"uint256"}],"name":"setTokenPricePresaleSecond","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"val","type":"uint256"}],"name":"setTokenPricePublicSale","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"URI","type":"string"}],"name":"setURIExtension","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"URI","type":"string"}],"name":"setUnrevealedURI","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"_whitelistRoot","type":"bytes32"}],"name":"setWhitelistRootFirst","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"_whitelistRoot","type":"bytes32"}],"name":"setWhitelistRootSecond","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":[],"name":"tokenBaseURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"target","type":"address"},{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"}],"name":"tokenPrice","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"tokenPricePresaleFirst","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"tokenPricePresaleSecond","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"tokenPricePublicSale","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":[],"name":"unrevealedURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"account","type":"address"},{"internalType":"bytes32[]","name":"proof","type":"bytes32[]"}],"name":"verify","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"whitelistRootFirst","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"whitelistRootSecond","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"withdraw","outputs":[],"stateMutability":"nonpayable","type":"function"}]

608060405260026009556002600a556001600b5566d529ae9e860000600c5567013fbe85edc90000600d5567013fbe85edc90000600e5560405180602001604052806000815250600f90805190602001906200005d9291906200031e565b506040518060200160405280600081525060109080519060200190620000859291906200031e565b506040518060400160405280600581526020017f2e6a736f6e00000000000000000000000000000000000000000000000000000081525060119080519060200190620000d39291906200031e565b506000601260006101000a81548160ff0219169083151502179055506000601260016101000a81548160ff02191690831515021790555060006013557fc06ec807c2f6a93e9b8ba7f83191025eb1dcd9f530a813541a769518fefd9bfe60001b6014557f14d15c29b384f640304629354ca55f4e328b0e3b110cebff1ab28b70492b366860001b6015553480156200016a57600080fd5b506040518060400160405280600981526020017f4f73686172654e465400000000000000000000000000000000000000000000008152506040518060400160405280600681526020017f4f534841524500000000000000000000000000000000000000000000000000008152508160029080519060200190620001ef9291906200031e565b508060039080519060200190620002089291906200031e565b50620002196200024760201b60201c565b600081905550505062000241620002356200025060201b60201c565b6200025860201b60201c565b62000433565b60006001905090565b600033905090565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b8280546200032c90620003ce565b90600052602060002090601f0160209004810192826200035057600085556200039c565b82601f106200036b57805160ff19168380011785556200039c565b828001600101855582156200039c579182015b828111156200039b5782518255916020019190600101906200037e565b5b509050620003ab9190620003af565b5090565b5b80821115620003ca576000816000905550600101620003b0565b5090565b60006002820490506001821680620003e757607f821691505b60208210811415620003fe57620003fd62000404565b5b50919050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b61497c80620004436000396000f3fe6080604052600436106102ff5760003560e01c8063762cda3c11610190578063b0220015116100dc578063c87b56dd11610095578063f2fde38b1161006f578063f2fde38b14610b6f578063fab55c5314610b98578063fdd4b0f014610bc3578063fe2c7fee14610bee576102ff565b8063c87b56dd14610acc578063e985e9c514610b09578063e98cfcc114610b46576102ff565b8063b0220015146109cb578063b323b01b146109f6578063b76a0df414610a21578063b88d4fde14610a5e578063ba41b0c614610a87578063c54e73e314610aa3576102ff565b80639a6b7da211610149578063a22cb46511610123578063a22cb4651461090f578063a6d21bc614610938578063ab73e50c14610963578063ae3aa72f1461098e576102ff565b80639a6b7da2146108925780639f95608c146108bb578063a106a577146108e4576102ff565b8063762cda3c1461079457806378c5fe37146107bd5780638da5cb5b146107e85780639070975114610813578063945da7891461083c57806395d89b4114610867576102ff565b806346c4dc271161024f5780635c1cd692116102085780637035bf18116101e25780637035bf18146106d857806370a0823114610703578063715018a61461074057806372def46e14610757576102ff565b80635c1cd692146106455780635cfbd28b146106705780636352211e1461069b576102ff565b806346c4dc271461053757806348df7424146105605780634e99b8001461059d5780635406e251146105c857806355f804b3146105f35780635aca1bb61461061c576102ff565b806317465471116102bc5780633ccfd60b116102965780633ccfd60b146104a357806342842e0e146104ba57806344f92221146104e357806345c3274f1461050c576102ff565b8063174654711461042457806318160ddd1461044f57806323b872dd1461047a576102ff565b806301ffc9a71461030457806303b8807814610341578063069520dd1461036a57806306fdde0314610393578063081812fc146103be578063095ea7b3146103fb575b600080fd5b34801561031057600080fd5b5061032b60048036038101906103269190613ba7565b610c17565b604051610338919061403a565b60405180910390f35b34801561034d57600080fd5b5061036860048036038101906103639190613c4e565b610cf9565b005b34801561037657600080fd5b50610391600480360381019061038c9190613c4e565b610d7f565b005b34801561039f57600080fd5b506103a8610e05565b6040516103b59190614070565b60405180910390f35b3480156103ca57600080fd5b506103e560048036038101906103e09190613c4e565b610e97565b6040516103f29190613fd3565b60405180910390f35b34801561040757600080fd5b50610422600480360381019061041d9190613b0d565b610f13565b005b34801561043057600080fd5b5061043961101e565b60405161044691906141b2565b60405180910390f35b34801561045b57600080fd5b50610464611024565b60405161047191906141b2565b60405180910390f35b34801561048657600080fd5b506104a1600480360381019061049c919061399b565b61103b565b005b3480156104af57600080fd5b506104b861104b565b005b3480156104c657600080fd5b506104e160048036038101906104dc919061399b565b611107565b005b3480156104ef57600080fd5b5061050a60048036038101906105059190613c4e565b611127565b005b34801561051857600080fd5b506105216111ad565b60405161052e91906141b2565b60405180910390f35b34801561054357600080fd5b5061055e60048036038101906105599190613c4e565b6111b3565b005b34801561056c57600080fd5b506105876004803603810190610582919061392e565b611239565b60405161059491906141b2565b60405180910390f35b3480156105a957600080fd5b506105b2611251565b6040516105bf9190614070565b60405180910390f35b3480156105d457600080fd5b506105dd6112df565b6040516105ea91906141b2565b60405180910390f35b3480156105ff57600080fd5b5061061a60048036038101906106159190613c01565b6112e5565b005b34801561062857600080fd5b50610643600480360381019061063e9190613b4d565b611377565b005b34801561065157600080fd5b5061065a611410565b6040516106679190614055565b60405180910390f35b34801561067c57600080fd5b50610685611416565b6040516106929190614070565b60405180910390f35b3480156106a757600080fd5b506106c260048036038101906106bd9190613c4e565b6114a4565b6040516106cf9190613fd3565b60405180910390f35b3480156106e457600080fd5b506106ed6114ba565b6040516106fa9190614070565b60405180910390f35b34801561070f57600080fd5b5061072a6004803603810190610725919061392e565b611548565b60405161073791906141b2565b60405180910390f35b34801561074c57600080fd5b50610755611618565b005b34801561076357600080fd5b5061077e60048036038101906107799190613a71565b6116a0565b60405161078b91906141b2565b60405180910390f35b3480156107a057600080fd5b506107bb60048036038101906107b69190613c4e565b611732565b005b3480156107c957600080fd5b506107d26117b8565b6040516107df91906141b2565b60405180910390f35b3480156107f457600080fd5b506107fd6117be565b60405161080a9190613fd3565b60405180910390f35b34801561081f57600080fd5b5061083a60048036038101906108359190613c01565b6117e8565b005b34801561084857600080fd5b5061085161187a565b60405161085e91906141b2565b60405180910390f35b34801561087357600080fd5b5061087c611880565b6040516108899190614070565b60405180910390f35b34801561089e57600080fd5b506108b960048036038101906108b49190613b7a565b611912565b005b3480156108c757600080fd5b506108e260048036038101906108dd9190613b7a565b611998565b005b3480156108f057600080fd5b506108f9611a1e565b60405161090691906141b2565b60405180910390f35b34801561091b57600080fd5b5061093660048036038101906109319190613acd565b611a24565b005b34801561094457600080fd5b5061094d611b9c565b60405161095a91906141b2565b60405180910390f35b34801561096f57600080fd5b50610978611ba2565b6040516109859190614055565b60405180910390f35b34801561099a57600080fd5b506109b560048036038101906109b09190613a71565b611ba8565b6040516109c291906141b2565b60405180910390f35b3480156109d757600080fd5b506109e0611c3a565b6040516109ed919061403a565b60405180910390f35b348015610a0257600080fd5b50610a0b611c4d565b604051610a1891906141b2565b60405180910390f35b348015610a2d57600080fd5b50610a486004803603810190610a439190613a71565b611c52565b604051610a55919061403a565b60405180910390f35b348015610a6a57600080fd5b50610a856004803603810190610a8091906139ee565b611ca8565b005b610aa16004803603810190610a9c9190613c7b565b611d24565b005b348015610aaf57600080fd5b50610aca6004803603810190610ac59190613b4d565b612007565b005b348015610ad857600080fd5b50610af36004803603810190610aee9190613c4e565b6120a0565b604051610b009190614070565b60405180910390f35b348015610b1557600080fd5b50610b306004803603810190610b2b919061395b565b6121c5565b604051610b3d919061403a565b60405180910390f35b348015610b5257600080fd5b50610b6d6004803603810190610b689190613c4e565b612259565b005b348015610b7b57600080fd5b50610b966004803603810190610b91919061392e565b6122df565b005b348015610ba457600080fd5b50610bad6123d7565b604051610bba91906141b2565b60405180910390f35b348015610bcf57600080fd5b50610bd86123dd565b604051610be5919061403a565b60405180910390f35b348015610bfa57600080fd5b50610c156004803603810190610c109190613c01565b6123f0565b005b60007f80ac58cd000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff19161480610ce257507f5b5e139f000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b80610cf25750610cf182612482565b5b9050919050565b610d016124ec565b73ffffffffffffffffffffffffffffffffffffffff16610d1f6117be565b73ffffffffffffffffffffffffffffffffffffffff1614610d75576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610d6c90614132565b60405180910390fd5b80600a8190555050565b610d876124ec565b73ffffffffffffffffffffffffffffffffffffffff16610da56117be565b73ffffffffffffffffffffffffffffffffffffffff1614610dfb576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610df290614132565b60405180910390fd5b80600d8190555050565b606060028054610e149061447c565b80601f0160208091040260200160405190810160405280929190818152602001828054610e409061447c565b8015610e8d5780601f10610e6257610100808354040283529160200191610e8d565b820191906000526020600020905b815481529060010190602001808311610e7057829003601f168201915b5050505050905090565b6000610ea2826124f4565b610ed8576040517fcf4700e400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6006600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff169050919050565b6000610f1e826114a4565b90508073ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff161415610f86576040517f943f7b8c00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8073ffffffffffffffffffffffffffffffffffffffff16610fa56124ec565b73ffffffffffffffffffffffffffffffffffffffff1614158015610fd75750610fd581610fd06124ec565b6121c5565b155b1561100e576040517fcfb3b94200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b611019838383612542565b505050565b600b5481565b600061102e6125f4565b6001546000540303905090565b6110468383836125fd565b505050565b6110536124ec565b73ffffffffffffffffffffffffffffffffffffffff166110716117be565b73ffffffffffffffffffffffffffffffffffffffff16146110c7576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016110be90614132565b60405180910390fd5b3373ffffffffffffffffffffffffffffffffffffffff166108fc479081150290604051600060405180830381858888f1935050505061110557600080fd5b565b61112283838360405180602001604052806000815250611ca8565b505050565b61112f6124ec565b73ffffffffffffffffffffffffffffffffffffffff1661114d6117be565b73ffffffffffffffffffffffffffffffffffffffff16146111a3576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161119a90614132565b60405180910390fd5b8060098190555050565b60135481565b6111bb6124ec565b73ffffffffffffffffffffffffffffffffffffffff166111d96117be565b73ffffffffffffffffffffffffffffffffffffffff161461122f576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161122690614132565b60405180910390fd5b80600e8190555050565b60166020528060005260406000206000915090505481565b600f805461125e9061447c565b80601f016020809104026020016040519081016040528092919081815260200182805461128a9061447c565b80156112d75780601f106112ac576101008083540402835291602001916112d7565b820191906000526020600020905b8154815290600101906020018083116112ba57829003601f168201915b505050505081565b600d5481565b6112ed6124ec565b73ffffffffffffffffffffffffffffffffffffffff1661130b6117be565b73ffffffffffffffffffffffffffffffffffffffff1614611361576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161135890614132565b60405180910390fd5b8181600f9190611372929190613666565b505050565b61137f6124ec565b73ffffffffffffffffffffffffffffffffffffffff1661139d6117be565b73ffffffffffffffffffffffffffffffffffffffff16146113f3576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016113ea90614132565b60405180910390fd5b80601260016101000a81548160ff02191690831515021790555050565b60145481565b601180546114239061447c565b80601f016020809104026020016040519081016040528092919081815260200182805461144f9061447c565b801561149c5780601f106114715761010080835404028352916020019161149c565b820191906000526020600020905b81548152906001019060200180831161147f57829003601f168201915b505050505081565b60006114af82612aee565b600001519050919050565b601080546114c79061447c565b80601f01602080910402602001604051908101604052809291908181526020018280546114f39061447c565b80156115405780601f1061151557610100808354040283529160200191611540565b820191906000526020600020905b81548152906001019060200180831161152357829003601f168201915b505050505081565b60008073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff1614156115b0576040517f8f4eb60400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600560008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160009054906101000a900467ffffffffffffffff1667ffffffffffffffff169050919050565b6116206124ec565b73ffffffffffffffffffffffffffffffffffffffff1661163e6117be565b73ffffffffffffffffffffffffffffffffffffffff1614611694576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161168b90614132565b60405180910390fd5b61169e6000612d7d565b565b600080836040516020016116b49190613f87565b604051602081830303815290604052805190602001209050601260019054906101000a900460ff16156116ec57600b5491505061172c565b6116f98360145483612e43565b156117095760095491505061172c565b6117168360155483612e43565b1561172657600a5491505061172c565b60009150505b92915050565b61173a6124ec565b73ffffffffffffffffffffffffffffffffffffffff166117586117be565b73ffffffffffffffffffffffffffffffffffffffff16146117ae576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016117a590614132565b60405180910390fd5b80600b8190555050565b600e5481565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b6117f06124ec565b73ffffffffffffffffffffffffffffffffffffffff1661180e6117be565b73ffffffffffffffffffffffffffffffffffffffff1614611864576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161185b90614132565b60405180910390fd5b818160119190611875929190613666565b505050565b600a5481565b60606003805461188f9061447c565b80601f01602080910402602001604051908101604052809291908181526020018280546118bb9061447c565b80156119085780601f106118dd57610100808354040283529160200191611908565b820191906000526020600020905b8154815290600101906020018083116118eb57829003601f168201915b5050505050905090565b61191a6124ec565b73ffffffffffffffffffffffffffffffffffffffff166119386117be565b73ffffffffffffffffffffffffffffffffffffffff161461198e576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161198590614132565b60405180910390fd5b8060148190555050565b6119a06124ec565b73ffffffffffffffffffffffffffffffffffffffff166119be6117be565b73ffffffffffffffffffffffffffffffffffffffff1614611a14576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611a0b90614132565b60405180910390fd5b8060158190555050565b600c5481565b611a2c6124ec565b73ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415611a91576040517fb06307db00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8060076000611a9e6124ec565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060006101000a81548160ff0219169083151502179055508173ffffffffffffffffffffffffffffffffffffffff16611b4b6124ec565b73ffffffffffffffffffffffffffffffffffffffff167f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c3183604051611b90919061403a565b60405180910390a35050565b61177081565b60155481565b60008083604051602001611bbc9190613f87565b604051602081830303815290604052805190602001209050601260019054906101000a900460ff1615611bf457600e54915050611c34565b611c018360145483612e43565b15611c1157600c54915050611c34565b611c1e8360155483612e43565b15611c2e57600d54915050611c34565b60009150505b92915050565b601260009054906101000a900460ff1681565b600181565b60008083604051602001611c669190613f87565b604051602081830303815290604052805190602001209050611c8b8360145483612e43565b80611c9f5750611c9e8360155483612e43565b5b91505092915050565b611cb38484846125fd565b611cd28373ffffffffffffffffffffffffffffffffffffffff16612e5a565b8015611ce75750611ce584848484612e7d565b155b15611d1e576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b50505050565b81611d2f3383611ba8565b611d39919061432e565b341015611d7b576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611d72906140f2565b60405180910390fd5b601260009054906101000a900460ff16611dca576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611dc190614092565b60405180910390fd5b601260019054906101000a900460ff1680611deb5750611dea3382611c52565b5b611e2a576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611e2190614112565b60405180910390fd5b611e3433826116a0565b821115611e76576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611e6d906140b2565b60405180910390fd5b61177082601354611e8791906142a7565b1115611ec8576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611ebf90614172565b60405180910390fd5b601260019054906101000a900460ff1680611f365750611ee833826116a0565b82601660003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054611f3391906142a7565b11155b611f75576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611f6c90614192565b60405180910390fd5b611f7f3383612fdd565b601260019054906101000a900460ff16611fea5781601660003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254611fe291906142a7565b925050819055505b8160136000828254611ffc91906142a7565b925050819055505050565b61200f6124ec565b73ffffffffffffffffffffffffffffffffffffffff1661202d6117be565b73ffffffffffffffffffffffffffffffffffffffff1614612083576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161207a90614132565b60405180910390fd5b80601260006101000a81548160ff02191690831515021790555050565b60606120ab826124f4565b6120ea576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016120e190614152565b60405180910390fd5b60006120f4612ffb565b9050600081511161218f576010805461210c9061447c565b80601f01602080910402602001604051908101604052809291908181526020018280546121389061447c565b80156121855780601f1061215a57610100808354040283529160200191612185565b820191906000526020600020905b81548152906001019060200180831161216857829003601f168201915b50505050506121bd565b806121998461308d565b60116040516020016121ad93929190613fa2565b6040516020818303038152906040525b915050919050565b6000600760008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff16905092915050565b6122616124ec565b73ffffffffffffffffffffffffffffffffffffffff1661227f6117be565b73ffffffffffffffffffffffffffffffffffffffff16146122d5576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016122cc90614132565b60405180910390fd5b80600c8190555050565b6122e76124ec565b73ffffffffffffffffffffffffffffffffffffffff166123056117be565b73ffffffffffffffffffffffffffffffffffffffff161461235b576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161235290614132565b60405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff1614156123cb576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016123c2906140d2565b60405180910390fd5b6123d481612d7d565b50565b60095481565b601260019054906101000a900460ff1681565b6123f86124ec565b73ffffffffffffffffffffffffffffffffffffffff166124166117be565b73ffffffffffffffffffffffffffffffffffffffff161461246c576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161246390614132565b60405180910390fd5b81816010919061247d929190613666565b505050565b60007f01ffc9a7000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916149050919050565b600033905090565b6000816124ff6125f4565b1115801561250e575060005482105b801561253b575060046000838152602001908152602001600020600001601c9054906101000a900460ff16155b9050919050565b826006600084815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550818373ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff167f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92560405160405180910390a4505050565b60006001905090565b600061260882612aee565b90506000816000015173ffffffffffffffffffffffffffffffffffffffff1661262f6124ec565b73ffffffffffffffffffffffffffffffffffffffff1614806126625750612661826000015161265c6124ec565b6121c5565b5b806126a757506126706124ec565b73ffffffffffffffffffffffffffffffffffffffff1661268f84610e97565b73ffffffffffffffffffffffffffffffffffffffff16145b9050806126e0576040517f59c896be00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8473ffffffffffffffffffffffffffffffffffffffff16826000015173ffffffffffffffffffffffffffffffffffffffff1614612749576040517fa114810000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff1614156127b0576040517fea553b3400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6127bd85858560016131ee565b6127cd6000848460000151612542565b6001600560008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160392506101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055506001600560008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff160217905550836004600085815260200190815260200160002060000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550426004600085815260200190815260200160002060000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055506000600184019050600073ffffffffffffffffffffffffffffffffffffffff166004600083815260200190815260200160002060000160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff161415612a7e57600054811015612a7d5782600001516004600083815260200190815260200160002060000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555082602001516004600083815260200190815260200160002060000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055505b5b50828473ffffffffffffffffffffffffffffffffffffffff168673ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4612ae785858560016131f4565b5050505050565b612af66136ec565b600082905080612b046125f4565b11158015612b13575060005481105b15612d46576000600460008381526020019081526020016000206040518060600160405290816000820160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020016000820160149054906101000a900467ffffffffffffffff1667ffffffffffffffff1667ffffffffffffffff16815260200160008201601c9054906101000a900460ff16151515158152505090508060400151612d4457600073ffffffffffffffffffffffffffffffffffffffff16816000015173ffffffffffffffffffffffffffffffffffffffff1614612c28578092505050612d78565b5b600115612d4357818060019003925050600460008381526020019081526020016000206040518060600160405290816000820160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020016000820160149054906101000a900467ffffffffffffffff1667ffffffffffffffff1667ffffffffffffffff16815260200160008201601c9054906101000a900460ff1615151515815250509050600073ffffffffffffffffffffffffffffffffffffffff16816000015173ffffffffffffffffffffffffffffffffffffffff1614612d3e578092505050612d78565b612c29565b5b505b6040517fdf2d9b4200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b919050565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b600082612e5085846131fa565b1490509392505050565b6000808273ffffffffffffffffffffffffffffffffffffffff163b119050919050565b60008373ffffffffffffffffffffffffffffffffffffffff1663150b7a02612ea36124ec565b8786866040518563ffffffff1660e01b8152600401612ec59493929190613fee565b602060405180830381600087803b158015612edf57600080fd5b505af1925050508015612f1057506040513d601f19601f82011682018060405250810190612f0d9190613bd4565b60015b612f8a573d8060008114612f40576040519150601f19603f3d011682016040523d82523d6000602084013e612f45565b606091505b50600081511415612f82576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b805181602001fd5b63150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916817bffffffffffffffffffffffffffffffffffffffffffffffffffffffff191614915050949350505050565b612ff782826040518060200160405280600081525061326f565b5050565b6060600f805461300a9061447c565b80601f01602080910402602001604051908101604052809291908181526020018280546130369061447c565b80156130835780601f1061305857610100808354040283529160200191613083565b820191906000526020600020905b81548152906001019060200180831161306657829003601f168201915b5050505050905090565b606060008214156130d5576040518060400160405280600181526020017f300000000000000000000000000000000000000000000000000000000000000081525090506131e9565b600082905060005b600082146131075780806130f0906144df565b915050600a8261310091906142fd565b91506130dd565b60008167ffffffffffffffff81111561312357613122614639565b5b6040519080825280601f01601f1916602001820160405280156131555781602001600182028036833780820191505090505b5090505b600085146131e25760018261316e9190614388565b9150600a8561317d919061454c565b603061318991906142a7565b60f81b81838151811061319f5761319e61460a565b5b60200101907effffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916908160001a905350600a856131db91906142fd565b9450613159565b8093505050505b919050565b50505050565b50505050565b60008082905060005b84518110156132645760008582815181106132215761322061460a565b5b602002602001015190508083116132435761323c8382613281565b9250613250565b61324d8184613281565b92505b50808061325c906144df565b915050613203565b508091505092915050565b61327c8383836001613298565b505050565b600082600052816020526040600020905092915050565b600080549050600073ffffffffffffffffffffffffffffffffffffffff168573ffffffffffffffffffffffffffffffffffffffff161415613305576040517f2e07630000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6000841415613340576040517fb562e8dd00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b61334d60008683876131ee565b83600560008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff16021790555083600560008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160088282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff160217905550846004600083815260200190815260200160002060000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550426004600083815260200190815260200160002060000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff16021790555060008190506000858201905083801561351757506135168773ffffffffffffffffffffffffffffffffffffffff16612e5a565b5b156135dd575b818773ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a461358c6000888480600101955088612e7d565b6135c2576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8082141561351d5782600054146135d857600080fd5b613649565b5b818060010192508773ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4808214156135de575b81600081905550505061365f60008683876131f4565b5050505050565b8280546136729061447c565b90600052602060002090601f01602090048101928261369457600085556136db565b82601f106136ad57803560ff19168380011785556136db565b828001600101855582156136db579182015b828111156136da5782358255916020019190600101906136bf565b5b5090506136e8919061372f565b5090565b6040518060600160405280600073ffffffffffffffffffffffffffffffffffffffff168152602001600067ffffffffffffffff1681526020016000151581525090565b5b80821115613748576000816000905550600101613730565b5090565b600061375f61375a846141f2565b6141cd565b9050808382526020820190508285602086028201111561378257613781614672565b5b60005b858110156137b257816137988882613856565b845260208401935060208301925050600181019050613785565b5050509392505050565b60006137cf6137ca8461421e565b6141cd565b9050828152602081018484840111156137eb576137ea614677565b5b6137f684828561443a565b509392505050565b60008135905061380d816148d3565b92915050565b600082601f8301126138285761382761466d565b5b813561383884826020860161374c565b91505092915050565b600081359050613850816148ea565b92915050565b60008135905061386581614901565b92915050565b60008135905061387a81614918565b92915050565b60008151905061388f81614918565b92915050565b600082601f8301126138aa576138a961466d565b5b81356138ba8482602086016137bc565b91505092915050565b60008083601f8401126138d9576138d861466d565b5b8235905067ffffffffffffffff8111156138f6576138f5614668565b5b60208301915083600182028301111561391257613911614672565b5b9250929050565b6000813590506139288161492f565b92915050565b60006020828403121561394457613943614681565b5b6000613952848285016137fe565b91505092915050565b6000806040838503121561397257613971614681565b5b6000613980858286016137fe565b9250506020613991858286016137fe565b9150509250929050565b6000806000606084860312156139b4576139b3614681565b5b60006139c2868287016137fe565b93505060206139d3868287016137fe565b92505060406139e486828701613919565b9150509250925092565b60008060008060808587031215613a0857613a07614681565b5b6000613a16878288016137fe565b9450506020613a27878288016137fe565b9350506040613a3887828801613919565b925050606085013567ffffffffffffffff811115613a5957613a5861467c565b5b613a6587828801613895565b91505092959194509250565b60008060408385031215613a8857613a87614681565b5b6000613a96858286016137fe565b925050602083013567ffffffffffffffff811115613ab757613ab661467c565b5b613ac385828601613813565b9150509250929050565b60008060408385031215613ae457613ae3614681565b5b6000613af2858286016137fe565b9250506020613b0385828601613841565b9150509250929050565b60008060408385031215613b2457613b23614681565b5b6000613b32858286016137fe565b9250506020613b4385828601613919565b9150509250929050565b600060208284031215613b6357613b62614681565b5b6000613b7184828501613841565b91505092915050565b600060208284031215613b9057613b8f614681565b5b6000613b9e84828501613856565b91505092915050565b600060208284031215613bbd57613bbc614681565b5b6000613bcb8482850161386b565b91505092915050565b600060208284031215613bea57613be9614681565b5b6000613bf884828501613880565b91505092915050565b60008060208385031215613c1857613c17614681565b5b600083013567ffffffffffffffff811115613c3657613c3561467c565b5b613c42858286016138c3565b92509250509250929050565b600060208284031215613c6457613c63614681565b5b6000613c7284828501613919565b91505092915050565b60008060408385031215613c9257613c91614681565b5b6000613ca085828601613919565b925050602083013567ffffffffffffffff811115613cc157613cc061467c565b5b613ccd85828601613813565b9150509250929050565b613ce0816143bc565b82525050565b613cf7613cf2826143bc565b614528565b82525050565b613d06816143ce565b82525050565b613d15816143da565b82525050565b6000613d2682614264565b613d30818561427a565b9350613d40818560208601614449565b613d4981614686565b840191505092915050565b6000613d5f8261426f565b613d69818561428b565b9350613d79818560208601614449565b613d8281614686565b840191505092915050565b6000613d988261426f565b613da2818561429c565b9350613db2818560208601614449565b80840191505092915050565b60008154613dcb8161447c565b613dd5818661429c565b94506001821660008114613df05760018114613e0157613e34565b60ff19831686528186019350613e34565b613e0a8561424f565b60005b83811015613e2c57815481890152600182019150602081019050613e0d565b838801955050505b50505092915050565b6000613e4a601a8361428b565b9150613e55826146a4565b602082019050919050565b6000613e6d602d8361428b565b9150613e78826146cd565b604082019050919050565b6000613e9060268361428b565b9150613e9b8261471c565b604082019050919050565b6000613eb3600d8361428b565b9150613ebe8261476b565b602082019050919050565b6000613ed660218361428b565b9150613ee182614794565b604082019050919050565b6000613ef960208361428b565b9150613f04826147e3565b602082019050919050565b6000613f1c602f8361428b565b9150613f278261480c565b604082019050919050565b6000613f3f601a8361428b565b9150613f4a8261485b565b602082019050919050565b6000613f62603c8361428b565b9150613f6d82614884565b604082019050919050565b613f8181614430565b82525050565b6000613f938284613ce6565b60148201915081905092915050565b6000613fae8286613d8d565b9150613fba8285613d8d565b9150613fc68284613dbe565b9150819050949350505050565b6000602082019050613fe86000830184613cd7565b92915050565b60006080820190506140036000830187613cd7565b6140106020830186613cd7565b61401d6040830185613f78565b818103606083015261402f8184613d1b565b905095945050505050565b600060208201905061404f6000830184613cfd565b92915050565b600060208201905061406a6000830184613d0c565b92915050565b6000602082019050818103600083015261408a8184613d54565b905092915050565b600060208201905081810360008301526140ab81613e3d565b9050919050565b600060208201905081810360008301526140cb81613e60565b9050919050565b600060208201905081810360008301526140eb81613e83565b9050919050565b6000602082019050818103600083015261410b81613ea6565b9050919050565b6000602082019050818103600083015261412b81613ec9565b9050919050565b6000602082019050818103600083015261414b81613eec565b9050919050565b6000602082019050818103600083015261416b81613f0f565b9050919050565b6000602082019050818103600083015261418b81613f32565b9050919050565b600060208201905081810360008301526141ab81613f55565b9050919050565b60006020820190506141c76000830184613f78565b92915050565b60006141d76141e8565b90506141e382826144ae565b919050565b6000604051905090565b600067ffffffffffffffff82111561420d5761420c614639565b5b602082029050602081019050919050565b600067ffffffffffffffff82111561423957614238614639565b5b61424282614686565b9050602081019050919050565b60008190508160005260206000209050919050565b600081519050919050565b600081519050919050565b600082825260208201905092915050565b600082825260208201905092915050565b600081905092915050565b60006142b282614430565b91506142bd83614430565b9250827fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff038211156142f2576142f161457d565b5b828201905092915050565b600061430882614430565b915061431383614430565b925082614323576143226145ac565b5b828204905092915050565b600061433982614430565b915061434483614430565b9250817fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff048311821515161561437d5761437c61457d565b5b828202905092915050565b600061439382614430565b915061439e83614430565b9250828210156143b1576143b061457d565b5b828203905092915050565b60006143c782614410565b9050919050565b60008115159050919050565b6000819050919050565b60007fffffffff0000000000000000000000000000000000000000000000000000000082169050919050565b600073ffffffffffffffffffffffffffffffffffffffff82169050919050565b6000819050919050565b82818337600083830152505050565b60005b8381101561446757808201518184015260208101905061444c565b83811115614476576000848401525b50505050565b6000600282049050600182168061449457607f821691505b602082108114156144a8576144a76145db565b5b50919050565b6144b782614686565b810181811067ffffffffffffffff821117156144d6576144d5614639565b5b80604052505050565b60006144ea82614430565b91507fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff82141561451d5761451c61457d565b5b600182019050919050565b60006145338261453a565b9050919050565b600061454582614697565b9050919050565b600061455782614430565b915061456283614430565b925082614572576145716145ac565b5b828206905092915050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b600080fd5b600080fd5b600080fd5b600080fd5b600080fd5b600080fd5b6000601f19601f8301169050919050565b60008160601b9050919050565b7f43616e6e6f74206d696e74206265666f72652070726573616c65000000000000600082015250565b7f43616e6e6f74206d696e74206d6f7265207468616e20746865206d617820746f60008201527f6b656e7320706572206d696e7400000000000000000000000000000000000000602082015250565b7f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160008201527f6464726573730000000000000000000000000000000000000000000000000000602082015250565b7f496e636f72726563742045544800000000000000000000000000000000000000600082015250565b7f4275796572206e6f742077686974656c697374656420666f722070726573616c60008201527f6500000000000000000000000000000000000000000000000000000000000000602082015250565b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b7f4552433732314d657461646174613a2055524920717565727920666f72206e6f60008201527f6e6578697374656e7420746f6b656e0000000000000000000000000000000000602082015250565b7f4e6f20746f6b656e73206c65667420666f72206d696e74696e67000000000000600082015250565b7f43616e6e6f74206d696e74206d6f7265207468616e20746865206d617820746f60008201527f6b656e73207065722077686974656c6973746564206164647265737300000000602082015250565b6148dc816143bc565b81146148e757600080fd5b50565b6148f3816143ce565b81146148fe57600080fd5b50565b61490a816143da565b811461491557600080fd5b50565b614921816143e4565b811461492c57600080fd5b50565b61493881614430565b811461494357600080fd5b5056fea2646970667358221220a137902ff01c4043f1820d1de508c92bd130a0eb471ec1dfad4606c141c9b55e64736f6c63430008070033

Deployed Bytecode

0x6080604052600436106102ff5760003560e01c8063762cda3c11610190578063b0220015116100dc578063c87b56dd11610095578063f2fde38b1161006f578063f2fde38b14610b6f578063fab55c5314610b98578063fdd4b0f014610bc3578063fe2c7fee14610bee576102ff565b8063c87b56dd14610acc578063e985e9c514610b09578063e98cfcc114610b46576102ff565b8063b0220015146109cb578063b323b01b146109f6578063b76a0df414610a21578063b88d4fde14610a5e578063ba41b0c614610a87578063c54e73e314610aa3576102ff565b80639a6b7da211610149578063a22cb46511610123578063a22cb4651461090f578063a6d21bc614610938578063ab73e50c14610963578063ae3aa72f1461098e576102ff565b80639a6b7da2146108925780639f95608c146108bb578063a106a577146108e4576102ff565b8063762cda3c1461079457806378c5fe37146107bd5780638da5cb5b146107e85780639070975114610813578063945da7891461083c57806395d89b4114610867576102ff565b806346c4dc271161024f5780635c1cd692116102085780637035bf18116101e25780637035bf18146106d857806370a0823114610703578063715018a61461074057806372def46e14610757576102ff565b80635c1cd692146106455780635cfbd28b146106705780636352211e1461069b576102ff565b806346c4dc271461053757806348df7424146105605780634e99b8001461059d5780635406e251146105c857806355f804b3146105f35780635aca1bb61461061c576102ff565b806317465471116102bc5780633ccfd60b116102965780633ccfd60b146104a357806342842e0e146104ba57806344f92221146104e357806345c3274f1461050c576102ff565b8063174654711461042457806318160ddd1461044f57806323b872dd1461047a576102ff565b806301ffc9a71461030457806303b8807814610341578063069520dd1461036a57806306fdde0314610393578063081812fc146103be578063095ea7b3146103fb575b600080fd5b34801561031057600080fd5b5061032b60048036038101906103269190613ba7565b610c17565b604051610338919061403a565b60405180910390f35b34801561034d57600080fd5b5061036860048036038101906103639190613c4e565b610cf9565b005b34801561037657600080fd5b50610391600480360381019061038c9190613c4e565b610d7f565b005b34801561039f57600080fd5b506103a8610e05565b6040516103b59190614070565b60405180910390f35b3480156103ca57600080fd5b506103e560048036038101906103e09190613c4e565b610e97565b6040516103f29190613fd3565b60405180910390f35b34801561040757600080fd5b50610422600480360381019061041d9190613b0d565b610f13565b005b34801561043057600080fd5b5061043961101e565b60405161044691906141b2565b60405180910390f35b34801561045b57600080fd5b50610464611024565b60405161047191906141b2565b60405180910390f35b34801561048657600080fd5b506104a1600480360381019061049c919061399b565b61103b565b005b3480156104af57600080fd5b506104b861104b565b005b3480156104c657600080fd5b506104e160048036038101906104dc919061399b565b611107565b005b3480156104ef57600080fd5b5061050a60048036038101906105059190613c4e565b611127565b005b34801561051857600080fd5b506105216111ad565b60405161052e91906141b2565b60405180910390f35b34801561054357600080fd5b5061055e60048036038101906105599190613c4e565b6111b3565b005b34801561056c57600080fd5b506105876004803603810190610582919061392e565b611239565b60405161059491906141b2565b60405180910390f35b3480156105a957600080fd5b506105b2611251565b6040516105bf9190614070565b60405180910390f35b3480156105d457600080fd5b506105dd6112df565b6040516105ea91906141b2565b60405180910390f35b3480156105ff57600080fd5b5061061a60048036038101906106159190613c01565b6112e5565b005b34801561062857600080fd5b50610643600480360381019061063e9190613b4d565b611377565b005b34801561065157600080fd5b5061065a611410565b6040516106679190614055565b60405180910390f35b34801561067c57600080fd5b50610685611416565b6040516106929190614070565b60405180910390f35b3480156106a757600080fd5b506106c260048036038101906106bd9190613c4e565b6114a4565b6040516106cf9190613fd3565b60405180910390f35b3480156106e457600080fd5b506106ed6114ba565b6040516106fa9190614070565b60405180910390f35b34801561070f57600080fd5b5061072a6004803603810190610725919061392e565b611548565b60405161073791906141b2565b60405180910390f35b34801561074c57600080fd5b50610755611618565b005b34801561076357600080fd5b5061077e60048036038101906107799190613a71565b6116a0565b60405161078b91906141b2565b60405180910390f35b3480156107a057600080fd5b506107bb60048036038101906107b69190613c4e565b611732565b005b3480156107c957600080fd5b506107d26117b8565b6040516107df91906141b2565b60405180910390f35b3480156107f457600080fd5b506107fd6117be565b60405161080a9190613fd3565b60405180910390f35b34801561081f57600080fd5b5061083a60048036038101906108359190613c01565b6117e8565b005b34801561084857600080fd5b5061085161187a565b60405161085e91906141b2565b60405180910390f35b34801561087357600080fd5b5061087c611880565b6040516108899190614070565b60405180910390f35b34801561089e57600080fd5b506108b960048036038101906108b49190613b7a565b611912565b005b3480156108c757600080fd5b506108e260048036038101906108dd9190613b7a565b611998565b005b3480156108f057600080fd5b506108f9611a1e565b60405161090691906141b2565b60405180910390f35b34801561091b57600080fd5b5061093660048036038101906109319190613acd565b611a24565b005b34801561094457600080fd5b5061094d611b9c565b60405161095a91906141b2565b60405180910390f35b34801561096f57600080fd5b50610978611ba2565b6040516109859190614055565b60405180910390f35b34801561099a57600080fd5b506109b560048036038101906109b09190613a71565b611ba8565b6040516109c291906141b2565b60405180910390f35b3480156109d757600080fd5b506109e0611c3a565b6040516109ed919061403a565b60405180910390f35b348015610a0257600080fd5b50610a0b611c4d565b604051610a1891906141b2565b60405180910390f35b348015610a2d57600080fd5b50610a486004803603810190610a439190613a71565b611c52565b604051610a55919061403a565b60405180910390f35b348015610a6a57600080fd5b50610a856004803603810190610a8091906139ee565b611ca8565b005b610aa16004803603810190610a9c9190613c7b565b611d24565b005b348015610aaf57600080fd5b50610aca6004803603810190610ac59190613b4d565b612007565b005b348015610ad857600080fd5b50610af36004803603810190610aee9190613c4e565b6120a0565b604051610b009190614070565b60405180910390f35b348015610b1557600080fd5b50610b306004803603810190610b2b919061395b565b6121c5565b604051610b3d919061403a565b60405180910390f35b348015610b5257600080fd5b50610b6d6004803603810190610b689190613c4e565b612259565b005b348015610b7b57600080fd5b50610b966004803603810190610b91919061392e565b6122df565b005b348015610ba457600080fd5b50610bad6123d7565b604051610bba91906141b2565b60405180910390f35b348015610bcf57600080fd5b50610bd86123dd565b604051610be5919061403a565b60405180910390f35b348015610bfa57600080fd5b50610c156004803603810190610c109190613c01565b6123f0565b005b60007f80ac58cd000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff19161480610ce257507f5b5e139f000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b80610cf25750610cf182612482565b5b9050919050565b610d016124ec565b73ffffffffffffffffffffffffffffffffffffffff16610d1f6117be565b73ffffffffffffffffffffffffffffffffffffffff1614610d75576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610d6c90614132565b60405180910390fd5b80600a8190555050565b610d876124ec565b73ffffffffffffffffffffffffffffffffffffffff16610da56117be565b73ffffffffffffffffffffffffffffffffffffffff1614610dfb576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610df290614132565b60405180910390fd5b80600d8190555050565b606060028054610e149061447c565b80601f0160208091040260200160405190810160405280929190818152602001828054610e409061447c565b8015610e8d5780601f10610e6257610100808354040283529160200191610e8d565b820191906000526020600020905b815481529060010190602001808311610e7057829003601f168201915b5050505050905090565b6000610ea2826124f4565b610ed8576040517fcf4700e400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6006600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff169050919050565b6000610f1e826114a4565b90508073ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff161415610f86576040517f943f7b8c00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8073ffffffffffffffffffffffffffffffffffffffff16610fa56124ec565b73ffffffffffffffffffffffffffffffffffffffff1614158015610fd75750610fd581610fd06124ec565b6121c5565b155b1561100e576040517fcfb3b94200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b611019838383612542565b505050565b600b5481565b600061102e6125f4565b6001546000540303905090565b6110468383836125fd565b505050565b6110536124ec565b73ffffffffffffffffffffffffffffffffffffffff166110716117be565b73ffffffffffffffffffffffffffffffffffffffff16146110c7576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016110be90614132565b60405180910390fd5b3373ffffffffffffffffffffffffffffffffffffffff166108fc479081150290604051600060405180830381858888f1935050505061110557600080fd5b565b61112283838360405180602001604052806000815250611ca8565b505050565b61112f6124ec565b73ffffffffffffffffffffffffffffffffffffffff1661114d6117be565b73ffffffffffffffffffffffffffffffffffffffff16146111a3576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161119a90614132565b60405180910390fd5b8060098190555050565b60135481565b6111bb6124ec565b73ffffffffffffffffffffffffffffffffffffffff166111d96117be565b73ffffffffffffffffffffffffffffffffffffffff161461122f576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161122690614132565b60405180910390fd5b80600e8190555050565b60166020528060005260406000206000915090505481565b600f805461125e9061447c565b80601f016020809104026020016040519081016040528092919081815260200182805461128a9061447c565b80156112d75780601f106112ac576101008083540402835291602001916112d7565b820191906000526020600020905b8154815290600101906020018083116112ba57829003601f168201915b505050505081565b600d5481565b6112ed6124ec565b73ffffffffffffffffffffffffffffffffffffffff1661130b6117be565b73ffffffffffffffffffffffffffffffffffffffff1614611361576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161135890614132565b60405180910390fd5b8181600f9190611372929190613666565b505050565b61137f6124ec565b73ffffffffffffffffffffffffffffffffffffffff1661139d6117be565b73ffffffffffffffffffffffffffffffffffffffff16146113f3576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016113ea90614132565b60405180910390fd5b80601260016101000a81548160ff02191690831515021790555050565b60145481565b601180546114239061447c565b80601f016020809104026020016040519081016040528092919081815260200182805461144f9061447c565b801561149c5780601f106114715761010080835404028352916020019161149c565b820191906000526020600020905b81548152906001019060200180831161147f57829003601f168201915b505050505081565b60006114af82612aee565b600001519050919050565b601080546114c79061447c565b80601f01602080910402602001604051908101604052809291908181526020018280546114f39061447c565b80156115405780601f1061151557610100808354040283529160200191611540565b820191906000526020600020905b81548152906001019060200180831161152357829003601f168201915b505050505081565b60008073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff1614156115b0576040517f8f4eb60400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600560008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160009054906101000a900467ffffffffffffffff1667ffffffffffffffff169050919050565b6116206124ec565b73ffffffffffffffffffffffffffffffffffffffff1661163e6117be565b73ffffffffffffffffffffffffffffffffffffffff1614611694576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161168b90614132565b60405180910390fd5b61169e6000612d7d565b565b600080836040516020016116b49190613f87565b604051602081830303815290604052805190602001209050601260019054906101000a900460ff16156116ec57600b5491505061172c565b6116f98360145483612e43565b156117095760095491505061172c565b6117168360155483612e43565b1561172657600a5491505061172c565b60009150505b92915050565b61173a6124ec565b73ffffffffffffffffffffffffffffffffffffffff166117586117be565b73ffffffffffffffffffffffffffffffffffffffff16146117ae576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016117a590614132565b60405180910390fd5b80600b8190555050565b600e5481565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b6117f06124ec565b73ffffffffffffffffffffffffffffffffffffffff1661180e6117be565b73ffffffffffffffffffffffffffffffffffffffff1614611864576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161185b90614132565b60405180910390fd5b818160119190611875929190613666565b505050565b600a5481565b60606003805461188f9061447c565b80601f01602080910402602001604051908101604052809291908181526020018280546118bb9061447c565b80156119085780601f106118dd57610100808354040283529160200191611908565b820191906000526020600020905b8154815290600101906020018083116118eb57829003601f168201915b5050505050905090565b61191a6124ec565b73ffffffffffffffffffffffffffffffffffffffff166119386117be565b73ffffffffffffffffffffffffffffffffffffffff161461198e576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161198590614132565b60405180910390fd5b8060148190555050565b6119a06124ec565b73ffffffffffffffffffffffffffffffffffffffff166119be6117be565b73ffffffffffffffffffffffffffffffffffffffff1614611a14576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611a0b90614132565b60405180910390fd5b8060158190555050565b600c5481565b611a2c6124ec565b73ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415611a91576040517fb06307db00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8060076000611a9e6124ec565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060006101000a81548160ff0219169083151502179055508173ffffffffffffffffffffffffffffffffffffffff16611b4b6124ec565b73ffffffffffffffffffffffffffffffffffffffff167f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c3183604051611b90919061403a565b60405180910390a35050565b61177081565b60155481565b60008083604051602001611bbc9190613f87565b604051602081830303815290604052805190602001209050601260019054906101000a900460ff1615611bf457600e54915050611c34565b611c018360145483612e43565b15611c1157600c54915050611c34565b611c1e8360155483612e43565b15611c2e57600d54915050611c34565b60009150505b92915050565b601260009054906101000a900460ff1681565b600181565b60008083604051602001611c669190613f87565b604051602081830303815290604052805190602001209050611c8b8360145483612e43565b80611c9f5750611c9e8360155483612e43565b5b91505092915050565b611cb38484846125fd565b611cd28373ffffffffffffffffffffffffffffffffffffffff16612e5a565b8015611ce75750611ce584848484612e7d565b155b15611d1e576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b50505050565b81611d2f3383611ba8565b611d39919061432e565b341015611d7b576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611d72906140f2565b60405180910390fd5b601260009054906101000a900460ff16611dca576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611dc190614092565b60405180910390fd5b601260019054906101000a900460ff1680611deb5750611dea3382611c52565b5b611e2a576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611e2190614112565b60405180910390fd5b611e3433826116a0565b821115611e76576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611e6d906140b2565b60405180910390fd5b61177082601354611e8791906142a7565b1115611ec8576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611ebf90614172565b60405180910390fd5b601260019054906101000a900460ff1680611f365750611ee833826116a0565b82601660003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054611f3391906142a7565b11155b611f75576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611f6c90614192565b60405180910390fd5b611f7f3383612fdd565b601260019054906101000a900460ff16611fea5781601660003373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254611fe291906142a7565b925050819055505b8160136000828254611ffc91906142a7565b925050819055505050565b61200f6124ec565b73ffffffffffffffffffffffffffffffffffffffff1661202d6117be565b73ffffffffffffffffffffffffffffffffffffffff1614612083576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161207a90614132565b60405180910390fd5b80601260006101000a81548160ff02191690831515021790555050565b60606120ab826124f4565b6120ea576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016120e190614152565b60405180910390fd5b60006120f4612ffb565b9050600081511161218f576010805461210c9061447c565b80601f01602080910402602001604051908101604052809291908181526020018280546121389061447c565b80156121855780601f1061215a57610100808354040283529160200191612185565b820191906000526020600020905b81548152906001019060200180831161216857829003601f168201915b50505050506121bd565b806121998461308d565b60116040516020016121ad93929190613fa2565b6040516020818303038152906040525b915050919050565b6000600760008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff16905092915050565b6122616124ec565b73ffffffffffffffffffffffffffffffffffffffff1661227f6117be565b73ffffffffffffffffffffffffffffffffffffffff16146122d5576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016122cc90614132565b60405180910390fd5b80600c8190555050565b6122e76124ec565b73ffffffffffffffffffffffffffffffffffffffff166123056117be565b73ffffffffffffffffffffffffffffffffffffffff161461235b576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161235290614132565b60405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff1614156123cb576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016123c2906140d2565b60405180910390fd5b6123d481612d7d565b50565b60095481565b601260019054906101000a900460ff1681565b6123f86124ec565b73ffffffffffffffffffffffffffffffffffffffff166124166117be565b73ffffffffffffffffffffffffffffffffffffffff161461246c576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161246390614132565b60405180910390fd5b81816010919061247d929190613666565b505050565b60007f01ffc9a7000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916149050919050565b600033905090565b6000816124ff6125f4565b1115801561250e575060005482105b801561253b575060046000838152602001908152602001600020600001601c9054906101000a900460ff16155b9050919050565b826006600084815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550818373ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff167f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92560405160405180910390a4505050565b60006001905090565b600061260882612aee565b90506000816000015173ffffffffffffffffffffffffffffffffffffffff1661262f6124ec565b73ffffffffffffffffffffffffffffffffffffffff1614806126625750612661826000015161265c6124ec565b6121c5565b5b806126a757506126706124ec565b73ffffffffffffffffffffffffffffffffffffffff1661268f84610e97565b73ffffffffffffffffffffffffffffffffffffffff16145b9050806126e0576040517f59c896be00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8473ffffffffffffffffffffffffffffffffffffffff16826000015173ffffffffffffffffffffffffffffffffffffffff1614612749576040517fa114810000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff1614156127b0576040517fea553b3400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6127bd85858560016131ee565b6127cd6000848460000151612542565b6001600560008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160392506101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055506001600560008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff160217905550836004600085815260200190815260200160002060000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550426004600085815260200190815260200160002060000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055506000600184019050600073ffffffffffffffffffffffffffffffffffffffff166004600083815260200190815260200160002060000160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff161415612a7e57600054811015612a7d5782600001516004600083815260200190815260200160002060000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555082602001516004600083815260200190815260200160002060000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055505b5b50828473ffffffffffffffffffffffffffffffffffffffff168673ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4612ae785858560016131f4565b5050505050565b612af66136ec565b600082905080612b046125f4565b11158015612b13575060005481105b15612d46576000600460008381526020019081526020016000206040518060600160405290816000820160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020016000820160149054906101000a900467ffffffffffffffff1667ffffffffffffffff1667ffffffffffffffff16815260200160008201601c9054906101000a900460ff16151515158152505090508060400151612d4457600073ffffffffffffffffffffffffffffffffffffffff16816000015173ffffffffffffffffffffffffffffffffffffffff1614612c28578092505050612d78565b5b600115612d4357818060019003925050600460008381526020019081526020016000206040518060600160405290816000820160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020016000820160149054906101000a900467ffffffffffffffff1667ffffffffffffffff1667ffffffffffffffff16815260200160008201601c9054906101000a900460ff1615151515815250509050600073ffffffffffffffffffffffffffffffffffffffff16816000015173ffffffffffffffffffffffffffffffffffffffff1614612d3e578092505050612d78565b612c29565b5b505b6040517fdf2d9b4200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b919050565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b600082612e5085846131fa565b1490509392505050565b6000808273ffffffffffffffffffffffffffffffffffffffff163b119050919050565b60008373ffffffffffffffffffffffffffffffffffffffff1663150b7a02612ea36124ec565b8786866040518563ffffffff1660e01b8152600401612ec59493929190613fee565b602060405180830381600087803b158015612edf57600080fd5b505af1925050508015612f1057506040513d601f19601f82011682018060405250810190612f0d9190613bd4565b60015b612f8a573d8060008114612f40576040519150601f19603f3d011682016040523d82523d6000602084013e612f45565b606091505b50600081511415612f82576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b805181602001fd5b63150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916817bffffffffffffffffffffffffffffffffffffffffffffffffffffffff191614915050949350505050565b612ff782826040518060200160405280600081525061326f565b5050565b6060600f805461300a9061447c565b80601f01602080910402602001604051908101604052809291908181526020018280546130369061447c565b80156130835780601f1061305857610100808354040283529160200191613083565b820191906000526020600020905b81548152906001019060200180831161306657829003601f168201915b5050505050905090565b606060008214156130d5576040518060400160405280600181526020017f300000000000000000000000000000000000000000000000000000000000000081525090506131e9565b600082905060005b600082146131075780806130f0906144df565b915050600a8261310091906142fd565b91506130dd565b60008167ffffffffffffffff81111561312357613122614639565b5b6040519080825280601f01601f1916602001820160405280156131555781602001600182028036833780820191505090505b5090505b600085146131e25760018261316e9190614388565b9150600a8561317d919061454c565b603061318991906142a7565b60f81b81838151811061319f5761319e61460a565b5b60200101907effffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916908160001a905350600a856131db91906142fd565b9450613159565b8093505050505b919050565b50505050565b50505050565b60008082905060005b84518110156132645760008582815181106132215761322061460a565b5b602002602001015190508083116132435761323c8382613281565b9250613250565b61324d8184613281565b92505b50808061325c906144df565b915050613203565b508091505092915050565b61327c8383836001613298565b505050565b600082600052816020526040600020905092915050565b600080549050600073ffffffffffffffffffffffffffffffffffffffff168573ffffffffffffffffffffffffffffffffffffffff161415613305576040517f2e07630000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6000841415613340576040517fb562e8dd00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b61334d60008683876131ee565b83600560008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff16021790555083600560008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160088282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff160217905550846004600083815260200190815260200160002060000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550426004600083815260200190815260200160002060000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff16021790555060008190506000858201905083801561351757506135168773ffffffffffffffffffffffffffffffffffffffff16612e5a565b5b156135dd575b818773ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a461358c6000888480600101955088612e7d565b6135c2576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8082141561351d5782600054146135d857600080fd5b613649565b5b818060010192508773ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4808214156135de575b81600081905550505061365f60008683876131f4565b5050505050565b8280546136729061447c565b90600052602060002090601f01602090048101928261369457600085556136db565b82601f106136ad57803560ff19168380011785556136db565b828001600101855582156136db579182015b828111156136da5782358255916020019190600101906136bf565b5b5090506136e8919061372f565b5090565b6040518060600160405280600073ffffffffffffffffffffffffffffffffffffffff168152602001600067ffffffffffffffff1681526020016000151581525090565b5b80821115613748576000816000905550600101613730565b5090565b600061375f61375a846141f2565b6141cd565b9050808382526020820190508285602086028201111561378257613781614672565b5b60005b858110156137b257816137988882613856565b845260208401935060208301925050600181019050613785565b5050509392505050565b60006137cf6137ca8461421e565b6141cd565b9050828152602081018484840111156137eb576137ea614677565b5b6137f684828561443a565b509392505050565b60008135905061380d816148d3565b92915050565b600082601f8301126138285761382761466d565b5b813561383884826020860161374c565b91505092915050565b600081359050613850816148ea565b92915050565b60008135905061386581614901565b92915050565b60008135905061387a81614918565b92915050565b60008151905061388f81614918565b92915050565b600082601f8301126138aa576138a961466d565b5b81356138ba8482602086016137bc565b91505092915050565b60008083601f8401126138d9576138d861466d565b5b8235905067ffffffffffffffff8111156138f6576138f5614668565b5b60208301915083600182028301111561391257613911614672565b5b9250929050565b6000813590506139288161492f565b92915050565b60006020828403121561394457613943614681565b5b6000613952848285016137fe565b91505092915050565b6000806040838503121561397257613971614681565b5b6000613980858286016137fe565b9250506020613991858286016137fe565b9150509250929050565b6000806000606084860312156139b4576139b3614681565b5b60006139c2868287016137fe565b93505060206139d3868287016137fe565b92505060406139e486828701613919565b9150509250925092565b60008060008060808587031215613a0857613a07614681565b5b6000613a16878288016137fe565b9450506020613a27878288016137fe565b9350506040613a3887828801613919565b925050606085013567ffffffffffffffff811115613a5957613a5861467c565b5b613a6587828801613895565b91505092959194509250565b60008060408385031215613a8857613a87614681565b5b6000613a96858286016137fe565b925050602083013567ffffffffffffffff811115613ab757613ab661467c565b5b613ac385828601613813565b9150509250929050565b60008060408385031215613ae457613ae3614681565b5b6000613af2858286016137fe565b9250506020613b0385828601613841565b9150509250929050565b60008060408385031215613b2457613b23614681565b5b6000613b32858286016137fe565b9250506020613b4385828601613919565b9150509250929050565b600060208284031215613b6357613b62614681565b5b6000613b7184828501613841565b91505092915050565b600060208284031215613b9057613b8f614681565b5b6000613b9e84828501613856565b91505092915050565b600060208284031215613bbd57613bbc614681565b5b6000613bcb8482850161386b565b91505092915050565b600060208284031215613bea57613be9614681565b5b6000613bf884828501613880565b91505092915050565b60008060208385031215613c1857613c17614681565b5b600083013567ffffffffffffffff811115613c3657613c3561467c565b5b613c42858286016138c3565b92509250509250929050565b600060208284031215613c6457613c63614681565b5b6000613c7284828501613919565b91505092915050565b60008060408385031215613c9257613c91614681565b5b6000613ca085828601613919565b925050602083013567ffffffffffffffff811115613cc157613cc061467c565b5b613ccd85828601613813565b9150509250929050565b613ce0816143bc565b82525050565b613cf7613cf2826143bc565b614528565b82525050565b613d06816143ce565b82525050565b613d15816143da565b82525050565b6000613d2682614264565b613d30818561427a565b9350613d40818560208601614449565b613d4981614686565b840191505092915050565b6000613d5f8261426f565b613d69818561428b565b9350613d79818560208601614449565b613d8281614686565b840191505092915050565b6000613d988261426f565b613da2818561429c565b9350613db2818560208601614449565b80840191505092915050565b60008154613dcb8161447c565b613dd5818661429c565b94506001821660008114613df05760018114613e0157613e34565b60ff19831686528186019350613e34565b613e0a8561424f565b60005b83811015613e2c57815481890152600182019150602081019050613e0d565b838801955050505b50505092915050565b6000613e4a601a8361428b565b9150613e55826146a4565b602082019050919050565b6000613e6d602d8361428b565b9150613e78826146cd565b604082019050919050565b6000613e9060268361428b565b9150613e9b8261471c565b604082019050919050565b6000613eb3600d8361428b565b9150613ebe8261476b565b602082019050919050565b6000613ed660218361428b565b9150613ee182614794565b604082019050919050565b6000613ef960208361428b565b9150613f04826147e3565b602082019050919050565b6000613f1c602f8361428b565b9150613f278261480c565b604082019050919050565b6000613f3f601a8361428b565b9150613f4a8261485b565b602082019050919050565b6000613f62603c8361428b565b9150613f6d82614884565b604082019050919050565b613f8181614430565b82525050565b6000613f938284613ce6565b60148201915081905092915050565b6000613fae8286613d8d565b9150613fba8285613d8d565b9150613fc68284613dbe565b9150819050949350505050565b6000602082019050613fe86000830184613cd7565b92915050565b60006080820190506140036000830187613cd7565b6140106020830186613cd7565b61401d6040830185613f78565b818103606083015261402f8184613d1b565b905095945050505050565b600060208201905061404f6000830184613cfd565b92915050565b600060208201905061406a6000830184613d0c565b92915050565b6000602082019050818103600083015261408a8184613d54565b905092915050565b600060208201905081810360008301526140ab81613e3d565b9050919050565b600060208201905081810360008301526140cb81613e60565b9050919050565b600060208201905081810360008301526140eb81613e83565b9050919050565b6000602082019050818103600083015261410b81613ea6565b9050919050565b6000602082019050818103600083015261412b81613ec9565b9050919050565b6000602082019050818103600083015261414b81613eec565b9050919050565b6000602082019050818103600083015261416b81613f0f565b9050919050565b6000602082019050818103600083015261418b81613f32565b9050919050565b600060208201905081810360008301526141ab81613f55565b9050919050565b60006020820190506141c76000830184613f78565b92915050565b60006141d76141e8565b90506141e382826144ae565b919050565b6000604051905090565b600067ffffffffffffffff82111561420d5761420c614639565b5b602082029050602081019050919050565b600067ffffffffffffffff82111561423957614238614639565b5b61424282614686565b9050602081019050919050565b60008190508160005260206000209050919050565b600081519050919050565b600081519050919050565b600082825260208201905092915050565b600082825260208201905092915050565b600081905092915050565b60006142b282614430565b91506142bd83614430565b9250827fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff038211156142f2576142f161457d565b5b828201905092915050565b600061430882614430565b915061431383614430565b925082614323576143226145ac565b5b828204905092915050565b600061433982614430565b915061434483614430565b9250817fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff048311821515161561437d5761437c61457d565b5b828202905092915050565b600061439382614430565b915061439e83614430565b9250828210156143b1576143b061457d565b5b828203905092915050565b60006143c782614410565b9050919050565b60008115159050919050565b6000819050919050565b60007fffffffff0000000000000000000000000000000000000000000000000000000082169050919050565b600073ffffffffffffffffffffffffffffffffffffffff82169050919050565b6000819050919050565b82818337600083830152505050565b60005b8381101561446757808201518184015260208101905061444c565b83811115614476576000848401525b50505050565b6000600282049050600182168061449457607f821691505b602082108114156144a8576144a76145db565b5b50919050565b6144b782614686565b810181811067ffffffffffffffff821117156144d6576144d5614639565b5b80604052505050565b60006144ea82614430565b91507fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff82141561451d5761451c61457d565b5b600182019050919050565b60006145338261453a565b9050919050565b600061454582614697565b9050919050565b600061455782614430565b915061456283614430565b925082614572576145716145ac565b5b828206905092915050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b600080fd5b600080fd5b600080fd5b600080fd5b600080fd5b600080fd5b6000601f19601f8301169050919050565b60008160601b9050919050565b7f43616e6e6f74206d696e74206265666f72652070726573616c65000000000000600082015250565b7f43616e6e6f74206d696e74206d6f7265207468616e20746865206d617820746f60008201527f6b656e7320706572206d696e7400000000000000000000000000000000000000602082015250565b7f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160008201527f6464726573730000000000000000000000000000000000000000000000000000602082015250565b7f496e636f72726563742045544800000000000000000000000000000000000000600082015250565b7f4275796572206e6f742077686974656c697374656420666f722070726573616c60008201527f6500000000000000000000000000000000000000000000000000000000000000602082015250565b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b7f4552433732314d657461646174613a2055524920717565727920666f72206e6f60008201527f6e6578697374656e7420746f6b656e0000000000000000000000000000000000602082015250565b7f4e6f20746f6b656e73206c65667420666f72206d696e74696e67000000000000600082015250565b7f43616e6e6f74206d696e74206d6f7265207468616e20746865206d617820746f60008201527f6b656e73207065722077686974656c6973746564206164647265737300000000602082015250565b6148dc816143bc565b81146148e757600080fd5b50565b6148f3816143ce565b81146148fe57600080fd5b50565b61490a816143da565b811461491557600080fd5b50565b614921816143e4565b811461492c57600080fd5b50565b61493881614430565b811461494357600080fd5b5056fea2646970667358221220a137902ff01c4043f1820d1de508c92bd130a0eb471ec1dfad4606c141c9b55e64736f6c63430008070033

Deployed Bytecode Sourcemap

79446:5728:0:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;61908:305;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;81357:142;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;80963:116;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;65293:100;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;66796:204;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;66359:371;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;79651:35;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;61157:303;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;67653:170;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;85055:114;;;;;;;;;;;;;:::i;:::-;;67894:185;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;81209:140;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;80186:31;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;81091:110;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;80441:60;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;79868:31;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;79752:51;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;84618:97;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;83065;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;80226:100;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;79945:36;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;65102:124;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;79906:32;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;62277:206;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;16686:103;;;;;;;;;;;;;:::i;:::-;;82312:536;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;82856:102;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;79811:48;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;16035:87;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;84835:102;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;79589:55;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;65462:104;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;80571:126;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;80705:128;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;79695:50;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;67072:279;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;80132:47;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;80333:101;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;81799:505;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;79990:37;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;80083:42;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;81507:284;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;68150:369;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;83170:948;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;82966:91;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;84248:359;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;67422:164;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;80841:114;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;16944:201;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;79528:54;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;80034:40;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;84723:104;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;61908:305;62010:4;62062:25;62047:40;;;:11;:40;;;;:105;;;;62119:33;62104:48;;;:11;:48;;;;62047:105;:158;;;;62169:36;62193:11;62169:23;:36::i;:::-;62047:158;62027:178;;61908:305;;;:::o;81357:142::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;81488:3:::1;81449:36;:42;;;;81357:142:::0;:::o;80963:116::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;81068:3:::1;81042:23;:29;;;;80963:116:::0;:::o;65293:100::-;65347:13;65380:5;65373:12;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;65293:100;:::o;66796:204::-;66864:7;66889:16;66897:7;66889;:16::i;:::-;66884:64;;66914:34;;;;;;;;;;;;;;66884:64;66968:15;:24;66984:7;66968:24;;;;;;;;;;;;;;;;;;;;;66961:31;;66796:204;;;:::o;66359:371::-;66432:13;66448:24;66464:7;66448:15;:24::i;:::-;66432:40;;66493:5;66487:11;;:2;:11;;;66483:48;;;66507:24;;;;;;;;;;;;;;66483:48;66564:5;66548:21;;:12;:10;:12::i;:::-;:21;;;;:63;;;;;66574:37;66591:5;66598:12;:10;:12::i;:::-;66574:16;:37::i;:::-;66573:38;66548:63;66544:138;;;66635:35;;;;;;;;;;;;;;66544:138;66694:28;66703:2;66707:7;66716:5;66694:8;:28::i;:::-;66421:309;66359:371;;:::o;79651:35::-;;;;:::o;61157:303::-;61201:7;61426:15;:13;:15::i;:::-;61411:12;;61395:13;;:28;:46;61388:53;;61157:303;:::o;67653:170::-;67787:28;67797:4;67803:2;67807:7;67787:9;:28::i;:::-;67653:170;;;:::o;85055:114::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;85121:10:::1;85113:24;;:47;85138:21;85113:47;;;;;;;;;;;;;;;;;;;;;;;85105:56;;;::::0;::::1;;85055:114::o:0;67894:185::-;68032:39;68049:4;68055:2;68059:7;68032:39;;;;;;;;;;;;:16;:39::i;:::-;67894:185;;;:::o;81209:140::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;81338:3:::1;81300:35;:41;;;;81209:140:::0;:::o;80186:31::-;;;;:::o;81091:110::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;81190:3:::1;81167:20;:26;;;;81091:110:::0;:::o;80441:60::-;;;;;;;;;;;;;;;;;:::o;79868:31::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;79752:51::-;;;;:::o;84618:97::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;84704:3:::1;;84689:12;:18;;;;;;;:::i;:::-;;84618:97:::0;;:::o;83065:::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;83151:3:::1;83128:20;;:26;;;;;;;;;;;;;;;;;;83065:97:::0;:::o;80226:100::-;;;;:::o;79945:36::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;65102:124::-;65166:7;65193:20;65205:7;65193:11;:20::i;:::-;:25;;;65186:32;;65102:124;;;:::o;79906:32::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;62277:206::-;62341:7;62382:1;62365:19;;:5;:19;;;62361:60;;;62393:28;;;;;;;;;;;;;;62361:60;62447:12;:19;62460:5;62447:19;;;;;;;;;;;;;;;:27;;;;;;;;;;;;62439:36;;62432:43;;62277:206;;;:::o;16686:103::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;16751:30:::1;16778:1;16751:18;:30::i;:::-;16686:103::o:0;82312:536::-;82402:7;82422:12;82464:6;82447:24;;;;;;;;:::i;:::-;;;;;;;;;;;;;82437:35;;;;;;82422:50;;82487:20;;;;;;;;;;;82483:339;;;82531:16;;82524:23;;;;;82483:339;82567:51;82586:5;82593:18;;82613:4;82567:18;:51::i;:::-;82564:258;;;82642:35;;82635:42;;;;;82564:258;82698:52;82717:5;82724:19;;82745:4;82698:18;:52::i;:::-;82694:128;;;82774:36;;82767:43;;;;;82694:128;82839:1;82832:8;;;82312:536;;;;;:::o;82856:102::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;82947:3:::1;82928:16;:22;;;;82856:102:::0;:::o;79811:48::-;;;;:::o;16035:87::-;16081:7;16108:6;;;;;;;;;;;16101:13;;16035:87;:::o;84835:102::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;84926:3:::1;;84911:12;:18;;;;;;;:::i;:::-;;84835:102:::0;;:::o;79589:55::-;;;;:::o;65462:104::-;65518:13;65551:7;65544:14;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;65462:104;:::o;80571:126::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;80675:14:::1;80654:18;:35;;;;80571:126:::0;:::o;80705:128::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;80811:14:::1;80789:19;:36;;;;80705:128:::0;:::o;79695:50::-;;;;:::o;67072:279::-;67175:12;:10;:12::i;:::-;67163:24;;:8;:24;;;67159:54;;;67196:17;;;;;;;;;;;;;;67159:54;67271:8;67226:18;:32;67245:12;:10;:12::i;:::-;67226:32;;;;;;;;;;;;;;;:42;67259:8;67226:42;;;;;;;;;;;;;;;;:53;;;;;;;;;;;;;;;;;;67324:8;67295:48;;67310:12;:10;:12::i;:::-;67295:48;;;67334:8;67295:48;;;;;;:::i;:::-;;;;;;;;67072:279;;:::o;80132:47::-;80175:4;80132:47;:::o;80333:101::-;;;;:::o;81799:505::-;81880:7;81900:12;81942:6;81925:24;;;;;;;;:::i;:::-;;;;;;;;;;;;;81915:35;;;;;;81900:50;;81965:20;;;;;;;;;;;81961:317;;;82009:20;;82002:27;;;;;81961:317;82049:51;82068:5;82075:18;;82095:4;82049:18;:51::i;:::-;82046:232;;;82124:22;;82117:29;;;;;82046:232;82167:52;82186:5;82193:19;;82214:4;82167:18;:52::i;:::-;82163:115;;;82243:23;;82236:30;;;;;82163:115;82295:1;82288:8;;;81799:505;;;;;:::o;79990:37::-;;;;;;;;;;;;;:::o;80083:42::-;80124:1;80083:42;:::o;81507:284::-;81585:4;81607:12;81649:7;81632:25;;;;;;;;:::i;:::-;;;;;;;;;;;;;81622:36;;;;;;81607:51;;81676;81695:5;81702:18;;81722:4;81676:18;:51::i;:::-;:107;;;;81731:52;81750:5;81757:19;;81778:4;81731:18;:52::i;:::-;81676:107;81669:114;;;81507:284;;;;:::o;68150:369::-;68317:28;68327:4;68333:2;68337:7;68317:9;:28::i;:::-;68360:15;:2;:13;;;:15::i;:::-;:76;;;;;68380:56;68411:4;68417:2;68421:7;68430:5;68380:30;:56::i;:::-;68379:57;68360:76;68356:156;;;68460:40;;;;;;;;;;;;;;68356:156;68150:369;;;;:::o;83170:948::-;83305:6;83273:29;83284:10;83296:5;83273:10;:29::i;:::-;:38;;;;:::i;:::-;83260:9;:51;;83252:77;;;;;;;;;;;;:::i;:::-;;;;;;;;;83348:17;;;;;;;;;;;83340:56;;;;;;;;;;;;:::i;:::-;;;;;;;;;83415:20;;;;;;;;;;;:49;;;;83439:25;83446:10;83458:5;83439:6;:25::i;:::-;83415:49;83407:95;;;;;;;;;;;;:::i;:::-;;;;;;;;;83531:38;83551:10;83563:5;83531:19;:38::i;:::-;83521:6;:48;;83513:106;;;;;;;;;;;;:::i;:::-;;;;;;;;;80175:4;83653:6;83638:12;;:21;;;;:::i;:::-;:41;;83630:80;;;;;;;;;;;;:::i;:::-;;;;;;;;;83729:20;;;;;;;;;;;:114;;;;83804:38;83824:10;83836:5;83804:19;:38::i;:::-;83794:6;83754:25;:37;83780:10;83754:37;;;;;;;;;;;;;;;;:46;;;;:::i;:::-;:88;;83729:114;83721:198;;;;;;;;;;;;:::i;:::-;;;;;;;;;83933:29;83943:10;83955:6;83933:9;:29::i;:::-;83980:20;;;;;;;;;;;83975:101;;84058:6;84017:25;:37;84043:10;84017:37;;;;;;;;;;;;;;;;:47;;;;;;;:::i;:::-;;;;;;;;83975:101;84104:6;84088:12;;:22;;;;;;;:::i;:::-;;;;;;;;83170:948;;:::o;82966:91::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;83046:3:::1;83026:17;;:23;;;;;;;;;;;;;;;;;;82966:91:::0;:::o;84248:359::-;84322:13;84356:16;84364:7;84356;:16::i;:::-;84348:76;;;;;;;;;;;;:::i;:::-;;;;;;;;;84435:21;84459:10;:8;:10::i;:::-;84435:34;;84512:1;84494:7;84488:21;:25;:111;;84586:13;84488:111;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;84540:7;84549:18;:7;:16;:18::i;:::-;84569:12;84523:59;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;84488:111;84481:118;;;84248:359;;;:::o;67422:164::-;67519:4;67543:18;:25;67562:5;67543:25;;;;;;;;;;;;;;;:35;67569:8;67543:35;;;;;;;;;;;;;;;;;;;;;;;;;67536:42;;67422:164;;;;:::o;80841:114::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;80944:3:::1;80919:22;:28;;;;80841:114:::0;:::o;16944:201::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;17053:1:::1;17033:22;;:8;:22;;;;17025:73;;;;;;;;;;;;:::i;:::-;;;;;;;;;17109:28;17128:8;17109:18;:28::i;:::-;16944:201:::0;:::o;79528:54::-;;;;:::o;80034:40::-;;;;;;;;;;;;;:::o;84723:104::-;16266:12;:10;:12::i;:::-;16255:23;;:7;:5;:7::i;:::-;:23;;;16247:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;84816:3:::1;;84800:13;:19;;;;;;;:::i;:::-;;84723:104:::0;;:::o;28819:157::-;28904:4;28943:25;28928:40;;;:11;:40;;;;28921:47;;28819:157;;;:::o;14759:98::-;14812:7;14839:10;14832:17;;14759:98;:::o;68774:187::-;68831:4;68874:7;68855:15;:13;:15::i;:::-;:26;;:53;;;;;68895:13;;68885:7;:23;68855:53;:98;;;;;68926:11;:20;68938:7;68926:20;;;;;;;;;;;:27;;;;;;;;;;;;68925:28;68855:98;68848:105;;68774:187;;;:::o;76385:196::-;76527:2;76500:15;:24;76516:7;76500:24;;;;;;;;;;;;:29;;;;;;;;;;;;;;;;;;76565:7;76561:2;76545:28;;76554:5;76545:28;;;;;;;;;;;;76385:196;;;:::o;84945:102::-;85011:7;85038:1;85031:8;;84945:102;:::o;71887:2112::-;72002:35;72040:20;72052:7;72040:11;:20::i;:::-;72002:58;;72073:22;72115:13;:18;;;72099:34;;:12;:10;:12::i;:::-;:34;;;:101;;;;72150:50;72167:13;:18;;;72187:12;:10;:12::i;:::-;72150:16;:50::i;:::-;72099:101;:154;;;;72241:12;:10;:12::i;:::-;72217:36;;:20;72229:7;72217:11;:20::i;:::-;:36;;;72099:154;72073:181;;72272:17;72267:66;;72298:35;;;;;;;;;;;;;;72267:66;72370:4;72348:26;;:13;:18;;;:26;;;72344:67;;72383:28;;;;;;;;;;;;;;72344:67;72440:1;72426:16;;:2;:16;;;72422:52;;;72451:23;;;;;;;;;;;;;;72422:52;72487:43;72509:4;72515:2;72519:7;72528:1;72487:21;:43::i;:::-;72595:49;72612:1;72616:7;72625:13;:18;;;72595:8;:49::i;:::-;72970:1;72940:12;:18;72953:4;72940:18;;;;;;;;;;;;;;;:26;;;:31;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;73014:1;72986:12;:16;72999:2;72986:16;;;;;;;;;;;;;;;:24;;;:29;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;73060:2;73032:11;:20;73044:7;73032:20;;;;;;;;;;;:25;;;:30;;;;;;;;;;;;;;;;;;73122:15;73077:11;:20;73089:7;73077:20;;;;;;;;;;;:35;;;:61;;;;;;;;;;;;;;;;;;73390:19;73422:1;73412:7;:11;73390:33;;73483:1;73442:43;;:11;:24;73454:11;73442:24;;;;;;;;;;;:29;;;;;;;;;;;;:43;;;73438:445;;;73667:13;;73653:11;:27;73649:219;;;73737:13;:18;;;73705:11;:24;73717:11;73705:24;;;;;;;;;;;:29;;;:50;;;;;;;;;;;;;;;;;;73820:13;:28;;;73778:11;:24;73790:11;73778:24;;;;;;;;;;;:39;;;:70;;;;;;;;;;;;;;;;;;73649:219;73438:445;72915:979;73930:7;73926:2;73911:27;;73920:4;73911:27;;;;;;;;;;;;73949:42;73970:4;73976:2;73980:7;73989:1;73949:20;:42::i;:::-;71991:2008;;71887:2112;;;:::o;63932:1108::-;63993:21;;:::i;:::-;64027:12;64042:7;64027:22;;64110:4;64091:15;:13;:15::i;:::-;:23;;:47;;;;;64125:13;;64118:4;:20;64091:47;64087:886;;;64159:31;64193:11;:17;64205:4;64193:17;;;;;;;;;;;64159:51;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;64234:9;:16;;;64229:729;;64305:1;64279:28;;:9;:14;;;:28;;;64275:101;;64343:9;64336:16;;;;;;64275:101;64678:261;64685:4;64678:261;;;64718:6;;;;;;;;64763:11;:17;64775:4;64763:17;;;;;;;;;;;64751:29;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;64837:1;64811:28;;:9;:14;;;:28;;;64807:109;;64879:9;64872:16;;;;;;64807:109;64678:261;;;64229:729;64140:833;64087:886;65001:31;;;;;;;;;;;;;;63932:1108;;;;:::o;17305:191::-;17379:16;17398:6;;;;;;;;;;;17379:25;;17424:8;17415:6;;:17;;;;;;;;;;;;;;;;;;17479:8;17448:40;;17469:8;17448:40;;;;;;;;;;;;17368:128;17305:191;:::o;956:190::-;1081:4;1134;1105:25;1118:5;1125:4;1105:12;:25::i;:::-;:33;1098:40;;956:190;;;;;:::o;18736:326::-;18796:4;19053:1;19031:7;:19;;;:23;19024:30;;18736:326;;;:::o;77073:667::-;77236:4;77273:2;77257:36;;;77294:12;:10;:12::i;:::-;77308:4;77314:7;77323:5;77257:72;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;77253:480;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;77508:1;77491:6;:13;:18;77487:235;;;77537:40;;;;;;;;;;;;;;77487:235;77680:6;77674:13;77665:6;77661:2;77657:15;77650:38;77253:480;77386:45;;;77376:55;;;:6;:55;;;;77369:62;;;77073:667;;;;;;:::o;68969:104::-;69038:27;69048:2;69052:8;69038:27;;;;;;;;;;;;:9;:27::i;:::-;68969:104;;:::o;84126:114::-;84187:13;84220:12;84213:19;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;84126:114;:::o;2787:723::-;2843:13;3073:1;3064:5;:10;3060:53;;;3091:10;;;;;;;;;;;;;;;;;;;;;3060:53;3123:12;3138:5;3123:20;;3154:14;3179:78;3194:1;3186:4;:9;3179:78;;3212:8;;;;;:::i;:::-;;;;3243:2;3235:10;;;;;:::i;:::-;;;3179:78;;;3267:19;3299:6;3289:17;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;3267:39;;3317:154;3333:1;3324:5;:10;3317:154;;3361:1;3351:11;;;;;:::i;:::-;;;3428:2;3420:5;:10;;;;:::i;:::-;3407:2;:24;;;;:::i;:::-;3394:39;;3377:6;3384;3377:14;;;;;;;;:::i;:::-;;;;;:56;;;;;;;;;;;3457:2;3448:11;;;;;:::i;:::-;;;3317:154;;;3495:6;3481:21;;;;;2787:723;;;;:::o;78388:159::-;;;;;:::o;79206:158::-;;;;;:::o;1508:675::-;1591:7;1611:20;1634:4;1611:27;;1654:9;1649:497;1673:5;:12;1669:1;:16;1649:497;;;1707:20;1730:5;1736:1;1730:8;;;;;;;;:::i;:::-;;;;;;;;1707:31;;1773:12;1757;:28;1753:382;;1900:42;1915:12;1929;1900:14;:42::i;:::-;1885:57;;1753:382;;;2077:42;2092:12;2106;2077:14;:42::i;:::-;2062:57;;1753:382;1692:454;1687:3;;;;;:::i;:::-;;;;1649:497;;;;2163:12;2156:19;;;1508:675;;;;:::o;69436:163::-;69559:32;69565:2;69569:8;69579:5;69586:4;69559:5;:32::i;:::-;69436:163;;;:::o;2191:224::-;2259:13;2322:1;2316:4;2309:15;2351:1;2345:4;2338:15;2392:4;2386;2376:21;2367:30;;2191:224;;;;:::o;69858:1775::-;69997:20;70020:13;;69997:36;;70062:1;70048:16;;:2;:16;;;70044:48;;;70073:19;;;;;;;;;;;;;;70044:48;70119:1;70107:8;:13;70103:44;;;70129:18;;;;;;;;;;;;;;70103:44;70160:61;70190:1;70194:2;70198:12;70212:8;70160:21;:61::i;:::-;70533:8;70498:12;:16;70511:2;70498:16;;;;;;;;;;;;;;;:24;;;:44;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;70597:8;70557:12;:16;70570:2;70557:16;;;;;;;;;;;;;;;:29;;;:49;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;70656:2;70623:11;:25;70635:12;70623:25;;;;;;;;;;;:30;;;:35;;;;;;;;;;;;;;;;;;70723:15;70673:11;:25;70685:12;70673:25;;;;;;;;;;;:40;;;:66;;;;;;;;;;;;;;;;;;70756:20;70779:12;70756:35;;70806:11;70835:8;70820:12;:23;70806:37;;70864:4;:23;;;;;70872:15;:2;:13;;;:15::i;:::-;70864:23;70860:641;;;70908:314;70964:12;70960:2;70939:38;;70956:1;70939:38;;;;;;;;;;;;71005:69;71044:1;71048:2;71052:14;;;;;;71068:5;71005:30;:69::i;:::-;71000:174;;71110:40;;;;;;;;;;;;;;71000:174;71217:3;71201:12;:19;;70908:314;;71303:12;71286:13;;:29;71282:43;;71317:8;;;71282:43;70860:641;;;71366:120;71422:14;;;;;;71418:2;71397:40;;71414:1;71397:40;;;;;;;;;;;;71481:3;71465:12;:19;;71366:120;;70860:641;71531:12;71515:13;:28;;;;70473:1082;;71565:60;71594:1;71598:2;71602:12;71616:8;71565:20;:60::i;:::-;69986:1647;69858:1775;;;;:::o;-1:-1:-1:-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;:::o;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;:::-;;;;;;;;;;;;;;;;;;;;;:::o;24:722:1:-;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:143;;;404:79;;:::i;:::-;350:143;517:1;502:238;527:6;524:1;521:13;502:238;;;595:3;624:37;657:3;645:10;624:37;:::i;:::-;619:3;612:50;691:4;686:3;682:14;675:21;;725:4;720:3;716:14;709:21;;562:178;549:1;546;542:9;537:14;;502:238;;;506:14;126:620;;24:722;;;;;:::o;752:410::-;829:5;854:65;870:48;911:6;870:48;:::i;:::-;854:65;:::i;:::-;845:74;;942:6;935:5;928:21;980:4;973:5;969:16;1018:3;1009:6;1004:3;1000:16;997:25;994:112;;;1025:79;;:::i;:::-;994:112;1115:41;1149:6;1144:3;1139;1115:41;:::i;:::-;835:327;752:410;;;;;:::o;1168:139::-;1214:5;1252:6;1239:20;1230:29;;1268:33;1295:5;1268:33;:::i;:::-;1168:139;;;;:::o;1330:370::-;1401:5;1450:3;1443:4;1435:6;1431:17;1427:27;1417:122;;1458:79;;:::i;:::-;1417:122;1575:6;1562:20;1600:94;1690:3;1682:6;1675:4;1667:6;1663:17;1600:94;:::i;:::-;1591:103;;1407:293;1330:370;;;;:::o;1706:133::-;1749:5;1787:6;1774:20;1765:29;;1803:30;1827:5;1803:30;:::i;:::-;1706:133;;;;:::o;1845:139::-;1891:5;1929:6;1916:20;1907:29;;1945:33;1972:5;1945:33;:::i;:::-;1845:139;;;;:::o;1990:137::-;2035:5;2073:6;2060:20;2051:29;;2089:32;2115:5;2089:32;:::i;:::-;1990:137;;;;:::o;2133:141::-;2189:5;2220:6;2214:13;2205:22;;2236:32;2262:5;2236:32;:::i;:::-;2133:141;;;;:::o;2293:338::-;2348:5;2397:3;2390:4;2382:6;2378:17;2374:27;2364:122;;2405:79;;:::i;:::-;2364:122;2522:6;2509:20;2547:78;2621:3;2613:6;2606:4;2598:6;2594:17;2547:78;:::i;:::-;2538:87;;2354:277;2293:338;;;;:::o;2651:553::-;2709:8;2719:6;2769:3;2762:4;2754:6;2750:17;2746:27;2736:122;;2777:79;;:::i;:::-;2736:122;2890:6;2877:20;2867:30;;2920:18;2912:6;2909:30;2906:117;;;2942:79;;:::i;:::-;2906:117;3056:4;3048:6;3044:17;3032:29;;3110:3;3102:4;3094:6;3090:17;3080:8;3076:32;3073:41;3070:128;;;3117:79;;:::i;:::-;3070:128;2651:553;;;;;:::o;3210:139::-;3256:5;3294:6;3281:20;3272:29;;3310:33;3337:5;3310:33;:::i;:::-;3210:139;;;;:::o;3355:329::-;3414:6;3463:2;3451:9;3442:7;3438:23;3434:32;3431:119;;;3469:79;;:::i;:::-;3431:119;3589:1;3614:53;3659:7;3650:6;3639:9;3635:22;3614:53;:::i;:::-;3604:63;;3560:117;3355:329;;;;:::o;3690:474::-;3758:6;3766;3815:2;3803:9;3794:7;3790:23;3786:32;3783:119;;;3821:79;;:::i;:::-;3783:119;3941:1;3966:53;4011:7;4002:6;3991:9;3987:22;3966:53;:::i;:::-;3956:63;;3912:117;4068:2;4094:53;4139:7;4130:6;4119:9;4115:22;4094:53;:::i;:::-;4084:63;;4039:118;3690:474;;;;;:::o;4170:619::-;4247:6;4255;4263;4312:2;4300:9;4291:7;4287:23;4283:32;4280:119;;;4318:79;;:::i;:::-;4280:119;4438:1;4463:53;4508:7;4499:6;4488:9;4484:22;4463:53;:::i;:::-;4453:63;;4409:117;4565:2;4591:53;4636:7;4627:6;4616:9;4612:22;4591:53;:::i;:::-;4581:63;;4536:118;4693:2;4719:53;4764:7;4755:6;4744:9;4740:22;4719:53;:::i;:::-;4709:63;;4664:118;4170:619;;;;;:::o;4795:943::-;4890:6;4898;4906;4914;4963:3;4951:9;4942:7;4938:23;4934:33;4931:120;;;4970:79;;:::i;:::-;4931:120;5090:1;5115:53;5160:7;5151:6;5140:9;5136:22;5115:53;:::i;:::-;5105:63;;5061:117;5217:2;5243:53;5288:7;5279:6;5268:9;5264:22;5243:53;:::i;:::-;5233:63;;5188:118;5345:2;5371:53;5416:7;5407:6;5396:9;5392:22;5371:53;:::i;:::-;5361:63;;5316:118;5501:2;5490:9;5486:18;5473:32;5532:18;5524:6;5521:30;5518:117;;;5554:79;;:::i;:::-;5518:117;5659:62;5713:7;5704:6;5693:9;5689:22;5659:62;:::i;:::-;5649:72;;5444:287;4795:943;;;;;;;:::o;5744:684::-;5837:6;5845;5894:2;5882:9;5873:7;5869:23;5865:32;5862:119;;;5900:79;;:::i;:::-;5862:119;6020:1;6045:53;6090:7;6081:6;6070:9;6066:22;6045:53;:::i;:::-;6035:63;;5991:117;6175:2;6164:9;6160:18;6147:32;6206:18;6198:6;6195:30;6192:117;;;6228:79;;:::i;:::-;6192:117;6333:78;6403:7;6394:6;6383:9;6379:22;6333:78;:::i;:::-;6323:88;;6118:303;5744:684;;;;;:::o;6434:468::-;6499:6;6507;6556:2;6544:9;6535:7;6531:23;6527:32;6524:119;;;6562:79;;:::i;:::-;6524:119;6682:1;6707:53;6752:7;6743:6;6732:9;6728:22;6707:53;:::i;:::-;6697:63;;6653:117;6809:2;6835:50;6877:7;6868:6;6857:9;6853:22;6835:50;:::i;:::-;6825:60;;6780:115;6434:468;;;;;:::o;6908:474::-;6976:6;6984;7033:2;7021:9;7012:7;7008:23;7004:32;7001:119;;;7039:79;;:::i;:::-;7001:119;7159:1;7184:53;7229:7;7220:6;7209:9;7205:22;7184:53;:::i;:::-;7174:63;;7130:117;7286:2;7312:53;7357:7;7348:6;7337:9;7333:22;7312:53;:::i;:::-;7302:63;;7257:118;6908:474;;;;;:::o;7388:323::-;7444:6;7493:2;7481:9;7472:7;7468:23;7464:32;7461:119;;;7499:79;;:::i;:::-;7461:119;7619:1;7644:50;7686:7;7677:6;7666:9;7662:22;7644:50;:::i;:::-;7634:60;;7590:114;7388:323;;;;:::o;7717:329::-;7776:6;7825:2;7813:9;7804:7;7800:23;7796:32;7793:119;;;7831:79;;:::i;:::-;7793:119;7951:1;7976:53;8021:7;8012:6;8001:9;7997:22;7976:53;:::i;:::-;7966:63;;7922:117;7717:329;;;;:::o;8052:327::-;8110:6;8159:2;8147:9;8138:7;8134:23;8130:32;8127:119;;;8165:79;;:::i;:::-;8127:119;8285:1;8310:52;8354:7;8345:6;8334:9;8330:22;8310:52;:::i;:::-;8300:62;;8256:116;8052:327;;;;:::o;8385:349::-;8454:6;8503:2;8491:9;8482:7;8478:23;8474:32;8471:119;;;8509:79;;:::i;:::-;8471:119;8629:1;8654:63;8709:7;8700:6;8689:9;8685:22;8654:63;:::i;:::-;8644:73;;8600:127;8385:349;;;;:::o;8740:529::-;8811:6;8819;8868:2;8856:9;8847:7;8843:23;8839:32;8836:119;;;8874:79;;:::i;:::-;8836:119;9022:1;9011:9;9007:17;8994:31;9052:18;9044:6;9041:30;9038:117;;;9074:79;;:::i;:::-;9038:117;9187:65;9244:7;9235:6;9224:9;9220:22;9187:65;:::i;:::-;9169:83;;;;8965:297;8740:529;;;;;:::o;9275:329::-;9334:6;9383:2;9371:9;9362:7;9358:23;9354:32;9351:119;;;9389:79;;:::i;:::-;9351:119;9509:1;9534:53;9579:7;9570:6;9559:9;9555:22;9534:53;:::i;:::-;9524:63;;9480:117;9275:329;;;;:::o;9610:684::-;9703:6;9711;9760:2;9748:9;9739:7;9735:23;9731:32;9728:119;;;9766:79;;:::i;:::-;9728:119;9886:1;9911:53;9956:7;9947:6;9936:9;9932:22;9911:53;:::i;:::-;9901:63;;9857:117;10041:2;10030:9;10026:18;10013:32;10072:18;10064:6;10061:30;10058:117;;;10094:79;;:::i;:::-;10058:117;10199:78;10269:7;10260:6;10249:9;10245:22;10199:78;:::i;:::-;10189:88;;9984:303;9610:684;;;;;:::o;10300:118::-;10387:24;10405:5;10387:24;:::i;:::-;10382:3;10375:37;10300:118;;:::o;10424:157::-;10529:45;10549:24;10567:5;10549:24;:::i;:::-;10529:45;:::i;:::-;10524:3;10517:58;10424:157;;:::o;10587:109::-;10668:21;10683:5;10668:21;:::i;:::-;10663:3;10656:34;10587:109;;:::o;10702:118::-;10789:24;10807:5;10789:24;:::i;:::-;10784:3;10777:37;10702:118;;:::o;10826:360::-;10912:3;10940:38;10972:5;10940:38;:::i;:::-;10994:70;11057:6;11052:3;10994:70;:::i;:::-;10987:77;;11073:52;11118:6;11113:3;11106:4;11099:5;11095:16;11073:52;:::i;:::-;11150:29;11172:6;11150:29;:::i;:::-;11145:3;11141:39;11134:46;;10916:270;10826:360;;;;:::o;11192:364::-;11280:3;11308:39;11341:5;11308:39;:::i;:::-;11363:71;11427:6;11422:3;11363:71;:::i;:::-;11356:78;;11443:52;11488:6;11483:3;11476:4;11469:5;11465:16;11443:52;:::i;:::-;11520:29;11542:6;11520:29;:::i;:::-;11515:3;11511:39;11504:46;;11284:272;11192:364;;;;:::o;11562:377::-;11668:3;11696:39;11729:5;11696:39;:::i;:::-;11751:89;11833:6;11828:3;11751:89;:::i;:::-;11744:96;;11849:52;11894:6;11889:3;11882:4;11875:5;11871:16;11849:52;:::i;:::-;11926:6;11921:3;11917:16;11910:23;;11672:267;11562:377;;;;:::o;11969:845::-;12072:3;12109:5;12103:12;12138:36;12164:9;12138:36;:::i;:::-;12190:89;12272:6;12267:3;12190:89;:::i;:::-;12183:96;;12310:1;12299:9;12295:17;12326:1;12321:137;;;;12472:1;12467:341;;;;12288:520;;12321:137;12405:4;12401:9;12390;12386:25;12381:3;12374:38;12441:6;12436:3;12432:16;12425:23;;12321:137;;12467:341;12534:38;12566:5;12534:38;:::i;:::-;12594:1;12608:154;12622:6;12619:1;12616:13;12608:154;;;12696:7;12690:14;12686:1;12681:3;12677:11;12670:35;12746:1;12737:7;12733:15;12722:26;;12644:4;12641:1;12637:12;12632:17;;12608:154;;;12791:6;12786:3;12782:16;12775:23;;12474:334;;12288:520;;12076:738;;11969:845;;;;:::o;12820:366::-;12962:3;12983:67;13047:2;13042:3;12983:67;:::i;:::-;12976:74;;13059:93;13148:3;13059:93;:::i;:::-;13177:2;13172:3;13168:12;13161:19;;12820:366;;;:::o;13192:::-;13334:3;13355:67;13419:2;13414:3;13355:67;:::i;:::-;13348:74;;13431:93;13520:3;13431:93;:::i;:::-;13549:2;13544:3;13540:12;13533:19;;13192:366;;;:::o;13564:::-;13706:3;13727:67;13791:2;13786:3;13727:67;:::i;:::-;13720:74;;13803:93;13892:3;13803:93;:::i;:::-;13921:2;13916:3;13912:12;13905:19;;13564:366;;;:::o;13936:::-;14078:3;14099:67;14163:2;14158:3;14099:67;:::i;:::-;14092:74;;14175:93;14264:3;14175:93;:::i;:::-;14293:2;14288:3;14284:12;14277:19;;13936:366;;;:::o;14308:::-;14450:3;14471:67;14535:2;14530:3;14471:67;:::i;:::-;14464:74;;14547:93;14636:3;14547:93;:::i;:::-;14665:2;14660:3;14656:12;14649:19;;14308:366;;;:::o;14680:::-;14822:3;14843:67;14907:2;14902:3;14843:67;:::i;:::-;14836:74;;14919:93;15008:3;14919:93;:::i;:::-;15037:2;15032:3;15028:12;15021:19;;14680:366;;;:::o;15052:::-;15194:3;15215:67;15279:2;15274:3;15215:67;:::i;:::-;15208:74;;15291:93;15380:3;15291:93;:::i;:::-;15409:2;15404:3;15400:12;15393:19;;15052:366;;;:::o;15424:::-;15566:3;15587:67;15651:2;15646:3;15587:67;:::i;:::-;15580:74;;15663:93;15752:3;15663:93;:::i;:::-;15781:2;15776:3;15772:12;15765:19;;15424:366;;;:::o;15796:::-;15938:3;15959:67;16023:2;16018:3;15959:67;:::i;:::-;15952:74;;16035:93;16124:3;16035:93;:::i;:::-;16153:2;16148:3;16144:12;16137:19;;15796:366;;;:::o;16168:118::-;16255:24;16273:5;16255:24;:::i;:::-;16250:3;16243:37;16168:118;;:::o;16292:256::-;16404:3;16419:75;16490:3;16481:6;16419:75;:::i;:::-;16519:2;16514:3;16510:12;16503:19;;16539:3;16532:10;;16292:256;;;;:::o;16554:589::-;16779:3;16801:95;16892:3;16883:6;16801:95;:::i;:::-;16794:102;;16913:95;17004:3;16995:6;16913:95;:::i;:::-;16906:102;;17025:92;17113:3;17104:6;17025:92;:::i;:::-;17018:99;;17134:3;17127:10;;16554:589;;;;;;:::o;17149:222::-;17242:4;17280:2;17269:9;17265:18;17257:26;;17293:71;17361:1;17350:9;17346:17;17337:6;17293:71;:::i;:::-;17149:222;;;;:::o;17377:640::-;17572:4;17610:3;17599:9;17595:19;17587:27;;17624:71;17692:1;17681:9;17677:17;17668:6;17624:71;:::i;:::-;17705:72;17773:2;17762:9;17758:18;17749:6;17705:72;:::i;:::-;17787;17855:2;17844:9;17840:18;17831:6;17787:72;:::i;:::-;17906:9;17900:4;17896:20;17891:2;17880:9;17876:18;17869:48;17934:76;18005:4;17996:6;17934:76;:::i;:::-;17926:84;;17377:640;;;;;;;:::o;18023:210::-;18110:4;18148:2;18137:9;18133:18;18125:26;;18161:65;18223:1;18212:9;18208:17;18199:6;18161:65;:::i;:::-;18023:210;;;;:::o;18239:222::-;18332:4;18370:2;18359:9;18355:18;18347:26;;18383:71;18451:1;18440:9;18436:17;18427:6;18383:71;:::i;:::-;18239:222;;;;:::o;18467:313::-;18580:4;18618:2;18607:9;18603:18;18595:26;;18667:9;18661:4;18657:20;18653:1;18642:9;18638:17;18631:47;18695:78;18768:4;18759:6;18695:78;:::i;:::-;18687:86;;18467:313;;;;:::o;18786:419::-;18952:4;18990:2;18979:9;18975:18;18967:26;;19039:9;19033:4;19029:20;19025:1;19014:9;19010:17;19003:47;19067:131;19193:4;19067:131;:::i;:::-;19059:139;;18786:419;;;:::o;19211:::-;19377:4;19415:2;19404:9;19400:18;19392:26;;19464:9;19458:4;19454:20;19450:1;19439:9;19435:17;19428:47;19492:131;19618:4;19492:131;:::i;:::-;19484:139;;19211:419;;;:::o;19636:::-;19802:4;19840:2;19829:9;19825:18;19817:26;;19889:9;19883:4;19879:20;19875:1;19864:9;19860:17;19853:47;19917:131;20043:4;19917:131;:::i;:::-;19909:139;;19636:419;;;:::o;20061:::-;20227:4;20265:2;20254:9;20250:18;20242:26;;20314:9;20308:4;20304:20;20300:1;20289:9;20285:17;20278:47;20342:131;20468:4;20342:131;:::i;:::-;20334:139;;20061:419;;;:::o;20486:::-;20652:4;20690:2;20679:9;20675:18;20667:26;;20739:9;20733:4;20729:20;20725:1;20714:9;20710:17;20703:47;20767:131;20893:4;20767:131;:::i;:::-;20759:139;;20486:419;;;:::o;20911:::-;21077:4;21115:2;21104:9;21100:18;21092:26;;21164:9;21158:4;21154:20;21150:1;21139:9;21135:17;21128:47;21192:131;21318:4;21192:131;:::i;:::-;21184:139;;20911:419;;;:::o;21336:::-;21502:4;21540:2;21529:9;21525:18;21517:26;;21589:9;21583:4;21579:20;21575:1;21564:9;21560:17;21553:47;21617:131;21743:4;21617:131;:::i;:::-;21609:139;;21336:419;;;:::o;21761:::-;21927:4;21965:2;21954:9;21950:18;21942:26;;22014:9;22008:4;22004:20;22000:1;21989:9;21985:17;21978:47;22042:131;22168:4;22042:131;:::i;:::-;22034:139;;21761:419;;;:::o;22186:::-;22352:4;22390:2;22379:9;22375:18;22367:26;;22439:9;22433:4;22429:20;22425:1;22414:9;22410:17;22403:47;22467:131;22593:4;22467:131;:::i;:::-;22459:139;;22186:419;;;:::o;22611:222::-;22704:4;22742:2;22731:9;22727:18;22719:26;;22755:71;22823:1;22812:9;22808:17;22799:6;22755:71;:::i;:::-;22611:222;;;;:::o;22839:129::-;22873:6;22900:20;;:::i;:::-;22890:30;;22929:33;22957:4;22949:6;22929:33;:::i;:::-;22839:129;;;:::o;22974:75::-;23007:6;23040:2;23034:9;23024:19;;22974:75;:::o;23055:311::-;23132:4;23222:18;23214:6;23211:30;23208:56;;;23244:18;;:::i;:::-;23208:56;23294:4;23286:6;23282:17;23274:25;;23354:4;23348;23344:15;23336:23;;23055:311;;;:::o;23372:307::-;23433:4;23523:18;23515:6;23512:30;23509:56;;;23545:18;;:::i;:::-;23509:56;23583:29;23605:6;23583:29;:::i;:::-;23575:37;;23667:4;23661;23657:15;23649:23;;23372:307;;;:::o;23685:141::-;23734:4;23757:3;23749:11;;23780:3;23777:1;23770:14;23814:4;23811:1;23801:18;23793:26;;23685:141;;;:::o;23832:98::-;23883:6;23917:5;23911:12;23901:22;;23832:98;;;:::o;23936:99::-;23988:6;24022:5;24016:12;24006:22;;23936:99;;;:::o;24041:168::-;24124:11;24158:6;24153:3;24146:19;24198:4;24193:3;24189:14;24174:29;;24041:168;;;;:::o;24215:169::-;24299:11;24333:6;24328:3;24321:19;24373:4;24368:3;24364:14;24349:29;;24215:169;;;;:::o;24390:148::-;24492:11;24529:3;24514:18;;24390:148;;;;:::o;24544:305::-;24584:3;24603:20;24621:1;24603:20;:::i;:::-;24598:25;;24637:20;24655:1;24637:20;:::i;:::-;24632:25;;24791:1;24723:66;24719:74;24716:1;24713:81;24710:107;;;24797:18;;:::i;:::-;24710:107;24841:1;24838;24834:9;24827:16;;24544:305;;;;:::o;24855:185::-;24895:1;24912:20;24930:1;24912:20;:::i;:::-;24907:25;;24946:20;24964:1;24946:20;:::i;:::-;24941:25;;24985:1;24975:35;;24990:18;;:::i;:::-;24975:35;25032:1;25029;25025:9;25020:14;;24855:185;;;;:::o;25046:348::-;25086:7;25109:20;25127:1;25109:20;:::i;:::-;25104:25;;25143:20;25161:1;25143:20;:::i;:::-;25138:25;;25331:1;25263:66;25259:74;25256:1;25253:81;25248:1;25241:9;25234:17;25230:105;25227:131;;;25338:18;;:::i;:::-;25227:131;25386:1;25383;25379:9;25368:20;;25046:348;;;;:::o;25400:191::-;25440:4;25460:20;25478:1;25460:20;:::i;:::-;25455:25;;25494:20;25512:1;25494:20;:::i;:::-;25489:25;;25533:1;25530;25527:8;25524:34;;;25538:18;;:::i;:::-;25524:34;25583:1;25580;25576:9;25568:17;;25400:191;;;;:::o;25597:96::-;25634:7;25663:24;25681:5;25663:24;:::i;:::-;25652:35;;25597:96;;;:::o;25699:90::-;25733:7;25776:5;25769:13;25762:21;25751:32;;25699:90;;;:::o;25795:77::-;25832:7;25861:5;25850:16;;25795:77;;;:::o;25878:149::-;25914:7;25954:66;25947:5;25943:78;25932:89;;25878:149;;;:::o;26033:126::-;26070:7;26110:42;26103:5;26099:54;26088:65;;26033:126;;;:::o;26165:77::-;26202:7;26231:5;26220:16;;26165:77;;;:::o;26248:154::-;26332:6;26327:3;26322;26309:30;26394:1;26385:6;26380:3;26376:16;26369:27;26248:154;;;:::o;26408:307::-;26476:1;26486:113;26500:6;26497:1;26494:13;26486:113;;;26585:1;26580:3;26576:11;26570:18;26566:1;26561:3;26557:11;26550:39;26522:2;26519:1;26515:10;26510:15;;26486:113;;;26617:6;26614:1;26611:13;26608:101;;;26697:1;26688:6;26683:3;26679:16;26672:27;26608:101;26457:258;26408:307;;;:::o;26721:320::-;26765:6;26802:1;26796:4;26792:12;26782:22;;26849:1;26843:4;26839:12;26870:18;26860:81;;26926:4;26918:6;26914:17;26904:27;;26860:81;26988:2;26980:6;26977:14;26957:18;26954:38;26951:84;;;27007:18;;:::i;:::-;26951:84;26772:269;26721:320;;;:::o;27047:281::-;27130:27;27152:4;27130:27;:::i;:::-;27122:6;27118:40;27260:6;27248:10;27245:22;27224:18;27212:10;27209:34;27206:62;27203:88;;;27271:18;;:::i;:::-;27203:88;27311:10;27307:2;27300:22;27090:238;27047:281;;:::o;27334:233::-;27373:3;27396:24;27414:5;27396:24;:::i;:::-;27387:33;;27442:66;27435:5;27432:77;27429:103;;;27512:18;;:::i;:::-;27429:103;27559:1;27552:5;27548:13;27541:20;;27334:233;;;:::o;27573:100::-;27612:7;27641:26;27661:5;27641:26;:::i;:::-;27630:37;;27573:100;;;:::o;27679:94::-;27718:7;27747:20;27761:5;27747:20;:::i;:::-;27736:31;;27679:94;;;:::o;27779:176::-;27811:1;27828:20;27846:1;27828:20;:::i;:::-;27823:25;;27862:20;27880:1;27862:20;:::i;:::-;27857:25;;27901:1;27891:35;;27906:18;;:::i;:::-;27891:35;27947:1;27944;27940:9;27935:14;;27779:176;;;;:::o;27961:180::-;28009:77;28006:1;27999:88;28106:4;28103:1;28096:15;28130:4;28127:1;28120:15;28147:180;28195:77;28192:1;28185:88;28292:4;28289:1;28282:15;28316:4;28313:1;28306:15;28333:180;28381:77;28378:1;28371:88;28478:4;28475:1;28468:15;28502:4;28499:1;28492:15;28519:180;28567:77;28564:1;28557:88;28664:4;28661:1;28654:15;28688:4;28685:1;28678:15;28705:180;28753:77;28750:1;28743:88;28850:4;28847:1;28840:15;28874:4;28871:1;28864:15;28891:117;29000:1;28997;28990:12;29014:117;29123:1;29120;29113:12;29137:117;29246:1;29243;29236:12;29260:117;29369:1;29366;29359:12;29383:117;29492:1;29489;29482:12;29506:117;29615:1;29612;29605:12;29629:102;29670:6;29721:2;29717:7;29712:2;29705:5;29701:14;29697:28;29687:38;;29629:102;;;:::o;29737:94::-;29770:8;29818:5;29814:2;29810:14;29789:35;;29737:94;;;:::o;29837:176::-;29977:28;29973:1;29965:6;29961:14;29954:52;29837:176;:::o;30019:232::-;30159:34;30155:1;30147:6;30143:14;30136:58;30228:15;30223:2;30215:6;30211:15;30204:40;30019:232;:::o;30257:225::-;30397:34;30393:1;30385:6;30381:14;30374:58;30466:8;30461:2;30453:6;30449:15;30442:33;30257:225;:::o;30488:163::-;30628:15;30624:1;30616:6;30612:14;30605:39;30488:163;:::o;30657:220::-;30797:34;30793:1;30785:6;30781:14;30774:58;30866:3;30861:2;30853:6;30849:15;30842:28;30657:220;:::o;30883:182::-;31023:34;31019:1;31011:6;31007:14;31000:58;30883:182;:::o;31071:234::-;31211:34;31207:1;31199:6;31195:14;31188:58;31280:17;31275:2;31267:6;31263:15;31256:42;31071:234;:::o;31311:176::-;31451:28;31447:1;31439:6;31435:14;31428:52;31311:176;:::o;31493:247::-;31633:34;31629:1;31621:6;31617:14;31610:58;31702:30;31697:2;31689:6;31685:15;31678:55;31493:247;:::o;31746:122::-;31819:24;31837:5;31819:24;:::i;:::-;31812:5;31809:35;31799:63;;31858:1;31855;31848:12;31799:63;31746:122;:::o;31874:116::-;31944:21;31959:5;31944:21;:::i;:::-;31937:5;31934:32;31924:60;;31980:1;31977;31970:12;31924:60;31874:116;:::o;31996:122::-;32069:24;32087:5;32069:24;:::i;:::-;32062:5;32059:35;32049:63;;32108:1;32105;32098:12;32049:63;31996:122;:::o;32124:120::-;32196:23;32213:5;32196:23;:::i;:::-;32189:5;32186:34;32176:62;;32234:1;32231;32224:12;32176:62;32124:120;:::o;32250:122::-;32323:24;32341:5;32323:24;:::i;:::-;32316:5;32313:35;32303:63;;32362:1;32359;32352:12;32303:63;32250:122;:::o

Swarm Source

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