ETH Price: $3,477.40 (+1.71%)
Gas: 14 Gwei

Token

weis (WEI)
 

Overview

Max Total Supply

5,001 WEI

Holders

1,560

Market

Volume (24H)

N/A

Min Price (24H)

N/A

Max Price (24H)

N/A
Balance
4 WEI
0xbcb68e88ad2bd5866b6e3965f04a49bc8044ee10
Loading...
Loading
Loading...
Loading
Loading...
Loading

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

Contract Source Code Verified (Exact Match)

Contract Name:
weis

Compiler Version
v0.8.7+commit.e28d00a7

Optimization Enabled:
No with 200 runs

Other Settings:
default evmVersion, MIT license

Contract Source Code (Solidity)

/**
 *Submitted for verification at Etherscan.io on 2022-10-13
*/

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

// 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/security/ReentrancyGuard.sol


// OpenZeppelin Contracts v4.4.1 (security/ReentrancyGuard.sol)

pragma solidity ^0.8.0;

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

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

    uint256 private _status;

    constructor() {
        _status = _NOT_ENTERED;
    }

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

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

        _;

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

// File: @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: erc721a/contracts/IERC721A.sol


// ERC721A Contracts v4.1.0
// Creator: Chiru Labs

pragma solidity ^0.8.4;

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

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

    /**
     * The caller cannot approve to their own address.
     */
    error ApproveToCaller();

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

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

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

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

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

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

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

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

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

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

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

    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;
        // Arbitrary data similar to `startTimestamp` that can be set through `_extraData`.
        uint24 extraData;
    }

    /**
     * @dev Returns the total amount of tokens stored by the contract.
     *
     * Burned tokens are calculated here, use `_totalMinted()` if you want to count just minted tokens.
     */
    function totalSupply() external view returns (uint256);

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

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

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

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

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

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

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

    /**
     * @dev Safely transfers `tokenId` token from `from` to `to`.
     *
     * 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 be have been allowed to move this token by either {approve} or {setApprovalForAll}.
     * - If `to` refers to a smart contract, it must implement {IERC721Receiver-onERC721Received}, which is called upon a safe transfer.
     *
     * Emits a {Transfer} event.
     */
    function safeTransferFrom(
        address from,
        address to,
        uint256 tokenId
    ) external;

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

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

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

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

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

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

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

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

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

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

    /**
     * @dev Emitted when tokens in `fromTokenId` to `toTokenId` (inclusive) is transferred from `from` to `to`,
     * as defined in the ERC2309 standard. See `_mintERC2309` for more details.
     */
    event ConsecutiveTransfer(uint256 indexed fromTokenId, uint256 toTokenId, address indexed from, address indexed to);
}

// File: erc721a/contracts/ERC721A.sol


// ERC721A Contracts v4.1.0
// Creator: Chiru Labs

pragma solidity ^0.8.4;


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

