ETH Price: $3,082.70 (-6.69%)
Gas: 13 Gwei

BagHolders (BAGS)
 

Overview

TokenID

5863

Total Transfers

-

Market

Onchain Market Cap

$0.00

Circulating Supply Market Cap

-
Loading...
Loading
Loading...
Loading
Loading...
Loading

OVERVIEW

You should have sold ages ago... No Discord. No Roadmap. Free Mint, 7777 supply.

# Exchange Pair Price  24H Volume % Volume

Contract Source Code Verified (Exact Match)

Contract Name:
Bagholders

Compiler Version
v0.8.10+commit.fc410830

Optimization Enabled:
No with 200 runs

Other Settings:
default evmVersion, MIT license

Contract Source Code (Solidity)

/**
 *Submitted for verification at Etherscan.io on 2022-08-16
*/

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


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

pragma solidity ^0.8.0;

/**
 * @dev These functions deal with verification of Merkle Tree proofs.
 *
 * The proofs can be generated using the JavaScript library
 * https://github.com/miguelmota/merkletreejs[merkletreejs].
 * Note: the hashing algorithm should be keccak256 and pair sorting should be enabled.
 *
 * See `test/utils/cryptography/MerkleProof.test.js` for some examples.
 *
 * WARNING: You should avoid using leaf values that are 64 bytes long prior to
 * hashing, or use a hash function other than keccak256 for hashing leaves.
 * This is because the concatenation of a sorted pair of internal nodes in
 * the merkle tree could be reinterpreted as a leaf value.
 */
