LLVM API Documentation
Functions | |
bool | isFPImm (const APFloat &Val, uint32_t &Imm8Bits) |
bool | isFPImm (const APFloat &Val) |
bool | isLogicalImm (unsigned RegWidth, uint64_t Imm, uint32_t &Bits) |
bool | isLogicalImmBits (unsigned RegWidth, uint32_t Bits, uint64_t &Imm) |
bool | isMOVZImm (int RegWidth, uint64_t Value, int &UImm16, int &Shift) |
bool | isMOVNImm (int RegWidth, uint64_t Value, int &UImm16, int &Shift) |
bool | isOnlyMOVNImm (int RegWidth, uint64_t Value, int &UImm16, int &Shift) |
uint64_t | decodeNeonModImm (unsigned Val, unsigned OpCmode, unsigned &EltBits) |
bool | decodeNeonModShiftImm (unsigned OpCmode, unsigned &ShiftImm, unsigned &ShiftOnesIn) |
Definition at line 1144 of file AArch64BaseInfo.cpp.
References llvm_unreachable.
bool llvm::A64Imms::decodeNeonModShiftImm | ( | unsigned | OpCmode, |
unsigned & | ShiftImm, | ||
unsigned & | ShiftOnesIn | ||
) |
Definition at line 1112 of file AArch64BaseInfo.cpp.
References llvm_unreachable.
Definition at line 872 of file AArch64BaseInfo.cpp.
References llvm::APFloat::bitcastToAPInt(), llvm::tgtok::Bits, llvm::APInt::getLimitedValue(), llvm::APFloat::getSemantics(), llvm::APFloat::isNegative(), llvm_unreachable, and llvm::APFloat::semanticsPrecision().
Referenced by isFPImm(), and llvm::AArch64TargetLowering::LowerBUILD_VECTOR().
|
inline |
Definition at line 1116 of file AArch64BaseInfo.h.
References llvm::X86II::Imm8, and isFPImm().
Definition at line 946 of file AArch64BaseInfo.cpp.
References llvm::CountLeadingOnes_32(), llvm::CountLeadingOnes_64(), llvm::CountTrailingOnes_64(), llvm::countTrailingZeros(), llvm::isMask_64(), and N.
Referenced by llvm::AArch64TargetLowering::LowerAsmOperandForConstraint().
Definition at line 1021 of file AArch64BaseInfo.cpp.
References N.
Referenced by DecodeLogicalImmOperand(), and llvm::AArch64InstPrinter::printLogicalImmOperand().
bool llvm::A64Imms::isMOVNImm | ( | int | RegWidth, |
uint64_t | Value, | ||
int & | UImm16, | ||
int & | Shift | ||
) |
Definition at line 1087 of file AArch64BaseInfo.cpp.
References isMOVZImm().
Referenced by isOnlyMOVNImm().
bool llvm::A64Imms::isMOVZImm | ( | int | RegWidth, |
uint64_t | Value, | ||
int & | UImm16, | ||
int & | Shift | ||
) |
Definition at line 1070 of file AArch64BaseInfo.cpp.
Referenced by isMOVNImm(), and isOnlyMOVNImm().
bool llvm::A64Imms::isOnlyMOVNImm | ( | int | RegWidth, |
uint64_t | Value, | ||
int & | UImm16, | ||
int & | Shift | ||
) |
Definition at line 1101 of file AArch64BaseInfo.cpp.
References isMOVNImm(), and isMOVZImm().