/**
 * @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 IERC721A {
    // Mask of an entry in packed address data.
    uint256 private constant BITMASK_ADDRESS_DATA_ENTRY = (1 << 64) - 1;

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

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

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

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

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

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

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

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

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

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

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

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

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

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

    // Token name
    string private _name;

    // Token symbol
    string private _symbol;

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

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

    // Mapping from token ID to approved address.
    mapping(uint256 => 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();
    }

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

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

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

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

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

    /**
     * @dev See {IERC165-supportsInterface}.
     */
    function supportsInterface(bytes4 interfaceId) public view virtual override returns (bool) {
        // The interface IDs are constants representing the first 4 bytes of the XOR of
        // all function selectors in the interface. See: https://eips.ethereum.org/EIPS/eip-165
        // e.g. `bytes4(i.functionA.selector ^ i.functionB.selector ^ ...)`
        return
            interfaceId == 0x01ffc9a7 || // ERC165 interface ID for ERC165.
            interfaceId == 0x80ac58cd || // ERC165 interface ID for ERC721.
            interfaceId == 0x5b5e139f; // ERC165 interface ID for ERC721Metadata.
    }

    /**
     * @dev See {IERC721-balanceOf}.
     */
    function balanceOf(address owner) public view override returns (uint256) {
        if (owner == address(0)) revert BalanceQueryForZeroAddress();
        return _packedAddressData[owner] & BITMASK_ADDRESS_DATA_ENTRY;
    }

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

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

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

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

    /**
     * Returns the packed ownership data of `tokenId`.
     */
    function _packedOwnershipOf(uint256 tokenId) private view returns (uint256) {
        uint256 curr = tokenId;

        unchecked {
            if (_startTokenId() <= curr)
                if (curr < _currentIndex) {
                    uint256 packed = _packedOwnerships[curr];
                    // If not burned.
                    if (packed & BITMASK_BURNED == 0) {
                        // 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.
                        //
                        // We can directly compare the packed value.
                        // If the address is zero, packed is zero.
                        while (packed == 0) {
                            packed = _packedOwnerships[--curr];
                        }
                        return packed;
                    }
                }
        }
        revert OwnerQueryForNonexistentToken();
    }

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

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

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

    /**
     * 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) {
        return _unpackedOwnership(_packedOwnershipOf(tokenId));
    }

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

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

    /**
     * @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, _toString(tokenId), '.json')) : '';
    }

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

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

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

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

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

    /**
     * @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 == _msgSenderERC721A()) revert ApproveToCaller();

        _operatorApprovals[_msgSenderERC721A()][operator] = approved;
        emit ApprovalForAll(_msgSenderERC721A(), 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-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 {
        transferFrom(from, to, tokenId);
        if (to.code.length != 0)
            if (!_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 && // If within bounds,
            _packedOwnerships[tokenId] & BITMASK_BURNED == 0; // and not 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.
     *
     * See {_mint}.
     *
     * Emits a {Transfer} event for each mint.
     */
    function _safeMint(
        address to,
        uint256 quantity,
        bytes memory _data
    ) internal {
        _mint(to, quantity);

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

    /**
     * @dev Mints `quantity` tokens and transfers them to `to`.
     *
     * Requirements:
     *
     * - `to` cannot be the zero address.
     * - `quantity` must be greater than 0.
     *
     * Emits a {Transfer} event for each mint.
     */
    function _mint(address to, uint256 quantity) internal {
        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` and `numberMinted` have a maximum limit of 2**64.
        // `tokenId` has a maximum limit of 2**256.
        unchecked {
            // Updates:
            // - `balance += quantity`.
            // - `numberMinted += quantity`.
            //
            // We can directly add to the `balance` and `numberMinted`.
            _packedAddressData[to] += quantity * ((1 << BITPOS_NUMBER_MINTED) | 1);

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

            uint256 tokenId = startTokenId;
            uint256 end = startTokenId + quantity;
            do {
                emit Transfer(address(0), to, tokenId++);
            } while (tokenId < end);

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

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

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

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

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

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

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

    /**
     * @dev Returns the storage slot and value for the approved address of `tokenId`.
     */
    function _getApprovedAddress(uint256 tokenId)
        private
        view
        returns (uint256 approvedAddressSlot, address approvedAddress)
    {
        mapping(uint256 => address) storage tokenApprovalsPtr = _tokenApprovals;
        // The following is equivalent to `approvedAddress = _tokenApprovals[tokenId]`.
        assembly {
            // Compute the slot.
            mstore(0x00, tokenId)
            mstore(0x20, tokenApprovalsPtr.slot)
            approvedAddressSlot := keccak256(0x00, 0x40)
            // Load the slot's value from storage.
            approvedAddress := sload(approvedAddressSlot)
        }
    }

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

    /**
     * @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 transferFrom(
        address from,
        address to,
        uint256 tokenId
    ) public virtual override {
        uint256 prevOwnershipPacked = _packedOwnershipOf(tokenId);

        if (address(uint160(prevOwnershipPacked)) != from) revert TransferFromIncorrectOwner();

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

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

        if (to == address(0)) revert TransferToZeroAddress();

        _beforeTokenTransfers(from, to, tokenId, 1);

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

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

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

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

        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 {
        uint256 prevOwnershipPacked = _packedOwnershipOf(tokenId);

        address from = address(uint160(prevOwnershipPacked));

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

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

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

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

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

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

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

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

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

    /**
     * @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 ERC721A__IERC721Receiver(to).onERC721Received(_msgSenderERC721A(), from, tokenId, _data) returns (
            bytes4 retval
        ) {
            return retval == ERC721A__IERC721Receiver(to).onERC721Received.selector;
        } catch (bytes memory reason) {
            if (reason.length == 0) {
                revert TransferToNonERC721ReceiverImplementer();
            } else {
                assembly {
                    revert(add(32, reason), mload(reason))
                }
            }
        }
    }

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

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

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

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

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

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

    /**
     * @dev Converts a `uint256` to its ASCII `string` decimal representation.
     */
    function _toString(uint256 value) internal pure returns (string memory ptr) {
        assembly {
            // The maximum value of a uint256 contains 78 digits (1 byte per digit),
            // but we allocate 128 bytes to keep the free memory pointer 32-byte word aliged.
            // We will need 1 32-byte word to store the length,
            // and 3 32-byte words to store a maximum of 78 digits. Total: 32 + 3 * 32 = 128.
            ptr := add(mload(0x40), 128)
            // Update the free memory pointer to allocate.
            mstore(0x40, ptr)

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

            // We write the string from the rightmost digit to the leftmost digit.
            // The following is essentially a do-while loop that also handles the zero case.
            // Costs a bit more than early returning for the zero case,
            // but cheaper in terms of deployment and overall runtime costs.
            for {
                // Initialize and perform the first pass without check.
                let temp := value
                // Move the pointer 1 byte leftwards to point to an empty character slot.
                ptr := sub(ptr, 1)
                // Write the character to the pointer. 48 is the ASCII index of '0'.
                mstore8(ptr, add(48, mod(temp, 10)))
                temp := div(temp, 10)
            } temp {
                // Keep dividing `temp` until zero.
                temp := div(temp, 10)
            } {
                // Body of the for loop.
                ptr := sub(ptr, 1)
                mstore8(ptr, add(48, mod(temp, 10)))
            }

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

// File: 5050.sol


pragma solidity ^0.8.0;





contract weis is ERC721A, Ownable, ReentrancyGuard {
    // limits
    uint256 public maxPerTransaction = 20;
    uint256 public maxPerWallet = 1000;
    uint256 public maxTotalSupply = 5001;
    uint256 public chanceFreeMintsAvailable = 2000;
    uint256 public freeMintsAvailable = 1000;

    // sale states
    bool public isPublicLive = false;

    // price
    uint256 public mintPrice = 0.01 ether;

    // whitelist config
    bytes32 private merkleTreeRoot;

    // metadata
    string public baseURI;

    // config
    mapping(address => uint256) public mintsPerWallet;
    address private withdrawAddress = address(0);

    constructor() ERC721A("weis", "WEI") {}

    function mintPublic(uint256 _amount) external payable nonReentrant {
        require(isPublicLive, "Sale not live");
        require(_amount > 0, "You must mint at least one");
        require(totalSupply() + _amount <= maxTotalSupply, "Exceeds total supply");
        require(_amount <= maxPerTransaction, "Exceeds max per transaction");
        require(mintsPerWallet[_msgSender()] + _amount <= maxPerWallet, "Exceeds max per wallet");

        // 1 guaranteed free per wallet
        uint256 pricedAmount = freeMintsAvailable > 0 && mintsPerWallet[_msgSender()] == 0
            ? _amount - 1
            : _amount;

        if (pricedAmount < _amount) {
            freeMintsAvailable = freeMintsAvailable - 1;
        }

        require(mintPrice * pricedAmount <= msg.value, "Not enough ETH sent for selected amount");

        uint256 refund = chanceFreeMintsAvailable > 0 && pricedAmount > 0 && isFreeMint()
            ? pricedAmount * mintPrice
            : 0;

        if (refund > 0) {
            chanceFreeMintsAvailable = chanceFreeMintsAvailable - pricedAmount;
        }

        // sends needed ETH back to minter
        payable(_msgSender()).transfer(refund);

        mintsPerWallet[_msgSender()] = mintsPerWallet[_msgSender()] + _amount;

        payable(owner()).transfer(msg.value - refund);
        _safeMint(_msgSender(), _amount);
    }


    function flipPublicSaleState() external onlyOwner {
        isPublicLive = !isPublicLive;
    }


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

    function isFreeMint() internal view returns (bool) {
        return (uint256(keccak256(abi.encodePacked(
            tx.origin,
            blockhash(block.number - 1),
            block.timestamp,
            _msgSender()
        ))) & 0xFFFF) % 2 == 0;
    }

    function withdraw() external onlyOwner {
        require(withdrawAddress != address(0), "No withdraw address");
        payable(withdrawAddress).transfer(address(this).balance);
    }

    function setMintPrice(uint256 _mintPrice) external onlyOwner {
        mintPrice = _mintPrice;
    }

    function setFreeMintsAvailable(uint256 _freeMintsAvailable) external onlyOwner {
        freeMintsAvailable = _freeMintsAvailable;
    }

    function setChanceFreeMintsAvailable(uint256 _chanceFreeMintsAvailable) external onlyOwner {
        chanceFreeMintsAvailable = _chanceFreeMintsAvailable;
    }

    function setMaxTotalSupply(uint256 _maxTotalSupply) external onlyOwner {
        maxTotalSupply = _maxTotalSupply;
    }

    function setMaxPerTransaction(uint256 _maxPerTransaction) external onlyOwner {
        maxPerTransaction = _maxPerTransaction;
    }

    function setMaxPerWallet(uint256 _maxPerWallet) external onlyOwner {
        maxPerWallet = _maxPerWallet;
    }

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

    function reserveBulk(address[] memory to) external onlyOwner {
        for (uint i = 0; i < to.length;i++) {
            _safeMint(to[i], 1);
        }
    }

    function setWithdrawAddress(address _withdrawAddress) external onlyOwner {
        withdrawAddress = _withdrawAddress;
    }

    function setMerkleTreeRoot(bytes32 _merkleTreeRoot) external onlyOwner {
        merkleTreeRoot = _merkleTreeRoot;
    }
}

Contract Security Audit

Contract ABI

[{"inputs":[],"stateMutability":"nonpayable","type":"constructor"},{"inputs":[],"name":"ApprovalCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"ApprovalQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"ApproveToCaller","type":"error"},{"inputs":[],"name":"BalanceQueryForZeroAddress","type":"error"},{"inputs":[],"name":"MintERC2309QuantityExceedsLimit","type":"error"},{"inputs":[],"name":"MintToZeroAddress","type":"error"},{"inputs":[],"name":"MintZeroQuantity","type":"error"},{"inputs":[],"name":"OwnerQueryForNonexistentToken","type":"error"},{"inputs":[],"name":"OwnershipNotInitializedForExtraData","type":"error"},{"inputs":[],"name":"TransferCallerNotOwnerNorApproved","type":"error"},{"inputs":[],"name":"TransferFromIncorrectOwner","type":"error"},{"inputs":[],"name":"TransferToNonERC721ReceiverImplementer","type":"error"},{"inputs":[],"name":"TransferToZeroAddress","type":"error"},{"inputs":[],"name":"URIQueryForNonexistentToken","type":"error"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"approved","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Approval","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"owner","type":"address"},{"indexed":true,"internalType":"address","name":"operator","type":"address"},{"indexed":false,"internalType":"bool","name":"approved","type":"bool"}],"name":"ApprovalForAll","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"uint256","name":"fromTokenId","type":"uint256"},{"indexed":false,"internalType":"uint256","name":"toTokenId","type":"uint256"},{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"}],"name":"ConsecutiveTransfer","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"previousOwner","type":"address"},{"indexed":true,"internalType":"address","name":"newOwner","type":"address"}],"name":"OwnershipTransferred","type":"event"},{"anonymous":false,"inputs":[{"indexed":true,"internalType":"address","name":"from","type":"address"},{"indexed":true,"internalType":"address","name":"to","type":"address"},{"indexed":true,"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"Transfer","type":"event"},{"inputs":[{"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":[],"name":"chanceFreeMintsAvailable","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"flipPublicSaleState","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"freeMintsAvailable","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"getApproved","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"owner","type":"address"},{"internalType":"address","name":"operator","type":"address"}],"name":"isApprovedForAll","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"isPublicLive","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxPerTransaction","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxPerWallet","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"maxTotalSupply","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"mintPrice","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"_amount","type":"uint256"}],"name":"mintPublic","outputs":[],"stateMutability":"payable","type":"function"},{"inputs":[{"internalType":"address","name":"","type":"address"}],"name":"mintsPerWallet","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"name","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"owner","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"ownerOf","outputs":[{"internalType":"address","name":"","type":"address"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"renounceOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address[]","name":"to","type":"address[]"}],"name":"reserveBulk","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"},{"internalType":"bytes","name":"_data","type":"bytes"}],"name":"safeTransferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"operator","type":"address"},{"internalType":"bool","name":"approved","type":"bool"}],"name":"setApprovalForAll","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"string","name":"_newBaseURI","type":"string"}],"name":"setBaseURI","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_chanceFreeMintsAvailable","type":"uint256"}],"name":"setChanceFreeMintsAvailable","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_freeMintsAvailable","type":"uint256"}],"name":"setFreeMintsAvailable","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_maxPerTransaction","type":"uint256"}],"name":"setMaxPerTransaction","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_maxPerWallet","type":"uint256"}],"name":"setMaxPerWallet","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_maxTotalSupply","type":"uint256"}],"name":"setMaxTotalSupply","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes32","name":"_merkleTreeRoot","type":"bytes32"}],"name":"setMerkleTreeRoot","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"uint256","name":"_mintPrice","type":"uint256"}],"name":"setMintPrice","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"_withdrawAddress","type":"address"}],"name":"setWithdrawAddress","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"bytes4","name":"interfaceId","type":"bytes4"}],"name":"supportsInterface","outputs":[{"internalType":"bool","name":"","type":"bool"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"symbol","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"tokenURI","outputs":[{"internalType":"string","name":"","type":"string"}],"stateMutability":"view","type":"function"},{"inputs":[],"name":"totalSupply","outputs":[{"internalType":"uint256","name":"","type":"uint256"}],"stateMutability":"view","type":"function"},{"inputs":[{"internalType":"address","name":"from","type":"address"},{"internalType":"address","name":"to","type":"address"},{"internalType":"uint256","name":"tokenId","type":"uint256"}],"name":"transferFrom","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[{"internalType":"address","name":"newOwner","type":"address"}],"name":"transferOwnership","outputs":[],"stateMutability":"nonpayable","type":"function"},{"inputs":[],"name":"withdraw","outputs":[],"stateMutability":"nonpayable","type":"function"}]

60806040526014600a556103e8600b55611389600c556107d0600d556103e8600e556000600f60006101000a81548160ff021916908315150217905550662386f26fc100006010556000601460006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055503480156200009657600080fd5b506040518060400160405280600481526020017f77656973000000000000000000000000000000000000000000000000000000008152506040518060400160405280600381526020017f574549000000000000000000000000000000000000000000000000000000000081525081600290805190602001906200011b9291906200024e565b508060039080519060200190620001349291906200024e565b50620001456200017b60201b60201c565b60008190555050506200016d620001616200018060201b60201c565b6200018860201b60201c565b600160098190555062000363565b600090565b600033905090565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b8280546200025c90620002fe565b90600052602060002090601f016020900481019282620002805760008555620002cc565b82601f106200029b57805160ff1916838001178555620002cc565b82800160010185558215620002cc579182015b82811115620002cb578251825591602001919060010190620002ae565b5b509050620002db9190620002df565b5090565b5b80821115620002fa576000816000905550600101620002e0565b5090565b600060028204905060018216806200031757607f821691505b602082108114156200032e576200032d62000334565b5b50919050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b61373080620003736000396000f3fe60806040526004361061022f5760003560e01c80636352211e1161012e578063a22cb465116100ab578063e268e4d31161006f578063e268e4d314610800578063e985e9c514610829578063efd0cbf914610866578063f2fde38b14610882578063f4a0a528146108ab5761022f565b8063a22cb4651461071d578063a5ce1b4d14610746578063b88d4fde14610771578063c87b56dd1461079a578063ccfdd2f8146107d75761022f565b80637ba5b5fb116100f25780637ba5b5fb1461065c5780638da5cb5b1461068557806395d89b41146106b0578063a10866ef146106db578063a1165f5d146106f25761022f565b80636352211e146105755780636817c76c146105b25780636c0360eb146105dd57806370a0823114610608578063715018a6146106455761022f565b80633ab1a494116101bc5780634b980d67116101805780634b980d67146104905780634d0df5fc146104bb57806350dc4656146104f857806355f804b3146105215780635e5f3ce41461054a5761022f565b80633ab1a494146103d35780633ccfd60b146103fc5780633f3e4c111461041357806342842e0e1461043c578063453c2310146104655761022f565b8063095ea7b311610203578063095ea7b3146103025780630964617e1461032b57806318160ddd1461035457806323b872dd1461037f5780632ab4d052146103a85761022f565b8062d759191461023457806301ffc9a71461025d57806306fdde031461029a578063081812fc146102c5575b600080fd5b34801561024057600080fd5b5061025b60048036038101906102569190612a68565b6108d4565b005b34801561026957600080fd5b50610284600480360381019061027f91906129c5565b6108e6565b6040516102919190612e0f565b60405180910390f35b3480156102a657600080fd5b506102af610978565b6040516102bc9190612e2a565b60405180910390f35b3480156102d157600080fd5b506102ec60048036038101906102e79190612a68565b610a0a565b6040516102f99190612da8565b60405180910390f35b34801561030e57600080fd5b506103296004803603810190610324919061290f565b610a86565b005b34801561033757600080fd5b50610352600480360381019061034d9190612a68565b610bc7565b005b34801561036057600080fd5b50610369610bd9565b6040516103769190612f8c565b60405180910390f35b34801561038b57600080fd5b506103a660048036038101906103a191906127f9565b610bf0565b005b3480156103b457600080fd5b506103bd610f15565b6040516103ca9190612f8c565b60405180910390f35b3480156103df57600080fd5b506103fa60048036038101906103f5919061278c565b610f1b565b005b34801561040857600080fd5b50610411610f67565b005b34801561041f57600080fd5b5061043a60048036038101906104359190612a68565b61106c565b005b34801561044857600080fd5b50610463600480360381019061045e91906127f9565b61107e565b005b34801561047157600080fd5b5061047a61109e565b6040516104879190612f8c565b60405180910390f35b34801561049c57600080fd5b506104a56110a4565b6040516104b29190612f8c565b60405180910390f35b3480156104c757600080fd5b506104e260048036038101906104dd919061278c565b6110aa565b6040516104ef9190612f8c565b60405180910390f35b34801561050457600080fd5b5061051f600480360381019061051a9190612998565b6110c2565b005b34801561052d57600080fd5b5061054860048036038101906105439190612a1f565b6110d4565b005b34801561055657600080fd5b5061055f6110f6565b60405161056c9190612e0f565b60405180910390f35b34801561058157600080fd5b5061059c60048036038101906105979190612a68565b611109565b6040516105a99190612da8565b60405180910390f35b3480156105be57600080fd5b506105c761111b565b6040516105d49190612f8c565b60405180910390f35b3480156105e957600080fd5b506105f2611121565b6040516105ff9190612e2a565b60405180910390f35b34801561061457600080fd5b5061062f600480360381019061062a919061278c565b6111af565b60405161063c9190612f8c565b60405180910390f35b34801561065157600080fd5b5061065a611268565b005b34801561066857600080fd5b50610683600480360381019061067e919061294f565b61127c565b005b34801561069157600080fd5b5061069a6112cc565b6040516106a79190612da8565b60405180910390f35b3480156106bc57600080fd5b506106c56112f6565b6040516106d29190612e2a565b60405180910390f35b3480156106e757600080fd5b506106f0611388565b005b3480156106fe57600080fd5b506107076113bc565b6040516107149190612f8c565b60405180910390f35b34801561072957600080fd5b50610744600480360381019061073f91906128cf565b6113c2565b005b34801561075257600080fd5b5061075b61153a565b6040516107689190612f8c565b60405180910390f35b34801561077d57600080fd5b506107986004803603810190610793919061284c565b611540565b005b3480156107a657600080fd5b506107c160048036038101906107bc9190612a68565b6115b3565b6040516107ce9190612e2a565b60405180910390f35b3480156107e357600080fd5b506107fe60048036038101906107f99190612a68565b611652565b005b34801561080c57600080fd5b5061082760048036038101906108229190612a68565b611664565b005b34801561083557600080fd5b50610850600480360381019061084b91906127b9565b611676565b60405161085d9190612e0f565b60405180910390f35b610880600480360381019061087b9190612a68565b61170a565b005b34801561088e57600080fd5b506108a960048036038101906108a4919061278c565b611bbb565b005b3480156108b757600080fd5b506108d260048036038101906108cd9190612a68565b611c3f565b005b6108dc611c51565b80600d8190555050565b60006301ffc9a760e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916148061094157506380ac58cd60e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b806109715750635b5e139f60e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b9050919050565b60606002805461098790613241565b80601f01602080910402602001604051908101604052809291908181526020018280546109b390613241565b8015610a005780601f106109d557610100808354040283529160200191610a00565b820191906000526020600020905b8154815290600101906020018083116109e357829003601f168201915b5050505050905090565b6000610a1582611ccf565b610a4b576040517fcf4700e400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6006600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff169050919050565b6000610a9182611109565b90508073ffffffffffffffffffffffffffffffffffffffff16610ab2611d2e565b73ffffffffffffffffffffffffffffffffffffffff1614610b1557610ade81610ad9611d2e565b611676565b610b14576040517fcfb3b94200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b5b826006600084815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550818373ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff167f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92560405160405180910390a4505050565b610bcf611c51565b80600e8190555050565b6000610be3611d36565b6001546000540303905090565b6000610bfb82611d3b565b90508373ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff1614610c62576040517fa114810000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600080610c6e84611e09565b91509150610c848187610c7f611d2e565b611e2b565b610cd057610c9986610c94611d2e565b611676565b610ccf576040517f59c896be00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b5b600073ffffffffffffffffffffffffffffffffffffffff168573ffffffffffffffffffffffffffffffffffffffff161415610d37576040517fea553b3400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b610d448686866001611e6f565b8015610d4f57600082555b600560008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600081546001900391905081905550600560008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000815460010191905081905550610e1d85610df9888887611e75565b7c020000000000000000000000000000000000000000000000000000000017611e9d565b600460008681526020019081526020016000208190555060007c020000000000000000000000000000000000000000000000000000000084161415610ea5576000600185019050600060046000838152602001908152602001600020541415610ea3576000548114610ea2578360046000838152602001908152602001600020819055505b5b505b838573ffffffffffffffffffffffffffffffffffffffff168773ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4610f0d8686866001611ec8565b505050505050565b600c5481565b610f23611c51565b80601460006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555050565b610f6f611c51565b600073ffffffffffffffffffffffffffffffffffffffff16601460009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff161415611001576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610ff890612e6c565b60405180910390fd5b601460009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff166108fc479081150290604051600060405180830381858888f19350505050158015611069573d6000803e3d6000fd5b50565b611074611c51565b80600c8190555050565b61109983838360405180602001604052806000815250611540565b505050565b600b5481565b600a5481565b60136020528060005260406000206000915090505481565b6110ca611c51565b8060118190555050565b6110dc611c51565b80601290805190602001906110f29291906124ed565b5050565b600f60009054906101000a900460ff1681565b600061111482611d3b565b9050919050565b60105481565b6012805461112e90613241565b80601f016020809104026020016040519081016040528092919081815260200182805461115a90613241565b80156111a75780601f1061117c576101008083540402835291602001916111a7565b820191906000526020600020905b81548152906001019060200180831161118a57829003601f168201915b505050505081565b60008073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415611217576040517f8f4eb60400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b67ffffffffffffffff600560008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054169050919050565b611270611c51565b61127a6000611ece565b565b611284611c51565b60005b81518110156112c8576112b58282815181106112a6576112a56133e3565b5b60200260200101516001611f94565b80806112c0906132a4565b915050611287565b5050565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b60606003805461130590613241565b80601f016020809104026020016040519081016040528092919081815260200182805461133190613241565b801561137e5780601f106113535761010080835404028352916020019161137e565b820191906000526020600020905b81548152906001019060200180831161136157829003601f168201915b5050505050905090565b611390611c51565b600f60009054906101000a900460ff1615600f60006101000a81548160ff021916908315150217905550565b600e5481565b6113ca611d2e565b73ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff16141561142f576040517fb06307db00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b806007600061143c611d2e565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060006101000a81548160ff0219169083151502179055508173ffffffffffffffffffffffffffffffffffffffff166114e9611d2e565b73ffffffffffffffffffffffffffffffffffffffff167f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c318360405161152e9190612e0f565b60405180910390a35050565b600d5481565b61154b848484610bf0565b60008373ffffffffffffffffffffffffffffffffffffffff163b146115ad5761157684848484611fb2565b6115ac576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b5b50505050565b60606115be82611ccf565b6115f4576040517fa14c4b5000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b60006115fe612112565b905060008151141561161f576040518060200160405280600081525061164a565b80611629846121a4565b60405160200161163a929190612d79565b6040516020818303038152906040525b915050919050565b61165a611c51565b80600a8190555050565b61166c611c51565b80600b8190555050565b6000600760008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff16905092915050565b60026009541415611750576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161174790612f6c565b60405180910390fd5b6002600981905550600f60009054906101000a900460ff166117a7576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161179e90612ecc565b60405180910390fd5b600081116117ea576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016117e190612eac565b60405180910390fd5b600c54816117f6610bd9565b611800919061309d565b1115611841576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161183890612e8c565b60405180910390fd5b600a54811115611886576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161187d90612f2c565b60405180910390fd5b600b5481601360006118966121fe565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020546118db919061309d565b111561191c576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161191390612f4c565b60405180910390fd5b600080600e5411801561197557506000601360006119386121fe565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054145b61197f578161198d565b60018261198c919061314d565b5b9050818110156119ad576001600e546119a6919061314d565b600e819055505b34816010546119bc91906130f3565b11156119fd576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016119f490612f0c565b60405180910390fd5b600080600d54118015611a105750600082115b8015611a205750611a1f612206565b5b611a2b576000611a3a565b60105482611a3991906130f3565b5b90506000811115611a5a5781600d54611a53919061314d565b600d819055505b611a626121fe565b73ffffffffffffffffffffffffffffffffffffffff166108fc829081150290604051600060405180830381858888f19350505050158015611aa7573d6000803e3d6000fd5b508260136000611ab56121fe565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054611afa919061309d565b60136000611b066121fe565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002081905550611b4c6112cc565b73ffffffffffffffffffffffffffffffffffffffff166108fc8234611b71919061314d565b9081150290604051600060405180830381858888f19350505050158015611b9c573d6000803e3d6000fd5b50611bae611ba86121fe565b84611f94565b5050600160098190555050565b611bc3611c51565b600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff161415611c33576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611c2a90612e4c565b60405180910390fd5b611c3c81611ece565b50565b611c47611c51565b8060108190555050565b611c596121fe565b73ffffffffffffffffffffffffffffffffffffffff16611c776112cc565b73ffffffffffffffffffffffffffffffffffffffff1614611ccd576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611cc490612eec565b60405180910390fd5b565b600081611cda611d36565b11158015611ce9575060005482105b8015611d27575060007c0100000000000000000000000000000000000000000000000000000000600460008581526020019081526020016000205416145b9050919050565b600033905090565b600090565b60008082905080611d4a611d36565b11611dd257600054811015611dd15760006004600083815260200190815260200160002054905060007c010000000000000000000000000000000000000000000000000000000082161415611dcf575b6000811415611dc5576004600083600190039350838152602001908152602001600020549050611d9a565b8092505050611e04565b505b5b6040517fdf2d9b4200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b919050565b6000806000600690508360005280602052604060002092508254915050915091565b600073ffffffffffffffffffffffffffffffffffffffff8316925073ffffffffffffffffffffffffffffffffffffffff821691508382148383141790509392505050565b50505050565b60008060e883901c905060e8611e8c868684612263565b62ffffff16901b9150509392505050565b600073ffffffffffffffffffffffffffffffffffffffff83169250814260a01b178317905092915050565b50505050565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b611fae82826040518060200160405280600081525061226c565b5050565b60008373ffffffffffffffffffffffffffffffffffffffff1663150b7a02611fd8611d2e565b8786866040518563ffffffff1660e01b8152600401611ffa9493929190612dc3565b602060405180830381600087803b15801561201457600080fd5b505af192505050801561204557506040513d601f19601f8201168201806040525081019061204291906129f2565b60015b6120bf573d8060008114612075576040519150601f19603f3d011682016040523d82523d6000602084013e61207a565b606091505b506000815114156120b7576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b805181602001fd5b63150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916817bffffffffffffffffffffffffffffffffffffffffffffffffffffffff191614915050949350505050565b60606012805461212190613241565b80601f016020809104026020016040519081016040528092919081815260200182805461214d90613241565b801561219a5780601f1061216f5761010080835404028352916020019161219a565b820191906000526020600020905b81548152906001019060200180831161217d57829003601f168201915b5050505050905090565b60606080604051019050806040528082600183039250600a81066030018353600a810490505b80156121ea57600183039250600a81066030018353600a810490506121ca565b508181036020830392508083525050919050565b600033905090565b600080600261ffff3260014361221c919061314d565b40426122266121fe565b6040516020016122399493929190612d2b565b6040516020818303038152906040528051906020012060001c1661225d9190613325565b14905090565b60009392505050565b6122768383612309565b60008373ffffffffffffffffffffffffffffffffffffffff163b1461230457600080549050600083820390505b6122b66000868380600101945086611fb2565b6122ec576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8181106122a357816000541461230157600080fd5b50505b505050565b600080549050600073ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff161415612376576040517f2e07630000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b60008214156123b1576040517fb562e8dd00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6123be6000848385611e6f565b600160406001901b178202600560008573ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282540192505081905550612435836124266000866000611e75565b61242f856124dd565b17611e9d565b60046000838152602001908152602001600020819055506000819050600083830190505b818060010192508573ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4808210612459578060008190555050506124d86000848385611ec8565b505050565b60006001821460e11b9050919050565b8280546124f990613241565b90600052602060002090601f01602090048101928261251b5760008555612562565b82601f1061253457805160ff1916838001178555612562565b82800160010185558215612562579182015b82811115612561578251825591602001919060010190612546565b5b50905061256f9190612573565b5090565b5b8082111561258c576000816000905550600101612574565b5090565b60006125a361259e84612fcc565b612fa7565b905080838252602082019050828560208602820111156125c6576125c5613446565b5b60005b858110156125f657816125dc8882612684565b8452602084019350602083019250506001810190506125c9565b5050509392505050565b600061261361260e84612ff8565b612fa7565b90508281526020810184848401111561262f5761262e61344b565b5b61263a8482856131ff565b509392505050565b600061265561265084613029565b612fa7565b9050828152602081018484840111156126715761267061344b565b5b61267c8482856131ff565b509392505050565b60008135905061269381613687565b92915050565b600082601f8301126126ae576126ad613441565b5b81356126be848260208601612590565b91505092915050565b6000813590506126d68161369e565b92915050565b6000813590506126eb816136b5565b92915050565b600081359050612700816136cc565b92915050565b600081519050612715816136cc565b92915050565b600082601f8301126127305761272f613441565b5b8135612740848260208601612600565b91505092915050565b600082601f83011261275e5761275d613441565b5b813561276e848260208601612642565b91505092915050565b600081359050612786816136e3565b92915050565b6000602082840312156127a2576127a1613455565b5b60006127b084828501612684565b91505092915050565b600080604083850312156127d0576127cf613455565b5b60006127de85828601612684565b92505060206127ef85828601612684565b9150509250929050565b60008060006060848603121561281257612811613455565b5b600061282086828701612684565b935050602061283186828701612684565b925050604061284286828701612777565b9150509250925092565b6000806000806080858703121561286657612865613455565b5b600061287487828801612684565b945050602061288587828801612684565b935050604061289687828801612777565b925050606085013567ffffffffffffffff8111156128b7576128b6613450565b5b6128c38782880161271b565b91505092959194509250565b600080604083850312156128e6576128e5613455565b5b60006128f485828601612684565b9250506020612905858286016126c7565b9150509250929050565b6000806040838503121561292657612925613455565b5b600061293485828601612684565b925050602061294585828601612777565b9150509250929050565b60006020828403121561296557612964613455565b5b600082013567ffffffffffffffff81111561298357612982613450565b5b61298f84828501612699565b91505092915050565b6000602082840312156129ae576129ad613455565b5b60006129bc848285016126dc565b91505092915050565b6000602082840312156129db576129da613455565b5b60006129e9848285016126f1565b91505092915050565b600060208284031215612a0857612a07613455565b5b6000612a1684828501612706565b91505092915050565b600060208284031215612a3557612a34613455565b5b600082013567ffffffffffffffff811115612a5357612a52613450565b5b612a5f84828501612749565b91505092915050565b600060208284031215612a7e57612a7d613455565b5b6000612a8c84828501612777565b91505092915050565b612a9e81613181565b82525050565b612ab5612ab082613181565b6132ed565b82525050565b612ac481613193565b82525050565b612adb612ad68261319f565b6132ff565b82525050565b6000612aec8261305a565b612af68185613070565b9350612b0681856020860161320e565b612b0f8161345a565b840191505092915050565b6000612b2582613065565b612b2f8185613081565b9350612b3f81856020860161320e565b612b488161345a565b840191505092915050565b6000612b5e82613065565b612b688185613092565b9350612b7881856020860161320e565b80840191505092915050565b6000612b91602683613081565b9150612b9c82613478565b604082019050919050565b6000612bb4601383613081565b9150612bbf826134c7565b602082019050919050565b6000612bd7601483613081565b9150612be2826134f0565b602082019050919050565b6000612bfa601a83613081565b9150612c0582613519565b602082019050919050565b6000612c1d600d83613081565b9150612c2882613542565b602082019050919050565b6000612c40600583613092565b9150612c4b8261356b565b600582019050919050565b6000612c63602083613081565b9150612c6e82613594565b602082019050919050565b6000612c86602783613081565b9150612c91826135bd565b604082019050919050565b6000612ca9601b83613081565b9150612cb48261360c565b602082019050919050565b6000612ccc601683613081565b9150612cd782613635565b602082019050919050565b6000612cef601f83613081565b9150612cfa8261365e565b602082019050919050565b612d0e816131f5565b82525050565b612d25612d20826131f5565b61331b565b82525050565b6000612d378287612aa4565b601482019150612d478286612aca565b602082019150612d578285612d14565b602082019150612d678284612aa4565b60148201915081905095945050505050565b6000612d858285612b53565b9150612d918284612b53565b9150612d9c82612c33565b91508190509392505050565b6000602082019050612dbd6000830184612a95565b92915050565b6000608082019050612dd86000830187612a95565b612de56020830186612a95565b612df26040830185612d05565b8181036060830152612e048184612ae1565b905095945050505050565b6000602082019050612e246000830184612abb565b92915050565b60006020820190508181036000830152612e448184612b1a565b905092915050565b60006020820190508181036000830152612e6581612b84565b9050919050565b60006020820190508181036000830152612e8581612ba7565b9050919050565b60006020820190508181036000830152612ea581612bca565b9050919050565b60006020820190508181036000830152612ec581612bed565b9050919050565b60006020820190508181036000830152612ee581612c10565b9050919050565b60006020820190508181036000830152612f0581612c56565b9050919050565b60006020820190508181036000830152612f2581612c79565b9050919050565b60006020820190508181036000830152612f4581612c9c565b9050919050565b60006020820190508181036000830152612f6581612cbf565b9050919050565b60006020820190508181036000830152612f8581612ce2565b9050919050565b6000602082019050612fa16000830184612d05565b92915050565b6000612fb1612fc2565b9050612fbd8282613273565b919050565b6000604051905090565b600067ffffffffffffffff821115612fe757612fe6613412565b5b602082029050602081019050919050565b600067ffffffffffffffff82111561301357613012613412565b5b61301c8261345a565b9050602081019050919050565b600067ffffffffffffffff82111561304457613043613412565b5b61304d8261345a565b9050602081019050919050565b600081519050919050565b600081519050919050565b600082825260208201905092915050565b600082825260208201905092915050565b600081905092915050565b60006130a8826131f5565b91506130b3836131f5565b9250827fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff038211156130e8576130e7613356565b5b828201905092915050565b60006130fe826131f5565b9150613109836131f5565b9250817fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff048311821515161561314257613141613356565b5b828202905092915050565b6000613158826131f5565b9150613163836131f5565b92508282101561317657613175613356565b5b828203905092915050565b600061318c826131d5565b9050919050565b60008115159050919050565b6000819050919050565b60007fffffffff0000000000000000000000000000000000000000000000000000000082169050919050565b600073ffffffffffffffffffffffffffffffffffffffff82169050919050565b6000819050919050565b82818337600083830152505050565b60005b8381101561322c578082015181840152602081019050613211565b8381111561323b576000848401525b50505050565b6000600282049050600182168061325957607f821691505b6020821081141561326d5761326c6133b4565b5b50919050565b61327c8261345a565b810181811067ffffffffffffffff8211171561329b5761329a613412565b5b80604052505050565b60006132af826131f5565b91507fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff8214156132e2576132e1613356565b5b600182019050919050565b60006132f882613309565b9050919050565b6000819050919050565b60006133148261346b565b9050919050565b6000819050919050565b6000613330826131f5565b915061333b836131f5565b92508261334b5761334a613385565b5b828206905092915050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b600080fd5b600080fd5b600080fd5b600080fd5b600080fd5b6000601f19601f8301169050919050565b60008160601b9050919050565b7f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160008201527f6464726573730000000000000000000000000000000000000000000000000000602082015250565b7f4e6f207769746864726177206164647265737300000000000000000000000000600082015250565b7f4578636565647320746f74616c20737570706c79000000000000000000000000600082015250565b7f596f75206d757374206d696e74206174206c65617374206f6e65000000000000600082015250565b7f53616c65206e6f74206c69766500000000000000000000000000000000000000600082015250565b7f2e6a736f6e000000000000000000000000000000000000000000000000000000600082015250565b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b7f4e6f7420656e6f756768204554482073656e7420666f722073656c656374656460008201527f20616d6f756e7400000000000000000000000000000000000000000000000000602082015250565b7f45786365656473206d617820706572207472616e73616374696f6e0000000000600082015250565b7f45786365656473206d6178207065722077616c6c657400000000000000000000600082015250565b7f5265656e7472616e637947756172643a207265656e7472616e742063616c6c00600082015250565b61369081613181565b811461369b57600080fd5b50565b6136a781613193565b81146136b257600080fd5b50565b6136be8161319f565b81146136c957600080fd5b50565b6136d5816131a9565b81146136e057600080fd5b50565b6136ec816131f5565b81146136f757600080fd5b5056fea26469706673582212200f945f0933d4034fec5e31f4bc52cfc69eac34357e2c3040e07ff0f9bd8f8a4a64736f6c63430008070033

Deployed Bytecode

0x60806040526004361061022f5760003560e01c80636352211e1161012e578063a22cb465116100ab578063e268e4d31161006f578063e268e4d314610800578063e985e9c514610829578063efd0cbf914610866578063f2fde38b14610882578063f4a0a528146108ab5761022f565b8063a22cb4651461071d578063a5ce1b4d14610746578063b88d4fde14610771578063c87b56dd1461079a578063ccfdd2f8146107d75761022f565b80637ba5b5fb116100f25780637ba5b5fb1461065c5780638da5cb5b1461068557806395d89b41146106b0578063a10866ef146106db578063a1165f5d146106f25761022f565b80636352211e146105755780636817c76c146105b25780636c0360eb146105dd57806370a0823114610608578063715018a6146106455761022f565b80633ab1a494116101bc5780634b980d67116101805780634b980d67146104905780634d0df5fc146104bb57806350dc4656146104f857806355f804b3146105215780635e5f3ce41461054a5761022f565b80633ab1a494146103d35780633ccfd60b146103fc5780633f3e4c111461041357806342842e0e1461043c578063453c2310146104655761022f565b8063095ea7b311610203578063095ea7b3146103025780630964617e1461032b57806318160ddd1461035457806323b872dd1461037f5780632ab4d052146103a85761022f565b8062d759191461023457806301ffc9a71461025d57806306fdde031461029a578063081812fc146102c5575b600080fd5b34801561024057600080fd5b5061025b60048036038101906102569190612a68565b6108d4565b005b34801561026957600080fd5b50610284600480360381019061027f91906129c5565b6108e6565b6040516102919190612e0f565b60405180910390f35b3480156102a657600080fd5b506102af610978565b6040516102bc9190612e2a565b60405180910390f35b3480156102d157600080fd5b506102ec60048036038101906102e79190612a68565b610a0a565b6040516102f99190612da8565b60405180910390f35b34801561030e57600080fd5b506103296004803603810190610324919061290f565b610a86565b005b34801561033757600080fd5b50610352600480360381019061034d9190612a68565b610bc7565b005b34801561036057600080fd5b50610369610bd9565b6040516103769190612f8c565b60405180910390f35b34801561038b57600080fd5b506103a660048036038101906103a191906127f9565b610bf0565b005b3480156103b457600080fd5b506103bd610f15565b6040516103ca9190612f8c565b60405180910390f35b3480156103df57600080fd5b506103fa60048036038101906103f5919061278c565b610f1b565b005b34801561040857600080fd5b50610411610f67565b005b34801561041f57600080fd5b5061043a60048036038101906104359190612a68565b61106c565b005b34801561044857600080fd5b50610463600480360381019061045e91906127f9565b61107e565b005b34801561047157600080fd5b5061047a61109e565b6040516104879190612f8c565b60405180910390f35b34801561049c57600080fd5b506104a56110a4565b6040516104b29190612f8c565b60405180910390f35b3480156104c757600080fd5b506104e260048036038101906104dd919061278c565b6110aa565b6040516104ef9190612f8c565b60405180910390f35b34801561050457600080fd5b5061051f600480360381019061051a9190612998565b6110c2565b005b34801561052d57600080fd5b5061054860048036038101906105439190612a1f565b6110d4565b005b34801561055657600080fd5b5061055f6110f6565b60405161056c9190612e0f565b60405180910390f35b34801561058157600080fd5b5061059c60048036038101906105979190612a68565b611109565b6040516105a99190612da8565b60405180910390f35b3480156105be57600080fd5b506105c761111b565b6040516105d49190612f8c565b60405180910390f35b3480156105e957600080fd5b506105f2611121565b6040516105ff9190612e2a565b60405180910390f35b34801561061457600080fd5b5061062f600480360381019061062a919061278c565b6111af565b60405161063c9190612f8c565b60405180910390f35b34801561065157600080fd5b5061065a611268565b005b34801561066857600080fd5b50610683600480360381019061067e919061294f565b61127c565b005b34801561069157600080fd5b5061069a6112cc565b6040516106a79190612da8565b60405180910390f35b3480156106bc57600080fd5b506106c56112f6565b6040516106d29190612e2a565b60405180910390f35b3480156106e757600080fd5b506106f0611388565b005b3480156106fe57600080fd5b506107076113bc565b6040516107149190612f8c565b60405180910390f35b34801561072957600080fd5b50610744600480360381019061073f91906128cf565b6113c2565b005b34801561075257600080fd5b5061075b61153a565b6040516107689190612f8c565b60405180910390f35b34801561077d57600080fd5b506107986004803603810190610793919061284c565b611540565b005b3480156107a657600080fd5b506107c160048036038101906107bc9190612a68565b6115b3565b6040516107ce9190612e2a565b60405180910390f35b3480156107e357600080fd5b506107fe60048036038101906107f99190612a68565b611652565b005b34801561080c57600080fd5b5061082760048036038101906108229190612a68565b611664565b005b34801561083557600080fd5b50610850600480360381019061084b91906127b9565b611676565b60405161085d9190612e0f565b60405180910390f35b610880600480360381019061087b9190612a68565b61170a565b005b34801561088e57600080fd5b506108a960048036038101906108a4919061278c565b611bbb565b005b3480156108b757600080fd5b506108d260048036038101906108cd9190612a68565b611c3f565b005b6108dc611c51565b80600d8190555050565b60006301ffc9a760e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916148061094157506380ac58cd60e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b806109715750635b5e139f60e01b827bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916145b9050919050565b60606002805461098790613241565b80601f01602080910402602001604051908101604052809291908181526020018280546109b390613241565b8015610a005780601f106109d557610100808354040283529160200191610a00565b820191906000526020600020905b8154815290600101906020018083116109e357829003601f168201915b5050505050905090565b6000610a1582611ccf565b610a4b576040517fcf4700e400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6006600083815260200190815260200160002060009054906101000a900473ffffffffffffffffffffffffffffffffffffffff169050919050565b6000610a9182611109565b90508073ffffffffffffffffffffffffffffffffffffffff16610ab2611d2e565b73ffffffffffffffffffffffffffffffffffffffff1614610b1557610ade81610ad9611d2e565b611676565b610b14576040517fcfb3b94200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b5b826006600084815260200190815260200160002060006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff160217905550818373ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff167f8c5be1e5ebec7d5bd14f71427d1e84f3dd0314c0f7b2291e5b200ac8c7c3b92560405160405180910390a4505050565b610bcf611c51565b80600e8190555050565b6000610be3611d36565b6001546000540303905090565b6000610bfb82611d3b565b90508373ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff1614610c62576040517fa114810000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b600080610c6e84611e09565b91509150610c848187610c7f611d2e565b611e2b565b610cd057610c9986610c94611d2e565b611676565b610ccf576040517f59c896be00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b5b600073ffffffffffffffffffffffffffffffffffffffff168573ffffffffffffffffffffffffffffffffffffffff161415610d37576040517fea553b3400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b610d448686866001611e6f565b8015610d4f57600082555b600560008773ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020600081546001900391905081905550600560008673ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff1681526020019081526020016000206000815460010191905081905550610e1d85610df9888887611e75565b7c020000000000000000000000000000000000000000000000000000000017611e9d565b600460008681526020019081526020016000208190555060007c020000000000000000000000000000000000000000000000000000000084161415610ea5576000600185019050600060046000838152602001908152602001600020541415610ea3576000548114610ea2578360046000838152602001908152602001600020819055505b5b505b838573ffffffffffffffffffffffffffffffffffffffff168773ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4610f0d8686866001611ec8565b505050505050565b600c5481565b610f23611c51565b80601460006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff16021790555050565b610f6f611c51565b600073ffffffffffffffffffffffffffffffffffffffff16601460009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff161415611001576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401610ff890612e6c565b60405180910390fd5b601460009054906101000a900473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff166108fc479081150290604051600060405180830381858888f19350505050158015611069573d6000803e3d6000fd5b50565b611074611c51565b80600c8190555050565b61109983838360405180602001604052806000815250611540565b505050565b600b5481565b600a5481565b60136020528060005260406000206000915090505481565b6110ca611c51565b8060118190555050565b6110dc611c51565b80601290805190602001906110f29291906124ed565b5050565b600f60009054906101000a900460ff1681565b600061111482611d3b565b9050919050565b60105481565b6012805461112e90613241565b80601f016020809104026020016040519081016040528092919081815260200182805461115a90613241565b80156111a75780601f1061117c576101008083540402835291602001916111a7565b820191906000526020600020905b81548152906001019060200180831161118a57829003601f168201915b505050505081565b60008073ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff161415611217576040517f8f4eb60400000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b67ffffffffffffffff600560008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054169050919050565b611270611c51565b61127a6000611ece565b565b611284611c51565b60005b81518110156112c8576112b58282815181106112a6576112a56133e3565b5b60200260200101516001611f94565b80806112c0906132a4565b915050611287565b5050565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905090565b60606003805461130590613241565b80601f016020809104026020016040519081016040528092919081815260200182805461133190613241565b801561137e5780601f106113535761010080835404028352916020019161137e565b820191906000526020600020905b81548152906001019060200180831161136157829003601f168201915b5050505050905090565b611390611c51565b600f60009054906101000a900460ff1615600f60006101000a81548160ff021916908315150217905550565b600e5481565b6113ca611d2e565b73ffffffffffffffffffffffffffffffffffffffff168273ffffffffffffffffffffffffffffffffffffffff16141561142f576040517fb06307db00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b806007600061143c611d2e565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060006101000a81548160ff0219169083151502179055508173ffffffffffffffffffffffffffffffffffffffff166114e9611d2e565b73ffffffffffffffffffffffffffffffffffffffff167f17307eab39ab6107e8899845ad3d59bd9653f200f220920489ca2b5937696c318360405161152e9190612e0f565b60405180910390a35050565b600d5481565b61154b848484610bf0565b60008373ffffffffffffffffffffffffffffffffffffffff163b146115ad5761157684848484611fb2565b6115ac576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b5b50505050565b60606115be82611ccf565b6115f4576040517fa14c4b5000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b60006115fe612112565b905060008151141561161f576040518060200160405280600081525061164a565b80611629846121a4565b60405160200161163a929190612d79565b6040516020818303038152906040525b915050919050565b61165a611c51565b80600a8190555050565b61166c611c51565b80600b8190555050565b6000600760008473ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008373ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060009054906101000a900460ff16905092915050565b60026009541415611750576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161174790612f6c565b60405180910390fd5b6002600981905550600f60009054906101000a900460ff166117a7576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161179e90612ecc565b60405180910390fd5b600081116117ea576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016117e190612eac565b60405180910390fd5b600c54816117f6610bd9565b611800919061309d565b1115611841576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161183890612e8c565b60405180910390fd5b600a54811115611886576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161187d90612f2c565b60405180910390fd5b600b5481601360006118966121fe565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff168152602001908152602001600020546118db919061309d565b111561191c576040517f08c379a000000000000000000000000000000000000000000000000000000000815260040161191390612f4c565b60405180910390fd5b600080600e5411801561197557506000601360006119386121fe565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054145b61197f578161198d565b60018261198c919061314d565b5b9050818110156119ad576001600e546119a6919061314d565b600e819055505b34816010546119bc91906130f3565b11156119fd576040517f08c379a00000000000000000000000000000000000000000000000000000000081526004016119f490612f0c565b60405180910390fd5b600080600d54118015611a105750600082115b8015611a205750611a1f612206565b5b611a2b576000611a3a565b60105482611a3991906130f3565b5b90506000811115611a5a5781600d54611a53919061314d565b600d819055505b611a626121fe565b73ffffffffffffffffffffffffffffffffffffffff166108fc829081150290604051600060405180830381858888f19350505050158015611aa7573d6000803e3d6000fd5b508260136000611ab56121fe565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002054611afa919061309d565b60136000611b066121fe565b73ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002081905550611b4c6112cc565b73ffffffffffffffffffffffffffffffffffffffff166108fc8234611b71919061314d565b9081150290604051600060405180830381858888f19350505050158015611b9c573d6000803e3d6000fd5b50611bae611ba86121fe565b84611f94565b5050600160098190555050565b611bc3611c51565b600073ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff161415611c33576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611c2a90612e4c565b60405180910390fd5b611c3c81611ece565b50565b611c47611c51565b8060108190555050565b611c596121fe565b73ffffffffffffffffffffffffffffffffffffffff16611c776112cc565b73ffffffffffffffffffffffffffffffffffffffff1614611ccd576040517f08c379a0000000000000000000000000000000000000000000000000000000008152600401611cc490612eec565b60405180910390fd5b565b600081611cda611d36565b11158015611ce9575060005482105b8015611d27575060007c0100000000000000000000000000000000000000000000000000000000600460008581526020019081526020016000205416145b9050919050565b600033905090565b600090565b60008082905080611d4a611d36565b11611dd257600054811015611dd15760006004600083815260200190815260200160002054905060007c010000000000000000000000000000000000000000000000000000000082161415611dcf575b6000811415611dc5576004600083600190039350838152602001908152602001600020549050611d9a565b8092505050611e04565b505b5b6040517fdf2d9b4200000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b919050565b6000806000600690508360005280602052604060002092508254915050915091565b600073ffffffffffffffffffffffffffffffffffffffff8316925073ffffffffffffffffffffffffffffffffffffffff821691508382148383141790509392505050565b50505050565b60008060e883901c905060e8611e8c868684612263565b62ffffff16901b9150509392505050565b600073ffffffffffffffffffffffffffffffffffffffff83169250814260a01b178317905092915050565b50505050565b6000600860009054906101000a900473ffffffffffffffffffffffffffffffffffffffff16905081600860006101000a81548173ffffffffffffffffffffffffffffffffffffffff021916908373ffffffffffffffffffffffffffffffffffffffff1602179055508173ffffffffffffffffffffffffffffffffffffffff168173ffffffffffffffffffffffffffffffffffffffff167f8be0079c531659141344cd1fd0a4f28419497f9722a3daafe3b4186f6b6457e060405160405180910390a35050565b611fae82826040518060200160405280600081525061226c565b5050565b60008373ffffffffffffffffffffffffffffffffffffffff1663150b7a02611fd8611d2e565b8786866040518563ffffffff1660e01b8152600401611ffa9493929190612dc3565b602060405180830381600087803b15801561201457600080fd5b505af192505050801561204557506040513d601f19601f8201168201806040525081019061204291906129f2565b60015b6120bf573d8060008114612075576040519150601f19603f3d011682016040523d82523d6000602084013e61207a565b606091505b506000815114156120b7576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b805181602001fd5b63150b7a0260e01b7bffffffffffffffffffffffffffffffffffffffffffffffffffffffff1916817bffffffffffffffffffffffffffffffffffffffffffffffffffffffff191614915050949350505050565b60606012805461212190613241565b80601f016020809104026020016040519081016040528092919081815260200182805461214d90613241565b801561219a5780601f1061216f5761010080835404028352916020019161219a565b820191906000526020600020905b81548152906001019060200180831161217d57829003601f168201915b5050505050905090565b60606080604051019050806040528082600183039250600a81066030018353600a810490505b80156121ea57600183039250600a81066030018353600a810490506121ca565b508181036020830392508083525050919050565b600033905090565b600080600261ffff3260014361221c919061314d565b40426122266121fe565b6040516020016122399493929190612d2b565b6040516020818303038152906040528051906020012060001c1661225d9190613325565b14905090565b60009392505050565b6122768383612309565b60008373ffffffffffffffffffffffffffffffffffffffff163b1461230457600080549050600083820390505b6122b66000868380600101945086611fb2565b6122ec576040517fd1a57ed600000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b8181106122a357816000541461230157600080fd5b50505b505050565b600080549050600073ffffffffffffffffffffffffffffffffffffffff168373ffffffffffffffffffffffffffffffffffffffff161415612376576040517f2e07630000000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b60008214156123b1576040517fb562e8dd00000000000000000000000000000000000000000000000000000000815260040160405180910390fd5b6123be6000848385611e6f565b600160406001901b178202600560008573ffffffffffffffffffffffffffffffffffffffff1673ffffffffffffffffffffffffffffffffffffffff16815260200190815260200160002060008282540192505081905550612435836124266000866000611e75565b61242f856124dd565b17611e9d565b60046000838152602001908152602001600020819055506000819050600083830190505b818060010192508573ffffffffffffffffffffffffffffffffffffffff16600073ffffffffffffffffffffffffffffffffffffffff167fddf252ad1be2c89b69c2b068fc378daa952ba7f163c4a11628f55a4df523b3ef60405160405180910390a4808210612459578060008190555050506124d86000848385611ec8565b505050565b60006001821460e11b9050919050565b8280546124f990613241565b90600052602060002090601f01602090048101928261251b5760008555612562565b82601f1061253457805160ff1916838001178555612562565b82800160010185558215612562579182015b82811115612561578251825591602001919060010190612546565b5b50905061256f9190612573565b5090565b5b8082111561258c576000816000905550600101612574565b5090565b60006125a361259e84612fcc565b612fa7565b905080838252602082019050828560208602820111156125c6576125c5613446565b5b60005b858110156125f657816125dc8882612684565b8452602084019350602083019250506001810190506125c9565b5050509392505050565b600061261361260e84612ff8565b612fa7565b90508281526020810184848401111561262f5761262e61344b565b5b61263a8482856131ff565b509392505050565b600061265561265084613029565b612fa7565b9050828152602081018484840111156126715761267061344b565b5b61267c8482856131ff565b509392505050565b60008135905061269381613687565b92915050565b600082601f8301126126ae576126ad613441565b5b81356126be848260208601612590565b91505092915050565b6000813590506126d68161369e565b92915050565b6000813590506126eb816136b5565b92915050565b600081359050612700816136cc565b92915050565b600081519050612715816136cc565b92915050565b600082601f8301126127305761272f613441565b5b8135612740848260208601612600565b91505092915050565b600082601f83011261275e5761275d613441565b5b813561276e848260208601612642565b91505092915050565b600081359050612786816136e3565b92915050565b6000602082840312156127a2576127a1613455565b5b60006127b084828501612684565b91505092915050565b600080604083850312156127d0576127cf613455565b5b60006127de85828601612684565b92505060206127ef85828601612684565b9150509250929050565b60008060006060848603121561281257612811613455565b5b600061282086828701612684565b935050602061283186828701612684565b925050604061284286828701612777565b9150509250925092565b6000806000806080858703121561286657612865613455565b5b600061287487828801612684565b945050602061288587828801612684565b935050604061289687828801612777565b925050606085013567ffffffffffffffff8111156128b7576128b6613450565b5b6128c38782880161271b565b91505092959194509250565b600080604083850312156128e6576128e5613455565b5b60006128f485828601612684565b9250506020612905858286016126c7565b9150509250929050565b6000806040838503121561292657612925613455565b5b600061293485828601612684565b925050602061294585828601612777565b9150509250929050565b60006020828403121561296557612964613455565b5b600082013567ffffffffffffffff81111561298357612982613450565b5b61298f84828501612699565b91505092915050565b6000602082840312156129ae576129ad613455565b5b60006129bc848285016126dc565b91505092915050565b6000602082840312156129db576129da613455565b5b60006129e9848285016126f1565b91505092915050565b600060208284031215612a0857612a07613455565b5b6000612a1684828501612706565b91505092915050565b600060208284031215612a3557612a34613455565b5b600082013567ffffffffffffffff811115612a5357612a52613450565b5b612a5f84828501612749565b91505092915050565b600060208284031215612a7e57612a7d613455565b5b6000612a8c84828501612777565b91505092915050565b612a9e81613181565b82525050565b612ab5612ab082613181565b6132ed565b82525050565b612ac481613193565b82525050565b612adb612ad68261319f565b6132ff565b82525050565b6000612aec8261305a565b612af68185613070565b9350612b0681856020860161320e565b612b0f8161345a565b840191505092915050565b6000612b2582613065565b612b2f8185613081565b9350612b3f81856020860161320e565b612b488161345a565b840191505092915050565b6000612b5e82613065565b612b688185613092565b9350612b7881856020860161320e565b80840191505092915050565b6000612b91602683613081565b9150612b9c82613478565b604082019050919050565b6000612bb4601383613081565b9150612bbf826134c7565b602082019050919050565b6000612bd7601483613081565b9150612be2826134f0565b602082019050919050565b6000612bfa601a83613081565b9150612c0582613519565b602082019050919050565b6000612c1d600d83613081565b9150612c2882613542565b602082019050919050565b6000612c40600583613092565b9150612c4b8261356b565b600582019050919050565b6000612c63602083613081565b9150612c6e82613594565b602082019050919050565b6000612c86602783613081565b9150612c91826135bd565b604082019050919050565b6000612ca9601b83613081565b9150612cb48261360c565b602082019050919050565b6000612ccc601683613081565b9150612cd782613635565b602082019050919050565b6000612cef601f83613081565b9150612cfa8261365e565b602082019050919050565b612d0e816131f5565b82525050565b612d25612d20826131f5565b61331b565b82525050565b6000612d378287612aa4565b601482019150612d478286612aca565b602082019150612d578285612d14565b602082019150612d678284612aa4565b60148201915081905095945050505050565b6000612d858285612b53565b9150612d918284612b53565b9150612d9c82612c33565b91508190509392505050565b6000602082019050612dbd6000830184612a95565b92915050565b6000608082019050612dd86000830187612a95565b612de56020830186612a95565b612df26040830185612d05565b8181036060830152612e048184612ae1565b905095945050505050565b6000602082019050612e246000830184612abb565b92915050565b60006020820190508181036000830152612e448184612b1a565b905092915050565b60006020820190508181036000830152612e6581612b84565b9050919050565b60006020820190508181036000830152612e8581612ba7565b9050919050565b60006020820190508181036000830152612ea581612bca565b9050919050565b60006020820190508181036000830152612ec581612bed565b9050919050565b60006020820190508181036000830152612ee581612c10565b9050919050565b60006020820190508181036000830152612f0581612c56565b9050919050565b60006020820190508181036000830152612f2581612c79565b9050919050565b60006020820190508181036000830152612f4581612c9c565b9050919050565b60006020820190508181036000830152612f6581612cbf565b9050919050565b60006020820190508181036000830152612f8581612ce2565b9050919050565b6000602082019050612fa16000830184612d05565b92915050565b6000612fb1612fc2565b9050612fbd8282613273565b919050565b6000604051905090565b600067ffffffffffffffff821115612fe757612fe6613412565b5b602082029050602081019050919050565b600067ffffffffffffffff82111561301357613012613412565b5b61301c8261345a565b9050602081019050919050565b600067ffffffffffffffff82111561304457613043613412565b5b61304d8261345a565b9050602081019050919050565b600081519050919050565b600081519050919050565b600082825260208201905092915050565b600082825260208201905092915050565b600081905092915050565b60006130a8826131f5565b91506130b3836131f5565b9250827fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff038211156130e8576130e7613356565b5b828201905092915050565b60006130fe826131f5565b9150613109836131f5565b9250817fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff048311821515161561314257613141613356565b5b828202905092915050565b6000613158826131f5565b9150613163836131f5565b92508282101561317657613175613356565b5b828203905092915050565b600061318c826131d5565b9050919050565b60008115159050919050565b6000819050919050565b60007fffffffff0000000000000000000000000000000000000000000000000000000082169050919050565b600073ffffffffffffffffffffffffffffffffffffffff82169050919050565b6000819050919050565b82818337600083830152505050565b60005b8381101561322c578082015181840152602081019050613211565b8381111561323b576000848401525b50505050565b6000600282049050600182168061325957607f821691505b6020821081141561326d5761326c6133b4565b5b50919050565b61327c8261345a565b810181811067ffffffffffffffff8211171561329b5761329a613412565b5b80604052505050565b60006132af826131f5565b91507fffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffffff8214156132e2576132e1613356565b5b600182019050919050565b60006132f882613309565b9050919050565b6000819050919050565b60006133148261346b565b9050919050565b6000819050919050565b6000613330826131f5565b915061333b836131f5565b92508261334b5761334a613385565b5b828206905092915050565b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601160045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052601260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052602260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052603260045260246000fd5b7f4e487b7100000000000000000000000000000000000000000000000000000000600052604160045260246000fd5b600080fd5b600080fd5b600080fd5b600080fd5b600080fd5b6000601f19601f8301169050919050565b60008160601b9050919050565b7f4f776e61626c653a206e6577206f776e657220697320746865207a65726f206160008201527f6464726573730000000000000000000000000000000000000000000000000000602082015250565b7f4e6f207769746864726177206164647265737300000000000000000000000000600082015250565b7f4578636565647320746f74616c20737570706c79000000000000000000000000600082015250565b7f596f75206d757374206d696e74206174206c65617374206f6e65000000000000600082015250565b7f53616c65206e6f74206c69766500000000000000000000000000000000000000600082015250565b7f2e6a736f6e000000000000000000000000000000000000000000000000000000600082015250565b7f4f776e61626c653a2063616c6c6572206973206e6f7420746865206f776e6572600082015250565b7f4e6f7420656e6f756768204554482073656e7420666f722073656c656374656460008201527f20616d6f756e7400000000000000000000000000000000000000000000000000602082015250565b7f45786365656473206d617820706572207472616e73616374696f6e0000000000600082015250565b7f45786365656473206d6178207065722077616c6c657400000000000000000000600082015250565b7f5265656e7472616e637947756172643a207265656e7472616e742063616c6c00600082015250565b61369081613181565b811461369b57600080fd5b50565b6136a781613193565b81146136b257600080fd5b50565b6136be8161319f565b81146136c957600080fd5b50565b6136d5816131a9565b81146136e057600080fd5b50565b6136ec816131f5565b81146136f757600080fd5b5056fea26469706673582212200f945f0933d4034fec5e31f4bc52cfc69eac34357e2c3040e07ff0f9bd8f8a4a64736f6c63430008070033

Deployed Bytecode Sourcemap

59899:4167:0:-:0;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;62960:162;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;29700:615;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;35347:100;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;37302:204;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;36850:386;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;62814:138;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;28754:315;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;46567:2800;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;60057:36;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;63807:126;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;62510:186;;;;;;;;;;;;;:::i;:::-;;63130:122;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;38192:185;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;60016:34;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;59972:37;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;60449:49;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;63941:122;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;63524:106;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;60222:32;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;35136:144;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;60277:37;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;60404:21;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;30379:224;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;14291:103;;;;;;;;;;;;;:::i;:::-;;63638:161;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;13643:87;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;35516:104;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;62012:97;;;;;;;;;;;;;:::i;:::-;;60153:40;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;37578:308;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;60100:46;;;;;;;;;;;;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;38448:399;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;35691:327;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;63260:134;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;63402:114;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;37957:164;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;;;;;;:::i;:::-;;;;;;;;60605:1397;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;14549:201;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;62704:102;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;:::i;:::-;;62960:162;13529:13;:11;:13::i;:::-;63089:25:::1;63062:24;:52;;;;62960:162:::0;:::o;29700:615::-;29785:4;30100:10;30085:25;;:11;:25;;;;:102;;;;30177:10;30162:25;;:11;:25;;;;30085:102;:179;;;;30254:10;30239:25;;:11;:25;;;;30085:179;30065:199;;29700:615;;;:::o;35347:100::-;35401:13;35434:5;35427:12;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;35347:100;:::o;37302:204::-;37370:7;37395:16;37403:7;37395;:16::i;:::-;37390:64;;37420:34;;;;;;;;;;;;;;37390:64;37474:15;:24;37490:7;37474:24;;;;;;;;;;;;;;;;;;;;;37467:31;;37302:204;;;:::o;36850:386::-;36923:13;36939:16;36947:7;36939;:16::i;:::-;36923:32;;36995:5;36972:28;;:19;:17;:19::i;:::-;:28;;;36968:175;;37020:44;37037:5;37044:19;:17;:19::i;:::-;37020:16;:44::i;:::-;37015:128;;37092:35;;;;;;;;;;;;;;37015:128;36968:175;37182:2;37155:15;:24;37171:7;37155:24;;;;;;;;;;;;:29;;;;;;;;;;;;;;;;;;37220:7;37216:2;37200:28;;37209:5;37200:28;;;;;;;;;;;;36912:324;36850:386;;:::o;62814:138::-;13529:13;:11;:13::i;:::-;62925:19:::1;62904:18;:40;;;;62814:138:::0;:::o;28754:315::-;28807:7;29035:15;:13;:15::i;:::-;29020:12;;29004:13;;:28;:46;28997:53;;28754:315;:::o;46567:2800::-;46701:27;46731;46750:7;46731:18;:27::i;:::-;46701:57;;46816:4;46775:45;;46791:19;46775:45;;;46771:86;;46829:28;;;;;;;;;;;;;;46771:86;46871:27;46900:23;46927:28;46947:7;46927:19;:28::i;:::-;46870:85;;;;47055:62;47074:15;47091:4;47097:19;:17;:19::i;:::-;47055:18;:62::i;:::-;47050:174;;47137:43;47154:4;47160:19;:17;:19::i;:::-;47137:16;:43::i;:::-;47132:92;;47189:35;;;;;;;;;;;;;;47132:92;47050:174;47255:1;47241:16;;:2;:16;;;47237:52;;;47266:23;;;;;;;;;;;;;;47237:52;47302:43;47324:4;47330:2;47334:7;47343:1;47302:21;:43::i;:::-;47438:15;47435:160;;;47578:1;47557:19;47550:30;47435:160;47973:18;:24;47992:4;47973:24;;;;;;;;;;;;;;;;47971:26;;;;;;;;;;;;48042:18;:22;48061:2;48042:22;;;;;;;;;;;;;;;;48040:24;;;;;;;;;;;48364:145;48401:2;48449:45;48464:4;48470:2;48474:19;48449:14;:45::i;:::-;25982:8;48422:72;48364:18;:145::i;:::-;48335:17;:26;48353:7;48335:26;;;;;;;;;;;:174;;;;48679:1;25982:8;48629:19;:46;:51;48625:626;;;48701:19;48733:1;48723:7;:11;48701:33;;48890:1;48856:17;:30;48874:11;48856:30;;;;;;;;;;;;:35;48852:384;;;48994:13;;48979:11;:28;48975:242;;49174:19;49141:17;:30;49159:11;49141:30;;;;;;;;;;;:52;;;;48975:242;48852:384;48682:569;48625:626;49298:7;49294:2;49279:27;;49288:4;49279:27;;;;;;;;;;;;49317:42;49338:4;49344:2;49348:7;49357:1;49317:20;:42::i;:::-;46690:2677;;;46567:2800;;;:::o;60057:36::-;;;;:::o;63807:126::-;13529:13;:11;:13::i;:::-;63909:16:::1;63891:15;;:34;;;;;;;;;;;;;;;;;;63807:126:::0;:::o;62510:186::-;13529:13;:11;:13::i;:::-;62595:1:::1;62568:29;;:15;;;;;;;;;;;:29;;;;62560:61;;;;;;;;;;;;:::i;:::-;;;;;;;;;62640:15;;;;;;;;;;;62632:33;;:56;62666:21;62632:56;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;::::0;::::1;;;;;;62510:186::o:0;63130:122::-;13529:13;:11;:13::i;:::-;63229:15:::1;63212:14;:32;;;;63130:122:::0;:::o;38192:185::-;38330:39;38347:4;38353:2;38357:7;38330:39;;;;;;;;;;;;:16;:39::i;:::-;38192:185;;;:::o;60016:34::-;;;;:::o;59972:37::-;;;;:::o;60449:49::-;;;;;;;;;;;;;;;;;:::o;63941:122::-;13529:13;:11;:13::i;:::-;64040:15:::1;64023:14;:32;;;;63941:122:::0;:::o;63524:106::-;13529:13;:11;:13::i;:::-;63611:11:::1;63601:7;:21;;;;;;;;;;;;:::i;:::-;;63524:106:::0;:::o;60222:32::-;;;;;;;;;;;;;:::o;35136:144::-;35200:7;35243:27;35262:7;35243:18;:27::i;:::-;35220:52;;35136:144;;;:::o;60277:37::-;;;;:::o;60404:21::-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::o;30379:224::-;30443:7;30484:1;30467:19;;:5;:19;;;30463:60;;;30495:28;;;;;;;;;;;;;;30463:60;24934:13;30541:18;:25;30560:5;30541:25;;;;;;;;;;;;;;;;:54;30534:61;;30379:224;;;:::o;14291:103::-;13529:13;:11;:13::i;:::-;14356:30:::1;14383:1;14356:18;:30::i;:::-;14291:103::o:0;63638:161::-;13529:13;:11;:13::i;:::-;63715:6:::1;63710:82;63731:2;:9;63727:1;:13;63710:82;;;63761:19;63771:2;63774:1;63771:5;;;;;;;;:::i;:::-;;;;;;;;63778:1;63761:9;:19::i;:::-;63741:3;;;;;:::i;:::-;;;;63710:82;;;;63638:161:::0;:::o;13643:87::-;13689:7;13716:6;;;;;;;;;;;13709:13;;13643:87;:::o;35516:104::-;35572:13;35605:7;35598:14;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;35516:104;:::o;62012:97::-;13529:13;:11;:13::i;:::-;62089:12:::1;;;;;;;;;;;62088:13;62073:12;;:28;;;;;;;;;;;;;;;;;;62012:97::o:0;60153:40::-;;;;:::o;37578:308::-;37689:19;:17;:19::i;:::-;37677:31;;:8;:31;;;37673:61;;;37717:17;;;;;;;;;;;;;;37673:61;37799:8;37747:18;:39;37766:19;:17;:19::i;:::-;37747:39;;;;;;;;;;;;;;;:49;37787:8;37747:49;;;;;;;;;;;;;;;;:60;;;;;;;;;;;;;;;;;;37859:8;37823:55;;37838:19;:17;:19::i;:::-;37823:55;;;37869:8;37823:55;;;;;;:::i;:::-;;;;;;;;37578:308;;:::o;60100:46::-;;;;:::o;38448:399::-;38615:31;38628:4;38634:2;38638:7;38615:12;:31::i;:::-;38679:1;38661:2;:14;;;:19;38657:183;;38700:56;38731:4;38737:2;38741:7;38750:5;38700:30;:56::i;:::-;38695:145;;38784:40;;;;;;;;;;;;;;38695:145;38657:183;38448:399;;;;:::o;35691:327::-;35764:13;35795:16;35803:7;35795;:16::i;:::-;35790:59;;35820:29;;;;;;;;;;;;;;35790:59;35862:21;35886:10;:8;:10::i;:::-;35862:34;;35939:1;35920:7;35914:21;:26;;:96;;;;;;;;;;;;;;;;;35967:7;35976:18;35986:7;35976:9;:18::i;:::-;35950:54;;;;;;;;;:::i;:::-;;;;;;;;;;;;;35914:96;35907:103;;;35691:327;;;:::o;63260:134::-;13529:13;:11;:13::i;:::-;63368:18:::1;63348:17;:38;;;;63260:134:::0;:::o;63402:114::-;13529:13;:11;:13::i;:::-;63495::::1;63480:12;:28;;;;63402:114:::0;:::o;37957:164::-;38054:4;38078:18;:25;38097:5;38078:25;;;;;;;;;;;;;;;:35;38104:8;38078:35;;;;;;;;;;;;;;;;;;;;;;;;;38071:42;;37957:164;;;;:::o;60605:1397::-;10568:1;11166:7;;:19;;11158:63;;;;;;;;;;;;:::i;:::-;;;;;;;;;10568:1;11299:7;:18;;;;60691:12:::1;;;;;;;;;;;60683:38;;;;;;;;;;;;:::i;:::-;;;;;;;;;60750:1;60740:7;:11;60732:50;;;;;;;;;;;;:::i;:::-;;;;;;;;;60828:14;;60817:7;60801:13;:11;:13::i;:::-;:23;;;;:::i;:::-;:41;;60793:74;;;;;;;;;;;;:::i;:::-;;;;;;;;;60897:17;;60886:7;:28;;60878:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;61007:12;;60996:7;60965:14;:28;60980:12;:10;:12::i;:::-;60965:28;;;;;;;;;;;;;;;;:38;;;;:::i;:::-;:54;;60957:89;;;;;;;;;;;;:::i;:::-;;;;;;;;;61100:20;61144:1:::0;61123:18:::1;;:22;:59;;;;;61181:1;61149:14;:28;61164:12;:10;:12::i;:::-;61149:28;;;;;;;;;;;;;;;;:33;61123:59;:109;;61225:7;61123:109;;;61208:1;61198:7;:11;;;;:::i;:::-;61123:109;61100:132;;61264:7;61249:12;:22;61245:98;;;61330:1;61309:18;;:22;;;;:::i;:::-;61288:18;:43;;;;61245:98;61391:9;61375:12;61363:9;;:24;;;;:::i;:::-;:37;;61355:89;;;;;;;;;;;;:::i;:::-;;;;;;;;;61457:14;61501:1:::0;61474:24:::1;;:28;:48;;;;;61521:1;61506:12;:16;61474:48;:64;;;;;61526:12;:10;:12::i;:::-;61474:64;:121;;61594:1;61474:121;;;61569:9;;61554:12;:24;;;;:::i;:::-;61474:121;61457:138;;61621:1;61612:6;:10;61608:109;;;61693:12;61666:24;;:39;;;;:::i;:::-;61639:24;:66;;;;61608:109;61781:12;:10;:12::i;:::-;61773:30;;:38;61804:6;61773:38;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;::::0;::::1;;;;;;61886:7;61855:14;:28;61870:12;:10;:12::i;:::-;61855:28;;;;;;;;;;;;;;;;:38;;;;:::i;:::-;61824:14;:28;61839:12;:10;:12::i;:::-;61824:28;;;;;;;;;;;;;;;:69;;;;61914:7;:5;:7::i;:::-;61906:25;;:45;61944:6;61932:9;:18;;;;:::i;:::-;61906:45;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;::::0;::::1;;;;;;61962:32;61972:12;:10;:12::i;:::-;61986:7;61962:9;:32::i;:::-;60672:1330;;10524:1:::0;11478:7;:22;;;;60605:1397;:::o;14549:201::-;13529:13;:11;:13::i;:::-;14658:1:::1;14638:22;;:8;:22;;;;14630:73;;;;;;;;;;;;:::i;:::-;;;;;;;;;14714:28;14733:8;14714:18;:28::i;:::-;14549:201:::0;:::o;62704:102::-;13529:13;:11;:13::i;:::-;62788:10:::1;62776:9;:22;;;;62704:102:::0;:::o;13808:132::-;13883:12;:10;:12::i;:::-;13872:23;;:7;:5;:7::i;:::-;:23;;;13864:68;;;;;;;;;;;;:::i;:::-;;;;;;;;;13808:132::o;39102:273::-;39159:4;39215:7;39196:15;:13;:15::i;:::-;:26;;:66;;;;;39249:13;;39239:7;:23;39196:66;:152;;;;;39347:1;25704:8;39300:17;:26;39318:7;39300:26;;;;;;;;;;;;:43;:48;39196:152;39176:172;;39102:273;;;:::o;57663:105::-;57723:7;57750:10;57743:17;;57663:105;:::o;28278:92::-;28334:7;28278:92;:::o;32053:1129::-;32120:7;32140:12;32155:7;32140:22;;32223:4;32204:15;:13;:15::i;:::-;:23;32200:915;;32257:13;;32250:4;:20;32246:869;;;32295:14;32312:17;:23;32330:4;32312:23;;;;;;;;;;;;32295:40;;32428:1;25704:8;32401:6;:23;:28;32397:699;;;32920:113;32937:1;32927:6;:11;32920:113;;;32980:17;:25;32998:6;;;;;;;32980:25;;;;;;;;;;;;32971:34;;32920:113;;;33066:6;33059:13;;;;;;32397:699;32272:843;32246:869;32200:915;33143:31;;;;;;;;;;;;;;32053:1129;;;;:::o;44903:652::-;44998:27;45027:23;45068:53;45124:15;45068:71;;45310:7;45304:4;45297:21;45345:22;45339:4;45332:36;45421:4;45415;45405:21;45382:44;;45517:19;45511:26;45492:45;;45248:300;44903:652;;;:::o;45668:645::-;45810:11;45972:15;45966:4;45962:26;45954:34;;46131:15;46120:9;46116:31;46103:44;;46278:15;46267:9;46264:30;46257:4;46246:9;46243:19;46240:55;46230:65;;45668:645;;;;;:::o;56496:159::-;;;;;:::o;54808:309::-;54943:7;54963:16;26105:3;54989:19;:40;;54963:67;;26105:3;55056:31;55067:4;55073:2;55077:9;55056:10;:31::i;:::-;55048:40;;:61;;55041:68;;;54808:309;;;;;:::o;34627:447::-;34707:14;34875:15;34868:5;34864:27;34855:36;;35049:5;35035:11;35011:22;35007:40;35004:51;34997:5;34994:62;34984:72;;34627:447;;;;:::o;57314:158::-;;;;;:::o;14910:191::-;14984:16;15003:6;;;;;;;;;;;14984:25;;15029:8;15020:6;;:17;;;;;;;;;;;;;;;;;;15084:8;15053:40;;15074:8;15053:40;;;;;;;;;;;;14973:128;14910:191;:::o;39459:104::-;39528:27;39538:2;39542:8;39528:27;;;;;;;;;;;;:9;:27::i;:::-;39459:104;;:::o;53318:716::-;53481:4;53527:2;53502:45;;;53548:19;:17;:19::i;:::-;53569:4;53575:7;53584:5;53502:88;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;53498:529;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;53802:1;53785:6;:13;:18;53781:235;;;53831:40;;;;;;;;;;;;;;53781:235;53974:6;53968:13;53959:6;53955:2;53951:15;53944:38;53498:529;53671:54;;;53661:64;;;:6;:64;;;;53654:71;;;53318:716;;;;;;:::o;62119:108::-;62179:13;62212:7;62205:14;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;62119:108;:::o;57874:1960::-;57931:17;58350:3;58343:4;58337:11;58333:21;58326:28;;58441:3;58435:4;58428:17;58547:3;59003:5;59133:1;59128:3;59124:11;59117:18;;59270:2;59264:4;59260:13;59256:2;59252:22;59247:3;59239:36;59311:2;59305:4;59301:13;59293:21;;58895:697;59330:4;58895:697;;;59521:1;59516:3;59512:11;59505:18;;59572:2;59566:4;59562:13;59558:2;59554:22;59549:3;59541:36;59425:2;59419:4;59415:13;59407:21;;58895:697;;;58899:430;59631:3;59626;59622:13;59746:2;59741:3;59737:12;59730:19;;59809:6;59804:3;59797:19;57970:1857;;57874:1960;;;:::o;12194:98::-;12247:7;12274:10;12267:17;;12194:98;:::o;62235:267::-;62280:4;62493:1;62488;62478:6;62354:9;62403:1;62388:12;:16;;;;:::i;:::-;62378:27;62420:15;62450:12;:10;:12::i;:::-;62323:150;;;;;;;;;;;:::i;:::-;;;;;;;;;;;;;62313:161;;;;;;62305:170;;:179;62304:185;;;;:::i;:::-;:190;62297:197;;62235:267;:::o;55693:147::-;55830:6;55693:147;;;;;:::o;39979:681::-;40102:19;40108:2;40112:8;40102:5;:19::i;:::-;40181:1;40163:2;:14;;;:19;40159:483;;40203:11;40217:13;;40203:27;;40249:13;40271:8;40265:3;:14;40249:30;;40298:233;40329:62;40368:1;40372:2;40376:7;;;;;;40385:5;40329:30;:62::i;:::-;40324:167;;40427:40;;;;;;;;;;;;;;40324:167;40526:3;40518:5;:11;40298:233;;40613:3;40596:13;;:20;40592:34;;40618:8;;;40592:34;40184:458;;40159:483;39979:681;;;:::o;40933:1529::-;40998:20;41021:13;;40998:36;;41063:1;41049:16;;:2;:16;;;41045:48;;;41074:19;;;;;;;;;;;;;;41045:48;41120:1;41108:8;:13;41104:44;;;41130:18;;;;;;;;;;;;;;41104:44;41161:61;41191:1;41195:2;41199:12;41213:8;41161:21;:61::i;:::-;41704:1;25071:2;41675:1;:25;;41674:31;41662:8;:44;41636:18;:22;41655:2;41636:22;;;;;;;;;;;;;;;;:70;;;;;;;;;;;41983:139;42020:2;42074:33;42097:1;42101:2;42105:1;42074:14;:33::i;:::-;42041:30;42062:8;42041:20;:30::i;:::-;:66;41983:18;:139::i;:::-;41949:17;:31;41967:12;41949:31;;;;;;;;;;;:173;;;;42139:15;42157:12;42139:30;;42184:11;42213:8;42198:12;:23;42184:37;;42236:101;42288:9;;;;;;42284:2;42263:35;;42280:1;42263:35;;;;;;;;;;;;42332:3;42322:7;:13;42236:101;;42369:3;42353:13;:19;;;;41410:974;;42394:60;42423:1;42427:2;42431:12;42445:8;42394:20;:60::i;:::-;40987:1475;40933:1529;;:::o;36466:322::-;36536:14;36767:1;36757:8;36754:15;36729:23;36725:45;36715:55;;36466:322;;;:::o;-1:-1:-1:-;;;;;;;:::i;:::-;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;;:::i;:::-;;;:::o;:::-;;;;;;;;;;;;;;;;;;;;;:::o;24:722:1:-;120:5;145:81;161:64;218:6;161:64;:::i;:::-;145:81;:::i;:::-;136:90;;246:5;275:6;268:5;261:21;309:4;302:5;298:16;291:23;;335:6;385:3;377:4;369:6;365:17;360:3;356:27;353:36;350:143;;;404:79;;:::i;:::-;350:143;517:1;502:238;527:6;524:1;521:13;502:238;;;595:3;624:37;657:3;645:10;624:37;:::i;:::-;619:3;612:50;691:4;686:3;682:14;675:21;;725:4;720:3;716:14;709:21;;562:178;549:1;546;542:9;537:14;;502:238;;;506:14;126:620;;24:722;;;;;:::o;752:410::-;829:5;854:65;870:48;911:6;870:48;:::i;:::-;854:65;:::i;:::-;845:74;;942:6;935:5;928:21;980:4;973:5;969:16;1018:3;1009:6;1004:3;1000:16;997:25;994:112;;;1025:79;;:::i;:::-;994:112;1115:41;1149:6;1144:3;1139;1115:41;:::i;:::-;835:327;752:410;;;;;:::o;1168:412::-;1246:5;1271:66;1287:49;1329:6;1287:49;:::i;:::-;1271:66;:::i;:::-;1262:75;;1360:6;1353:5;1346:21;1398:4;1391:5;1387:16;1436:3;1427:6;1422:3;1418:16;1415:25;1412:112;;;1443:79;;:::i;:::-;1412:112;1533:41;1567:6;1562:3;1557;1533:41;:::i;:::-;1252:328;1168:412;;;;;:::o;1586:139::-;1632:5;1670:6;1657:20;1648:29;;1686:33;1713:5;1686:33;:::i;:::-;1586:139;;;;:::o;1748:370::-;1819:5;1868:3;1861:4;1853:6;1849:17;1845:27;1835:122;;1876:79;;:::i;:::-;1835:122;1993:6;1980:20;2018:94;2108:3;2100:6;2093:4;2085:6;2081:17;2018:94;:::i;:::-;2009:103;;1825:293;1748:370;;;;:::o;2124:133::-;2167:5;2205:6;2192:20;2183:29;;2221:30;2245:5;2221:30;:::i;:::-;2124:133;;;;:::o;2263:139::-;2309:5;2347:6;2334:20;2325:29;;2363:33;2390:5;2363:33;:::i;:::-;2263:139;;;;:::o;2408:137::-;2453:5;2491:6;2478:20;2469:29;;2507:32;2533:5;2507:32;:::i;:::-;2408:137;;;;:::o;2551:141::-;2607:5;2638:6;2632:13;2623:22;;2654:32;2680:5;2654:32;:::i;:::-;2551:141;;;;:::o;2711:338::-;2766:5;2815:3;2808:4;2800:6;2796:17;2792:27;2782:122;;2823:79;;:::i;:::-;2782:122;2940:6;2927:20;2965:78;3039:3;3031:6;3024:4;3016:6;3012:17;2965:78;:::i;:::-;2956:87;;2772:277;2711:338;;;;:::o;3069:340::-;3125:5;3174:3;3167:4;3159:6;3155:17;3151:27;3141:122;;3182:79;;:::i;:::-;3141:122;3299:6;3286:20;3324:79;3399:3;3391:6;3384:4;3376:6;3372:17;3324:79;:::i;:::-;3315:88;;3131:278;3069:340;;;;:::o;3415:139::-;3461:5;3499:6;3486:20;3477:29;;3515:33;3542:5;3515:33;:::i;:::-;3415:139;;;;:::o;3560:329::-;3619:6;3668:2;3656:9;3647:7;3643:23;3639:32;3636:119;;;3674:79;;:::i;:::-;3636:119;3794:1;3819:53;3864:7;3855:6;3844:9;3840:22;3819:53;:::i;:::-;3809:63;;3765:117;3560:329;;;;:::o;3895:474::-;3963:6;3971;4020:2;4008:9;3999:7;3995:23;3991:32;3988:119;;;4026:79;;:::i;:::-;3988:119;4146:1;4171:53;4216:7;4207:6;4196:9;4192:22;4171:53;:::i;:::-;4161:63;;4117:117;4273:2;4299:53;4344:7;4335:6;4324:9;4320:22;4299:53;:::i;:::-;4289:63;;4244:118;3895:474;;;;;:::o;4375:619::-;4452:6;4460;4468;4517:2;4505:9;4496:7;4492:23;4488:32;4485:119;;;4523:79;;:::i;:::-;4485:119;4643:1;4668:53;4713:7;4704:6;4693:9;4689:22;4668:53;:::i;:::-;4658:63;;4614:117;4770:2;4796:53;4841:7;4832:6;4821:9;4817:22;4796:53;:::i;:::-;4786:63;;4741:118;4898:2;4924:53;4969:7;4960:6;4949:9;4945:22;4924:53;:::i;:::-;4914:63;;4869:118;4375:619;;;;;:::o;5000:943::-;5095:6;5103;5111;5119;5168:3;5156:9;5147:7;5143:23;5139:33;5136:120;;;5175:79;;:::i;:::-;5136:120;5295:1;5320:53;5365:7;5356:6;5345:9;5341:22;5320:53;:::i;:::-;5310:63;;5266:117;5422:2;5448:53;5493:7;5484:6;5473:9;5469:22;5448:53;:::i;:::-;5438:63;;5393:118;5550:2;5576:53;5621:7;5612:6;5601:9;5597:22;5576:53;:::i;:::-;5566:63;;5521:118;5706:2;5695:9;5691:18;5678:32;5737:18;5729:6;5726:30;5723:117;;;5759:79;;:::i;:::-;5723:117;5864:62;5918:7;5909:6;5898:9;5894:22;5864:62;:::i;:::-;5854:72;;5649:287;5000:943;;;;;;;:::o;5949:468::-;6014:6;6022;6071:2;6059:9;6050:7;6046:23;6042:32;6039:119;;;6077:79;;:::i;:::-;6039:119;6197:1;6222:53;6267:7;6258:6;6247:9;6243:22;6222:53;:::i;:::-;6212:63;;6168:117;6324:2;6350:50;6392:7;6383:6;6372:9;6368:22;6350:50;:::i;:::-;6340:60;;6295:115;5949:468;;;;;:::o;6423:474::-;6491:6;6499;6548:2;6536:9;6527:7;6523:23;6519:32;6516:119;;;6554:79;;:::i;:::-;6516:119;6674:1;6699:53;6744:7;6735:6;6724:9;6720:22;6699:53;:::i;:::-;6689:63;;6645:117;6801:2;6827:53;6872:7;6863:6;6852:9;6848:22;6827:53;:::i;:::-;6817:63;;6772:118;6423:474;;;;;:::o;6903:539::-;6987:6;7036:2;7024:9;7015:7;7011:23;7007:32;7004:119;;;7042:79;;:::i;:::-;7004:119;7190:1;7179:9;7175:17;7162:31;7220:18;7212:6;7209:30;7206:117;;;7242:79;;:::i;:::-;7206:117;7347:78;7417:7;7408:6;7397:9;7393:22;7347:78;:::i;:::-;7337:88;;7133:302;6903:539;;;;:::o;7448:329::-;7507:6;7556:2;7544:9;7535:7;7531:23;7527:32;7524:119;;;7562:79;;:::i;:::-;7524:119;7682:1;7707:53;7752:7;7743:6;7732:9;7728:22;7707:53;:::i;:::-;7697:63;;7653:117;7448:329;;;;:::o;7783:327::-;7841:6;7890:2;7878:9;7869:7;7865:23;7861:32;7858:119;;;7896:79;;:::i;:::-;7858:119;8016:1;8041:52;8085:7;8076:6;8065:9;8061:22;8041:52;:::i;:::-;8031:62;;7987:116;7783:327;;;;:::o;8116:349::-;8185:6;8234:2;8222:9;8213:7;8209:23;8205:32;8202:119;;;8240:79;;:::i;:::-;8202:119;8360:1;8385:63;8440:7;8431:6;8420:9;8416:22;8385:63;:::i;:::-;8375:73;;8331:127;8116:349;;;;:::o;8471:509::-;8540:6;8589:2;8577:9;8568:7;8564:23;8560:32;8557:119;;;8595:79;;:::i;:::-;8557:119;8743:1;8732:9;8728:17;8715:31;8773:18;8765:6;8762:30;8759:117;;;8795:79;;:::i;:::-;8759:117;8900:63;8955:7;8946:6;8935:9;8931:22;8900:63;:::i;:::-;8890:73;;8686:287;8471:509;;;;:::o;8986:329::-;9045:6;9094:2;9082:9;9073:7;9069:23;9065:32;9062:119;;;9100:79;;:::i;:::-;9062:119;9220:1;9245:53;9290:7;9281:6;9270:9;9266:22;9245:53;:::i;:::-;9235:63;;9191:117;8986:329;;;;:::o;9321:118::-;9408:24;9426:5;9408:24;:::i;:::-;9403:3;9396:37;9321:118;;:::o;9445:157::-;9550:45;9570:24;9588:5;9570:24;:::i;:::-;9550:45;:::i;:::-;9545:3;9538:58;9445:157;;:::o;9608:109::-;9689:21;9704:5;9689:21;:::i;:::-;9684:3;9677:34;9608:109;;:::o;9723:157::-;9828:45;9848:24;9866:5;9848:24;:::i;:::-;9828:45;:::i;:::-;9823:3;9816:58;9723:157;;:::o;9886:360::-;9972:3;10000:38;10032:5;10000:38;:::i;:::-;10054:70;10117:6;10112:3;10054:70;:::i;:::-;10047:77;;10133:52;10178:6;10173:3;10166:4;10159:5;10155:16;10133:52;:::i;:::-;10210:29;10232:6;10210:29;:::i;:::-;10205:3;10201:39;10194:46;;9976:270;9886:360;;;;:::o;10252:364::-;10340:3;10368:39;10401:5;10368:39;:::i;:::-;10423:71;10487:6;10482:3;10423:71;:::i;:::-;10416:78;;10503:52;10548:6;10543:3;10536:4;10529:5;10525:16;10503:52;:::i;:::-;10580:29;10602:6;10580:29;:::i;:::-;10575:3;10571:39;10564:46;;10344:272;10252:364;;;;:::o;10622:377::-;10728:3;10756:39;10789:5;10756:39;:::i;:::-;10811:89;10893:6;10888:3;10811:89;:::i;:::-;10804:96;;10909:52;10954:6;10949:3;10942:4;10935:5;10931:16;10909:52;:::i;:::-;10986:6;10981:3;10977:16;10970:23;;10732:267;10622:377;;;;:::o;11005:366::-;11147:3;11168:67;11232:2;11227:3;11168:67;:::i;:::-;11161:74;;11244:93;11333:3;11244:93;:::i;:::-;11362:2;11357:3;11353:12;11346:19;;11005:366;;;:::o;11377:::-;11519:3;11540:67;11604:2;11599:3;11540:67;:::i;:::-;11533:74;;11616:93;11705:3;11616:93;:::i;:::-;11734:2;11729:3;11725:12;11718:19;;11377:366;;;:::o;11749:::-;11891:3;11912:67;11976:2;11971:3;11912:67;:::i;:::-;11905:74;;11988:93;12077:3;11988:93;:::i;:::-;12106:2;12101:3;12097:12;12090:19;;11749:366;;;:::o;12121:::-;12263:3;12284:67;12348:2;12343:3;12284:67;:::i;:::-;12277:74;;12360:93;12449:3;12360:93;:::i;:::-;12478:2;12473:3;12469:12;12462:19;;12121:366;;;:::o;12493:::-;12635:3;12656:67;12720:2;12715:3;12656:67;:::i;:::-;12649:74;;12732:93;12821:3;12732:93;:::i;:::-;12850:2;12845:3;12841:12;12834:19;;12493:366;;;:::o;12865:400::-;13025:3;13046:84;13128:1;13123:3;13046:84;:::i;:::-;13039:91;;13139:93;13228:3;13139:93;:::i;:::-;13257:1;13252:3;13248:11;13241:18;;12865:400;;;:::o;13271:366::-;13413:3;13434:67;13498:2;13493:3;13434:67;:::i;:::-;13427:74;;13510:93;13599:3;13510:93;:::i;:::-;13628:2;13623:3;13619:12;13612:19;;13271:366;;;:::o;13643:::-;13785:3;13806:67;13870:2;13865:3;13806:67;:::i;:::-;13799:74;;13882:93;13971:3;13882:93;:::i;:::-;14000:2;13995:3;13991:12;13984:19;;13643:366;;;:::o;14015:::-;14157:3;14178:67;14242:2;14237:3;14178:67;:::i;:::-;14171:74;;14254:93;14343:3;14254:93;:::i;:::-;14372:2;14367:3;14363:12;14356:19;;14015:366;;;:::o;14387:::-;14529:3;14550:67;14614:2;14609:3;14550:67;:::i;:::-;14543:74;;14626:93;14715:3;14626:93;:::i;:::-;14744:2;14739:3;14735:12;14728:19;;14387:366;;;:::o;14759:::-;14901:3;14922:67;14986:2;14981:3;14922:67;:::i;:::-;14915:74;;14998:93;15087:3;14998:93;:::i;:::-;15116:2;15111:3;15107:12;15100:19;;14759:366;;;:::o;15131:118::-;15218:24;15236:5;15218:24;:::i;:::-;15213:3;15206:37;15131:118;;:::o;15255:157::-;15360:45;15380:24;15398:5;15380:24;:::i;:::-;15360:45;:::i;:::-;15355:3;15348:58;15255:157;;:::o;15418:679::-;15614:3;15629:75;15700:3;15691:6;15629:75;:::i;:::-;15729:2;15724:3;15720:12;15713:19;;15742:75;15813:3;15804:6;15742:75;:::i;:::-;15842:2;15837:3;15833:12;15826:19;;15855:75;15926:3;15917:6;15855:75;:::i;:::-;15955:2;15950:3;15946:12;15939:19;;15968:75;16039:3;16030:6;15968:75;:::i;:::-;16068:2;16063:3;16059:12;16052:19;;16088:3;16081:10;;15418:679;;;;;;;:::o;16103:701::-;16384:3;16406:95;16497:3;16488:6;16406:95;:::i;:::-;16399:102;;16518:95;16609:3;16600:6;16518:95;:::i;:::-;16511:102;;16630:148;16774:3;16630:148;:::i;:::-;16623:155;;16795:3;16788:10;;16103:701;;;;;:::o;16810:222::-;16903:4;16941:2;16930:9;16926:18;16918:26;;16954:71;17022:1;17011:9;17007:17;16998:6;16954:71;:::i;:::-;16810:222;;;;:::o;17038:640::-;17233:4;17271:3;17260:9;17256:19;17248:27;;17285:71;17353:1;17342:9;17338:17;17329:6;17285:71;:::i;:::-;17366:72;17434:2;17423:9;17419:18;17410:6;17366:72;:::i;:::-;17448;17516:2;17505:9;17501:18;17492:6;17448:72;:::i;:::-;17567:9;17561:4;17557:20;17552:2;17541:9;17537:18;17530:48;17595:76;17666:4;17657:6;17595:76;:::i;:::-;17587:84;;17038:640;;;;;;;:::o;17684:210::-;17771:4;17809:2;17798:9;17794:18;17786:26;;17822:65;17884:1;17873:9;17869:17;17860:6;17822:65;:::i;:::-;17684:210;;;;:::o;17900:313::-;18013:4;18051:2;18040:9;18036:18;18028:26;;18100:9;18094:4;18090:20;18086:1;18075:9;18071:17;18064:47;18128:78;18201:4;18192:6;18128:78;:::i;:::-;18120:86;;17900:313;;;;:::o;18219:419::-;18385:4;18423:2;18412:9;18408:18;18400:26;;18472:9;18466:4;18462:20;18458:1;18447:9;18443:17;18436:47;18500:131;18626:4;18500:131;:::i;:::-;18492:139;;18219:419;;;:::o;18644:::-;18810:4;18848:2;18837:9;18833:18;18825:26;;18897:9;18891:4;18887:20;18883:1;18872:9;18868:17;18861:47;18925:131;19051:4;18925:131;:::i;:::-;18917:139;;18644:419;;;:::o;19069:::-;19235:4;19273:2;19262:9;19258:18;19250:26;;19322:9;19316:4;19312:20;19308:1;19297:9;19293:17;19286:47;19350:131;19476:4;19350:131;:::i;:::-;19342:139;;19069:419;;;:::o;19494:::-;19660:4;19698:2;19687:9;19683:18;19675:26;;19747:9;19741:4;19737:20;19733:1;19722:9;19718:17;19711:47;19775:131;19901:4;19775:131;:::i;:::-;19767:139;;19494:419;;;:::o;19919:::-;20085:4;20123:2;20112:9;20108:18;20100:26;;20172:9;20166:4;20162:20;20158:1;20147:9;20143:17;20136:47;20200:131;20326:4;20200:131;:::i;:::-;20192:139;;19919:419;;;:::o;20344:::-;20510:4;20548:2;20537:9;20533:18;20525:26;;20597:9;20591:4;20587:20;20583:1;20572:9;20568:17;20561:47;20625:131;20751:4;20625:131;:::i;:::-;20617:139;;20344:419;;;:::o;20769:::-;20935:4;20973:2;20962:9;20958:18;20950:26;;21022:9;21016:4;21012:20;21008:1;20997:9;20993:17;20986:47;21050:131;21176:4;21050:131;:::i;:::-;21042:139;;20769:419;;;:::o;21194:::-;21360:4;21398:2;21387:9;21383:18;21375:26;;21447:9;21441:4;21437:20;21433:1;21422:9;21418:17;21411:47;21475:131;21601:4;21475:131;:::i;:::-;21467:139;;21194:419;;;:::o;21619:::-;21785:4;21823:2;21812:9;21808:18;21800:26;;21872:9;21866:4;21862:20;21858:1;21847:9;21843:17;21836:47;21900:131;22026:4;21900:131;:::i;:::-;21892:139;;21619:419;;;:::o;22044:::-;22210:4;22248:2;22237:9;22233:18;22225:26;;22297:9;22291:4;22287:20;22283:1;22272:9;22268:17;22261:47;22325:131;22451:4;22325:131;:::i;:::-;22317:139;;22044:419;;;:::o;22469:222::-;22562:4;22600:2;22589:9;22585:18;22577:26;;22613:71;22681:1;22670:9;22666:17;22657:6;22613:71;:::i;:::-;22469:222;;;;:::o;22697:129::-;22731:6;22758:20;;:::i;:::-;22748:30;;22787:33;22815:4;22807:6;22787:33;:::i;:::-;22697:129;;;:::o;22832:75::-;22865:6;22898:2;22892:9;22882:19;;22832:75;:::o;22913:311::-;22990:4;23080:18;23072:6;23069:30;23066:56;;;23102:18;;:::i;:::-;23066:56;23152:4;23144:6;23140:17;23132:25;;23212:4;23206;23202:15;23194:23;;22913:311;;;:::o;23230:307::-;23291:4;23381:18;23373:6;23370:30;23367:56;;;23403:18;;:::i;:::-;23367:56;23441:29;23463:6;23441:29;:::i;:::-;23433:37;;23525:4;23519;23515:15;23507:23;;23230:307;;;:::o;23543:308::-;23605:4;23695:18;23687:6;23684:30;23681:56;;;23717:18;;:::i;:::-;23681:56;23755:29;23777:6;23755:29;:::i;:::-;23747:37;;23839:4;23833;23829:15;23821:23;;23543:308;;;:::o;23857:98::-;23908:6;23942:5;23936:12;23926:22;;23857:98;;;:::o;23961:99::-;24013:6;24047:5;24041:12;24031:22;;23961:99;;;:::o;24066:168::-;24149:11;24183:6;24178:3;24171:19;24223:4;24218:3;24214:14;24199:29;;24066:168;;;;:::o;24240:169::-;24324:11;24358:6;24353:3;24346:19;24398:4;24393:3;24389:14;24374:29;;24240:169;;;;:::o;24415:148::-;24517:11;24554:3;24539:18;;24415:148;;;;:::o;24569:305::-;24609:3;24628:20;24646:1;24628:20;:::i;:::-;24623:25;;24662:20;24680:1;24662:20;:::i;:::-;24657:25;;24816:1;24748:66;24744:74;24741:1;24738:81;24735:107;;;24822:18;;:::i;:::-;24735:107;24866:1;24863;24859:9;24852:16;;24569:305;;;;:::o;24880:348::-;24920:7;24943:20;24961:1;24943:20;:::i;:::-;24938:25;;24977:20;24995:1;24977:20;:::i;:::-;24972:25;;25165:1;25097:66;25093:74;25090:1;25087:81;25082:1;25075:9;25068:17;25064:105;25061:131;;;25172:18;;:::i;:::-;25061:131;25220:1;25217;25213:9;25202:20;;24880:348;;;;:::o;25234:191::-;25274:4;25294:20;25312:1;25294:20;:::i;:::-;25289:25;;25328:20;25346:1;25328:20;:::i;:::-;25323:25;;25367:1;25364;25361:8;25358:34;;;25372:18;;:::i;:::-;25358:34;25417:1;25414;25410:9;25402:17;;25234:191;;;;:::o;25431:96::-;25468:7;25497:24;25515:5;25497:24;:::i;:::-;25486:35;;25431:96;;;:::o;25533:90::-;25567:7;25610:5;25603:13;25596:21;25585:32;;25533:90;;;:::o;25629:77::-;25666:7;25695:5;25684:16;;25629:77;;;:::o;25712:149::-;25748:7;25788:66;25781:5;25777:78;25766:89;;25712:149;;;:::o;25867:126::-;25904:7;25944:42;25937:5;25933:54;25922:65;;25867:126;;;:::o;25999:77::-;26036:7;26065:5;26054:16;;25999:77;;;:::o;26082:154::-;26166:6;26161:3;26156;26143:30;26228:1;26219:6;26214:3;26210:16;26203:27;26082:154;;;:::o;26242:307::-;26310:1;26320:113;26334:6;26331:1;26328:13;26320:113;;;26419:1;26414:3;26410:11;26404:18;26400:1;26395:3;26391:11;26384:39;26356:2;26353:1;26349:10;26344:15;;26320:113;;;26451:6;26448:1;26445:13;26442:101;;;26531:1;26522:6;26517:3;26513:16;26506:27;26442:101;26291:258;26242:307;;;:::o;26555:320::-;26599:6;26636:1;26630:4;26626:12;26616:22;;26683:1;26677:4;26673:12;26704:18;26694:81;;26760:4;26752:6;26748:17;26738:27;;26694:81;26822:2;26814:6;26811:14;26791:18;26788:38;26785:84;;;26841:18;;:::i;:::-;26785:84;26606:269;26555:320;;;:::o;26881:281::-;26964:27;26986:4;26964:27;:::i;:::-;26956:6;26952:40;27094:6;27082:10;27079:22;27058:18;27046:10;27043:34;27040:62;27037:88;;;27105:18;;:::i;:::-;27037:88;27145:10;27141:2;27134:22;26924:238;26881:281;;:::o;27168:233::-;27207:3;27230:24;27248:5;27230:24;:::i;:::-;27221:33;;27276:66;27269:5;27266:77;27263:103;;;27346:18;;:::i;:::-;27263:103;27393:1;27386:5;27382:13;27375:20;;27168:233;;;:::o;27407:100::-;27446:7;27475:26;27495:5;27475:26;:::i;:::-;27464:37;;27407:100;;;:::o;27513:79::-;27552:7;27581:5;27570:16;;27513:79;;;:::o;27598:94::-;27637:7;27666:20;27680:5;27666:20;:::i;:::-;27655:31;;27598:94;;;:::o;27698:79::-;27737:7;27766:5;27755:16;;27698:79;;;:::o;27783:176::-;27815:1;27832:20;27850:1;27832:20;:::i;:::-;27827:25;;27866:20;27884:1;27866:20;:::i;:::-;27861:25;;27905:1;27895:35;;27910:18;;:::i;:::-;27895:35;27951:1;27948;27944:9;27939:14;;27783:176;;;;:::o;27965:180::-;28013:77;28010:1;28003:88;28110:4;28107:1;28100:15;28134:4;28131:1;28124:15;28151:180;28199:77;28196:1;28189:88;28296:4;28293:1;28286:15;28320:4;28317:1;28310:15;28337:180;28385:77;28382:1;28375:88;28482:4;28479:1;28472:15;28506:4;28503:1;28496:15;28523:180;28571:77;28568:1;28561:88;28668:4;28665:1;28658:15;28692:4;28689:1;28682:15;28709:180;28757:77;28754:1;28747:88;28854:4;28851:1;28844:15;28878:4;28875:1;28868:15;28895:117;29004:1;29001;28994:12;29018:117;29127:1;29124;29117:12;29141:117;29250:1;29247;29240:12;29264:117;29373:1;29370;29363:12;29387:117;29496:1;29493;29486:12;29510:102;29551:6;29602:2;29598:7;29593:2;29586:5;29582:14;29578:28;29568:38;;29510:102;;;:::o;29618:94::-;29651:8;29699:5;29695:2;29691:14;29670:35;;29618:94;;;:::o;29718:225::-;29858:34;29854:1;29846:6;29842:14;29835:58;29927:8;29922:2;29914:6;29910:15;29903:33;29718:225;:::o;29949:169::-;30089:21;30085:1;30077:6;30073:14;30066:45;29949:169;:::o;30124:170::-;30264:22;30260:1;30252:6;30248:14;30241:46;30124:170;:::o;30300:176::-;30440:28;30436:1;30428:6;30424:14;30417:52;30300:176;:::o;30482:163::-;30622:15;30618:1;30610:6;30606:14;30599:39;30482:163;:::o;30651:155::-;30791:7;30787:1;30779:6;30775:14;30768:31;30651:155;:::o;30812:182::-;30952:34;30948:1;30940:6;30936:14;30929:58;30812:182;:::o;31000:226::-;31140:34;31136:1;31128:6;31124:14;31117:58;31209:9;31204:2;31196:6;31192:15;31185:34;31000:226;:::o;31232:177::-;31372:29;31368:1;31360:6;31356:14;31349:53;31232:177;:::o;31415:172::-;31555:24;31551:1;31543:6;31539:14;31532:48;31415:172;:::o;31593:181::-;31733:33;31729:1;31721:6;31717:14;31710:57;31593:181;:::o;31780:122::-;31853:24;31871:5;31853:24;:::i;:::-;31846:5;31843:35;31833:63;;31892:1;31889;31882:12;31833:63;31780:122;:::o;31908:116::-;31978:21;31993:5;31978:21;:::i;:::-;31971:5;31968:32;31958:60;;32014:1;32011;32004:12;31958:60;31908:116;:::o;32030:122::-;32103:24;32121:5;32103:24;:::i;:::-;32096:5;32093:35;32083:63;;32142:1;32139;32132:12;32083:63;32030:122;:::o;32158:120::-;32230:23;32247:5;32230:23;:::i;:::-;32223:5;32220:34;32210:62;;32268:1;32265;32258:12;32210:62;32158:120;:::o;32284:122::-;32357:24;32375:5;32357:24;:::i;:::-;32350:5;32347:35;32337:63;;32396:1;32393;32386:12;32337:63;32284:122;:::o

Swarm Source

ipfs://0f945f0933d4034fec5e31f4bc52cfc69eac34357e2c3040e07ff0f9bd8f8a4a
Loading...
Loading
Loading...
Loading
[ Download: CSV Export  ]
[ Download: CSV Export  ]

A token is a representation of an on-chain or off-chain asset. The token page shows information such as price, total supply, holders, transfers and social links. Learn more about this page in our Knowledge Base.