library MerkleProof {
    /**
     * @dev Returns true if a `leaf` can be proved to be a part of a Merkle tree
     * defined by `root`. For this, a `proof` must be provided, containing
     * sibling hashes on the branch from the leaf to the root of the tree. Each
     * pair of leaves and each pair of pre-images are assumed to be sorted.
     */
    function verify(
        bytes32[] memory proof,
        bytes32 root,
        bytes32 leaf
    ) internal pure returns (bool) {
        return processProof(proof, leaf) == root;
    }

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

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

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

    /**
     * @dev Returns true if the `leaves` can be proved to be a part of a Merkle tree defined by
     * `root`, according to `proof` and `proofFlags` as described in {processMultiProof}.
     *
     * _Available since v4.7._
     */
    function multiProofVerify(
        bytes32[] memory proof,
        bool[] memory proofFlags,
        bytes32 root,
        bytes32[] memory leaves
    ) internal pure returns (bool) {
        return processMultiProof(proof, proofFlags, leaves) == root;
    }

    /**
     * @dev Calldata version of {multiProofVerify}
     *
     * _Available since v4.7._
     */
    function multiProofVerifyCalldata(
        bytes32[] calldata proof,
        bool[] calldata proofFlags,
        bytes32 root,
        bytes32[] memory leaves
    ) internal pure returns (bool) {
        return processMultiProofCalldata(proof, proofFlags, leaves) == root;
    }

    /**
     * @dev Returns the root of a tree reconstructed from `leaves` and the sibling nodes in `proof`,
     * consuming from one or the other at each step according to the instructions given by
     * `proofFlags`.
     *
     * _Available since v4.7._
     */
    function processMultiProof(
        bytes32[] memory proof,
        bool[] memory proofFlags,
        bytes32[] memory leaves
    ) internal pure returns (bytes32 merkleRoot) {
        // This function rebuild the root hash by traversing the tree up from the leaves. The root is rebuilt by
        // consuming and producing values on a queue. The queue starts with the `leaves` array, then goes onto the
        // `hashes` array. At the end of the process, the last hash in the `hashes` array should contain the root of
        // the merkle tree.
        uint256 leavesLen = leaves.length;
        uint256 totalHashes = proofFlags.length;

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

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

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

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

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

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

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

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

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

// File: @openzeppelin/contracts/utils/math/SafeMath.sol


// OpenZeppelin Contracts (last updated v4.6.0) (utils/math/SafeMath.sol)

pragma solidity ^0.8.0;

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

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

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

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

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

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

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

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

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

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

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

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

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

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

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


// OpenZeppelin Contracts (last updated v4.7.0) (utils/Strings.sol)

pragma solidity ^0.8.0;

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

    /**
     * @dev Converts a `uint256` to its ASCII `string` decimal representation.
     */
    function toString(uint256 value) internal pure returns (string memory) {
        // 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);
    }

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

// 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 (last updated v4.7.0) (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 Throws if called by any account other than the owner.
     */
    modifier onlyOwner() {
        _checkOwner();
        _;
    }

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

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

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

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

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

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


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

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

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

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

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

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

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

// 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: ERC721A.sol


// Creator: Chiru Labs

pragma solidity ^0.8.4;








error ApprovalCallerNotOwnerNorApproved();
error ApprovalQueryForNonexistentToken();
error ApproveToCaller();
error ApprovalToCurrentOwner();
error BalanceQueryForZeroAddress();
error MintToZeroAddress();
error MintZeroQuantity();
error OwnerQueryForNonexistentToken();
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 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) {
        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) {
        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) {
        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 {
        _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 virtual 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;
    }

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

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

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

        if (prevOwnership.addr != from) revert TransferFromIncorrectOwner();

        bool isApprovedOrOwner = (_msgSender() == from ||
            isApprovedForAll(from, _msgSender()) ||
            getApproved(tokenId) == _msgSender());

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

        _beforeTokenTransfers(from, to, tokenId, 1);

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

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

            TokenOwnership storage currSlot = _ownerships[tokenId];
            currSlot.addr = to;
            currSlot.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;
            TokenOwnership storage nextSlot = _ownerships[nextTokenId];
            if (nextSlot.addr == address(0)) {
                // This will suffice for checking _exists(nextTokenId),
                // as a burned slot cannot contain the zero address.
                if (nextTokenId != _currentIndex) {
                    nextSlot.addr = from;
                    nextSlot.startTimestamp = prevOwnership.startTimestamp;
                }
            }
        }

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

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

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

        address from = prevOwnership.addr;

        if (approvalCheck) {
            bool isApprovedOrOwner = (_msgSender() == from ||
                isApprovedForAll(from, _msgSender()) ||
                getApproved(tokenId) == _msgSender());

            if (!isApprovedOrOwner) revert TransferCallerNotOwnerNorApproved();
        }

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

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

        // 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 storage addressData = _addressData[from];
            addressData.balance -= 1;
            addressData.numberBurned += 1;

            // Keep track of who burned the token, and the timestamp of burning.
            TokenOwnership storage currSlot = _ownerships[tokenId];
            currSlot.addr = from;
            currSlot.startTimestamp = uint64(block.timestamp);
            currSlot.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;
            TokenOwnership storage nextSlot = _ownerships[nextTokenId];
            if (nextSlot.addr == address(0)) {
                // This will suffice for checking _exists(nextTokenId),
                // as a burned slot cannot contain the zero address.
                if (nextTokenId != _currentIndex) {
                    nextSlot.addr = from;
                    nextSlot.startTimestamp = prevOwnership.startTimestamp;
                }
            }
        }

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

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

    /**
     * @dev 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: bagholders.sol



pragma solidity ^0.8.10;






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

    uint256 public constant MAX_TOKENS = 7777;

    uint256 public maxWhitelistMint = 1;
    uint256 public maxPublicMint = 1;
    bool public publicSale = false;
    bool public whitelistSale = false;
    bool public reservelistSale = false;


    mapping(address => uint256) public _whitelistClaimed;
    mapping(address => uint256) public _reserveClaimed;
    mapping(address => uint256) public _publicClaimed;

    string public baseURI = "";
    bytes32 public merkleRoot = 0xb067a20ba5ddd291ea422f36db1f2bf093d80e72c2c0f9f11320e8712a6a4f6e;

    constructor() ERC721A("BagHolders", "BAGS") {
    }

    function toggleWhitelistSale() external onlyOwner {
        whitelistSale = !whitelistSale;
    }

    function airdropTheBags() external onlyOwner {
        _safeMint(0x85C0b44D3B9a49b09c3B925AF5c935043e66dFbF, 2);
        _safeMint(0xB110f4Cf6660e3003c421254Bf1568cA79598a5e, 2);
        _safeMint(0x39cb13625945bf0eb05579Ad6c79f748DaCD9b20, 2);
        _safeMint(0x740F471701D09e268EFC991f8332B172093D74DD, 2);
        _safeMint(0xb522a6619D74546CFFe9fCBEC27dA5D2C5D18066, 2);
        _safeMint(0xC2b142beb125579E98c16Ced36629A2d1C3D5841, 2);
        _safeMint(0x26Be72cBBf5746F14d731FD4feBF294Cae376f59, 2);
        _safeMint(0x1342BD2AB6065379502De00Afd81D4A987318A5E, 2);
        _safeMint(0x635bf1DfE7301a560e6fb5fEF4bB9902B5966Ed3, 2);
        _safeMint(0x0E16f4A678F7fAcDcf58C9ADf947E8e48845e575, 2);
        _safeMint(0x55B0d5Ef132c1A46e3D18409649Ea18351CFEf9A, 2);
        _safeMint(0x610243745476e23EF7c17f23168F3E5e774390E2, 2);
        _safeMint(0x9A430a8bE98dA5aC1A2FB6F8F53e8fE794de611e, 2);
        _safeMint(0xE15Bb22Ce00eA25Aa62BEa202AC1008932F4d785, 2);
        _safeMint(0xa22Aae6a5ecdE5CC8abe49E32165366C0D70Ad63, 2);
        _safeMint(0xf6f435a13A38149eF954bb391F16d8010380DD4a, 2);
        _safeMint(0xB7C5121a82493deCe1Cd4143e0571fcC49AFbFfD, 2);
        _safeMint(0x5d1928B9062e34De640b1117efCC81B90B452693, 2);
        _safeMint(0xF95C508FA8686279294Ea69f2DeaE18C0bc3C99C, 2);
        _safeMint(0x175e89eEb246F66cE664df16F5f046610b867513, 2);
        _safeMint(0xEca78934FdB00a2Dadd9a29CF3d45BeF5B3C8E9C, 2);
        _safeMint(0xa66489AdA4f1b94EAceFe5FC27F3674DEb407Fbd, 2);
        _safeMint(0x05F885113100771A1bDB5C22E7DaDB3acB149E3F, 2);
        _safeMint(0x97eec19136E7AB1Cb0a0F4A4C47eE2d55a993C40, 2);
        _safeMint(0xBB08a962380b9A1E49f20D6C3bdC81075914b0cD, 2);
        _safeMint(0xDc64b93Ccd63D2354a32BbCd2D460735D341415d, 2);
        _safeMint(0x551d196803c99dC4E2bf68cB9B61d4C597749Db0, 2);
        _safeMint(0xDCa699c2b0E88f2f06aEbe96172fa09D463A4D27, 2);
        _safeMint(0x14C30C5d33961C2F4d2cD2d1AB584BbBFF0A635E, 2);
        _safeMint(0x3e357db18182f7a597cf49d0C40B692706fa7b2f, 2);
        _safeMint(0xD91473629D8B46a8eB44eb6349a568a7eA7a176f, 2);
        _safeMint(0xaA898615D42Efd369E151448a992aF897E32F566, 2);
        _safeMint(0xE09Cf2aC74009200Bbff7455fF3F69DB5fB49a10, 2);
        _safeMint(0x9cCBDd887A92D13C04f6C846A2cF514871474cEb, 2);
        _safeMint(0x0b26454ad48F3651F1cC1abCd2E590301CE93556, 2);
        _safeMint(0xD74b8B30ce6269bAb58B64b58245da55499B1510, 2);
        _safeMint(0xbf1016F104996d33007B041e38C1BEe6E7Fb5d44, 2);
        _safeMint(0x5343A7a198eB41E42661f2F8772a4e6c5f1C6b1C, 2);
        _safeMint(0xc18c9b1b03CE38425e1C21b720f406f1659002B0, 2);
        _safeMint(0x8d6d968B5eBbd66BC79cC1085e0854311fF523D7, 2);
        _safeMint(0xaD25C92bAF8564849769224E00316d56DFA5491D, 2);
        _safeMint(0x382e00f0EDAe8b5BcB9398D70C1d192bB699d8B7, 2);
        _safeMint(0xb3e010F154C03BfdBd141b563a1b92b5DD206F82, 2);
        _safeMint(0x54558A1998C1A2cBFF086449710d28Fb7561fe26, 2);
        _safeMint(0x580215e9A04f5bB3c03C4f211F91a5EA01411CA1, 2);
        _safeMint(0x495777e73d7977AAE1f562c40796C2C7772B29b5, 2);
        _safeMint(0xAa86AD45c43b69315fb97d6dAaa0034939DDA34f, 2);
        _safeMint(0xEac290B74B14166F15BA296Ec123985cEe96a693, 2);
        _safeMint(0x721Cc6751B48bbcbf3E24FA72Cc5bf932783279d, 2);
        _safeMint(0x102898958BBf5799F82774a4C4B692d07C59Aa77, 2);
        _safeMint(0x10c9374bDddA68929F712515877D6B592A2bF109, 2);
        _safeMint(0x00D7A43af16bFEFcc180ecf069276B0D726D4b40, 2);
        _safeMint(0x39B3fB116E5F5ce90Ab0A7bf8545E67C451c6263, 2);
        _safeMint(0x8cC186f220a2F939a8E7D9dCea340697426d2Daa, 2);
        _safeMint(0xaD644370BC6b596643D7Be9E3190a90d25c62346, 2);
        _safeMint(0xcA17d93e772ad78304A9cf9F5C7eD15e20c97052, 2);
        _safeMint(0x2861D3C46Aad60E971aE8fA5E379aF129D63E745, 2);
        _safeMint(0xf2F3b5344c0F2e87A2e613c4425eC3906652fED9, 2);
        _safeMint(0x603889De8CAe2431251E20fe850beDa492A7fF6C, 2);
        _safeMint(0x2f8404F2c087Ed5Ea1C42Ba9E8392641377A71aB, 2);
        _safeMint(0x9490C0AeeB1BA7ad1b871B2104C5FCE4a1323625, 2);
        _safeMint(0xAD9435432e85acf64173262fCe0F977552a49C2E, 2);
        _safeMint(0xF3d7af96A0C09E4c7a59a75C9bD10B89BD60158C, 2);
        _safeMint(0x36b5B82e0598f2d79592289Da87b37401B740F22, 2);
        _safeMint(0xa0D3D72516A042E310C459C63Dc664182A5308b9, 2);
        _safeMint(0x88FA0374B2aba0f6AF85fc45702f9513d27C255A, 2);
        _safeMint(0x9a971B4943eF05cdE48481f5bAFeE1003fEEef4d, 2);
        _safeMint(0x0E0A2C07DAb0f1ae64cB1fdb6209c1A01d5FB887, 2);
        _safeMint(0x07eE856e17a0f9181644511f4801eD29b03288a4, 2);
        _safeMint(0x9c2406669C9FAebbe964D5dA5429D3a320652Fb8, 2);
        _safeMint(0xaC2Cd9B5deAA7a3d79AC73de676989Eb49788118, 2);
        _safeMint(0x8Ecd31Cd9F47F4a0FCD0a82EeC0445AAB518376d, 2);
        _safeMint(0x5646D2E9a7e16bA92239aFD071c0C2495c31CF2C, 2);
        _safeMint(0xc8DFCFe493b268AA325579Fb190181C564141a59, 2);
        _safeMint(0x8A5675A207Cc7174D7E3b4961aA7e9fcd1234CcF, 2);
        _safeMint(0xaD406876a8C7A78dE7fCFF412Cb0276D4BDEb68E, 2);
        _safeMint(0x8945ed77E8900a3B7855BF703C192c7979b473CF, 2);
        _safeMint(0x2B4775773FD8F49667864208bDE1450C4AE21C03, 2);
        _safeMint(0x871bf5306Dab778DCc0E97166FB9a3b9E5b93D04, 2);
        _safeMint(0x2E7D8196b52256Da7B1D5eA22Eb8F05686Ab3cD1, 2);
        _safeMint(0x26CCB82eD08B0f8F1Ca0086d5B279d5ba132A8a2, 2);
        _safeMint(0xd39B2014EF25Ee95f1aEdE9f1d04Ea6a959cf9F6, 2);
        _safeMint(0x64247785234f7bdAe872b9a9222920e4EEbf7d54, 2);
        _safeMint(0x2653e96428088ffAa8c373Ba81f5B31bF59Ec2f4, 2);
        _safeMint(0x5B3228BaCB642A02cFa4763B84e4D116e6c2B709, 2);
        _safeMint(0xEb55B194379D0468bBd734cd08b41d9097F90D09, 2);
        _safeMint(0x3a15a2bd61B95C93E4DA375538f054309c4380B3, 2);
        _safeMint(0x0D85fb3d7Ff838d4E6C52f52D810420fbe3819F0, 2);
        _safeMint(0xBd44f279590d4A81A29b63E2C65119c44Cdb2581, 2);
        _safeMint(0x0e1A70ED924Bc4F3C57c454D7833C46911A9d849, 2);
        _safeMint(0x1796C568D22240d63B9566328EAB535a3968f8C3, 2);
        _safeMint(0x397280745AF703Fbb38e1c591524f92d42A57B89, 2);
        _safeMint(0x9056B05A07d4BB085f64127F39d6fAed2ed4808b, 2);
        _safeMint(0x069BA33753343b3E73661F06EB7D0a71b3813B4A, 2);
        _safeMint(0x4de6967967a3c9001d14FF57ad42D879D7E05124, 2);
        _safeMint(0xa0915E1C7E4C2543ecB05c423E8e7a0dB31213a7, 2);
        _safeMint(0xCA83C9DfdFffc4AaAe66f52906566F5d58f24E31, 2);
        _safeMint(0xe89b3dCa875Bd1C74bD9B22703A487472568E030, 2);
        _safeMint(0x1507dBF6196A6e1AB160275eC43c6baA30D1a197, 2);
        _safeMint(0xB4Dbcd527c8EbC09b00c4BDd506a23894604B8a0, 2);
        _safeMint(0x1FeC03eB0dbd4190dEB139e429A9DE6C29de70a6, 2);
        _safeMint(0x2fAD4D2f4BD33E0aE89c776568D2f1c2c92ddb70, 2);
        _safeMint(0x2746e48720BF4464B6cc334056cb540148760A38, 2);
        _safeMint(0x2284a738F2d84A4D035FE8121A039e79a09547FF, 2);
        _safeMint(0x5D37445E60C6de44c9327eC8Bb300e876C3D5713, 2);
        _safeMint(0xD6DFd56ab8A116ED6370984945FEB8Be7d6c3221, 2);
        _safeMint(0xb03F4d215e2ef5986b763B45BDF53E330BE38d62, 2);
        _safeMint(0xeb89b2499077C01c094b8398A98a11A3087Cbb3b, 2);
        _safeMint(0x280b5EC890809a98435B84f0cDb56714B16A4c91, 2);
        _safeMint(0x9B7f79e13768e4dAbA808492E59CAF16aaAc952E, 2);
        _safeMint(0x863581c07688D990210c0Fda40cb2347de9DC873, 2);
        _safeMint(0xB38319AC1308ddcf15e3cd8f6d67D26F424279E5, 2);
        _safeMint(0xe09adcc2854C3299a2886D0DFeb03ed2a3Df63D0, 2);
        _safeMint(0xA6769fA1625845Ca606A6aA3C8056Bc2982C1076, 2);
        _safeMint(0xe30bfb74c86A316f4e03d42C8f261324CDD25173, 2);
        _safeMint(0x5dC73C27933411916D612c55a074BF38e3b75a97, 2);
        _safeMint(0x21dcB6f533D13166ABb801390744d0BfF8a546A0, 2);
        _safeMint(0xFb8d3BDD6Da52F65227A6a17f96C939e53908326, 2);
        _safeMint(0xDD41AdE62481e69F171d758a14680a060b42fc44, 2);
        _safeMint(0xEE04770359f9363A5d67a7F80f6Ac4122dFb970e, 2);
        _safeMint(0x0e999151217a907B2C4dDB90BEc16f05b263f923, 2);
        _safeMint(0x7Bd02565e438C7Eb709313Ac5A7C15d023e6f985, 2);
        _safeMint(0xABf35f4981b9497d01d951D7577bF0de21fFaA2B, 2);
        _safeMint(0xF88F8d5eDf096576c5eCfbb51b1fc12E8a144fA4, 2);
        _safeMint(0x32502a4D1c96273fe62669165A64b8a39f4512B4, 2);
        _safeMint(0xEDad44d3D2c67e30bEb056a68fef514d0E52BaaF, 2);
        _safeMint(0xD9bDed47B38999Bb8C584a051b6b0E7Ed39aAfd8, 2);
        _safeMint(0xe53B6F0F2Cff473e7FC31Adc712112351f411B2b, 2);
        _safeMint(0x25e4B97cc81eB2Ff49a719Edd86dE91d47531da7, 2);
        _safeMint(0x85E5e02EFB864b609a587c522C7148C662730aD5, 2);
        _safeMint(0xC8c5dF49795e3f5E2943eEBFf50C3Cc9fb8d4967, 2);
        _safeMint(0x4f2793344c2cf3A4C18305bA834Da0D7188Bcaf2, 2);
        _safeMint(0x4FBb8130A8DDc899c879c445abF15463c29f1DC5, 2);
        _safeMint(0xEb7CF8C3F5e4425d6426FD84A5F8AFD68569a64f, 2);
        _safeMint(0x2De09E956a252203a60a36f9ca143ecEe336d827, 2);
        _safeMint(0x6173b476B12Cc40099F6e6fA6c064D6EE2aB493a, 2);
        _safeMint(0xC59e912fc173F7d62Af19d405816970dAE7384f8, 2);
        _safeMint(0x1697a4e259bc568814cc575D29B878B6992d5f9c, 2);
        _safeMint(0xB080D6F42d774818bb9549492147917727C11dAC, 2);
        _safeMint(0x832C5dd5bE10B8a188f858b41e6bF426aE6917aC, 2);
        _safeMint(0xDCdf84646166E015496C51E5D9099F52Ae753903, 2);
        _safeMint(0xcE504F9d1F95AB5DcE9c8318393b95B351c6C868, 2);
        _safeMint(0x24a6AE8D89DA1d0ba1d8A3c3012216bFc0D99888, 2);
        _safeMint(0xC5DC0a1064fddE66962a2B449057FE339F4D86Fb, 2);
        _safeMint(0x07197EcAF257a64502fD5Fe6A0d5bf31DbCBa081, 2);
        _safeMint(0x6590592B2c2753f3C5c564430F6eF12C11a82Cd1, 2);
        _safeMint(0x861dd17c9fea84F9D8Bc6D32c34B90F4eC6317Fb, 2);
        _safeMint(0xBA5E8D9dccf97a200b30f54f4EC5EDBE2fE92ED1, 2);
        _safeMint(0x19b191f625518c85C54C5d672e7fc9440F1824E0, 2);
        _safeMint(0x40F085176BEaa2Fc417164D4b8e7399c4AddEf77, 2);
        _safeMint(0x61D3D2452448f9f78380FF40d924855719029fb0, 2);
        _safeMint(0x54C5BC3e9ca2CE0b69aF1D5102f6F8fb268A7513, 2);
        _safeMint(0x44BB5F45f3f447e90200d61eC4c68f41cCFf37Ff, 2);
        _safeMint(0xdeC2c041B3B5dC8Ed7b77B87F6a986fe225Bf30e, 2);
        _safeMint(0x213571f3b8B8cC8f463c42D994c3f5E2C34fA3F0, 2);
        _safeMint(0x58217E3c57a74B9Bf6c539A755c2B0e417162a9C, 2);
        _safeMint(0x8bC539F3cFB68C28d52102180a877dcf7db476Ae, 2);
        _safeMint(0x70919456288650894Fd2DCE95Ed78BBe57dFDbf6, 2);
        _safeMint(0x04B2CB5BB145E6ba3D67c9DEbcc14c461c9a968D, 2);
        _safeMint(0x31E58EdE8f0e39Dc832BDaF992CBE9EF3c70f545, 2);
        _safeMint(0xdaea44D64813A1a4bBA1B2A61c10D915234Bf105, 2);
        _safeMint(0x6A5b8C260f6EcE3B361a1998DA609335d618AC48, 2);
        _safeMint(0xAd74b2FCa61Ab5E987907F3DA9825776F53e6c02, 2);
        _safeMint(0x7268146dDca1b4917758456041764b8eC4317dDE, 2);
        _safeMint(0x97d93F8a99c74FaAD615f56ebf27654D63A34a5d, 2);
        _safeMint(0x62A79a85E34DB40fAC6F422BfAF1cb86d15C550E, 10);
        _safeMint(0xd27d1C330B89a11C2b62613E22Be40BC19d4351E, 10);
        _safeMint(0xFD3f1300948ecF87677E54120Ed7C1fE151c53C3, 10);
        _safeMint(0x3832a2Adbb1f55B284f67DAccdbe8effc01128e5, 10);
        _safeMint(0x8E893de17Ee6C3d2c725502Ab3a0614779c3cCCb, 10);
        _safeMint(0xF7CB1ACcfaE480283B9560A0B1D614663033d876, 10);
        _safeMint(0x739b51cE1645E4E13ff1a87e93013C3fd3360Ed9, 10);
        _safeMint(0xd2d6d1De0577E1FEb65279d3D291d04Cff10f00D, 10);
        _safeMint(0x98845CFA79B5Fa7878cB7BC203b8bF1429Ec4e7e, 10);
        _safeMint(0xd83dFa6E5301A3A98972ef6F1109927Ed48aAbf9, 10);
        _safeMint(0x9590Ea8123396623d109ef502b05659E9Ab59584, 10);
        _safeMint(0xe818E86d00670559c15A0943F37280CfFca1CB2E, 10);
        _safeMint(0x5fA89a1a3fef2c4Ca7083d4Dd1f6509dEee25df7, 10);
        _safeMint(0x327993A6950c0BD11F2f31511E42949DA5E8DaFb, 10);
        _safeMint(0x95EBF2A0EfEbd053C576806bbfC007ab80fB9870, 10);
        _safeMint(0x565E5E99ECe7aD636bAeffd162a1D9B7A6e5aC8e, 10);
        _safeMint(0xd6FeB6d54a254D5408b072B5CB1E43606eeEb2f7, 10);
        _safeMint(0x7b50700534cc27bD9aD321A475Fd136f7Fc0a333, 10);
    }

    function togglePublicSale() external onlyOwner {
        publicSale = !publicSale;
    }

    function toggleReserveSale() external onlyOwner {
        reservelistSale = !reservelistSale;
    }

    function setBaseURI(string memory _newBaseURI) external onlyOwner {
        baseURI = _newBaseURI;
    }

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

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

    //change max mint for wl
    function setMaxWhitelistMint(uint256 _newMaxWhitelistMint) external onlyOwner {
        maxWhitelistMint = _newMaxWhitelistMint;
    }

    //change max mint for publix
    function setMaxPublicMint(uint256 _newMaxPublicMint) external onlyOwner {
        maxPublicMint = _newMaxPublicMint;
    }

    //wl only mint
    function whitelistMint(uint256 tokens, bytes32[] calldata merkleProof) external {
        require(whitelistSale, "BAGS: You can not mint right now");
        require(MerkleProof.verify(merkleProof, merkleRoot, keccak256(abi.encodePacked(msg.sender))), "BAGS: Please wait to mint on public sale");
        require(_whitelistClaimed[_msgSender()] + tokens <= maxWhitelistMint, "BAGS: Cannot mint this many BAGS");
        require(tokens > 0, "BAGS: Please mint at least 1 BAGS");

        _whitelistClaimed[_msgSender()] += tokens;
        _safeMint(_msgSender(), tokens);
    }

    //reserve only mint
    function reserveMint(uint256 tokens, bytes32[] calldata merkleProof) external {
        require(reservelistSale, "BAGS: You can not mint right now");
        require(MerkleProof.verify(merkleProof, merkleRoot, keccak256(abi.encodePacked(msg.sender))), "BAGS: Please wait to mint on public sale");
        require(_reserveClaimed[_msgSender()] + tokens <= maxWhitelistMint, "BAGS: Cannot mint this many BAGS");
        require(tokens > 0, "BAGS: Please mint at least 1 BAGS");

        _whitelistClaimed[_msgSender()] += tokens;
        _reserveClaimed[_msgSender()] += tokens;
        _safeMint(_msgSender(), tokens);
    }

    //mint function for public
    function mint(uint256 tokens) external {
        require(publicSale, "BAGS: Public sale has not started");
        require(totalSupply() + tokens <= MAX_TOKENS, "BAGS: Exceeded supply");
        require(_publicClaimed[_msgSender()] + tokens <= maxPublicMint, "BAGS: Cannot mint this many BAGS");
        require(tokens > 0, "BAGS: Please mint at least 1 BAGS");

        _publicClaimed[_msgSender()] +=tokens;
        _safeMint(_msgSender(), tokens);
    }

    // No restrictions. use for giveaways, airdrops, etc
    function airdrop(address to, uint256 tokens) external onlyOwner {
        require(totalSupply() + tokens <= MAX_TOKENS, "BAGS: Minting would exceed max supply");
        require(tokens > 0, "BAGS: Must mint at least one token");
        _safeMint(to, tokens);
    }
}

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"},{"inputs":[],"name":"URIQueryForNonexistentToken","type":"error"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"approved","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Approval","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"operator","type":"address"},{"indexed":false,"internalType":"bool","name":"approved","type":"bool"}],"name":"ApprovalForAll","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"previousOwner","type":"address"},{"indexed":true,"internalType":"address","name":"newOwner","type":"address"}],"name":"OwnershipTransferred","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Transfer","type":"event"},{"inputs":[],"name":"MAX_TOKENS","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"_publicClaimed","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"_reserveClaimed","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"_whitelistClaimed","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokens","type":"uint256"}],"name":"airdrop","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"airdropTheBags","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"approve","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"}],"name":"balanceOf","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"baseURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"getApproved","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"},{"internalType":"address","name":"operator","type":"address"}],"name":"isApprovedForAll","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxPublicMint","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxWhitelistMint","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"merkleRoot","outputs":[{"internalType":"bytes32","name":"","type":"bytes32"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokens","type":"uint256"}],"name":"mint","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"name","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"owner","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"ownerOf","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"publicSale","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokens","type":"uint256"},{"internalType":"bytes32[]","name":"merkleProof","type":"bytes32[]"}],"name":"reserveMint","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"reservelistSale","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"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":"_newBaseURI","type":"string"}],"name":"setBaseURI","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_newMaxPublicMint","type":"uint256"}],"name":"setMaxPublicMint","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_newMaxWhitelistMint","type":"uint256"}],"name":"setMaxWhitelistMint","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"_merkleRoot","type":"bytes32"}],"name":"setMerkleRoot","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes4","name":"interfaceId","type":"bytes4"}],"name":"supportsInterface","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"symbol","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"togglePublicSale","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"toggleReserveSale","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"toggleWhitelistSale","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"tokenURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"totalSupply","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"transferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"newOwner","type":"address"}],"name":"transferOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokens","type":"uint256"},{"internalType":"bytes32[]","name":"merkleProof","type":"bytes32[]"}],"name":"whitelistMint","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"whitelistSale","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"}]

608060405260016009556001600a556000600b60006101000a81548160ff0219169083151502179055506000600b60016101000a81548160ff0219169083151502179055506000600b60026101000a81548160ff02191690831515021790555060405180602001604052806000815250600f9080519060200190620000869291906200026b565b507fb067a20ba5ddd291ea422f36db1f2bf093d80e72c2c0f9f11320e8712a6a4f6e60001b601055348015620000bb57600080fd5b506040518060400160405280600a81526020017f426167486f6c64657273000000000000000000000000000000000000000000008152506040518060400160405280600481526020017f42414753000000000000000000000000000000000000000000000000000000008152508160029080519060200190620001409291906200026b565b508060039080519060200190620001599291906200026b565b506200016a6200019860201b60201c565b600081905550505062000192620001866200019d60201b60201c565b620001a560201b60201c565b62000380565b600090565b600033905090565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b82805462000279906200034a565b90600052602060002090601f0160209004810192826200029d5760008555620002e9565b82601f10620002b857805160ff1916838001178555620002e9565b82800160010185558215620002e9579182015b82811115620002e8578251825591602001919060010190620002cb565b5b509050620002f89190620002fc565b5090565b5b8082111562000317576000816000905550600101620002fd565b5090565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b600060028204905060018216806200036357607f821691505b602082108114156200037a57620003796200031b565b5b50919050565b6153a780620003906000396000f3fe608060405234801561001057600080fd5b50600436106102485760003560e01c806370a082311161013b578063a22cb465116100b8578063e222c7f91161007c578063e222c7f91461068f578063e985e9c514610699578063ee419b89146106c9578063f2fde38b146106e5578063f47c84c51461070157610248565b8063a22cb465146105ed578063b88d4fde14610609578063c87b56dd14610625578063cabadaa014610655578063d2cab0561461067357610248565b8063851a7708116100ff578063851a7708146105495780638ba4cc3c146105795780638da5cb5b1461059557806395d89b41146105b3578063a0712d68146105d157610248565b806370a08231146104a7578063715018a6146104d757806371978011146104e15780637cb64759146104fd5780637f09e66f1461051957610248565b806331ffd6f1116101c957806359eda1b51161018d57806359eda1b51461041557806363439e611461041f5780636352211e1461044f5780636c0360eb1461047f5780636f02f62c1461049d57610248565b806331ffd6f11461038357806333bc1c5c146103a1578063423f74c9146103bf57806342842e0e146103dd57806355f804b3146103f957610248565b806318160ddd1161021057806318160ddd146102f157806323b872dd1461030f578063270ab52c1461032b5780632eb4a7ab14610347578063309a36861461036557610248565b806301ffc9a71461024d578063034d77941461027d57806306fdde0314610287578063081812fc146102a5578063095ea7b3146102d5575b600080fd5b610267600480360381019061026291906142fe565b61071f565b6040516102749190614346565b60405180910390f35b610285610801565b005b61028f610835565b60405161029c91906143fa565b60405180910390f35b6102bf60048036038101906102ba9190614452565b6108c7565b6040516102cc91906144c0565b60405180910390f35b6102ef60048036038101906102ea9190614507565b610943565b005b6102f9610a4e565b6040516103069190614556565b60405180910390f35b61032960048036038101906103249190614571565b610a65565b005b61034560048036038101906103409190614452565b610a75565b005b61034f610a87565b60405161035c91906145dd565b60405180910390f35b61036d610a8d565b60405161037a9190614556565b60405180910390f35b61038b610a93565b6040516103989190614346565b60405180910390f35b6103a9610aa6565b6040516103b69190614346565b60405180910390f35b6103c7610ab9565b6040516103d49190614346565b60405180910390f35b6103f760048036038101906103f29190614571565b610acc565b005b610413600480360381019061040e919061472d565b610aec565b005b61041d610b0e565b005b61043960048036038101906104349190614776565b610b42565b6040516104469190614556565b60405180910390f35b61046960048036038101906104649190614452565b610b5a565b60405161047691906144c0565b60405180910390f35b610487610b70565b60405161049491906143fa565b60405180910390f35b6104a5610bfe565b005b6104c160048036038101906104bc9190614776565b612230565b6040516104ce9190614556565b60405180910390f35b6104df612300565b005b6104fb60048036038101906104f69190614452565b612314565b005b610517600480360381019061051291906147cf565b612326565b005b610533600480360381019061052e9190614776565b612338565b6040516105409190614556565b60405180910390f35b610563600480360381019061055e9190614776565b612350565b6040516105709190614556565b60405180910390f35b610593600480360381019061058e9190614507565b612368565b005b61059d612418565b6040516105aa91906144c0565b60405180910390f35b6105bb612442565b6040516105c891906143fa565b60405180910390f35b6105eb60048036038101906105e69190614452565b6124d4565b005b61060760048036038101906106029190614828565b6126c4565b005b610623600480360381019061061e9190614909565b61283c565b005b61063f600480360381019061063a9190614452565b6128b8565b60405161064c91906143fa565b60405180910390f35b61065d612957565b60405161066a9190614556565b60405180910390f35b61068d600480360381019061068891906149ec565b61295d565b005b610697612bab565b005b6106b360048036038101906106ae9190614a4c565b612bdf565b6040516106c09190614346565b60405180910390f35b6106e360048036038101906106de91906149ec565b612c73565b005b6106ff60048036038101906106fa9190614776565b612f1e565b005b610709612fa2565b6040516107169190614556565b60405180910390f35b60007f80ac58cd000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff191614806107ea57507f5b5e139f000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b806107fa57506107f982612fa8565b5b9050919050565b610809613012565b600b60029054906101000a900460ff1615600b60026101000a81548160ff021916908315150217905550565b60606002805461084490614abb565b80601f016020809104026020016040519081016040528092919081815260200182805461087090614abb565b80156108bd5780601f10610892576101008083540402835291602001916108bd565b820191906000526020600020905b8154815290600101906020018083116108a057829003601f168201915b5050505050905090565b60006108d282613090565b610908576040517fcf4700e400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6006600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff169050919050565b600061094e82610b5a565b90508073ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff1614156109b6576040517f943f7b8c00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8073ffffffffffffffffffffffffffffffffffffffff166109d56130de565b73ffffffffffffffffffffffffffffffffffffffff1614158015610a075750610a0581610a006130de565b612bdf565b155b15610a3e576040517fcfb3b94200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b610a498383836130e6565b505050565b6000610a58613198565b6001546000540303905090565b610a7083838361319d565b505050565b610a7d613012565b80600a8190555050565b60105481565b60095481565b600b60019054906101000a900460ff1681565b600b60009054906101000a900460ff1681565b600b60029054906101000a900460ff1681565b610ae78383836040518060200160405280600081525061283c565b505050565b610af4613012565b80600f9080519060200190610b0a9291906141ac565b5050565b610b16613012565b600b60019054906101000a900460ff1615600b60016101000a81548160ff021916908315150217905550565b600d6020528060005260406000206000915090505481565b6000610b6582613653565b600001519050919050565b600f8054610b7d90614abb565b80601f0160208091040260200160405190810160405280929190818152602001828054610ba990614abb565b8015610bf65780601f10610bcb57610100808354040283529160200191610bf6565b820191906000526020600020905b815481529060010190602001808311610bd957829003601f168201915b505050505081565b610c06613012565b610c257385c0b44d3b9a49b09c3b925af5c935043e66dfbf60026138e2565b610c4473b110f4cf6660e3003c421254bf1568ca79598a5e60026138e2565b610c637339cb13625945bf0eb05579ad6c79f748dacd9b2060026138e2565b610c8273740f471701d09e268efc991f8332b172093d74dd60026138e2565b610ca173b522a6619d74546cffe9fcbec27da5d2c5d1806660026138e2565b610cc073c2b142beb125579e98c16ced36629a2d1c3d584160026138e2565b610cdf7326be72cbbf5746f14d731fd4febf294cae376f5960026138e2565b610cfe731342bd2ab6065379502de00afd81d4a987318a5e60026138e2565b610d1d73635bf1dfe7301a560e6fb5fef4bb9902b5966ed360026138e2565b610d3c730e16f4a678f7facdcf58c9adf947e8e48845e57560026138e2565b610d5b7355b0d5ef132c1a46e3d18409649ea18351cfef9a60026138e2565b610d7a73610243745476e23ef7c17f23168f3e5e774390e260026138e2565b610d99739a430a8be98da5ac1a2fb6f8f53e8fe794de611e60026138e2565b610db873e15bb22ce00ea25aa62bea202ac1008932f4d78560026138e2565b610dd773a22aae6a5ecde5cc8abe49e32165366c0d70ad6360026138e2565b610df673f6f435a13a38149ef954bb391f16d8010380dd4a60026138e2565b610e1573b7c5121a82493dece1cd4143e0571fcc49afbffd60026138e2565b610e34735d1928b9062e34de640b1117efcc81b90b45269360026138e2565b610e5373f95c508fa8686279294ea69f2deae18c0bc3c99c60026138e2565b610e7273175e89eeb246f66ce664df16f5f046610b86751360026138e2565b610e9173eca78934fdb00a2dadd9a29cf3d45bef5b3c8e9c60026138e2565b610eb073a66489ada4f1b94eacefe5fc27f3674deb407fbd60026138e2565b610ecf7305f885113100771a1bdb5c22e7dadb3acb149e3f60026138e2565b610eee7397eec19136e7ab1cb0a0f4a4c47ee2d55a993c4060026138e2565b610f0d73bb08a962380b9a1e49f20d6c3bdc81075914b0cd60026138e2565b610f2c73dc64b93ccd63d2354a32bbcd2d460735d341415d60026138e2565b610f4b73551d196803c99dc4e2bf68cb9b61d4c597749db060026138e2565b610f6a73dca699c2b0e88f2f06aebe96172fa09d463a4d2760026138e2565b610f897314c30c5d33961c2f4d2cd2d1ab584bbbff0a635e60026138e2565b610fa8733e357db18182f7a597cf49d0c40b692706fa7b2f60026138e2565b610fc773d91473629d8b46a8eb44eb6349a568a7ea7a176f60026138e2565b610fe673aa898615d42efd369e151448a992af897e32f56660026138e2565b61100573e09cf2ac74009200bbff7455ff3f69db5fb49a1060026138e2565b611024739ccbdd887a92d13c04f6c846a2cf514871474ceb60026138e2565b611043730b26454ad48f3651f1cc1abcd2e590301ce9355660026138e2565b61106273d74b8b30ce6269bab58b64b58245da55499b151060026138e2565b61108173bf1016f104996d33007b041e38c1bee6e7fb5d4460026138e2565b6110a0735343a7a198eb41e42661f2f8772a4e6c5f1c6b1c60026138e2565b6110bf73c18c9b1b03ce38425e1c21b720f406f1659002b060026138e2565b6110de738d6d968b5ebbd66bc79cc1085e0854311ff523d760026138e2565b6110fd73ad25c92baf8564849769224e00316d56dfa5491d60026138e2565b61111c73382e00f0edae8b5bcb9398d70c1d192bb699d8b760026138e2565b61113b73b3e010f154c03bfdbd141b563a1b92b5dd206f8260026138e2565b61115a7354558a1998c1a2cbff086449710d28fb7561fe2660026138e2565b61117973580215e9a04f5bb3c03c4f211f91a5ea01411ca160026138e2565b61119873495777e73d7977aae1f562c40796c2c7772b29b560026138e2565b6111b773aa86ad45c43b69315fb97d6daaa0034939dda34f60026138e2565b6111d673eac290b74b14166f15ba296ec123985cee96a69360026138e2565b6111f573721cc6751b48bbcbf3e24fa72cc5bf932783279d60026138e2565b61121473102898958bbf5799f82774a4c4b692d07c59aa7760026138e2565b6112337310c9374bddda68929f712515877d6b592a2bf10960026138e2565b61125172d7a43af16bfefcc180ecf069276b0d726d4b4060026138e2565b6112707339b3fb116e5f5ce90ab0a7bf8545e67c451c626360026138e2565b61128f738cc186f220a2f939a8e7d9dcea340697426d2daa60026138e2565b6112ae73ad644370bc6b596643d7be9e3190a90d25c6234660026138e2565b6112cd73ca17d93e772ad78304a9cf9f5c7ed15e20c9705260026138e2565b6112ec732861d3c46aad60e971ae8fa5e379af129d63e74560026138e2565b61130b73f2f3b5344c0f2e87a2e613c4425ec3906652fed960026138e2565b61132a73603889de8cae2431251e20fe850beda492a7ff6c60026138e2565b611349732f8404f2c087ed5ea1c42ba9e8392641377a71ab60026138e2565b611368739490c0aeeb1ba7ad1b871b2104c5fce4a132362560026138e2565b61138773ad9435432e85acf64173262fce0f977552a49c2e60026138e2565b6113a673f3d7af96a0c09e4c7a59a75c9bd10b89bd60158c60026138e2565b6113c57336b5b82e0598f2d79592289da87b37401b740f2260026138e2565b6113e473a0d3d72516a042e310c459c63dc664182a5308b960026138e2565b6114037388fa0374b2aba0f6af85fc45702f9513d27c255a60026138e2565b611422739a971b4943ef05cde48481f5bafee1003feeef4d60026138e2565b611441730e0a2c07dab0f1ae64cb1fdb6209c1a01d5fb88760026138e2565b6114607307ee856e17a0f9181644511f4801ed29b03288a460026138e2565b61147f739c2406669c9faebbe964d5da5429d3a320652fb860026138e2565b61149e73ac2cd9b5deaa7a3d79ac73de676989eb4978811860026138e2565b6114bd738ecd31cd9f47f4a0fcd0a82eec0445aab518376d60026138e2565b6114dc735646d2e9a7e16ba92239afd071c0c2495c31cf2c60026138e2565b6114fb73c8dfcfe493b268aa325579fb190181c564141a5960026138e2565b61151a738a5675a207cc7174d7e3b4961aa7e9fcd1234ccf60026138e2565b61153973ad406876a8c7a78de7fcff412cb0276d4bdeb68e60026138e2565b611558738945ed77e8900a3b7855bf703c192c7979b473cf60026138e2565b611577732b4775773fd8f49667864208bde1450c4ae21c0360026138e2565b61159673871bf5306dab778dcc0e97166fb9a3b9e5b93d0460026138e2565b6115b5732e7d8196b52256da7b1d5ea22eb8f05686ab3cd160026138e2565b6115d47326ccb82ed08b0f8f1ca0086d5b279d5ba132a8a260026138e2565b6115f373d39b2014ef25ee95f1aede9f1d04ea6a959cf9f660026138e2565b6116127364247785234f7bdae872b9a9222920e4eebf7d5460026138e2565b611631732653e96428088ffaa8c373ba81f5b31bf59ec2f460026138e2565b611650735b3228bacb642a02cfa4763b84e4d116e6c2b70960026138e2565b61166f73eb55b194379d0468bbd734cd08b41d9097f90d0960026138e2565b61168e733a15a2bd61b95c93e4da375538f054309c4380b360026138e2565b6116ad730d85fb3d7ff838d4e6c52f52d810420fbe3819f060026138e2565b6116cc73bd44f279590d4a81a29b63e2c65119c44cdb258160026138e2565b6116eb730e1a70ed924bc4f3c57c454d7833c46911a9d84960026138e2565b61170a731796c568d22240d63b9566328eab535a3968f8c360026138e2565b61172973397280745af703fbb38e1c591524f92d42a57b8960026138e2565b611748739056b05a07d4bb085f64127f39d6faed2ed4808b60026138e2565b61176773069ba33753343b3e73661f06eb7d0a71b3813b4a60026138e2565b611786734de6967967a3c9001d14ff57ad42d879d7e0512460026138e2565b6117a573a0915e1c7e4c2543ecb05c423e8e7a0db31213a760026138e2565b6117c473ca83c9dfdfffc4aaae66f52906566f5d58f24e3160026138e2565b6117e373e89b3dca875bd1c74bd9b22703a487472568e03060026138e2565b611802731507dbf6196a6e1ab160275ec43c6baa30d1a19760026138e2565b61182173b4dbcd527c8ebc09b00c4bdd506a23894604b8a060026138e2565b611840731fec03eb0dbd4190deb139e429a9de6c29de70a660026138e2565b61185f732fad4d2f4bd33e0ae89c776568d2f1c2c92ddb7060026138e2565b61187e732746e48720bf4464b6cc334056cb540148760a3860026138e2565b61189d732284a738f2d84a4d035fe8121a039e79a09547ff60026138e2565b6118bc735d37445e60c6de44c9327ec8bb300e876c3d571360026138e2565b6118db73d6dfd56ab8a116ed6370984945feb8be7d6c322160026138e2565b6118fa73b03f4d215e2ef5986b763b45bdf53e330be38d6260026138e2565b61191973eb89b2499077c01c094b8398a98a11a3087cbb3b60026138e2565b61193873280b5ec890809a98435b84f0cdb56714b16a4c9160026138e2565b611957739b7f79e13768e4daba808492e59caf16aaac952e60026138e2565b61197673863581c07688d990210c0fda40cb2347de9dc87360026138e2565b61199573b38319ac1308ddcf15e3cd8f6d67d26f424279e560026138e2565b6119b473e09adcc2854c3299a2886d0dfeb03ed2a3df63d060026138e2565b6119d373a6769fa1625845ca606a6aa3c8056bc2982c107660026138e2565b6119f273e30bfb74c86a316f4e03d42c8f261324cdd2517360026138e2565b611a11735dc73c27933411916d612c55a074bf38e3b75a9760026138e2565b611a307321dcb6f533d13166abb801390744d0bff8a546a060026138e2565b611a4f73fb8d3bdd6da52f65227a6a17f96c939e5390832660026138e2565b611a6e73dd41ade62481e69f171d758a14680a060b42fc4460026138e2565b611a8d73ee04770359f9363a5d67a7f80f6ac4122dfb970e60026138e2565b611aac730e999151217a907b2c4ddb90bec16f05b263f92360026138e2565b611acb737bd02565e438c7eb709313ac5a7c15d023e6f98560026138e2565b611aea73abf35f4981b9497d01d951d7577bf0de21ffaa2b60026138e2565b611b0973f88f8d5edf096576c5ecfbb51b1fc12e8a144fa460026138e2565b611b287332502a4d1c96273fe62669165a64b8a39f4512b460026138e2565b611b4773edad44d3d2c67e30beb056a68fef514d0e52baaf60026138e2565b611b6673d9bded47b38999bb8c584a051b6b0e7ed39aafd860026138e2565b611b8573e53b6f0f2cff473e7fc31adc712112351f411b2b60026138e2565b611ba47325e4b97cc81eb2ff49a719edd86de91d47531da760026138e2565b611bc37385e5e02efb864b609a587c522c7148c662730ad560026138e2565b611be273c8c5df49795e3f5e2943eebff50c3cc9fb8d496760026138e2565b611c01734f2793344c2cf3a4c18305ba834da0d7188bcaf260026138e2565b611c20734fbb8130a8ddc899c879c445abf15463c29f1dc560026138e2565b611c3f73eb7cf8c3f5e4425d6426fd84a5f8afd68569a64f60026138e2565b611c5e732de09e956a252203a60a36f9ca143ecee336d82760026138e2565b611c7d736173b476b12cc40099f6e6fa6c064d6ee2ab493a60026138e2565b611c9c73c59e912fc173f7d62af19d405816970dae7384f860026138e2565b611cbb731697a4e259bc568814cc575d29b878b6992d5f9c60026138e2565b611cda73b080d6f42d774818bb9549492147917727c11dac60026138e2565b611cf973832c5dd5be10b8a188f858b41e6bf426ae6917ac60026138e2565b611d1873dcdf84646166e015496c51e5d9099f52ae75390360026138e2565b611d3773ce504f9d1f95ab5dce9c8318393b95b351c6c86860026138e2565b611d567324a6ae8d89da1d0ba1d8a3c3012216bfc0d9988860026138e2565b611d7573c5dc0a1064fdde66962a2b449057fe339f4d86fb60026138e2565b611d947307197ecaf257a64502fd5fe6a0d5bf31dbcba08160026138e2565b611db3736590592b2c2753f3c5c564430f6ef12c11a82cd160026138e2565b611dd273861dd17c9fea84f9d8bc6d32c34b90f4ec6317fb60026138e2565b611df173ba5e8d9dccf97a200b30f54f4ec5edbe2fe92ed160026138e2565b611e107319b191f625518c85c54c5d672e7fc9440f1824e060026138e2565b611e2f7340f085176beaa2fc417164d4b8e7399c4addef7760026138e2565b611e4e7361d3d2452448f9f78380ff40d924855719029fb060026138e2565b611e6d7354c5bc3e9ca2ce0b69af1d5102f6f8fb268a751360026138e2565b611e8c7344bb5f45f3f447e90200d61ec4c68f41ccff37ff60026138e2565b611eab73dec2c041b3b5dc8ed7b77b87f6a986fe225bf30e60026138e2565b611eca73213571f3b8b8cc8f463c42d994c3f5e2c34fa3f060026138e2565b611ee97358217e3c57a74b9bf6c539a755c2b0e417162a9c60026138e2565b611f08738bc539f3cfb68c28d52102180a877dcf7db476ae60026138e2565b611f277370919456288650894fd2dce95ed78bbe57dfdbf660026138e2565b611f467304b2cb5bb145e6ba3d67c9debcc14c461c9a968d60026138e2565b611f657331e58ede8f0e39dc832bdaf992cbe9ef3c70f54560026138e2565b611f8473daea44d64813a1a4bba1b2a61c10d915234bf10560026138e2565b611fa3736a5b8c260f6ece3b361a1998da609335d618ac4860026138e2565b611fc273ad74b2fca61ab5e987907f3da9825776f53e6c0260026138e2565b611fe1737268146ddca1b4917758456041764b8ec4317dde60026138e2565b6120007397d93f8a99c74faad615f56ebf27654d63a34a5d60026138e2565b61201f7362a79a85e34db40fac6f422bfaf1cb86d15c550e600a6138e2565b61203e73d27d1c330b89a11c2b62613e22be40bc19d4351e600a6138e2565b61205d73fd3f1300948ecf87677e54120ed7c1fe151c53c3600a6138e2565b61207c733832a2adbb1f55b284f67daccdbe8effc01128e5600a6138e2565b61209b738e893de17ee6c3d2c725502ab3a0614779c3cccb600a6138e2565b6120ba73f7cb1accfae480283b9560a0b1d614663033d876600a6138e2565b6120d973739b51ce1645e4e13ff1a87e93013c3fd3360ed9600a6138e2565b6120f873d2d6d1de0577e1feb65279d3d291d04cff10f00d600a6138e2565b6121177398845cfa79b5fa7878cb7bc203b8bf1429ec4e7e600a6138e2565b61213673d83dfa6e5301a3a98972ef6f1109927ed48aabf9600a6138e2565b612155739590ea8123396623d109ef502b05659e9ab59584600a6138e2565b61217473e818e86d00670559c15a0943f37280cffca1cb2e600a6138e2565b612193735fa89a1a3fef2c4ca7083d4dd1f6509deee25df7600a6138e2565b6121b273327993a6950c0bd11f2f31511e42949da5e8dafb600a6138e2565b6121d17395ebf2a0efebd053c576806bbfc007ab80fb9870600a6138e2565b6121f073565e5e99ece7ad636baeffd162a1d9b7a6e5ac8e600a6138e2565b61220f73d6feb6d54a254d5408b072b5cb1e43606eeeb2f7600a6138e2565b61222e737b50700534cc27bd9ad321a475fd136f7fc0a333600a6138e2565b565b60008073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415612298576040517f8f4eb60400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600560008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160009054906101000a900467ffffffffffffffff1667ffffffffffffffff169050919050565b612308613012565b6123126000613900565b565b61231c613012565b8060098190555050565b61232e613012565b8060108190555050565b600e6020528060005260406000206000915090505481565b600c6020528060005260406000206000915090505481565b612370613012565b611e618161237c610a4e565b6123869190614b1c565b11156123c7576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016123be90614be4565b60405180910390fd5b6000811161240a576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161240190614c76565b60405180910390fd5b61241482826138e2565b5050565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b60606003805461245190614abb565b80601f016020809104026020016040519081016040528092919081815260200182805461247d90614abb565b80156124ca5780601f1061249f576101008083540402835291602001916124ca565b820191906000526020600020905b8154815290600101906020018083116124ad57829003601f168201915b5050505050905090565b600b60009054906101000a900460ff16612523576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161251a90614d08565b60405180910390fd5b611e618161252f610a4e565b6125399190614b1c565b111561257a576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161257190614d74565b60405180910390fd5b600a5481600e600061258a6130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020546125cf9190614b1c565b1115612610576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161260790614de0565b60405180910390fd5b60008111612653576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161264a90614e72565b60405180910390fd5b80600e60006126606130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282546126a99190614b1c565b925050819055506126c16126bb6130de565b826138e2565b50565b6126cc6130de565b73ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415612731576040517fb06307db00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b806007600061273e6130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060006101000a81548160ff0219169083151502179055508173ffffffffffffffffffffffffffffffffffffffff166127eb6130de565b73ffffffffffffffffffffffffffffffffffffffff167f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31836040516128309190614346565b60405180910390a35050565b61284784848461319d565b6128668373ffffffffffffffffffffffffffffffffffffffff166139c6565b801561287b5750612879848484846139e9565b155b156128b2576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b50505050565b60606128c382613090565b6128f9576040517fa14c4b5000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6000612903613b3a565b9050600081511415612924576040518060200160405280600081525061294f565b8061292e84613bcc565b60405160200161293f929190614ece565b6040516020818303038152906040525b915050919050565b600a5481565b600b60019054906101000a900460ff166129ac576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016129a390614f3e565b60405180910390fd5b612a20828280806020026020016040519081016040528093929190818152602001838360200280828437600081840152601f19601f8201169050808301925050505050505060105433604051602001612a059190614fa6565b60405160208183030381529060405280519060200120613d2d565b612a5f576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612a5690615033565b60405180910390fd5b60095483600c6000612a6f6130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054612ab49190614b1c565b1115612af5576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612aec90614de0565b60405180910390fd5b60008311612b38576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612b2f90614e72565b60405180910390fd5b82600c6000612b456130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254612b8e9190614b1c565b92505081905550612ba6612ba06130de565b846138e2565b505050565b612bb3613012565b600b60009054906101000a900460ff1615600b60006101000a81548160ff021916908315150217905550565b6000600760008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff16905092915050565b600b60029054906101000a900460ff16612cc2576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612cb990614f3e565b60405180910390fd5b612d36828280806020026020016040519081016040528093929190818152602001838360200280828437600081840152601f19601f8201169050808301925050505050505060105433604051602001612d1b9190614fa6565b60405160208183030381529060405280519060200120613d2d565b612d75576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612d6c90615033565b60405180910390fd5b60095483600d6000612d856130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054612dca9190614b1c565b1115612e0b576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612e0290614de0565b60405180910390fd5b60008311612e4e576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612e4590614e72565b60405180910390fd5b82600c6000612e5b6130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254612ea49190614b1c565b9250508190555082600d6000612eb86130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254612f019190614b1c565b92505081905550612f19612f136130de565b846138e2565b505050565b612f26613012565b600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff161415612f96576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612f8d906150c5565b60405180910390fd5b612f9f81613900565b50565b611e6181565b60007f01ffc9a7000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916149050919050565b61301a6130de565b73ffffffffffffffffffffffffffffffffffffffff16613038612418565b73ffffffffffffffffffffffffffffffffffffffff161461308e576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161308590615131565b60405180910390fd5b565b60008161309b613198565b111580156130aa575060005482105b80156130d7575060046000838152602001908152602001600020600001601c9054906101000a900460ff16155b9050919050565b600033905090565b826006600084815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550818373ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff167f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92560405160405180910390a4505050565b600090565b60006131a882613653565b90508373ffffffffffffffffffffffffffffffffffffffff16816000015173ffffffffffffffffffffffffffffffffffffffff1614613213576040517fa114810000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b60008473ffffffffffffffffffffffffffffffffffffffff166132346130de565b73ffffffffffffffffffffffffffffffffffffffff16148061326357506132628561325d6130de565b612bdf565b5b806132a857506132716130de565b73ffffffffffffffffffffffffffffffffffffffff16613290846108c7565b73ffffffffffffffffffffffffffffffffffffffff16145b9050806132e1576040517f59c896be00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff161415613348576040517fea553b3400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6133558585856001613d44565b613361600084876130e6565b6001600560008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160392506101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055506001600560008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055506000600460008581526020019081526020016000209050848160000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550428160000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff16021790555060006001850190506000600460008381526020019081526020016000209050600073ffffffffffffffffffffffffffffffffffffffff168160000160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1614156135e15760005482146135e057878160000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555084602001518160000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055505b5b505050828473ffffffffffffffffffffffffffffffffffffffff168673ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a461364c8585856001613d4a565b5050505050565b61365b614232565b600082905080613669613198565b11158015613678575060005481105b156138ab576000600460008381526020019081526020016000206040518060600160405290816000820160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020016000820160149054906101000a900467ffffffffffffffff1667ffffffffffffffff1667ffffffffffffffff16815260200160008201601c9054906101000a900460ff161515151581525050905080604001516138a957600073ffffffffffffffffffffffffffffffffffffffff16816000015173ffffffffffffffffffffffffffffffffffffffff161461378d5780925050506138dd565b5b6001156138a857818060019003925050600460008381526020019081526020016000206040518060600160405290816000820160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020016000820160149054906101000a900467ffffffffffffffff1667ffffffffffffffff1667ffffffffffffffff16815260200160008201601c9054906101000a900460ff1615151515815250509050600073ffffffffffffffffffffffffffffffffffffffff16816000015173ffffffffffffffffffffffffffffffffffffffff16146138a35780925050506138dd565b61378e565b5b505b6040517fdf2d9b4200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b919050565b6138fc828260405180602001604052806000815250613d50565b5050565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b6000808273ffffffffffffffffffffffffffffffffffffffff163b119050919050565b60008373ffffffffffffffffffffffffffffffffffffffff1663150b7a02613a0f6130de565b8786866040518563ffffffff1660e01b8152600401613a3194939291906151a6565b6020604051808303816000875af1925050508015613a6d57506040513d601f19601f82011682018060405250810190613a6a9190615207565b60015b613ae7573d8060008114613a9d576040519150601f19603f3d011682016040523d82523d6000602084013e613aa2565b606091505b50600081511415613adf576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b805181602001fd5b63150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916817bffffffffffffffffffffffffffffffffffffffffffffffffffffffff191614915050949350505050565b6060600f8054613b4990614abb565b80601f0160208091040260200160405190810160405280929190818152602001828054613b7590614abb565b8015613bc25780601f10613b9757610100808354040283529160200191613bc2565b820191906000526020600020905b815481529060010190602001808311613ba557829003601f168201915b5050505050905090565b60606000821415613c14576040518060400160405280600181526020017f30000000000000000000000000000000000000000000000000000000000000008152509050613d28565b600082905060005b60008214613c46578080613c2f90615234565b915050600a82613c3f91906152ac565b9150613c1c565b60008167ffffffffffffffff811115613c6257613c61614602565b5b6040519080825280601f01601f191660200182016040528015613c945781602001600182028036833780820191505090505b5090505b60008514613d2157600182613cad91906152dd565b9150600a85613cbc9190615311565b6030613cc89190614b1c565b60f81b818381518110613cde57613cdd615342565b5b60200101907effffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916908160001a905350600a85613d1a91906152ac565b9450613c98565b8093505050505b919050565b600082613d3a8584614114565b1490509392505050565b50505050565b50505050565b600080549050600073ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff161415613dbd576040517f2e07630000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6000831415613df8576040517fb562e8dd00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b613e056000858386613d44565b82600560008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff16021790555082600560008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160088282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff160217905550836004600083815260200190815260200160002060000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550426004600083815260200190815260200160002060000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff160217905550600081905060008482019050613fc68673ffffffffffffffffffffffffffffffffffffffff166139c6565b1561408c575b818673ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a461403b60008784806001019550876139e9565b614071576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b80821415613fcc57826000541461408757600080fd5b6140f8565b5b818060010192508673ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a48082141561408d575b81600081905550505061410e6000858386613d4a565b50505050565b60008082905060005b845181101561415f5761414a8286838151811061413d5761413c615342565b5b602002602001015161416a565b9150808061415790615234565b91505061411d565b508091505092915050565b60008183106141825761417d8284614195565b61418d565b61418c8383614195565b5b905092915050565b600082600052816020526040600020905092915050565b8280546141b890614abb565b90600052602060002090601f0160209004810192826141da5760008555614221565b82601f106141f357805160ff1916838001178555614221565b82800160010185558215614221579182015b82811115614220578251825591602001919060010190614205565b5b50905061422e9190614275565b5090565b6040518060600160405280600073ffffffffffffffffffffffffffffffffffffffff168152602001600067ffffffffffffffff1681526020016000151581525090565b5b8082111561428e576000816000905550600101614276565b5090565b6000604051905090565b600080fd5b600080fd5b60007fffffffff0000000000000000000000000000000000000000000000000000000082169050919050565b6142db816142a6565b81146142e657600080fd5b50565b6000813590506142f8816142d2565b92915050565b6000602082840312156143145761431361429c565b5b6000614322848285016142e9565b91505092915050565b60008115159050919050565b6143408161432b565b82525050565b600060208201905061435b6000830184614337565b92915050565b600081519050919050565b600082825260208201905092915050565b60005b8381101561439b578082015181840152602081019050614380565b838111156143aa576000848401525b50505050565b6000601f19601f8301169050919050565b60006143cc82614361565b6143d6818561436c565b93506143e681856020860161437d565b6143ef816143b0565b840191505092915050565b6000602082019050818103600083015261441481846143c1565b905092915050565b6000819050919050565b61442f8161441c565b811461443a57600080fd5b50565b60008135905061444c81614426565b92915050565b6000602082840312156144685761446761429c565b5b60006144768482850161443d565b91505092915050565b600073ffffffffffffffffffffffffffffffffffffffff82169050919050565b60006144aa8261447f565b9050919050565b6144ba8161449f565b82525050565b60006020820190506144d560008301846144b1565b92915050565b6144e48161449f565b81146144ef57600080fd5b50565b600081359050614501816144db565b92915050565b6000806040838503121561451e5761451d61429c565b5b600061452c858286016144f2565b925050602061453d8582860161443d565b9150509250929050565b6145508161441c565b82525050565b600060208201905061456b6000830184614547565b92915050565b60008060006060848603121561458a5761458961429c565b5b6000614598868287016144f2565b93505060206145a9868287016144f2565b92505060406145ba8682870161443d565b9150509250925092565b6000819050919050565b6145d7816145c4565b82525050565b60006020820190506145f260008301846145ce565b92915050565b600080fd5b600080fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b61463a826143b0565b810181811067ffffffffffffffff8211171561465957614658614602565b5b80604052505050565b600061466c614292565b90506146788282614631565b919050565b600067ffffffffffffffff82111561469857614697614602565b5b6146a1826143b0565b9050602081019050919050565b82818337600083830152505050565b60006146d06146cb8461467d565b614662565b9050828152602081018484840111156146ec576146eb6145fd565b5b6146f78482856146ae565b509392505050565b600082601f830112614714576147136145f8565b5b81356147248482602086016146bd565b91505092915050565b6000602082840312156147435761474261429c565b5b600082013567ffffffffffffffff811115614761576147606142a1565b5b61476d848285016146ff565b91505092915050565b60006020828403121561478c5761478b61429c565b5b600061479a848285016144f2565b91505092915050565b6147ac816145c4565b81146147b757600080fd5b50565b6000813590506147c9816147a3565b92915050565b6000602082840312156147e5576147e461429c565b5b60006147f3848285016147ba565b91505092915050565b6148058161432b565b811461481057600080fd5b50565b600081359050614822816147fc565b92915050565b6000806040838503121561483f5761483e61429c565b5b600061484d858286016144f2565b925050602061485e85828601614813565b9150509250929050565b600067ffffffffffffffff82111561488357614882614602565b5b61488c826143b0565b9050602081019050919050565b60006148ac6148a784614868565b614662565b9050828152602081018484840111156148c8576148c76145fd565b5b6148d38482856146ae565b509392505050565b600082601f8301126148f0576148ef6145f8565b5b8135614900848260208601614899565b91505092915050565b600080600080608085870312156149235761492261429c565b5b6000614931878288016144f2565b9450506020614942878288016144f2565b93505060406149538782880161443d565b925050606085013567ffffffffffffffff811115614974576149736142a1565b5b614980878288016148db565b91505092959194509250565b600080fd5b600080fd5b60008083601f8401126149ac576149ab6145f8565b5b8235905067ffffffffffffffff8111156149c9576149c861498c565b5b6020830191508360208202830111156149e5576149e4614991565b5b9250929050565b600080600060408486031215614a0557614a0461429c565b5b6000614a138682870161443d565b935050602084013567ffffffffffffffff811115614a3457614a336142a1565b5b614a4086828701614996565b92509250509250925092565b60008060408385031215614a6357614a6261429c565b5b6000614a71858286016144f2565b9250506020614a82858286016144f2565b9150509250929050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b60006002820490506001821680614ad357607f821691505b60208210811415614ae757614ae6614a8c565b5b50919050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b6000614b278261441c565b9150614b328361441c565b9250827fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff03821115614b6757614b66614aed565b5b828201905092915050565b7f424147533a204d696e74696e6720776f756c6420657863656564206d6178207360008201527f7570706c79000000000000000000000000000000000000000000000000000000602082015250565b6000614bce60258361436c565b9150614bd982614b72565b604082019050919050565b60006020820190508181036000830152614bfd81614bc1565b9050919050565b7f424147533a204d757374206d696e74206174206c65617374206f6e6520746f6b60008201527f656e000000000000000000000000000000000000000000000000000000000000602082015250565b6000614c6060228361436c565b9150614c6b82614c04565b604082019050919050565b60006020820190508181036000830152614c8f81614c53565b9050919050565b7f424147533a205075626c69632073616c6520686173206e6f742073746172746560008201527f6400000000000000000000000000000000000000000000000000000000000000602082015250565b6000614cf260218361436c565b9150614cfd82614c96565b604082019050919050565b60006020820190508181036000830152614d2181614ce5565b9050919050565b7f424147533a20457863656564656420737570706c790000000000000000000000600082015250565b6000614d5e60158361436c565b9150614d6982614d28565b602082019050919050565b60006020820190508181036000830152614d8d81614d51565b9050919050565b7f424147533a2043616e6e6f74206d696e742074686973206d616e792042414753600082015250565b6000614dca60208361436c565b9150614dd582614d94565b602082019050919050565b60006020820190508181036000830152614df981614dbd565b9050919050565b7f424147533a20506c65617365206d696e74206174206c6561737420312042414760008201527f5300000000000000000000000000000000000000000000000000000000000000602082015250565b6000614e5c60218361436c565b9150614e6782614e00565b604082019050919050565b60006020820190508181036000830152614e8b81614e4f565b9050919050565b600081905092915050565b6000614ea882614361565b614eb28185614e92565b9350614ec281856020860161437d565b80840191505092915050565b6000614eda8285614e9d565b9150614ee68284614e9d565b91508190509392505050565b7f424147533a20596f752063616e206e6f74206d696e74207269676874206e6f77600082015250565b6000614f2860208361436c565b9150614f3382614ef2565b602082019050919050565b60006020820190508181036000830152614f5781614f1b565b9050919050565b60008160601b9050919050565b6000614f7682614f5e565b9050919050565b6000614f8882614f6b565b9050919050565b614fa0614f9b8261449f565b614f7d565b82525050565b6000614fb28284614f8f565b60148201915081905092915050565b7f424147533a20506c65617365207761697420746f206d696e74206f6e2070756260008201527f6c69632073616c65000000000000000000000000000000000000000000000000602082015250565b600061501d60288361436c565b915061502882614fc1565b604082019050919050565b6000602082019050818103600083015261504c81615010565b9050919050565b7f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160008201527f6464726573730000000000000000000000000000000000000000000000000000602082015250565b60006150af60268361436c565b91506150ba82615053565b604082019050919050565b600060208201905081810360008301526150de816150a2565b9050919050565b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b600061511b60208361436c565b9150615126826150e5565b602082019050919050565b6000602082019050818103600083015261514a8161510e565b9050919050565b600081519050919050565b600082825260208201905092915050565b600061517882615151565b615182818561515c565b935061519281856020860161437d565b61519b816143b0565b840191505092915050565b60006080820190506151bb60008301876144b1565b6151c860208301866144b1565b6151d56040830185614547565b81810360608301526151e7818461516d565b905095945050505050565b600081519050615201816142d2565b92915050565b60006020828403121561521d5761521c61429c565b5b600061522b848285016151f2565b91505092915050565b600061523f8261441c565b91507fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff82141561527257615271614aed565b5b600182019050919050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601260045260246000fd5b60006152b78261441c565b91506152c28361441c565b9250826152d2576152d161527d565b5b828204905092915050565b60006152e88261441c565b91506152f38361441c565b92508282101561530657615305614aed565b5b828203905092915050565b600061531c8261441c565b91506153278361441c565b9250826153375761533661527d565b5b828206905092915050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fdfea2646970667358221220963ff9dc601d0035f4df9879263a41a4c2b4a1154e2a4b6d28b8f72ee592067464736f6c634300080a0033

Deployed Bytecode

0x608060405234801561001057600080fd5b50600436106102485760003560e01c806370a082311161013b578063a22cb465116100b8578063e222c7f91161007c578063e222c7f91461068f578063e985e9c514610699578063ee419b89146106c9578063f2fde38b146106e5578063f47c84c51461070157610248565b8063a22cb465146105ed578063b88d4fde14610609578063c87b56dd14610625578063cabadaa014610655578063d2cab0561461067357610248565b8063851a7708116100ff578063851a7708146105495780638ba4cc3c146105795780638da5cb5b1461059557806395d89b41146105b3578063a0712d68146105d157610248565b806370a08231146104a7578063715018a6146104d757806371978011146104e15780637cb64759146104fd5780637f09e66f1461051957610248565b806331ffd6f1116101c957806359eda1b51161018d57806359eda1b51461041557806363439e611461041f5780636352211e1461044f5780636c0360eb1461047f5780636f02f62c1461049d57610248565b806331ffd6f11461038357806333bc1c5c146103a1578063423f74c9146103bf57806342842e0e146103dd57806355f804b3146103f957610248565b806318160ddd1161021057806318160ddd146102f157806323b872dd1461030f578063270ab52c1461032b5780632eb4a7ab14610347578063309a36861461036557610248565b806301ffc9a71461024d578063034d77941461027d57806306fdde0314610287578063081812fc146102a5578063095ea7b3146102d5575b600080fd5b610267600480360381019061026291906142fe565b61071f565b6040516102749190614346565b60405180910390f35b610285610801565b005b61028f610835565b60405161029c91906143fa565b60405180910390f35b6102bf60048036038101906102ba9190614452565b6108c7565b6040516102cc91906144c0565b60405180910390f35b6102ef60048036038101906102ea9190614507565b610943565b005b6102f9610a4e565b6040516103069190614556565b60405180910390f35b61032960048036038101906103249190614571565b610a65565b005b61034560048036038101906103409190614452565b610a75565b005b61034f610a87565b60405161035c91906145dd565b60405180910390f35b61036d610a8d565b60405161037a9190614556565b60405180910390f35b61038b610a93565b6040516103989190614346565b60405180910390f35b6103a9610aa6565b6040516103b69190614346565b60405180910390f35b6103c7610ab9565b6040516103d49190614346565b60405180910390f35b6103f760048036038101906103f29190614571565b610acc565b005b610413600480360381019061040e919061472d565b610aec565b005b61041d610b0e565b005b61043960048036038101906104349190614776565b610b42565b6040516104469190614556565b60405180910390f35b61046960048036038101906104649190614452565b610b5a565b60405161047691906144c0565b60405180910390f35b610487610b70565b60405161049491906143fa565b60405180910390f35b6104a5610bfe565b005b6104c160048036038101906104bc9190614776565b612230565b6040516104ce9190614556565b60405180910390f35b6104df612300565b005b6104fb60048036038101906104f69190614452565b612314565b005b610517600480360381019061051291906147cf565b612326565b005b610533600480360381019061052e9190614776565b612338565b6040516105409190614556565b60405180910390f35b610563600480360381019061055e9190614776565b612350565b6040516105709190614556565b60405180910390f35b610593600480360381019061058e9190614507565b612368565b005b61059d612418565b6040516105aa91906144c0565b60405180910390f35b6105bb612442565b6040516105c891906143fa565b60405180910390f35b6105eb60048036038101906105e69190614452565b6124d4565b005b61060760048036038101906106029190614828565b6126c4565b005b610623600480360381019061061e9190614909565b61283c565b005b61063f600480360381019061063a9190614452565b6128b8565b60405161064c91906143fa565b60405180910390f35b61065d612957565b60405161066a9190614556565b60405180910390f35b61068d600480360381019061068891906149ec565b61295d565b005b610697612bab565b005b6106b360048036038101906106ae9190614a4c565b612bdf565b6040516106c09190614346565b60405180910390f35b6106e360048036038101906106de91906149ec565b612c73565b005b6106ff60048036038101906106fa9190614776565b612f1e565b005b610709612fa2565b6040516107169190614556565b60405180910390f35b60007f80ac58cd000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff191614806107ea57507f5b5e139f000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b806107fa57506107f982612fa8565b5b9050919050565b610809613012565b600b60029054906101000a900460ff1615600b60026101000a81548160ff021916908315150217905550565b60606002805461084490614abb565b80601f016020809104026020016040519081016040528092919081815260200182805461087090614abb565b80156108bd5780601f10610892576101008083540402835291602001916108bd565b820191906000526020600020905b8154815290600101906020018083116108a057829003601f168201915b5050505050905090565b60006108d282613090565b610908576040517fcf4700e400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6006600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff169050919050565b600061094e82610b5a565b90508073ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff1614156109b6576040517f943f7b8c00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8073ffffffffffffffffffffffffffffffffffffffff166109d56130de565b73ffffffffffffffffffffffffffffffffffffffff1614158015610a075750610a0581610a006130de565b612bdf565b155b15610a3e576040517fcfb3b94200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b610a498383836130e6565b505050565b6000610a58613198565b6001546000540303905090565b610a7083838361319d565b505050565b610a7d613012565b80600a8190555050565b60105481565b60095481565b600b60019054906101000a900460ff1681565b600b60009054906101000a900460ff1681565b600b60029054906101000a900460ff1681565b610ae78383836040518060200160405280600081525061283c565b505050565b610af4613012565b80600f9080519060200190610b0a9291906141ac565b5050565b610b16613012565b600b60019054906101000a900460ff1615600b60016101000a81548160ff021916908315150217905550565b600d6020528060005260406000206000915090505481565b6000610b6582613653565b600001519050919050565b600f8054610b7d90614abb565b80601f0160208091040260200160405190810160405280929190818152602001828054610ba990614abb565b8015610bf65780601f10610bcb57610100808354040283529160200191610bf6565b820191906000526020600020905b815481529060010190602001808311610bd957829003601f168201915b505050505081565b610c06613012565b610c257385c0b44d3b9a49b09c3b925af5c935043e66dfbf60026138e2565b610c4473b110f4cf6660e3003c421254bf1568ca79598a5e60026138e2565b610c637339cb13625945bf0eb05579ad6c79f748dacd9b2060026138e2565b610c8273740f471701d09e268efc991f8332b172093d74dd60026138e2565b610ca173b522a6619d74546cffe9fcbec27da5d2c5d1806660026138e2565b610cc073c2b142beb125579e98c16ced36629a2d1c3d584160026138e2565b610cdf7326be72cbbf5746f14d731fd4febf294cae376f5960026138e2565b610cfe731342bd2ab6065379502de00afd81d4a987318a5e60026138e2565b610d1d73635bf1dfe7301a560e6fb5fef4bb9902b5966ed360026138e2565b610d3c730e16f4a678f7facdcf58c9adf947e8e48845e57560026138e2565b610d5b7355b0d5ef132c1a46e3d18409649ea18351cfef9a60026138e2565b610d7a73610243745476e23ef7c17f23168f3e5e774390e260026138e2565b610d99739a430a8be98da5ac1a2fb6f8f53e8fe794de611e60026138e2565b610db873e15bb22ce00ea25aa62bea202ac1008932f4d78560026138e2565b610dd773a22aae6a5ecde5cc8abe49e32165366c0d70ad6360026138e2565b610df673f6f435a13a38149ef954bb391f16d8010380dd4a60026138e2565b610e1573b7c5121a82493dece1cd4143e0571fcc49afbffd60026138e2565b610e34735d1928b9062e34de640b1117efcc81b90b45269360026138e2565b610e5373f95c508fa8686279294ea69f2deae18c0bc3c99c60026138e2565b610e7273175e89eeb246f66ce664df16f5f046610b86751360026138e2565b610e9173eca78934fdb00a2dadd9a29cf3d45bef5b3c8e9c60026138e2565b610eb073a66489ada4f1b94eacefe5fc27f3674deb407fbd60026138e2565b610ecf7305f885113100771a1bdb5c22e7dadb3acb149e3f60026138e2565b610eee7397eec19136e7ab1cb0a0f4a4c47ee2d55a993c4060026138e2565b610f0d73bb08a962380b9a1e49f20d6c3bdc81075914b0cd60026138e2565b610f2c73dc64b93ccd63d2354a32bbcd2d460735d341415d60026138e2565b610f4b73551d196803c99dc4e2bf68cb9b61d4c597749db060026138e2565b610f6a73dca699c2b0e88f2f06aebe96172fa09d463a4d2760026138e2565b610f897314c30c5d33961c2f4d2cd2d1ab584bbbff0a635e60026138e2565b610fa8733e357db18182f7a597cf49d0c40b692706fa7b2f60026138e2565b610fc773d91473629d8b46a8eb44eb6349a568a7ea7a176f60026138e2565b610fe673aa898615d42efd369e151448a992af897e32f56660026138e2565b61100573e09cf2ac74009200bbff7455ff3f69db5fb49a1060026138e2565b611024739ccbdd887a92d13c04f6c846a2cf514871474ceb60026138e2565b611043730b26454ad48f3651f1cc1abcd2e590301ce9355660026138e2565b61106273d74b8b30ce6269bab58b64b58245da55499b151060026138e2565b61108173bf1016f104996d33007b041e38c1bee6e7fb5d4460026138e2565b6110a0735343a7a198eb41e42661f2f8772a4e6c5f1c6b1c60026138e2565b6110bf73c18c9b1b03ce38425e1c21b720f406f1659002b060026138e2565b6110de738d6d968b5ebbd66bc79cc1085e0854311ff523d760026138e2565b6110fd73ad25c92baf8564849769224e00316d56dfa5491d60026138e2565b61111c73382e00f0edae8b5bcb9398d70c1d192bb699d8b760026138e2565b61113b73b3e010f154c03bfdbd141b563a1b92b5dd206f8260026138e2565b61115a7354558a1998c1a2cbff086449710d28fb7561fe2660026138e2565b61117973580215e9a04f5bb3c03c4f211f91a5ea01411ca160026138e2565b61119873495777e73d7977aae1f562c40796c2c7772b29b560026138e2565b6111b773aa86ad45c43b69315fb97d6daaa0034939dda34f60026138e2565b6111d673eac290b74b14166f15ba296ec123985cee96a69360026138e2565b6111f573721cc6751b48bbcbf3e24fa72cc5bf932783279d60026138e2565b61121473102898958bbf5799f82774a4c4b692d07c59aa7760026138e2565b6112337310c9374bddda68929f712515877d6b592a2bf10960026138e2565b61125172d7a43af16bfefcc180ecf069276b0d726d4b4060026138e2565b6112707339b3fb116e5f5ce90ab0a7bf8545e67c451c626360026138e2565b61128f738cc186f220a2f939a8e7d9dcea340697426d2daa60026138e2565b6112ae73ad644370bc6b596643d7be9e3190a90d25c6234660026138e2565b6112cd73ca17d93e772ad78304a9cf9f5c7ed15e20c9705260026138e2565b6112ec732861d3c46aad60e971ae8fa5e379af129d63e74560026138e2565b61130b73f2f3b5344c0f2e87a2e613c4425ec3906652fed960026138e2565b61132a73603889de8cae2431251e20fe850beda492a7ff6c60026138e2565b611349732f8404f2c087ed5ea1c42ba9e8392641377a71ab60026138e2565b611368739490c0aeeb1ba7ad1b871b2104c5fce4a132362560026138e2565b61138773ad9435432e85acf64173262fce0f977552a49c2e60026138e2565b6113a673f3d7af96a0c09e4c7a59a75c9bd10b89bd60158c60026138e2565b6113c57336b5b82e0598f2d79592289da87b37401b740f2260026138e2565b6113e473a0d3d72516a042e310c459c63dc664182a5308b960026138e2565b6114037388fa0374b2aba0f6af85fc45702f9513d27c255a60026138e2565b611422739a971b4943ef05cde48481f5bafee1003feeef4d60026138e2565b611441730e0a2c07dab0f1ae64cb1fdb6209c1a01d5fb88760026138e2565b6114607307ee856e17a0f9181644511f4801ed29b03288a460026138e2565b61147f739c2406669c9faebbe964d5da5429d3a320652fb860026138e2565b61149e73ac2cd9b5deaa7a3d79ac73de676989eb4978811860026138e2565b6114bd738ecd31cd9f47f4a0fcd0a82eec0445aab518376d60026138e2565b6114dc735646d2e9a7e16ba92239afd071c0c2495c31cf2c60026138e2565b6114fb73c8dfcfe493b268aa325579fb190181c564141a5960026138e2565b61151a738a5675a207cc7174d7e3b4961aa7e9fcd1234ccf60026138e2565b61153973ad406876a8c7a78de7fcff412cb0276d4bdeb68e60026138e2565b611558738945ed77e8900a3b7855bf703c192c7979b473cf60026138e2565b611577732b4775773fd8f49667864208bde1450c4ae21c0360026138e2565b61159673871bf5306dab778dcc0e97166fb9a3b9e5b93d0460026138e2565b6115b5732e7d8196b52256da7b1d5ea22eb8f05686ab3cd160026138e2565b6115d47326ccb82ed08b0f8f1ca0086d5b279d5ba132a8a260026138e2565b6115f373d39b2014ef25ee95f1aede9f1d04ea6a959cf9f660026138e2565b6116127364247785234f7bdae872b9a9222920e4eebf7d5460026138e2565b611631732653e96428088ffaa8c373ba81f5b31bf59ec2f460026138e2565b611650735b3228bacb642a02cfa4763b84e4d116e6c2b70960026138e2565b61166f73eb55b194379d0468bbd734cd08b41d9097f90d0960026138e2565b61168e733a15a2bd61b95c93e4da375538f054309c4380b360026138e2565b6116ad730d85fb3d7ff838d4e6c52f52d810420fbe3819f060026138e2565b6116cc73bd44f279590d4a81a29b63e2c65119c44cdb258160026138e2565b6116eb730e1a70ed924bc4f3c57c454d7833c46911a9d84960026138e2565b61170a731796c568d22240d63b9566328eab535a3968f8c360026138e2565b61172973397280745af703fbb38e1c591524f92d42a57b8960026138e2565b611748739056b05a07d4bb085f64127f39d6faed2ed4808b60026138e2565b61176773069ba33753343b3e73661f06eb7d0a71b3813b4a60026138e2565b611786734de6967967a3c9001d14ff57ad42d879d7e0512460026138e2565b6117a573a0915e1c7e4c2543ecb05c423e8e7a0db31213a760026138e2565b6117c473ca83c9dfdfffc4aaae66f52906566f5d58f24e3160026138e2565b6117e373e89b3dca875bd1c74bd9b22703a487472568e03060026138e2565b611802731507dbf6196a6e1ab160275ec43c6baa30d1a19760026138e2565b61182173b4dbcd527c8ebc09b00c4bdd506a23894604b8a060026138e2565b611840731fec03eb0dbd4190deb139e429a9de6c29de70a660026138e2565b61185f732fad4d2f4bd33e0ae89c776568d2f1c2c92ddb7060026138e2565b61187e732746e48720bf4464b6cc334056cb540148760a3860026138e2565b61189d732284a738f2d84a4d035fe8121a039e79a09547ff60026138e2565b6118bc735d37445e60c6de44c9327ec8bb300e876c3d571360026138e2565b6118db73d6dfd56ab8a116ed6370984945feb8be7d6c322160026138e2565b6118fa73b03f4d215e2ef5986b763b45bdf53e330be38d6260026138e2565b61191973eb89b2499077c01c094b8398a98a11a3087cbb3b60026138e2565b61193873280b5ec890809a98435b84f0cdb56714b16a4c9160026138e2565b611957739b7f79e13768e4daba808492e59caf16aaac952e60026138e2565b61197673863581c07688d990210c0fda40cb2347de9dc87360026138e2565b61199573b38319ac1308ddcf15e3cd8f6d67d26f424279e560026138e2565b6119b473e09adcc2854c3299a2886d0dfeb03ed2a3df63d060026138e2565b6119d373a6769fa1625845ca606a6aa3c8056bc2982c107660026138e2565b6119f273e30bfb74c86a316f4e03d42c8f261324cdd2517360026138e2565b611a11735dc73c27933411916d612c55a074bf38e3b75a9760026138e2565b611a307321dcb6f533d13166abb801390744d0bff8a546a060026138e2565b611a4f73fb8d3bdd6da52f65227a6a17f96c939e5390832660026138e2565b611a6e73dd41ade62481e69f171d758a14680a060b42fc4460026138e2565b611a8d73ee04770359f9363a5d67a7f80f6ac4122dfb970e60026138e2565b611aac730e999151217a907b2c4ddb90bec16f05b263f92360026138e2565b611acb737bd02565e438c7eb709313ac5a7c15d023e6f98560026138e2565b611aea73abf35f4981b9497d01d951d7577bf0de21ffaa2b60026138e2565b611b0973f88f8d5edf096576c5ecfbb51b1fc12e8a144fa460026138e2565b611b287332502a4d1c96273fe62669165a64b8a39f4512b460026138e2565b611b4773edad44d3d2c67e30beb056a68fef514d0e52baaf60026138e2565b611b6673d9bded47b38999bb8c584a051b6b0e7ed39aafd860026138e2565b611b8573e53b6f0f2cff473e7fc31adc712112351f411b2b60026138e2565b611ba47325e4b97cc81eb2ff49a719edd86de91d47531da760026138e2565b611bc37385e5e02efb864b609a587c522c7148c662730ad560026138e2565b611be273c8c5df49795e3f5e2943eebff50c3cc9fb8d496760026138e2565b611c01734f2793344c2cf3a4c18305ba834da0d7188bcaf260026138e2565b611c20734fbb8130a8ddc899c879c445abf15463c29f1dc560026138e2565b611c3f73eb7cf8c3f5e4425d6426fd84a5f8afd68569a64f60026138e2565b611c5e732de09e956a252203a60a36f9ca143ecee336d82760026138e2565b611c7d736173b476b12cc40099f6e6fa6c064d6ee2ab493a60026138e2565b611c9c73c59e912fc173f7d62af19d405816970dae7384f860026138e2565b611cbb731697a4e259bc568814cc575d29b878b6992d5f9c60026138e2565b611cda73b080d6f42d774818bb9549492147917727c11dac60026138e2565b611cf973832c5dd5be10b8a188f858b41e6bf426ae6917ac60026138e2565b611d1873dcdf84646166e015496c51e5d9099f52ae75390360026138e2565b611d3773ce504f9d1f95ab5dce9c8318393b95b351c6c86860026138e2565b611d567324a6ae8d89da1d0ba1d8a3c3012216bfc0d9988860026138e2565b611d7573c5dc0a1064fdde66962a2b449057fe339f4d86fb60026138e2565b611d947307197ecaf257a64502fd5fe6a0d5bf31dbcba08160026138e2565b611db3736590592b2c2753f3c5c564430f6ef12c11a82cd160026138e2565b611dd273861dd17c9fea84f9d8bc6d32c34b90f4ec6317fb60026138e2565b611df173ba5e8d9dccf97a200b30f54f4ec5edbe2fe92ed160026138e2565b611e107319b191f625518c85c54c5d672e7fc9440f1824e060026138e2565b611e2f7340f085176beaa2fc417164d4b8e7399c4addef7760026138e2565b611e4e7361d3d2452448f9f78380ff40d924855719029fb060026138e2565b611e6d7354c5bc3e9ca2ce0b69af1d5102f6f8fb268a751360026138e2565b611e8c7344bb5f45f3f447e90200d61ec4c68f41ccff37ff60026138e2565b611eab73dec2c041b3b5dc8ed7b77b87f6a986fe225bf30e60026138e2565b611eca73213571f3b8b8cc8f463c42d994c3f5e2c34fa3f060026138e2565b611ee97358217e3c57a74b9bf6c539a755c2b0e417162a9c60026138e2565b611f08738bc539f3cfb68c28d52102180a877dcf7db476ae60026138e2565b611f277370919456288650894fd2dce95ed78bbe57dfdbf660026138e2565b611f467304b2cb5bb145e6ba3d67c9debcc14c461c9a968d60026138e2565b611f657331e58ede8f0e39dc832bdaf992cbe9ef3c70f54560026138e2565b611f8473daea44d64813a1a4bba1b2a61c10d915234bf10560026138e2565b611fa3736a5b8c260f6ece3b361a1998da609335d618ac4860026138e2565b611fc273ad74b2fca61ab5e987907f3da9825776f53e6c0260026138e2565b611fe1737268146ddca1b4917758456041764b8ec4317dde60026138e2565b6120007397d93f8a99c74faad615f56ebf27654d63a34a5d60026138e2565b61201f7362a79a85e34db40fac6f422bfaf1cb86d15c550e600a6138e2565b61203e73d27d1c330b89a11c2b62613e22be40bc19d4351e600a6138e2565b61205d73fd3f1300948ecf87677e54120ed7c1fe151c53c3600a6138e2565b61207c733832a2adbb1f55b284f67daccdbe8effc01128e5600a6138e2565b61209b738e893de17ee6c3d2c725502ab3a0614779c3cccb600a6138e2565b6120ba73f7cb1accfae480283b9560a0b1d614663033d876600a6138e2565b6120d973739b51ce1645e4e13ff1a87e93013c3fd3360ed9600a6138e2565b6120f873d2d6d1de0577e1feb65279d3d291d04cff10f00d600a6138e2565b6121177398845cfa79b5fa7878cb7bc203b8bf1429ec4e7e600a6138e2565b61213673d83dfa6e5301a3a98972ef6f1109927ed48aabf9600a6138e2565b612155739590ea8123396623d109ef502b05659e9ab59584600a6138e2565b61217473e818e86d00670559c15a0943f37280cffca1cb2e600a6138e2565b612193735fa89a1a3fef2c4ca7083d4dd1f6509deee25df7600a6138e2565b6121b273327993a6950c0bd11f2f31511e42949da5e8dafb600a6138e2565b6121d17395ebf2a0efebd053c576806bbfc007ab80fb9870600a6138e2565b6121f073565e5e99ece7ad636baeffd162a1d9b7a6e5ac8e600a6138e2565b61220f73d6feb6d54a254d5408b072b5cb1e43606eeeb2f7600a6138e2565b61222e737b50700534cc27bd9ad321a475fd136f7fc0a333600a6138e2565b565b60008073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415612298576040517f8f4eb60400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600560008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160009054906101000a900467ffffffffffffffff1667ffffffffffffffff169050919050565b612308613012565b6123126000613900565b565b61231c613012565b8060098190555050565b61232e613012565b8060108190555050565b600e6020528060005260406000206000915090505481565b600c6020528060005260406000206000915090505481565b612370613012565b611e618161237c610a4e565b6123869190614b1c565b11156123c7576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016123be90614be4565b60405180910390fd5b6000811161240a576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161240190614c76565b60405180910390fd5b61241482826138e2565b5050565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b60606003805461245190614abb565b80601f016020809104026020016040519081016040528092919081815260200182805461247d90614abb565b80156124ca5780601f1061249f576101008083540402835291602001916124ca565b820191906000526020600020905b8154815290600101906020018083116124ad57829003601f168201915b5050505050905090565b600b60009054906101000a900460ff16612523576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161251a90614d08565b60405180910390fd5b611e618161252f610a4e565b6125399190614b1c565b111561257a576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161257190614d74565b60405180910390fd5b600a5481600e600061258a6130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020546125cf9190614b1c565b1115612610576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161260790614de0565b60405180910390fd5b60008111612653576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161264a90614e72565b60405180910390fd5b80600e60006126606130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282546126a99190614b1c565b925050819055506126c16126bb6130de565b826138e2565b50565b6126cc6130de565b73ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415612731576040517fb06307db00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b806007600061273e6130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060006101000a81548160ff0219169083151502179055508173ffffffffffffffffffffffffffffffffffffffff166127eb6130de565b73ffffffffffffffffffffffffffffffffffffffff167f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c31836040516128309190614346565b60405180910390a35050565b61284784848461319d565b6128668373ffffffffffffffffffffffffffffffffffffffff166139c6565b801561287b5750612879848484846139e9565b155b156128b2576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b50505050565b60606128c382613090565b6128f9576040517fa14c4b5000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6000612903613b3a565b9050600081511415612924576040518060200160405280600081525061294f565b8061292e84613bcc565b60405160200161293f929190614ece565b6040516020818303038152906040525b915050919050565b600a5481565b600b60019054906101000a900460ff166129ac576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016129a390614f3e565b60405180910390fd5b612a20828280806020026020016040519081016040528093929190818152602001838360200280828437600081840152601f19601f8201169050808301925050505050505060105433604051602001612a059190614fa6565b60405160208183030381529060405280519060200120613d2d565b612a5f576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612a5690615033565b60405180910390fd5b60095483600c6000612a6f6130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054612ab49190614b1c565b1115612af5576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612aec90614de0565b60405180910390fd5b60008311612b38576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612b2f90614e72565b60405180910390fd5b82600c6000612b456130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254612b8e9190614b1c565b92505081905550612ba6612ba06130de565b846138e2565b505050565b612bb3613012565b600b60009054906101000a900460ff1615600b60006101000a81548160ff021916908315150217905550565b6000600760008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff16905092915050565b600b60029054906101000a900460ff16612cc2576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612cb990614f3e565b60405180910390fd5b612d36828280806020026020016040519081016040528093929190818152602001838360200280828437600081840152601f19601f8201169050808301925050505050505060105433604051602001612d1b9190614fa6565b60405160208183030381529060405280519060200120613d2d565b612d75576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612d6c90615033565b60405180910390fd5b60095483600d6000612d856130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054612dca9190614b1c565b1115612e0b576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612e0290614de0565b60405180910390fd5b60008311612e4e576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612e4590614e72565b60405180910390fd5b82600c6000612e5b6130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254612ea49190614b1c565b9250508190555082600d6000612eb86130de565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000828254612f019190614b1c565b92505081905550612f19612f136130de565b846138e2565b505050565b612f26613012565b600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff161415612f96576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401612f8d906150c5565b60405180910390fd5b612f9f81613900565b50565b611e6181565b60007f01ffc9a7000000000000000000000000000000000000000000000000000000007bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916149050919050565b61301a6130de565b73ffffffffffffffffffffffffffffffffffffffff16613038612418565b73ffffffffffffffffffffffffffffffffffffffff161461308e576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161308590615131565b60405180910390fd5b565b60008161309b613198565b111580156130aa575060005482105b80156130d7575060046000838152602001908152602001600020600001601c9054906101000a900460ff16155b9050919050565b600033905090565b826006600084815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550818373ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff167f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92560405160405180910390a4505050565b600090565b60006131a882613653565b90508373ffffffffffffffffffffffffffffffffffffffff16816000015173ffffffffffffffffffffffffffffffffffffffff1614613213576040517fa114810000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b60008473ffffffffffffffffffffffffffffffffffffffff166132346130de565b73ffffffffffffffffffffffffffffffffffffffff16148061326357506132628561325d6130de565b612bdf565b5b806132a857506132716130de565b73ffffffffffffffffffffffffffffffffffffffff16613290846108c7565b73ffffffffffffffffffffffffffffffffffffffff16145b9050806132e1576040517f59c896be00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600073ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff161415613348576040517fea553b3400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6133558585856001613d44565b613361600084876130e6565b6001600560008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160392506101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055506001600560008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055506000600460008581526020019081526020016000209050848160000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550428160000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff16021790555060006001850190506000600460008381526020019081526020016000209050600073ffffffffffffffffffffffffffffffffffffffff168160000160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1614156135e15760005482146135e057878160000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555084602001518160000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff1602179055505b5b505050828473ffffffffffffffffffffffffffffffffffffffff168673ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a461364c8585856001613d4a565b5050505050565b61365b614232565b600082905080613669613198565b11158015613678575060005481105b156138ab576000600460008381526020019081526020016000206040518060600160405290816000820160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020016000820160149054906101000a900467ffffffffffffffff1667ffffffffffffffff1667ffffffffffffffff16815260200160008201601c9054906101000a900460ff161515151581525050905080604001516138a957600073ffffffffffffffffffffffffffffffffffffffff16816000015173ffffffffffffffffffffffffffffffffffffffff161461378d5780925050506138dd565b5b6001156138a857818060019003925050600460008381526020019081526020016000206040518060600160405290816000820160009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020016000820160149054906101000a900467ffffffffffffffff1667ffffffffffffffff1667ffffffffffffffff16815260200160008201601c9054906101000a900460ff1615151515815250509050600073ffffffffffffffffffffffffffffffffffffffff16816000015173ffffffffffffffffffffffffffffffffffffffff16146138a35780925050506138dd565b61378e565b5b505b6040517fdf2d9b4200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b919050565b6138fc828260405180602001604052806000815250613d50565b5050565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b6000808273ffffffffffffffffffffffffffffffffffffffff163b119050919050565b60008373ffffffffffffffffffffffffffffffffffffffff1663150b7a02613a0f6130de565b8786866040518563ffffffff1660e01b8152600401613a3194939291906151a6565b6020604051808303816000875af1925050508015613a6d57506040513d601f19601f82011682018060405250810190613a6a9190615207565b60015b613ae7573d8060008114613a9d576040519150601f19603f3d011682016040523d82523d6000602084013e613aa2565b606091505b50600081511415613adf576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b805181602001fd5b63150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916817bffffffffffffffffffffffffffffffffffffffffffffffffffffffff191614915050949350505050565b6060600f8054613b4990614abb565b80601f0160208091040260200160405190810160405280929190818152602001828054613b7590614abb565b8015613bc25780601f10613b9757610100808354040283529160200191613bc2565b820191906000526020600020905b815481529060010190602001808311613ba557829003601f168201915b5050505050905090565b60606000821415613c14576040518060400160405280600181526020017f30000000000000000000000000000000000000000000000000000000000000008152509050613d28565b600082905060005b60008214613c46578080613c2f90615234565b915050600a82613c3f91906152ac565b9150613c1c565b60008167ffffffffffffffff811115613c6257613c61614602565b5b6040519080825280601f01601f191660200182016040528015613c945781602001600182028036833780820191505090505b5090505b60008514613d2157600182613cad91906152dd565b9150600a85613cbc9190615311565b6030613cc89190614b1c565b60f81b818381518110613cde57613cdd615342565b5b60200101907effffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916908160001a905350600a85613d1a91906152ac565b9450613c98565b8093505050505b919050565b600082613d3a8584614114565b1490509392505050565b50505050565b50505050565b600080549050600073ffffffffffffffffffffffffffffffffffffffff168473ffffffffffffffffffffffffffffffffffffffff161415613dbd576040517f2e07630000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6000831415613df8576040517fb562e8dd00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b613e056000858386613d44565b82600560008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160008282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff16021790555082600560008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060000160088282829054906101000a900467ffffffffffffffff160192506101000a81548167ffffffffffffffff021916908367ffffffffffffffff160217905550836004600083815260200190815260200160002060000160006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550426004600083815260200190815260200160002060000160146101000a81548167ffffffffffffffff021916908367ffffffffffffffff160217905550600081905060008482019050613fc68673ffffffffffffffffffffffffffffffffffffffff166139c6565b1561408c575b818673ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a461403b60008784806001019550876139e9565b614071576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b80821415613fcc57826000541461408757600080fd5b6140f8565b5b818060010192508673ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a48082141561408d575b81600081905550505061410e6000858386613d4a565b50505050565b60008082905060005b845181101561415f5761414a8286838151811061413d5761413c615342565b5b602002602001015161416a565b9150808061415790615234565b91505061411d565b508091505092915050565b60008183106141825761417d8284614195565b61418d565b61418c8383614195565b5b905092915050565b600082600052816020526040600020905092915050565b8280546141b890614abb565b90600052602060002090601f0160209004810192826141da5760008555614221565b82601f106141f357805160ff1916838001178555614221565b82800160010185558215614221579182015b82811115614220578251825591602001919060010190614205565b5b50905061422e9190614275565b5090565b6040518060600160405280600073ffffffffffffffffffffffffffffffffffffffff168152602001600067ffffffffffffffff1681526020016000151581525090565b5b8082111561428e576000816000905550600101614276565b5090565b6000604051905090565b600080fd5b600080fd5b60007fffffffff0000000000000000000000000000000000000000000000000000000082169050919050565b6142db816142a6565b81146142e657600080fd5b50565b6000813590506142f8816142d2565b92915050565b6000602082840312156143145761431361429c565b5b6000614322848285016142e9565b91505092915050565b60008115159050919050565b6143408161432b565b82525050565b600060208201905061435b6000830184614337565b92915050565b600081519050919050565b600082825260208201905092915050565b60005b8381101561439b578082015181840152602081019050614380565b838111156143aa576000848401525b50505050565b6000601f19601f8301169050919050565b60006143cc82614361565b6143d6818561436c565b93506143e681856020860161437d565b6143ef816143b0565b840191505092915050565b6000602082019050818103600083015261441481846143c1565b905092915050565b6000819050919050565b61442f8161441c565b811461443a57600080fd5b50565b60008135905061444c81614426565b92915050565b6000602082840312156144685761446761429c565b5b60006144768482850161443d565b91505092915050565b600073ffffffffffffffffffffffffffffffffffffffff82169050919050565b60006144aa8261447f565b9050919050565b6144ba8161449f565b82525050565b60006020820190506144d560008301846144b1565b92915050565b6144e48161449f565b81146144ef57600080fd5b50565b600081359050614501816144db565b92915050565b6000806040838503121561451e5761451d61429c565b5b600061452c858286016144f2565b925050602061453d8582860161443d565b9150509250929050565b6145508161441c565b82525050565b600060208201905061456b6000830184614547565b92915050565b60008060006060848603121561458a5761458961429c565b5b6000614598868287016144f2565b93505060206145a9868287016144f2565b92505060406145ba8682870161443d565b9150509250925092565b6000819050919050565b6145d7816145c4565b82525050565b60006020820190506145f260008301846145ce565b92915050565b600080fd5b600080fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b61463a826143b0565b810181811067ffffffffffffffff8211171561465957614658614602565b5b80604052505050565b600061466c614292565b90506146788282614631565b919050565b600067ffffffffffffffff82111561469857614697614602565b5b6146a1826143b0565b9050602081019050919050565b82818337600083830152505050565b60006146d06146cb8461467d565b614662565b9050828152602081018484840111156146ec576146eb6145fd565b5b6146f78482856146ae565b509392505050565b600082601f830112614714576147136145f8565b5b81356147248482602086016146bd565b91505092915050565b6000602082840312156147435761474261429c565b5b600082013567ffffffffffffffff811115614761576147606142a1565b5b61476d848285016146ff565b91505092915050565b60006020828403121561478c5761478b61429c565b5b600061479a848285016144f2565b91505092915050565b6147ac816145c4565b81146147b757600080fd5b50565b6000813590506147c9816147a3565b92915050565b6000602082840312156147e5576147e461429c565b5b60006147f3848285016147ba565b91505092915050565b6148058161432b565b811461481057600080fd5b50565b600081359050614822816147fc565b92915050565b6000806040838503121561483f5761483e61429c565b5b600061484d858286016144f2565b925050602061485e85828601614813565b9150509250929050565b600067ffffffffffffffff82111561488357614882614602565b5b61488c826143b0565b9050602081019050919050565b60006148ac6148a784614868565b614662565b9050828152602081018484840111156148c8576148c76145fd565b5b6148d38482856146ae565b509392505050565b600082601f8301126148f0576148ef6145f8565b5b8135614900848260208601614899565b91505092915050565b600080600080608085870312156149235761492261429c565b5b6000614931878288016144f2565b9450506020614942878288016144f2565b93505060406149538782880161443d565b925050606085013567ffffffffffffffff811115614974576149736142a1565b5b614980878288016148db565b91505092959194509250565b600080fd5b600080fd5b60008083601f8401126149ac576149ab6145f8565b5b8235905067ffffffffffffffff8111156149c9576149c861498c565b5b6020830191508360208202830111156149e5576149e4614991565b5b9250929050565b600080600060408486031215614a0557614a0461429c565b5b6000614a138682870161443d565b935050602084013567ffffffffffffffff811115614a3457614a336142a1565b5b614a4086828701614996565b92509250509250925092565b60008060408385031215614a6357614a6261429c565b5b6000614a71858286016144f2565b9250506020614a82858286016144f2565b9150509250929050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b60006002820490506001821680614ad357607f821691505b60208210811415614ae757614ae6614a8c565b5b50919050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b6000614b278261441c565b9150614b328361441c565b9250827fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff03821115614b6757614b66614aed565b5b828201905092915050565b7f424147533a204d696e74696e6720776f756c6420657863656564206d6178207360008201527f7570706c79000000000000000000000000000000000000000000000000000000602082015250565b6000614bce60258361436c565b9150614bd982614b72565b604082019050919050565b60006020820190508181036000830152614bfd81614bc1565b9050919050565b7f424147533a204d757374206d696e74206174206c65617374206f6e6520746f6b60008201527f656e000000000000000000000000000000000000000000000000000000000000602082015250565b6000614c6060228361436c565b9150614c6b82614c04565b604082019050919050565b60006020820190508181036000830152614c8f81614c53565b9050919050565b7f424147533a205075626c69632073616c6520686173206e6f742073746172746560008201527f6400000000000000000000000000000000000000000000000000000000000000602082015250565b6000614cf260218361436c565b9150614cfd82614c96565b604082019050919050565b60006020820190508181036000830152614d2181614ce5565b9050919050565b7f424147533a20457863656564656420737570706c790000000000000000000000600082015250565b6000614d5e60158361436c565b9150614d6982614d28565b602082019050919050565b60006020820190508181036000830152614d8d81614d51565b9050919050565b7f424147533a2043616e6e6f74206d696e742074686973206d616e792042414753600082015250565b6000614dca60208361436c565b9150614dd582614d94565b602082019050919050565b60006020820190508181036000830152614df981614dbd565b9050919050565b7f424147533a20506c65617365206d696e74206174206c6561737420312042414760008201527f5300000000000000000000000000000000000000000000000000000000000000602082015250565b6000614e5c60218361436c565b9150614e6782614e00565b604082019050919050565b60006020820190508181036000830152614e8b81614e4f565b9050919050565b600081905092915050565b6000614ea882614361565b614eb28185614e92565b9350614ec281856020860161437d565b80840191505092915050565b6000614eda8285614e9d565b9150614ee68284614e9d565b91508190509392505050565b7f424147533a20596f752063616e206e6f74206d696e74207269676874206e6f77600082015250565b6000614f2860208361436c565b9150614f3382614ef2565b602082019050919050565b60006020820190508181036000830152614f5781614f1b565b9050919050565b60008160601b9050919050565b6000614f7682614f5e565b9050919050565b6000614f8882614f6b565b9050919050565b614fa0614f9b8261449f565b614f7d565b82525050565b6000614fb28284614f8f565b60148201915081905092915050565b7f424147533a20506c65617365207761697420746f206d696e74206f6e2070756260008201527f6c69632073616c65000000000000000000000000000000000000000000000000602082015250565b600061501d60288361436c565b915061502882614fc1565b604082019050919050565b6000602082019050818103600083015261504c81615010565b9050919050565b7f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160008201527f6464726573730000000000000000000000000000000000000000000000000000602082015250565b60006150af60268361436c565b91506150ba82615053565b604082019050919050565b600060208201905081810360008301526150de816150a2565b9050919050565b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b600061511b60208361436c565b9150615126826150e5565b602082019050919050565b6000602082019050818103600083015261514a8161510e565b9050919050565b600081519050919050565b600082825260208201905092915050565b600061517882615151565b615182818561515c565b935061519281856020860161437d565b61519b816143b0565b840191505092915050565b60006080820190506151bb60008301876144b1565b6151c860208301866144b1565b6151d56040830185614547565b81810360608301526151e7818461516d565b905095945050505050565b600081519050615201816142d2565b92915050565b60006020828403121561521d5761521c61429c565b5b600061522b848285016151f2565b91505092915050565b600061523f8261441c565b91507fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff82141561527257615271614aed565b5b600182019050919050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601260045260246000fd5b60006152b78261441c565b91506152c28361441c565b9250826152d2576152d161527d565b5b828204905092915050565b60006152e88261441c565b91506152f38361441c565b92508282101561530657615305614aed565b5b828203905092915050565b600061531c8261441c565b91506153278361441c565b9250826153375761533661527d565b5b828206905092915050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fdfea2646970667358221220963ff9dc601d0035f4df9879263a41a4c2b4a1154e2a4b6d28b8f72ee592067464736f6c634300080a0033

Deployed Bytecode Sourcemap

62229:16146:0:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;43348:305;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;75479:101;;;:::i;:::-;;46461:100;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;47964:204;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;47527:371;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;42597:303;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;48829:170;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;76132:124;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;62771:94;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;62360:35;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;62478:33;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;62441:30;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;62518:35;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;49070:185;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;75588:106;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;62934:99;;;:::i;:::-;;62623:50;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;46269:125;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;62738:26;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;63041:12332;;;:::i;:::-;;43717:206;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;21039:103;;;:::i;:::-;;75954:136;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;75702:106;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;62680:49;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;62564:52;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;78103:269;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;20391:87;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;46630:104;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;77573:464;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;48240:287;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;49326:369;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;46805:318;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;62402:32;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;76284:584;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;75381:90;;;:::i;:::-;;48598:164;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;76901:632;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;21297:201;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;62310:41;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;43348:305;43450:4;43502:25;43487:40;;;:11;:40;;;;:105;;;;43559:33;43544:48;;;:11;:48;;;;43487:105;:158;;;;43609:36;43633:11;43609:23;:36::i;:::-;43487:158;43467:178;;43348:305;;;:::o;75479:101::-;20277:13;:11;:13::i;:::-;75557:15:::1;;;;;;;;;;;75556:16;75538:15;;:34;;;;;;;;;;;;;;;;;;75479:101::o:0;46461:100::-;46515:13;46548:5;46541:12;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;46461:100;:::o;47964:204::-;48032:7;48057:16;48065:7;48057;:16::i;:::-;48052:64;;48082:34;;;;;;;;;;;;;;48052:64;48136:15;:24;48152:7;48136:24;;;;;;;;;;;;;;;;;;;;;48129:31;;47964:204;;;:::o;47527:371::-;47600:13;47616:24;47632:7;47616:15;:24::i;:::-;47600:40;;47661:5;47655:11;;:2;:11;;;47651:48;;;47675:24;;;;;;;;;;;;;;47651:48;47732:5;47716:21;;:12;:10;:12::i;:::-;:21;;;;:63;;;;;47742:37;47759:5;47766:12;:10;:12::i;:::-;47742:16;:37::i;:::-;47741:38;47716:63;47712:138;;;47803:35;;;;;;;;;;;;;;47712:138;47862:28;47871:2;47875:7;47884:5;47862:8;:28::i;:::-;47589:309;47527:371;;:::o;42597:303::-;42641:7;42866:15;:13;:15::i;:::-;42851:12;;42835:13;;:28;:46;42828:53;;42597:303;:::o;48829:170::-;48963:28;48973:4;48979:2;48983:7;48963:9;:28::i;:::-;48829:170;;;:::o;76132:124::-;20277:13;:11;:13::i;:::-;76231:17:::1;76215:13;:33;;;;76132:124:::0;:::o;62771:94::-;;;;:::o;62360:35::-;;;;:::o;62478:33::-;;;;;;;;;;;;;:::o;62441:30::-;;;;;;;;;;;;;:::o;62518:35::-;;;;;;;;;;;;;:::o;49070:185::-;49208:39;49225:4;49231:2;49235:7;49208:39;;;;;;;;;;;;:16;:39::i;:::-;49070:185;;;:::o;75588:106::-;20277:13;:11;:13::i;:::-;75675:11:::1;75665:7;:21;;;;;;;;;;;;:::i;:::-;;75588:106:::0;:::o;62934:99::-;20277:13;:11;:13::i;:::-;63012::::1;;;;;;;;;;;63011:14;62995:13;;:30;;;;;;;;;;;;;;;;;;62934:99::o:0;62623:50::-;;;;;;;;;;;;;;;;;:::o;46269:125::-;46333:7;46360:21;46373:7;46360:12;:21::i;:::-;:26;;;46353:33;;46269:125;;;:::o;62738:26::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;63041:12332::-;20277:13;:11;:13::i;:::-;63097:56:::1;63107:42;63151:1;63097:9;:56::i;:::-;63164;63174:42;63218:1;63164:9;:56::i;:::-;63231;63241:42;63285:1;63231:9;:56::i;:::-;63298;63308:42;63352:1;63298:9;:56::i;:::-;63365;63375:42;63419:1;63365:9;:56::i;:::-;63432;63442:42;63486:1;63432:9;:56::i;:::-;63499;63509:42;63553:1;63499:9;:56::i;:::-;63566;63576:42;63620:1;63566:9;:56::i;:::-;63633;63643:42;63687:1;63633:9;:56::i;:::-;63700;63710:42;63754:1;63700:9;:56::i;:::-;63767;63777:42;63821:1;63767:9;:56::i;:::-;63834;63844:42;63888:1;63834:9;:56::i;:::-;63901;63911:42;63955:1;63901:9;:56::i;:::-;63968;63978:42;64022:1;63968:9;:56::i;:::-;64035;64045:42;64089:1;64035:9;:56::i;:::-;64102;64112:42;64156:1;64102:9;:56::i;:::-;64169;64179:42;64223:1;64169:9;:56::i;:::-;64236;64246:42;64290:1;64236:9;:56::i;:::-;64303;64313:42;64357:1;64303:9;:56::i;:::-;64370;64380:42;64424:1;64370:9;:56::i;:::-;64437;64447:42;64491:1;64437:9;:56::i;:::-;64504;64514:42;64558:1;64504:9;:56::i;:::-;64571;64581:42;64625:1;64571:9;:56::i;:::-;64638;64648:42;64692:1;64638:9;:56::i;:::-;64705;64715:42;64759:1;64705:9;:56::i;:::-;64772;64782:42;64826:1;64772:9;:56::i;:::-;64839;64849:42;64893:1;64839:9;:56::i;:::-;64906;64916:42;64960:1;64906:9;:56::i;:::-;64973;64983:42;65027:1;64973:9;:56::i;:::-;65040;65050:42;65094:1;65040:9;:56::i;:::-;65107;65117:42;65161:1;65107:9;:56::i;:::-;65174;65184:42;65228:1;65174:9;:56::i;:::-;65241;65251:42;65295:1;65241:9;:56::i;:::-;65308;65318:42;65362:1;65308:9;:56::i;:::-;65375;65385:42;65429:1;65375:9;:56::i;:::-;65442;65452:42;65496:1;65442:9;:56::i;:::-;65509;65519:42;65563:1;65509:9;:56::i;:::-;65576;65586:42;65630:1;65576:9;:56::i;:::-;65643;65653:42;65697:1;65643:9;:56::i;:::-;65710;65720:42;65764:1;65710:9;:56::i;:::-;65777;65787:42;65831:1;65777:9;:56::i;:::-;65844;65854:42;65898:1;65844:9;:56::i;:::-;65911;65921:42;65965:1;65911:9;:56::i;:::-;65978;65988:42;66032:1;65978:9;:56::i;:::-;66045;66055:42;66099:1;66045:9;:56::i;:::-;66112;66122:42;66166:1;66112:9;:56::i;:::-;66179;66189:42;66233:1;66179:9;:56::i;:::-;66246;66256:42;66300:1;66246:9;:56::i;:::-;66313;66323:42;66367:1;66313:9;:56::i;:::-;66380;66390:42;66434:1;66380:9;:56::i;:::-;66447;66457:42;66501:1;66447:9;:56::i;:::-;66514;66524:42;66568:1;66514:9;:56::i;:::-;66581;66591:42;66635:1;66581:9;:56::i;:::-;66648;66658:42;66702:1;66648:9;:56::i;:::-;66715;66725:42;66769:1;66715:9;:56::i;:::-;66782;66792:42;66836:1;66782:9;:56::i;:::-;66849;66859:42;66903:1;66849:9;:56::i;:::-;66916;66926:42;66970:1;66916:9;:56::i;:::-;66983;66993:42;67037:1;66983:9;:56::i;:::-;67050;67060:42;67104:1;67050:9;:56::i;:::-;67117;67127:42;67171:1;67117:9;:56::i;:::-;67184;67194:42;67238:1;67184:9;:56::i;:::-;67251;67261:42;67305:1;67251:9;:56::i;:::-;67318;67328:42;67372:1;67318:9;:56::i;:::-;67385;67395:42;67439:1;67385:9;:56::i;:::-;67452;67462:42;67506:1;67452:9;:56::i;:::-;67519;67529:42;67573:1;67519:9;:56::i;:::-;67586;67596:42;67640:1;67586:9;:56::i;:::-;67653;67663:42;67707:1;67653:9;:56::i;:::-;67720;67730:42;67774:1;67720:9;:56::i;:::-;67787;67797:42;67841:1;67787:9;:56::i;:::-;67854;67864:42;67908:1;67854:9;:56::i;:::-;67921;67931:42;67975:1;67921:9;:56::i;:::-;67988;67998:42;68042:1;67988:9;:56::i;:::-;68055;68065:42;68109:1;68055:9;:56::i;:::-;68122;68132:42;68176:1;68122:9;:56::i;:::-;68189;68199:42;68243:1;68189:9;:56::i;:::-;68256;68266:42;68310:1;68256:9;:56::i;:::-;68323;68333:42;68377:1;68323:9;:56::i;:::-;68390;68400:42;68444:1;68390:9;:56::i;:::-;68457;68467:42;68511:1;68457:9;:56::i;:::-;68524;68534:42;68578:1;68524:9;:56::i;:::-;68591;68601:42;68645:1;68591:9;:56::i;:::-;68658;68668:42;68712:1;68658:9;:56::i;:::-;68725;68735:42;68779:1;68725:9;:56::i;:::-;68792;68802:42;68846:1;68792:9;:56::i;:::-;68859;68869:42;68913:1;68859:9;:56::i;:::-;68926;68936:42;68980:1;68926:9;:56::i;:::-;68993;69003:42;69047:1;68993:9;:56::i;:::-;69060;69070:42;69114:1;69060:9;:56::i;:::-;69127;69137:42;69181:1;69127:9;:56::i;:::-;69194;69204:42;69248:1;69194:9;:56::i;:::-;69261;69271:42;69315:1;69261:9;:56::i;:::-;69328;69338:42;69382:1;69328:9;:56::i;:::-;69395;69405:42;69449:1;69395:9;:56::i;:::-;69462;69472:42;69516:1;69462:9;:56::i;:::-;69529;69539:42;69583:1;69529:9;:56::i;:::-;69596;69606:42;69650:1;69596:9;:56::i;:::-;69663;69673:42;69717:1;69663:9;:56::i;:::-;69730;69740:42;69784:1;69730:9;:56::i;:::-;69797;69807:42;69851:1;69797:9;:56::i;:::-;69864;69874:42;69918:1;69864:9;:56::i;:::-;69931;69941:42;69985:1;69931:9;:56::i;:::-;69998;70008:42;70052:1;69998:9;:56::i;:::-;70065;70075:42;70119:1;70065:9;:56::i;:::-;70132;70142:42;70186:1;70132:9;:56::i;:::-;70199;70209:42;70253:1;70199:9;:56::i;:::-;70266;70276:42;70320:1;70266:9;:56::i;:::-;70333;70343:42;70387:1;70333:9;:56::i;:::-;70400;70410:42;70454:1;70400:9;:56::i;:::-;70467;70477:42;70521:1;70467:9;:56::i;:::-;70534;70544:42;70588:1;70534:9;:56::i;:::-;70601;70611:42;70655:1;70601:9;:56::i;:::-;70668;70678:42;70722:1;70668:9;:56::i;:::-;70735;70745:42;70789:1;70735:9;:56::i;:::-;70802;70812:42;70856:1;70802:9;:56::i;:::-;70869;70879:42;70923:1;70869:9;:56::i;:::-;70936;70946:42;70990:1;70936:9;:56::i;:::-;71003;71013:42;71057:1;71003:9;:56::i;:::-;71070;71080:42;71124:1;71070:9;:56::i;:::-;71137;71147:42;71191:1;71137:9;:56::i;:::-;71204;71214:42;71258:1;71204:9;:56::i;:::-;71271;71281:42;71325:1;71271:9;:56::i;:::-;71338;71348:42;71392:1;71338:9;:56::i;:::-;71405;71415:42;71459:1;71405:9;:56::i;:::-;71472;71482:42;71526:1;71472:9;:56::i;:::-;71539;71549:42;71593:1;71539:9;:56::i;:::-;71606;71616:42;71660:1;71606:9;:56::i;:::-;71673;71683:42;71727:1;71673:9;:56::i;:::-;71740;71750:42;71794:1;71740:9;:56::i;:::-;71807;71817:42;71861:1;71807:9;:56::i;:::-;71874;71884:42;71928:1;71874:9;:56::i;:::-;71941;71951:42;71995:1;71941:9;:56::i;:::-;72008;72018:42;72062:1;72008:9;:56::i;:::-;72075;72085:42;72129:1;72075:9;:56::i;:::-;72142;72152:42;72196:1;72142:9;:56::i;:::-;72209;72219:42;72263:1;72209:9;:56::i;:::-;72276;72286:42;72330:1;72276:9;:56::i;:::-;72343;72353:42;72397:1;72343:9;:56::i;:::-;72410;72420:42;72464:1;72410:9;:56::i;:::-;72477;72487:42;72531:1;72477:9;:56::i;:::-;72544;72554:42;72598:1;72544:9;:56::i;:::-;72611;72621:42;72665:1;72611:9;:56::i;:::-;72678;72688:42;72732:1;72678:9;:56::i;:::-;72745;72755:42;72799:1;72745:9;:56::i;:::-;72812;72822:42;72866:1;72812:9;:56::i;:::-;72879;72889:42;72933:1;72879:9;:56::i;:::-;72946;72956:42;73000:1;72946:9;:56::i;:::-;73013;73023:42;73067:1;73013:9;:56::i;:::-;73080;73090:42;73134:1;73080:9;:56::i;:::-;73147;73157:42;73201:1;73147:9;:56::i;:::-;73214;73224:42;73268:1;73214:9;:56::i;:::-;73281;73291:42;73335:1;73281:9;:56::i;:::-;73348;73358:42;73402:1;73348:9;:56::i;:::-;73415;73425:42;73469:1;73415:9;:56::i;:::-;73482;73492:42;73536:1;73482:9;:56::i;:::-;73549;73559:42;73603:1;73549:9;:56::i;:::-;73616;73626:42;73670:1;73616:9;:56::i;:::-;73683;73693:42;73737:1;73683:9;:56::i;:::-;73750;73760:42;73804:1;73750:9;:56::i;:::-;73817;73827:42;73871:1;73817:9;:56::i;:::-;73884;73894:42;73938:1;73884:9;:56::i;:::-;73951;73961:42;74005:1;73951:9;:56::i;:::-;74018;74028:42;74072:1;74018:9;:56::i;:::-;74085;74095:42;74139:1;74085:9;:56::i;:::-;74152:57;74162:42;74206:2;74152:9;:57::i;:::-;74220;74230:42;74274:2;74220:9;:57::i;:::-;74288;74298:42;74342:2;74288:9;:57::i;:::-;74356;74366:42;74410:2;74356:9;:57::i;:::-;74424;74434:42;74478:2;74424:9;:57::i;:::-;74492;74502:42;74546:2;74492:9;:57::i;:::-;74560;74570:42;74614:2;74560:9;:57::i;:::-;74628;74638:42;74682:2;74628:9;:57::i;:::-;74696;74706:42;74750:2;74696:9;:57::i;:::-;74764;74774:42;74818:2;74764:9;:57::i;:::-;74832;74842:42;74886:2;74832:9;:57::i;:::-;74900;74910:42;74954:2;74900:9;:57::i;:::-;74968;74978:42;75022:2;74968:9;:57::i;:::-;75036;75046:42;75090:2;75036:9;:57::i;:::-;75104;75114:42;75158:2;75104:9;:57::i;:::-;75172;75182:42;75226:2;75172:9;:57::i;:::-;75240;75250:42;75294:2;75240:9;:57::i;:::-;75308;75318:42;75362:2;75308:9;:57::i;:::-;63041:12332::o:0;43717:206::-;43781:7;43822:1;43805:19;;:5;:19;;;43801:60;;;43833:28;;;;;;;;;;;;;;43801:60;43887:12;:19;43900:5;43887:19;;;;;;;;;;;;;;;:27;;;;;;;;;;;;43879:36;;43872:43;;43717:206;;;:::o;21039:103::-;20277:13;:11;:13::i;:::-;21104:30:::1;21131:1;21104:18;:30::i;:::-;21039:103::o:0;75954:136::-;20277:13;:11;:13::i;:::-;76062:20:::1;76043:16;:39;;;;75954:136:::0;:::o;75702:106::-;20277:13;:11;:13::i;:::-;75789:11:::1;75776:10;:24;;;;75702:106:::0;:::o;62680:49::-;;;;;;;;;;;;;;;;;:::o;62564:52::-;;;;;;;;;;;;;;;;;:::o;78103:269::-;20277:13;:11;:13::i;:::-;62347:4:::1;78202:6;78186:13;:11;:13::i;:::-;:22;;;;:::i;:::-;:36;;78178:86;;;;;;;;;;;;:::i;:::-;;;;;;;;;78292:1;78283:6;:10;78275:57;;;;;;;;;;;;:::i;:::-;;;;;;;;;78343:21;78353:2;78357:6;78343:9;:21::i;:::-;78103:269:::0;;:::o;20391:87::-;20437:7;20464:6;;;;;;;;;;;20457:13;;20391:87;:::o;46630:104::-;46686:13;46719:7;46712:14;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;46630:104;:::o;77573:464::-;77631:10;;;;;;;;;;;77623:56;;;;;;;;;;;;:::i;:::-;;;;;;;;;62347:4;77714:6;77698:13;:11;:13::i;:::-;:22;;;;:::i;:::-;:36;;77690:70;;;;;;;;;;;;:::i;:::-;;;;;;;;;77820:13;;77810:6;77779:14;:28;77794:12;:10;:12::i;:::-;77779:28;;;;;;;;;;;;;;;;:37;;;;:::i;:::-;:54;;77771:99;;;;;;;;;;;;:::i;:::-;;;;;;;;;77898:1;77889:6;:10;77881:56;;;;;;;;;;;;:::i;:::-;;;;;;;;;77981:6;77950:14;:28;77965:12;:10;:12::i;:::-;77950:28;;;;;;;;;;;;;;;;:37;;;;;;;:::i;:::-;;;;;;;;77998:31;78008:12;:10;:12::i;:::-;78022:6;77998:9;:31::i;:::-;77573:464;:::o;48240:287::-;48351:12;:10;:12::i;:::-;48339:24;;:8;:24;;;48335:54;;;48372:17;;;;;;;;;;;;;;48335:54;48447:8;48402:18;:32;48421:12;:10;:12::i;:::-;48402:32;;;;;;;;;;;;;;;:42;48435:8;48402:42;;;;;;;;;;;;;;;;:53;;;;;;;;;;;;;;;;;;48500:8;48471:48;;48486:12;:10;:12::i;:::-;48471:48;;;48510:8;48471:48;;;;;;:::i;:::-;;;;;;;;48240:287;;:::o;49326:369::-;49493:28;49503:4;49509:2;49513:7;49493:9;:28::i;:::-;49536:15;:2;:13;;;:15::i;:::-;:76;;;;;49556:56;49587:4;49593:2;49597:7;49606:5;49556:30;:56::i;:::-;49555:57;49536:76;49532:156;;;49636:40;;;;;;;;;;;;;;49532:156;49326:369;;;;:::o;46805:318::-;46878:13;46909:16;46917:7;46909;:16::i;:::-;46904:59;;46934:29;;;;;;;;;;;;;;46904:59;46976:21;47000:10;:8;:10::i;:::-;46976:34;;47053:1;47034:7;47028:21;:26;;:87;;;;;;;;;;;;;;;;;47081:7;47090:18;:7;:16;:18::i;:::-;47064:45;;;;;;;;;:::i;:::-;;;;;;;;;;;;;47028:87;47021:94;;;46805:318;;;:::o;62402:32::-;;;;:::o;76284:584::-;76383:13;;;;;;;;;;;76375:58;;;;;;;;;;;;:::i;:::-;;;;;;;;;76452:84;76471:11;;76452:84;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;76484:10;;76523;76506:28;;;;;;;;:::i;:::-;;;;;;;;;;;;;76496:39;;;;;;76452:18;:84::i;:::-;76444:137;;;;;;;;;;;;:::i;:::-;;;;;;;;;76644:16;;76634:6;76600:17;:31;76618:12;:10;:12::i;:::-;76600:31;;;;;;;;;;;;;;;;:40;;;;:::i;:::-;:60;;76592:105;;;;;;;;;;;;:::i;:::-;;;;;;;;;76725:1;76716:6;:10;76708:56;;;;;;;;;;;;:::i;:::-;;;;;;;;;76812:6;76777:17;:31;76795:12;:10;:12::i;:::-;76777:31;;;;;;;;;;;;;;;;:41;;;;;;;:::i;:::-;;;;;;;;76829:31;76839:12;:10;:12::i;:::-;76853:6;76829:9;:31::i;:::-;76284:584;;;:::o;75381:90::-;20277:13;:11;:13::i;:::-;75453:10:::1;;;;;;;;;;;75452:11;75439:10;;:24;;;;;;;;;;;;;;;;;;75381:90::o:0;48598:164::-;48695:4;48719:18;:25;48738:5;48719:25;;;;;;;;;;;;;;;:35;48745:8;48719:35;;;;;;;;;;;;;;;;;;;;;;;;;48712:42;;48598:164;;;;:::o;76901:632::-;76998:15;;;;;;;;;;;76990:60;;;;;;;;;;;;:::i;:::-;;;;;;;;;77069:84;77088:11;;77069:84;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;77101:10;;77140;77123:28;;;;;;;;:::i;:::-;;;;;;;;;;;;;77113:39;;;;;;77069:18;:84::i;:::-;77061:137;;;;;;;;;;;;:::i;:::-;;;;;;;;;77259:16;;77249:6;77217:15;:29;77233:12;:10;:12::i;:::-;77217:29;;;;;;;;;;;;;;;;:38;;;;:::i;:::-;:58;;77209:103;;;;;;;;;;;;:::i;:::-;;;;;;;;;77340:1;77331:6;:10;77323:56;;;;;;;;;;;;:::i;:::-;;;;;;;;;77427:6;77392:17;:31;77410:12;:10;:12::i;:::-;77392:31;;;;;;;;;;;;;;;;:41;;;;;;;:::i;:::-;;;;;;;;77477:6;77444:15;:29;77460:12;:10;:12::i;:::-;77444:29;;;;;;;;;;;;;;;;:39;;;;;;;:::i;:::-;;;;;;;;77494:31;77504:12;:10;:12::i;:::-;77518:6;77494:9;:31::i;:::-;76901:632;;;:::o;21297:201::-;20277:13;:11;:13::i;:::-;21406:1:::1;21386:22;;:8;:22;;;;21378:73;;;;;;;;;;;;:::i;:::-;;;;;;;;;21462:28;21481:8;21462:18;:28::i;:::-;21297:201:::0;:::o;62310:41::-;62347:4;62310:41;:::o;33245:157::-;33330:4;33369:25;33354:40;;;:11;:40;;;;33347:47;;33245:157;;;:::o;20556:132::-;20631:12;:10;:12::i;:::-;20620:23;;:7;:5;:7::i;:::-;:23;;;20612:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;20556:132::o;49950:174::-;50007:4;50050:7;50031:15;:13;:15::i;:::-;:26;;:53;;;;;50071:13;;50061:7;:23;50031:53;:85;;;;;50089:11;:20;50101:7;50089:20;;;;;;;;;;;:27;;;;;;;;;;;;50088:28;50031:85;50024:92;;49950:174;;;:::o;18942:98::-;18995:7;19022:10;19015:17;;18942:98;:::o;59176:196::-;59318:2;59291:15;:24;59307:7;59291:24;;;;;;;;;;;;:29;;;;;;;;;;;;;;;;;;59356:7;59352:2;59336:28;;59345:5;59336:28;;;;;;;;;;;;59176:196;;;:::o;42371:92::-;42427:7;42371:92;:::o;54124:2130::-;54239:35;54277:21;54290:7;54277:12;:21::i;:::-;54239:59;;54337:4;54315:26;;:13;:18;;;:26;;;54311:67;;54350:28;;;;;;;;;;;;;;54311:67;54391:22;54433:4;54417:20;;:12;:10;:12::i;:::-;:20;;;:73;;;;54454:36;54471:4;54477:12;:10;:12::i;:::-;54454:16;:36::i;:::-;54417:73;:126;;;;54531:12;:10;:12::i;:::-;54507:36;;:20;54519:7;54507:11;:20::i;:::-;:36;;;54417:126;54391:153;;54562:17;54557:66;;54588:35;;;;;;;;;;;;;;54557:66;54652:1;54638:16;;:2;:16;;;54634:52;;;54663:23;;;;;;;;;;;;;;54634:52;54699:43;54721:4;54727:2;54731:7;54740:1;54699:21;:43::i;:::-;54807:35;54824:1;54828:7;54837:4;54807:8;:35::i;:::-;55168:1;55138:12;:18;55151:4;55138:18;;;;;;;;;;;;;;;:26;;;:31;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;55212:1;55184:12;:16;55197:2;55184:16;;;;;;;;;;;;;;;:24;;;:29;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;55230:31;55264:11;:20;55276:7;55264:20;;;;;;;;;;;55230:54;;55315:2;55299:8;:13;;;:18;;;;;;;;;;;;;;;;;;55365:15;55332:8;:23;;;:49;;;;;;;;;;;;;;;;;;55633:19;55665:1;55655:7;:11;55633:33;;55681:31;55715:11;:24;55727:11;55715:24;;;;;;;;;;;55681:58;;55783:1;55758:27;;:8;:13;;;;;;;;;;;;:27;;;55754:384;;;55968:13;;55953:11;:28;55949:174;;56022:4;56006:8;:13;;;:20;;;;;;;;;;;;;;;;;;56075:13;:28;;;56049:8;:23;;;:54;;;;;;;;;;;;;;;;;;55949:174;55754:384;55113:1036;;;56185:7;56181:2;56166:27;;56175:4;56166:27;;;;;;;;;;;;56204:42;56225:4;56231:2;56235:7;56244:1;56204:20;:42::i;:::-;54228:2026;;54124:2130;;;:::o;45098:1109::-;45160:21;;:::i;:::-;45194:12;45209:7;45194:22;;45277:4;45258:15;:13;:15::i;:::-;:23;;:47;;;;;45292:13;;45285:4;:20;45258:47;45254:886;;;45326:31;45360:11;:17;45372:4;45360:17;;;;;;;;;;;45326:51;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;45401:9;:16;;;45396:729;;45472:1;45446:28;;:9;:14;;;:28;;;45442:101;;45510:9;45503:16;;;;;;45442:101;45845:261;45852:4;45845:261;;;45885:6;;;;;;;;45930:11;:17;45942:4;45930:17;;;;;;;;;;;45918:29;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;46004:1;45978:28;;:9;:14;;;:28;;;45974:109;;46046:9;46039:16;;;;;;45974:109;45845:261;;;45396:729;45307:833;45254:886;46168:31;;;;;;;;;;;;;;45098:1109;;;;:::o;50208:104::-;50277:27;50287:2;50291:8;50277:27;;;;;;;;;;;;:9;:27::i;:::-;50208:104;;:::o;21658:191::-;21732:16;21751:6;;;;;;;;;;;21732:25;;21777:8;21768:6;;:17;;;;;;;;;;;;;;;;;;21832:8;21801:40;;21822:8;21801:40;;;;;;;;;;;;21721:128;21658:191;:::o;23089:326::-;23149:4;23406:1;23384:7;:19;;;:23;23377:30;;23089:326;;;:::o;59864:667::-;60027:4;60064:2;60048:36;;;60085:12;:10;:12::i;:::-;60099:4;60105:7;60114:5;60048:72;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;60044:480;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;60299:1;60282:6;:13;:18;60278:235;;;60328:40;;;;;;;;;;;;;;60278:235;60471:6;60465:13;60456:6;60452:2;60448:15;60441:38;60044:480;60177:45;;;60167:55;;;:6;:55;;;;60160:62;;;59864:667;;;;;;:::o;75816:100::-;75868:13;75901:7;75894:14;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;75816:100;:::o;16196:723::-;16252:13;16482:1;16473:5;:10;16469:53;;;16500:10;;;;;;;;;;;;;;;;;;;;;16469:53;16532:12;16547:5;16532:20;;16563:14;16588:78;16603:1;16595:4;:9;16588:78;;16621:8;;;;;:::i;:::-;;;;16652:2;16644:10;;;;;:::i;:::-;;;16588:78;;;16676:19;16708:6;16698:17;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;16676:39;;16726:154;16742:1;16733:5;:10;16726:154;;16770:1;16760:11;;;;;:::i;:::-;;;16837:2;16829:5;:10;;;;:::i;:::-;16816:2;:24;;;;:::i;:::-;16803:39;;16786:6;16793;16786:14;;;;;;;;:::i;:::-;;;;;:56;;;;;;;;;;;16866:2;16857:11;;;;;:::i;:::-;;;16726:154;;;16904:6;16890:21;;;;;16196:723;;;;:::o;1219:190::-;1344:4;1397;1368:25;1381:5;1388:4;1368:12;:25::i;:::-;:33;1361:40;;1219:190;;;;;:::o;61179:159::-;;;;;:::o;61997:158::-;;;;;:::o;50686:1751::-;50809:20;50832:13;;50809:36;;50874:1;50860:16;;:2;:16;;;50856:48;;;50885:19;;;;;;;;;;;;;;50856:48;50931:1;50919:8;:13;50915:44;;;50941:18;;;;;;;;;;;;;;50915:44;50972:61;51002:1;51006:2;51010:12;51024:8;50972:21;:61::i;:::-;51345:8;51310:12;:16;51323:2;51310:16;;;;;;;;;;;;;;;:24;;;:44;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;51409:8;51369:12;:16;51382:2;51369:16;;;;;;;;;;;;;;;:29;;;:49;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;51468:2;51435:11;:25;51447:12;51435:25;;;;;;;;;;;:30;;;:35;;;;;;;;;;;;;;;;;;51535:15;51485:11;:25;51497:12;51485:25;;;;;;;;;;;:40;;;:66;;;;;;;;;;;;;;;;;;51568:20;51591:12;51568:35;;51618:11;51647:8;51632:12;:23;51618:37;;51676:15;:2;:13;;;:15::i;:::-;51672:633;;;51712:314;51768:12;51764:2;51743:38;;51760:1;51743:38;;;;;;;;;;;;51809:69;51848:1;51852:2;51856:14;;;;;;51872:5;51809:30;:69::i;:::-;51804:174;;51914:40;;;;;;;;;;;;;;51804:174;52021:3;52005:12;:19;;51712:314;;52107:12;52090:13;;:29;52086:43;;52121:8;;;52086:43;51672:633;;;52170:120;52226:14;;;;;;52222:2;52201:40;;52218:1;52201:40;;;;;;;;;;;;52285:3;52269:12;:19;;52170:120;;51672:633;52335:12;52319:13;:28;;;;51285:1074;;52369:60;52398:1;52402:2;52406:12;52420:8;52369:20;:60::i;:::-;50798:1639;50686:1751;;;:::o;2086:296::-;2169:7;2189:20;2212:4;2189:27;;2232:9;2227:118;2251:5;:12;2247:1;:16;2227:118;;;2300:33;2310:12;2324:5;2330:1;2324:8;;;;;;;;:::i;:::-;;;;;;;;2300:9;:33::i;:::-;2285:48;;2265:3;;;;;:::i;:::-;;;;2227:118;;;;2362:12;2355:19;;;2086:296;;;;:::o;8293:149::-;8356:7;8387:1;8383;:5;:51;;8414:20;8429:1;8432;8414:14;:20::i;:::-;8383:51;;;8391:20;8406:1;8409;8391:14;:20::i;:::-;8383:51;8376:58;;8293:149;;;;:::o;8450:268::-;8518:13;8625:1;8619:4;8612:15;8654:1;8648:4;8641:15;8695:4;8689;8679:21;8670:30;;8450:268;;;;:::o;-1:-1:-1:-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;:::o;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;:::-;;;;;;;;;;;;;;;;;;;;;:::o;7:75:1:-;40:6;73:2;67:9;57:19;;7:75;:::o;88:117::-;197:1;194;187:12;211:117;320:1;317;310:12;334:149;370:7;410:66;403:5;399:78;388:89;;334:149;;;:::o;489:120::-;561:23;578:5;561:23;:::i;:::-;554:5;551:34;541:62;;599:1;596;589:12;541:62;489:120;:::o;615:137::-;660:5;698:6;685:20;676:29;;714:32;740:5;714:32;:::i;:::-;615:137;;;;:::o;758:327::-;816:6;865:2;853:9;844:7;840:23;836:32;833:119;;;871:79;;:::i;:::-;833:119;991:1;1016:52;1060:7;1051:6;1040:9;1036:22;1016:52;:::i;:::-;1006:62;;962:116;758:327;;;;:::o;1091:90::-;1125:7;1168:5;1161:13;1154:21;1143:32;;1091:90;;;:::o;1187:109::-;1268:21;1283:5;1268:21;:::i;:::-;1263:3;1256:34;1187:109;;:::o;1302:210::-;1389:4;1427:2;1416:9;1412:18;1404:26;;1440:65;1502:1;1491:9;1487:17;1478:6;1440:65;:::i;:::-;1302:210;;;;:::o;1518:99::-;1570:6;1604:5;1598:12;1588:22;;1518:99;;;:::o;1623:169::-;1707:11;1741:6;1736:3;1729:19;1781:4;1776:3;1772:14;1757:29;;1623:169;;;;:::o;1798:307::-;1866:1;1876:113;1890:6;1887:1;1884:13;1876:113;;;1975:1;1970:3;1966:11;1960:18;1956:1;1951:3;1947:11;1940:39;1912:2;1909:1;1905:10;1900:15;;1876:113;;;2007:6;2004:1;2001:13;1998:101;;;2087:1;2078:6;2073:3;2069:16;2062:27;1998:101;1847:258;1798:307;;;:::o;2111:102::-;2152:6;2203:2;2199:7;2194:2;2187:5;2183:14;2179:28;2169:38;;2111:102;;;:::o;2219:364::-;2307:3;2335:39;2368:5;2335:39;:::i;:::-;2390:71;2454:6;2449:3;2390:71;:::i;:::-;2383:78;;2470:52;2515:6;2510:3;2503:4;2496:5;2492:16;2470:52;:::i;:::-;2547:29;2569:6;2547:29;:::i;:::-;2542:3;2538:39;2531:46;;2311:272;2219:364;;;;:::o;2589:313::-;2702:4;2740:2;2729:9;2725:18;2717:26;;2789:9;2783:4;2779:20;2775:1;2764:9;2760:17;2753:47;2817:78;2890:4;2881:6;2817:78;:::i;:::-;2809:86;;2589:313;;;;:::o;2908:77::-;2945:7;2974:5;2963:16;;2908:77;;;:::o;2991:122::-;3064:24;3082:5;3064:24;:::i;:::-;3057:5;3054:35;3044:63;;3103:1;3100;3093:12;3044:63;2991:122;:::o;3119:139::-;3165:5;3203:6;3190:20;3181:29;;3219:33;3246:5;3219:33;:::i;:::-;3119:139;;;;:::o;3264:329::-;3323:6;3372:2;3360:9;3351:7;3347:23;3343:32;3340:119;;;3378:79;;:::i;:::-;3340:119;3498:1;3523:53;3568:7;3559:6;3548:9;3544:22;3523:53;:::i;:::-;3513:63;;3469:117;3264:329;;;;:::o;3599:126::-;3636:7;3676:42;3669:5;3665:54;3654:65;;3599:126;;;:::o;3731:96::-;3768:7;3797:24;3815:5;3797:24;:::i;:::-;3786:35;;3731:96;;;:::o;3833:118::-;3920:24;3938:5;3920:24;:::i;:::-;3915:3;3908:37;3833:118;;:::o;3957:222::-;4050:4;4088:2;4077:9;4073:18;4065:26;;4101:71;4169:1;4158:9;4154:17;4145:6;4101:71;:::i;:::-;3957:222;;;;:::o;4185:122::-;4258:24;4276:5;4258:24;:::i;:::-;4251:5;4248:35;4238:63;;4297:1;4294;4287:12;4238:63;4185:122;:::o;4313:139::-;4359:5;4397:6;4384:20;4375:29;;4413:33;4440:5;4413:33;:::i;:::-;4313:139;;;;:::o;4458:474::-;4526:6;4534;4583:2;4571:9;4562:7;4558:23;4554:32;4551:119;;;4589:79;;:::i;:::-;4551:119;4709:1;4734:53;4779:7;4770:6;4759:9;4755:22;4734:53;:::i;:::-;4724:63;;4680:117;4836:2;4862:53;4907:7;4898:6;4887:9;4883:22;4862:53;:::i;:::-;4852:63;;4807:118;4458:474;;;;;:::o;4938:118::-;5025:24;5043:5;5025:24;:::i;:::-;5020:3;5013:37;4938:118;;:::o;5062:222::-;5155:4;5193:2;5182:9;5178:18;5170:26;;5206:71;5274:1;5263:9;5259:17;5250:6;5206:71;:::i;:::-;5062:222;;;;:::o;5290:619::-;5367:6;5375;5383;5432:2;5420:9;5411:7;5407:23;5403:32;5400:119;;;5438:79;;:::i;:::-;5400:119;5558:1;5583:53;5628:7;5619:6;5608:9;5604:22;5583:53;:::i;:::-;5573:63;;5529:117;5685:2;5711:53;5756:7;5747:6;5736:9;5732:22;5711:53;:::i;:::-;5701:63;;5656:118;5813:2;5839:53;5884:7;5875:6;5864:9;5860:22;5839:53;:::i;:::-;5829:63;;5784:118;5290:619;;;;;:::o;5915:77::-;5952:7;5981:5;5970:16;;5915:77;;;:::o;5998:118::-;6085:24;6103:5;6085:24;:::i;:::-;6080:3;6073:37;5998:118;;:::o;6122:222::-;6215:4;6253:2;6242:9;6238:18;6230:26;;6266:71;6334:1;6323:9;6319:17;6310:6;6266:71;:::i;:::-;6122:222;;;;:::o;6350:117::-;6459:1;6456;6449:12;6473:117;6582:1;6579;6572:12;6596:180;6644:77;6641:1;6634:88;6741:4;6738:1;6731:15;6765:4;6762:1;6755:15;6782:281;6865:27;6887:4;6865:27;:::i;:::-;6857:6;6853:40;6995:6;6983:10;6980:22;6959:18;6947:10;6944:34;6941:62;6938:88;;;7006:18;;:::i;:::-;6938:88;7046:10;7042:2;7035:22;6825:238;6782:281;;:::o;7069:129::-;7103:6;7130:20;;:::i;:::-;7120:30;;7159:33;7187:4;7179:6;7159:33;:::i;:::-;7069:129;;;:::o;7204:308::-;7266:4;7356:18;7348:6;7345:30;7342:56;;;7378:18;;:::i;:::-;7342:56;7416:29;7438:6;7416:29;:::i;:::-;7408:37;;7500:4;7494;7490:15;7482:23;;7204:308;;;:::o;7518:154::-;7602:6;7597:3;7592;7579:30;7664:1;7655:6;7650:3;7646:16;7639:27;7518:154;;;:::o;7678:412::-;7756:5;7781:66;7797:49;7839:6;7797:49;:::i;:::-;7781:66;:::i;:::-;7772:75;;7870:6;7863:5;7856:21;7908:4;7901:5;7897:16;7946:3;7937:6;7932:3;7928:16;7925:25;7922:112;;;7953:79;;:::i;:::-;7922:112;8043:41;8077:6;8072:3;8067;8043:41;:::i;:::-;7762:328;7678:412;;;;;:::o;8110:340::-;8166:5;8215:3;8208:4;8200:6;8196:17;8192:27;8182:122;;8223:79;;:::i;:::-;8182:122;8340:6;8327:20;8365:79;8440:3;8432:6;8425:4;8417:6;8413:17;8365:79;:::i;:::-;8356:88;;8172:278;8110:340;;;;:::o;8456:509::-;8525:6;8574:2;8562:9;8553:7;8549:23;8545:32;8542:119;;;8580:79;;:::i;:::-;8542:119;8728:1;8717:9;8713:17;8700:31;8758:18;8750:6;8747:30;8744:117;;;8780:79;;:::i;:::-;8744:117;8885:63;8940:7;8931:6;8920:9;8916:22;8885:63;:::i;:::-;8875:73;;8671:287;8456:509;;;;:::o;8971:329::-;9030:6;9079:2;9067:9;9058:7;9054:23;9050:32;9047:119;;;9085:79;;:::i;:::-;9047:119;9205:1;9230:53;9275:7;9266:6;9255:9;9251:22;9230:53;:::i;:::-;9220:63;;9176:117;8971:329;;;;:::o;9306:122::-;9379:24;9397:5;9379:24;:::i;:::-;9372:5;9369:35;9359:63;;9418:1;9415;9408:12;9359:63;9306:122;:::o;9434:139::-;9480:5;9518:6;9505:20;9496:29;;9534:33;9561:5;9534:33;:::i;:::-;9434:139;;;;:::o;9579:329::-;9638:6;9687:2;9675:9;9666:7;9662:23;9658:32;9655:119;;;9693:79;;:::i;:::-;9655:119;9813:1;9838:53;9883:7;9874:6;9863:9;9859:22;9838:53;:::i;:::-;9828:63;;9784:117;9579:329;;;;:::o;9914:116::-;9984:21;9999:5;9984:21;:::i;:::-;9977:5;9974:32;9964:60;;10020:1;10017;10010:12;9964:60;9914:116;:::o;10036:133::-;10079:5;10117:6;10104:20;10095:29;;10133:30;10157:5;10133:30;:::i;:::-;10036:133;;;;:::o;10175:468::-;10240:6;10248;10297:2;10285:9;10276:7;10272:23;10268:32;10265:119;;;10303:79;;:::i;:::-;10265:119;10423:1;10448:53;10493:7;10484:6;10473:9;10469:22;10448:53;:::i;:::-;10438:63;;10394:117;10550:2;10576:50;10618:7;10609:6;10598:9;10594:22;10576:50;:::i;:::-;10566:60;;10521:115;10175:468;;;;;:::o;10649:307::-;10710:4;10800:18;10792:6;10789:30;10786:56;;;10822:18;;:::i;:::-;10786:56;10860:29;10882:6;10860:29;:::i;:::-;10852:37;;10944:4;10938;10934:15;10926:23;;10649:307;;;:::o;10962:410::-;11039:5;11064:65;11080:48;11121:6;11080:48;:::i;:::-;11064:65;:::i;:::-;11055:74;;11152:6;11145:5;11138:21;11190:4;11183:5;11179:16;11228:3;11219:6;11214:3;11210:16;11207:25;11204:112;;;11235:79;;:::i;:::-;11204:112;11325:41;11359:6;11354:3;11349;11325:41;:::i;:::-;11045:327;10962:410;;;;;:::o;11391:338::-;11446:5;11495:3;11488:4;11480:6;11476:17;11472:27;11462:122;;11503:79;;:::i;:::-;11462:122;11620:6;11607:20;11645:78;11719:3;11711:6;11704:4;11696:6;11692:17;11645:78;:::i;:::-;11636:87;;11452:277;11391:338;;;;:::o;11735:943::-;11830:6;11838;11846;11854;11903:3;11891:9;11882:7;11878:23;11874:33;11871:120;;;11910:79;;:::i;:::-;11871:120;12030:1;12055:53;12100:7;12091:6;12080:9;12076:22;12055:53;:::i;:::-;12045:63;;12001:117;12157:2;12183:53;12228:7;12219:6;12208:9;12204:22;12183:53;:::i;:::-;12173:63;;12128:118;12285:2;12311:53;12356:7;12347:6;12336:9;12332:22;12311:53;:::i;:::-;12301:63;;12256:118;12441:2;12430:9;12426:18;12413:32;12472:18;12464:6;12461:30;12458:117;;;12494:79;;:::i;:::-;12458:117;12599:62;12653:7;12644:6;12633:9;12629:22;12599:62;:::i;:::-;12589:72;;12384:287;11735:943;;;;;;;:::o;12684:117::-;12793:1;12790;12783:12;12807:117;12916:1;12913;12906:12;12947:568;13020:8;13030:6;13080:3;13073:4;13065:6;13061:17;13057:27;13047:122;;13088:79;;:::i;:::-;13047:122;13201:6;13188:20;13178:30;;13231:18;13223:6;13220:30;13217:117;;;13253:79;;:::i;:::-;13217:117;13367:4;13359:6;13355:17;13343:29;;13421:3;13413:4;13405:6;13401:17;13391:8;13387:32;13384:41;13381:128;;;13428:79;;:::i;:::-;13381:128;12947:568;;;;;:::o;13521:704::-;13616:6;13624;13632;13681:2;13669:9;13660:7;13656:23;13652:32;13649:119;;;13687:79;;:::i;:::-;13649:119;13807:1;13832:53;13877:7;13868:6;13857:9;13853:22;13832:53;:::i;:::-;13822:63;;13778:117;13962:2;13951:9;13947:18;13934:32;13993:18;13985:6;13982:30;13979:117;;;14015:79;;:::i;:::-;13979:117;14128:80;14200:7;14191:6;14180:9;14176:22;14128:80;:::i;:::-;14110:98;;;;13905:313;13521:704;;;;;:::o;14231:474::-;14299:6;14307;14356:2;14344:9;14335:7;14331:23;14327:32;14324:119;;;14362:79;;:::i;:::-;14324:119;14482:1;14507:53;14552:7;14543:6;14532:9;14528:22;14507:53;:::i;:::-;14497:63;;14453:117;14609:2;14635:53;14680:7;14671:6;14660:9;14656:22;14635:53;:::i;:::-;14625:63;;14580:118;14231:474;;;;;:::o;14711:180::-;14759:77;14756:1;14749:88;14856:4;14853:1;14846:15;14880:4;14877:1;14870:15;14897:320;14941:6;14978:1;14972:4;14968:12;14958:22;;15025:1;15019:4;15015:12;15046:18;15036:81;;15102:4;15094:6;15090:17;15080:27;;15036:81;15164:2;15156:6;15153:14;15133:18;15130:38;15127:84;;;15183:18;;:::i;:::-;15127:84;14948:269;14897:320;;;:::o;15223:180::-;15271:77;15268:1;15261:88;15368:4;15365:1;15358:15;15392:4;15389:1;15382:15;15409:305;15449:3;15468:20;15486:1;15468:20;:::i;:::-;15463:25;;15502:20;15520:1;15502:20;:::i;:::-;15497:25;;15656:1;15588:66;15584:74;15581:1;15578:81;15575:107;;;15662:18;;:::i;:::-;15575:107;15706:1;15703;15699:9;15692:16;;15409:305;;;;:::o;15720:224::-;15860:34;15856:1;15848:6;15844:14;15837:58;15929:7;15924:2;15916:6;15912:15;15905:32;15720:224;:::o;15950:366::-;16092:3;16113:67;16177:2;16172:3;16113:67;:::i;:::-;16106:74;;16189:93;16278:3;16189:93;:::i;:::-;16307:2;16302:3;16298:12;16291:19;;15950:366;;;:::o;16322:419::-;16488:4;16526:2;16515:9;16511:18;16503:26;;16575:9;16569:4;16565:20;16561:1;16550:9;16546:17;16539:47;16603:131;16729:4;16603:131;:::i;:::-;16595:139;;16322:419;;;:::o;16747:221::-;16887:34;16883:1;16875:6;16871:14;16864:58;16956:4;16951:2;16943:6;16939:15;16932:29;16747:221;:::o;16974:366::-;17116:3;17137:67;17201:2;17196:3;17137:67;:::i;:::-;17130:74;;17213:93;17302:3;17213:93;:::i;:::-;17331:2;17326:3;17322:12;17315:19;;16974:366;;;:::o;17346:419::-;17512:4;17550:2;17539:9;17535:18;17527:26;;17599:9;17593:4;17589:20;17585:1;17574:9;17570:17;17563:47;17627:131;17753:4;17627:131;:::i;:::-;17619:139;;17346:419;;;:::o;17771:220::-;17911:34;17907:1;17899:6;17895:14;17888:58;17980:3;17975:2;17967:6;17963:15;17956:28;17771:220;:::o;17997:366::-;18139:3;18160:67;18224:2;18219:3;18160:67;:::i;:::-;18153:74;;18236:93;18325:3;18236:93;:::i;:::-;18354:2;18349:3;18345:12;18338:19;;17997:366;;;:::o;18369:419::-;18535:4;18573:2;18562:9;18558:18;18550:26;;18622:9;18616:4;18612:20;18608:1;18597:9;18593:17;18586:47;18650:131;18776:4;18650:131;:::i;:::-;18642:139;;18369:419;;;:::o;18794:171::-;18934:23;18930:1;18922:6;18918:14;18911:47;18794:171;:::o;18971:366::-;19113:3;19134:67;19198:2;19193:3;19134:67;:::i;:::-;19127:74;;19210:93;19299:3;19210:93;:::i;:::-;19328:2;19323:3;19319:12;19312:19;;18971:366;;;:::o;19343:419::-;19509:4;19547:2;19536:9;19532:18;19524:26;;19596:9;19590:4;19586:20;19582:1;19571:9;19567:17;19560:47;19624:131;19750:4;19624:131;:::i;:::-;19616:139;;19343:419;;;:::o;19768:182::-;19908:34;19904:1;19896:6;19892:14;19885:58;19768:182;:::o;19956:366::-;20098:3;20119:67;20183:2;20178:3;20119:67;:::i;:::-;20112:74;;20195:93;20284:3;20195:93;:::i;:::-;20313:2;20308:3;20304:12;20297:19;;19956:366;;;:::o;20328:419::-;20494:4;20532:2;20521:9;20517:18;20509:26;;20581:9;20575:4;20571:20;20567:1;20556:9;20552:17;20545:47;20609:131;20735:4;20609:131;:::i;:::-;20601:139;;20328:419;;;:::o;20753:220::-;20893:34;20889:1;20881:6;20877:14;20870:58;20962:3;20957:2;20949:6;20945:15;20938:28;20753:220;:::o;20979:366::-;21121:3;21142:67;21206:2;21201:3;21142:67;:::i;:::-;21135:74;;21218:93;21307:3;21218:93;:::i;:::-;21336:2;21331:3;21327:12;21320:19;;20979:366;;;:::o;21351:419::-;21517:4;21555:2;21544:9;21540:18;21532:26;;21604:9;21598:4;21594:20;21590:1;21579:9;21575:17;21568:47;21632:131;21758:4;21632:131;:::i;:::-;21624:139;;21351:419;;;:::o;21776:148::-;21878:11;21915:3;21900:18;;21776:148;;;;:::o;21930:377::-;22036:3;22064:39;22097:5;22064:39;:::i;:::-;22119:89;22201:6;22196:3;22119:89;:::i;:::-;22112:96;;22217:52;22262:6;22257:3;22250:4;22243:5;22239:16;22217:52;:::i;:::-;22294:6;22289:3;22285:16;22278:23;;22040:267;21930:377;;;;:::o;22313:435::-;22493:3;22515:95;22606:3;22597:6;22515:95;:::i;:::-;22508:102;;22627:95;22718:3;22709:6;22627:95;:::i;:::-;22620:102;;22739:3;22732:10;;22313:435;;;;;:::o;22754:182::-;22894:34;22890:1;22882:6;22878:14;22871:58;22754:182;:::o;22942:366::-;23084:3;23105:67;23169:2;23164:3;23105:67;:::i;:::-;23098:74;;23181:93;23270:3;23181:93;:::i;:::-;23299:2;23294:3;23290:12;23283:19;;22942:366;;;:::o;23314:419::-;23480:4;23518:2;23507:9;23503:18;23495:26;;23567:9;23561:4;23557:20;23553:1;23542:9;23538:17;23531:47;23595:131;23721:4;23595:131;:::i;:::-;23587:139;;23314:419;;;:::o;23739:94::-;23772:8;23820:5;23816:2;23812:14;23791:35;;23739:94;;;:::o;23839:::-;23878:7;23907:20;23921:5;23907:20;:::i;:::-;23896:31;;23839:94;;;:::o;23939:100::-;23978:7;24007:26;24027:5;24007:26;:::i;:::-;23996:37;;23939:100;;;:::o;24045:157::-;24150:45;24170:24;24188:5;24170:24;:::i;:::-;24150:45;:::i;:::-;24145:3;24138:58;24045:157;;:::o;24208:256::-;24320:3;24335:75;24406:3;24397:6;24335:75;:::i;:::-;24435:2;24430:3;24426:12;24419:19;;24455:3;24448:10;;24208:256;;;;:::o;24470:227::-;24610:34;24606:1;24598:6;24594:14;24587:58;24679:10;24674:2;24666:6;24662:15;24655:35;24470:227;:::o;24703:366::-;24845:3;24866:67;24930:2;24925:3;24866:67;:::i;:::-;24859:74;;24942:93;25031:3;24942:93;:::i;:::-;25060:2;25055:3;25051:12;25044:19;;24703:366;;;:::o;25075:419::-;25241:4;25279:2;25268:9;25264:18;25256:26;;25328:9;25322:4;25318:20;25314:1;25303:9;25299:17;25292:47;25356:131;25482:4;25356:131;:::i;:::-;25348:139;;25075:419;;;:::o;25500:225::-;25640:34;25636:1;25628:6;25624:14;25617:58;25709:8;25704:2;25696:6;25692:15;25685:33;25500:225;:::o;25731:366::-;25873:3;25894:67;25958:2;25953:3;25894:67;:::i;:::-;25887:74;;25970:93;26059:3;25970:93;:::i;:::-;26088:2;26083:3;26079:12;26072:19;;25731:366;;;:::o;26103:419::-;26269:4;26307:2;26296:9;26292:18;26284:26;;26356:9;26350:4;26346:20;26342:1;26331:9;26327:17;26320:47;26384:131;26510:4;26384:131;:::i;:::-;26376:139;;26103:419;;;:::o;26528:182::-;26668:34;26664:1;26656:6;26652:14;26645:58;26528:182;:::o;26716:366::-;26858:3;26879:67;26943:2;26938:3;26879:67;:::i;:::-;26872:74;;26955:93;27044:3;26955:93;:::i;:::-;27073:2;27068:3;27064:12;27057:19;;26716:366;;;:::o;27088:419::-;27254:4;27292:2;27281:9;27277:18;27269:26;;27341:9;27335:4;27331:20;27327:1;27316:9;27312:17;27305:47;27369:131;27495:4;27369:131;:::i;:::-;27361:139;;27088:419;;;:::o;27513:98::-;27564:6;27598:5;27592:12;27582:22;;27513:98;;;:::o;27617:168::-;27700:11;27734:6;27729:3;27722:19;27774:4;27769:3;27765:14;27750:29;;27617:168;;;;:::o;27791:360::-;27877:3;27905:38;27937:5;27905:38;:::i;:::-;27959:70;28022:6;28017:3;27959:70;:::i;:::-;27952:77;;28038:52;28083:6;28078:3;28071:4;28064:5;28060:16;28038:52;:::i;:::-;28115:29;28137:6;28115:29;:::i;:::-;28110:3;28106:39;28099:46;;27881:270;27791:360;;;;:::o;28157:640::-;28352:4;28390:3;28379:9;28375:19;28367:27;;28404:71;28472:1;28461:9;28457:17;28448:6;28404:71;:::i;:::-;28485:72;28553:2;28542:9;28538:18;28529:6;28485:72;:::i;:::-;28567;28635:2;28624:9;28620:18;28611:6;28567:72;:::i;:::-;28686:9;28680:4;28676:20;28671:2;28660:9;28656:18;28649:48;28714:76;28785:4;28776:6;28714:76;:::i;:::-;28706:84;;28157:640;;;;;;;:::o;28803:141::-;28859:5;28890:6;28884:13;28875:22;;28906:32;28932:5;28906:32;:::i;:::-;28803:141;;;;:::o;28950:349::-;29019:6;29068:2;29056:9;29047:7;29043:23;29039:32;29036:119;;;29074:79;;:::i;:::-;29036:119;29194:1;29219:63;29274:7;29265:6;29254:9;29250:22;29219:63;:::i;:::-;29209:73;;29165:127;28950:349;;;;:::o;29305:233::-;29344:3;29367:24;29385:5;29367:24;:::i;:::-;29358:33;;29413:66;29406:5;29403:77;29400:103;;;29483:18;;:::i;:::-;29400:103;29530:1;29523:5;29519:13;29512:20;;29305:233;;;:::o;29544:180::-;29592:77;29589:1;29582:88;29689:4;29686:1;29679:15;29713:4;29710:1;29703:15;29730:185;29770:1;29787:20;29805:1;29787:20;:::i;:::-;29782:25;;29821:20;29839:1;29821:20;:::i;:::-;29816:25;;29860:1;29850:35;;29865:18;;:::i;:::-;29850:35;29907:1;29904;29900:9;29895:14;;29730:185;;;;:::o;29921:191::-;29961:4;29981:20;29999:1;29981:20;:::i;:::-;29976:25;;30015:20;30033:1;30015:20;:::i;:::-;30010:25;;30054:1;30051;30048:8;30045:34;;;30059:18;;:::i;:::-;30045:34;30104:1;30101;30097:9;30089:17;;29921:191;;;;:::o;30118:176::-;30150:1;30167:20;30185:1;30167:20;:::i;:::-;30162:25;;30201:20;30219:1;30201:20;:::i;:::-;30196:25;;30240:1;30230:35;;30245:18;;:::i;:::-;30230:35;30286:1;30283;30279:9;30274:14;;30118:176;;;;:::o;30300:180::-;30348:77;30345:1;30338:88;30445:4;30442:1;30435:15;30469:4;30466:1;30459:15

Swarm Source

ipfs://963ff9dc601d0035f4df9879263a41a4c2b4a1154e2a4b6d28b8f72ee5920674
Loading...
Loading
Loading...
Loading
[ 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.