Searched refs:SE (Results 1 - 25 of 161) sorted by relevance

1234567

/freebsd-11.0-release/contrib/llvm/include/llvm/ADT/
H A DSetOperations.h26 for (typename S2Ty::const_iterator SI = S2.begin(), SE = S2.end();
27 SI != SE; ++SI)
53 for (typename S1Ty::const_iterator SI = S1.begin(), SE = S1.end();
54 SI != SE; ++SI)
64 for (typename S2Ty::const_iterator SI = S2.begin(), SE = S2.end();
65 SI != SE; ++SI)
/freebsd-11.0-release/contrib/llvm/include/llvm/Analysis/
H A DScalarEvolutionAliasAnalysis.h28 ScalarEvolution &SE; member in class:llvm::SCEVAAResult
31 explicit SCEVAAResult(const TargetLibraryInfo &TLI, ScalarEvolution &SE) argument
32 : AAResultBase(TLI), SE(SE) {}
33 SCEVAAResult(SCEVAAResult &&Arg) : AAResultBase(std::move(Arg)), SE(Arg.SE) {}
H A DScalarEvolutionExpressions.h306 const SCEV *getStepRecurrence(ScalarEvolution &SE) const {
308 return SE.getAddRecExpr(SmallVector<const SCEV *, 3>(op_begin()+1,
339 const SCEV *evaluateAtIteration(const SCEV *It, ScalarEvolution &SE) const;
348 ScalarEvolution &SE) const;
352 const SCEVAddRecExpr *getPostIncExpr(ScalarEvolution &SE) const {
353 return cast<SCEVAddRecExpr>(SE.getAddExpr(this, getStepRecurrence(SE)));
415 /// SE - The parent ScalarEvolution value. This is used to update
418 ScalarEvolution *SE; member in class:llvm::final
426 SCEV(ID, scUnknown), CallbackVH(V), SE(s
561 ScalarEvolution &SE; member in class:llvm::SCEVRewriteVisitor
563 SCEVRewriteVisitor(ScalarEvolution &SE) argument
640 rewrite(const SCEV *Scev, ScalarEvolution &SE, ValueToValueMap &Map, bool InterpretConsts = false) argument
647 SCEVParameterRewriter(ScalarEvolution &SE, ValueToValueMap &M, bool C) argument
673 rewrite(const SCEV *Scev, LoopToScevMapT &Map, ScalarEvolution &SE) argument
679 SCEVLoopAddRecRewriter(ScalarEvolution &SE, LoopToScevMapT &M) argument
702 apply(const SCEV *Scev, LoopToScevMapT &Map, ScalarEvolution &SE) argument
[all...]
H A DScalarEvolutionNormalization.h73 ScalarEvolution &SE,
/freebsd-11.0-release/contrib/llvm/lib/Transforms/Utils/
H A DSimplifyIndVar.cpp49 ScalarEvolution *SE; member in class:__anon3290::SimplifyIndvar
57 SimplifyIndvar(Loop *Loop, ScalarEvolution *SE, DominatorTree *DT, argument
59 : L(Loop), LI(LI), SE(SE), DT(DT), DeadInsts(Dead), Changed(false) {
116 assert(SE->isSCEVable(IVSrc->getType()) && "Expect SCEVable IV operand");
128 FoldedExpr = SE->getUDivExpr(SE->getSCEV(IVSrc), SE->getSCEV(D));
131 if (!SE->isSCEVable(UseInst->getType()))
135 if (SE
498 isSimpleIVUser(Instruction *I, const Loop *L, ScalarEvolution *SE) argument
597 simplifyUsersOfIV(PHINode *CurrIV, ScalarEvolution *SE, DominatorTree *DT, LoopInfo *LI, SmallVectorImpl<WeakVH> &Dead, IVVisitor *V) argument
607 simplifyLoopIVs(Loop *L, ScalarEvolution *SE, DominatorTree *DT, LoopInfo *LI, SmallVectorImpl<WeakVH> &Dead) argument
[all...]
H A DLCSSA.cpp220 ScalarEvolution *SE) {
256 if (SE && Changed)
257 SE->forgetLoop(&L);
266 ScalarEvolution *SE) {
271 Changed |= formLCSSARecursively(*SubLoop, DT, LI, SE);
273 Changed |= formLCSSA(L, DT, LI, SE);
287 ScalarEvolution *SE; member in struct:__anon3277::LCSSA
326 SE = SEWP ? &SEWP->getSE() : nullptr;
330 Changed |= formLCSSARecursively(**I, *DT, LI, SE);
219 formLCSSA(Loop &L, DominatorTree &DT, LoopInfo *LI, ScalarEvolution *SE) argument
265 formLCSSARecursively(Loop &L, DominatorTree &DT, LoopInfo *LI, ScalarEvolution *SE) argument
/freebsd-11.0-release/contrib/llvm/lib/Analysis/
H A DScalarEvolutionNormalization.cpp70 ScalarEvolution &SE; member in class:__anon2416::PostIncTransform
78 Kind(kind), Loops(loops), SE(se), DT(dt) {}
99 case scZeroExtend: return SE.getZeroExtendExpr(N, S->getType());
100 case scSignExtend: return SE.getSignExtendExpr(N, S->getType());
101 case scTruncate: return SE.getTruncateExpr(N, S->getType());
119 const SCEV *Result = SE.getAddRecExpr(Operands, L, SCEV::FlagAnyWrap);
135 TransformSubExpr(AR->getStepRecurrence(SE),
137 Result = SE.getMinusSCEV(Result, TransformedStep);
166 TransformSubExpr(AR->getStepRecurrence(SE),
168 Result = SE
245 TransformForPostIncUse(TransformKind Kind, const SCEV *S, Instruction *User, Value *OperandValToReplace, PostIncLoopSet &Loops, ScalarEvolution &SE, DominatorTree &DT) argument
[all...]
H A DScalarEvolutionExpander.cpp83 assert(SE.DT.dominates(Ret, &*BIP));
120 assert(SE.getTypeSizeInBits(V->getType()) == SE.getTypeSizeInBits(Ty) &&
134 SE.getTypeSizeInBits(Ty) == SE.getTypeSizeInBits(V->getType())) {
138 SE.getTypeSizeInBits(CI->getType()) ==
139 SE.getTypeSizeInBits(CI->getOperand(0)->getType()))
144 SE.getTypeSizeInBits(CE->getType()) ==
145 SE.getTypeSizeInBits(CE->getOperand(0)->getType()))
204 while (const Loop *L = SE
228 FactorOutConstant(const SCEV *&S, const SCEV *&Remainder, const SCEV *Factor, ScalarEvolution &SE, const DataLayout &DL) argument
301 SimplifyAddOperands(SmallVectorImpl<const SCEV *> &Ops, Type *Ty, ScalarEvolution &SE) argument
330 SplitAddRecs(SmallVectorImpl<const SCEV *> &Ops, Type *Ty, ScalarEvolution &SE) argument
804 ExposePointerBase(const SCEV *&Base, const SCEV *&Rest, ScalarEvolution &SE) argument
1007 canBeCheaplyTransformed(ScalarEvolution &SE, const SCEVAddRecExpr *Phi, const SCEVAddRecExpr *Requested, bool &InvertStep) argument
1038 IsIncrementNSW(ScalarEvolution &SE, const SCEVAddRecExpr *AR) argument
1052 IsIncrementNUW(ScalarEvolution &SE, const SCEVAddRecExpr *AR) argument
1994 ScalarEvolution &SE; member in struct:__anon2415::SCEVFindUnsafe
2021 isSafeToExpand(const SCEV *S, ScalarEvolution &SE) argument
[all...]
H A DScalarEvolutionAliasAnalysis.cpp35 const SCEV *AS = SE.getSCEV(const_cast<Value *>(LocA.Ptr));
36 const SCEV *BS = SE.getSCEV(const_cast<Value *>(LocB.Ptr));
44 if (SE.getEffectiveSCEVType(AS->getType()) ==
45 SE.getEffectiveSCEVType(BS->getType())) {
46 unsigned BitWidth = SE.getTypeSizeInBits(AS->getType());
51 const SCEV *BA = SE.getMinusSCEV(BS, AS);
56 if (ASizeInt.ule(SE.getUnsignedRange(BA).getUnsignedMin()) &&
57 (-BSizeInt).uge(SE.getUnsignedRange(BA).getUnsignedMax()))
65 const SCEV *AB = SE.getMinusSCEV(AS, BS);
70 if (BSizeInt.ule(SE
[all...]
H A DDelinearization.cpp45 ScalarEvolution *SE; member in class:__anon2387::Delinearization
68 SE = &getAnalysis<ScalarEvolutionWrapperPass>().getSE();
97 const SCEV *AccessFn = SE->getSCEVAtScope(getPointerOperand(*Inst), L);
100 dyn_cast<SCEVUnknown>(SE->getPointerBase(AccessFn));
104 AccessFn = SE->getMinusSCEV(AccessFn, BasePointer);
112 SE->delinearize(AccessFn, Subscripts, Sizes, SE->getElementSize(Inst));
H A DDependenceAnalysis.cpp136 SE = &getAnalysis<ScalarEvolutionWrapperPass>().getSE();
338 return SE->getNegativeSCEV(C);
375 A = SE->getOne(D->getType());
376 B = SE->getNegativeSCEV(A);
377 C = SE->getNegativeSCEV(D);
388 SE = NewSE;
468 const SCEV *Prod1 = SE->getMulExpr(X->getA(), Y->getB());
469 const SCEV *Prod2 = SE->getMulExpr(X->getB(), Y->getA());
473 Prod1 = SE->getMulExpr(X->getC(), Y->getB());
474 Prod2 = SE
[all...]
H A DIVUsers.cpp54 ScalarEvolution *SE, LoopInfo *LI) {
62 SE->getSCEVAtScope(AR, LI->getLoopFor(I->getParent())) != AR);
66 return isInteresting(AR->getStart(), I, L, SE, LI) &&
67 !isInteresting(AR->getStepRecurrence(*SE), I, L, SE, LI);
75 if (isInteresting(*OI, I, L, SE, LI)) {
127 if (!SE->isSCEVable(I->getType()))
139 uint64_t Width = SE->getTypeSizeInBits(I->getType());
149 const SCEV *ISE = SE->getSCEV(I);
153 if (!isInteresting(ISE, I, L, SE, L
53 isInteresting(const SCEV *S, const Instruction *I, const Loop *L, ScalarEvolution *SE, LoopInfo *LI) argument
[all...]
/freebsd-11.0-release/contrib/llvm/include/llvm/Transforms/Utils/
H A DUnrollLoop.h34 LoopInfo *LI, ScalarEvolution *SE, DominatorTree *DT,
39 ScalarEvolution *SE, DominatorTree *DT,
H A DLoopVersioning.h43 DominatorTree *DT, ScalarEvolution *SE,
110 ScalarEvolution *SE; member in class:llvm::LoopVersioning
H A DSimplifyIndVar.h60 bool simplifyUsersOfIV(PHINode *CurrIV, ScalarEvolution *SE, DominatorTree *DT,
66 bool simplifyLoopIVs(Loop *L, ScalarEvolution *SE, DominatorTree *DT,
/freebsd-11.0-release/contrib/llvm/lib/Transforms/Scalar/
H A DAlignmentFromAssumptions.cpp76 ScalarEvolution *SE; member in struct:__anon3170::AlignmentFromAssumptions
107 ScalarEvolution *SE) {
109 const SCEV *DiffAlignDiv = SE->getUDivExpr(DiffSCEV, AlignSCEV);
110 const SCEV *DiffAlign = SE->getMulExpr(DiffAlignDiv, AlignSCEV);
111 const SCEV *DiffUnitsSCEV = SE->getMinusSCEV(DiffAlign, DiffSCEV);
142 ScalarEvolution *SE) {
143 const SCEV *PtrSCEV = SE->getSCEV(Ptr);
144 const SCEV *DiffSCEV = SE->getMinusSCEV(PtrSCEV, AASCEV);
148 DiffSCEV = SE->getNoopOrSignExtend(DiffSCEV, OffSCEV->getType());
152 DiffSCEV = SE
105 getNewAlignmentDiff(const SCEV *DiffSCEV, const SCEV *AlignSCEV, ScalarEvolution *SE) argument
140 getNewAlignment(const SCEV *AASCEV, const SCEV *AlignSCEV, const SCEV *OffSCEV, Value *Ptr, ScalarEvolution *SE) argument
[all...]
H A DInductiveRangeCheckElimination.cpp126 ScalarEvolution &SE, Value *&Index,
130 parseRangeCheck(Loop *L, ScalarEvolution &SE, Value *Condition,
192 Optional<Range> computeSafeIterationSpace(ScalarEvolution &SE,
199 Loop *L, ScalarEvolution &SE,
267 ScalarEvolution &SE, Value *&Index,
270 auto IsNonNegativeAndNotLoopVarying = [&SE, L](Value *V) {
271 const SCEV *S = SE.getSCEV(V);
275 return SE.getLoopDisposition(S, L) == ScalarEvolution::LoopInvariant &&
276 SE.isKnownNonNegative(S);
333 InductiveRangeCheck::parseRangeCheck(Loop *L, ScalarEvolution &SE, argument
266 parseRangeCheckICmp(Loop *L, ICmpInst *ICI, ScalarEvolution &SE, Value *&Index, Value *&Length) argument
391 create(InductiveRangeCheck::AllocatorTy &A, BranchInst *BI, Loop *L, ScalarEvolution &SE, BranchProbabilityInfo &BPI) argument
597 ScalarEvolution &SE; member in class:__anon3193::__anon3194::LoopConstrainer
617 LoopConstrainer(Loop &L, LoopInfo &LI, const LoopStructure &LS, ScalarEvolution &SE, InductiveRangeCheck::Range R) argument
637 CanBeSMax(ScalarEvolution &SE, const SCEV *S) argument
644 CanBeSMin(ScalarEvolution &SE, const SCEV *S) argument
652 parseLoopStructure(ScalarEvolution &SE, BranchProbabilityInfo &BPI, Loop &L, const char *&FailureReason) argument
1308 computeSafeIterationSpace(ScalarEvolution &SE, const SCEVAddRecExpr *IndVar, IRBuilder<> &) const argument
1376 IntersectRange(ScalarEvolution &SE, const Optional<InductiveRangeCheck::Range> &R1, const InductiveRangeCheck::Range &R2, IRBuilder<> &B) argument
1409 ScalarEvolution &SE = getAnalysis<ScalarEvolutionWrapperPass>().getSE(); local
[all...]
H A DIndVarSimplify.cpp92 ScalarEvolution *SE; member in class:__anon3187::IndVarSimplify
103 : LoopPass(ID), LI(nullptr), SE(nullptr), DT(nullptr), Changed(false) {
201 const SCEV *FromBase = SE->getPointerBase(SE->getSCEV(FromPtr));
202 const SCEV *ToBase = SE->getPointerBase(SE->getSCEV(ToPtr));
496 SE->forgetLoop(L);
593 SE->forgetValue(PN);
615 const SCEV *ExitValue = SE->getSCEVAtScope(Inst, L->getParentLoop());
616 if (!SE
787 visitIVCast(CastInst *Cast, WideIVInfo &WI, ScalarEvolution *SE, const TargetTransformInfo *TTI) argument
860 ScalarEvolution *SE; member in class:__anon3190::WidenIV
1453 ScalarEvolution *SE; member in class:__anon3191::IndVarSimplifyVisitor
1541 canExpandBackedgeTakenCount(Loop *L, ScalarEvolution *SE, SCEVExpander &Rewriter) argument
1720 FindLoopCounter(Loop *L, const SCEV *BECount, ScalarEvolution *SE, DominatorTree *DT) argument
1803 genLoopLimit(PHINode *IndVar, const SCEV *IVCount, Loop *L, SCEVExpander &Rewriter, ScalarEvolution *SE) argument
[all...]
H A DLoopStrengthReduce.cpp283 void initialMatch(const SCEV *S, Loop *L, ScalarEvolution &SE);
310 ScalarEvolution &SE) {
312 if (SE.properlyDominates(S, L->getHeader())) {
320 DoInitialMatch(S, L, Good, Bad, SE);
327 DoInitialMatch(AR->getStart(), L, Good, Bad, SE);
328 DoInitialMatch(SE.getAddRecExpr(SE.getConstant(AR->getType(), 0),
329 AR->getStepRecurrence(SE),
332 L, Good, Bad, SE);
340 const SCEV *NewMul = SE
307 DoInitialMatch(const SCEV *S, Loop *L, SmallVectorImpl<const SCEV *> &Good, SmallVectorImpl<const SCEV *> &Bad, ScalarEvolution &SE) argument
361 initialMatch(const SCEV *S, Loop *L, ScalarEvolution &SE) argument
509 isAddRecSExtable(const SCEVAddRecExpr *AR, ScalarEvolution &SE) argument
517 isAddSExtable(const SCEVAddExpr *A, ScalarEvolution &SE) argument
525 isMulSExtable(const SCEVMulExpr *M, ScalarEvolution &SE) argument
537 getExactSDiv(const SCEV *LHS, const SCEV *RHS, ScalarEvolution &SE, bool IgnoreSignificantBits = false) argument
624 ExtractImmediate(const SCEV *&S, ScalarEvolution &SE) argument
650 ExtractSymbol(const SCEV *&S, ScalarEvolution &SE) argument
731 isExistingPhi(const SCEVAddRecExpr *AR, ScalarEvolution &SE) argument
752 isHighCostExpansion(const SCEV *S, SmallPtrSetImpl<const SCEV*> &Processed, ScalarEvolution &SE) argument
925 RateRegister(const SCEV *Reg, SmallPtrSetImpl<const SCEV *> &Regs, const Loop *L, ScalarEvolution &SE, DominatorTree &DT) argument
973 RatePrimaryRegister(const SCEV *Reg, SmallPtrSetImpl<const SCEV *> &Regs, const Loop *L, ScalarEvolution &SE, DominatorTree &DT, SmallPtrSetImpl<const SCEV *> *LoserRegs) argument
989 RateFormula(const TargetTransformInfo &TTI, const Formula &F, SmallPtrSetImpl<const SCEV *> &Regs, const DenseSet<const SCEV *> &VisitedRegs, const Loop *L, const SmallVectorImpl<int64_t> &Offsets, ScalarEvolution &SE, DominatorTree &DT, const LSRUse &LU, SmallPtrSetImpl<const SCEV *> *LoserRegs) argument
1548 isAlwaysFoldable(const TargetTransformInfo &TTI, ScalarEvolution &SE, int64_t MinOffset, int64_t MaxOffset, LSRUse::KindType Kind, MemAccessTy AccessTy, const SCEV *S, bool HasBaseReg) argument
1643 ScalarEvolution &SE; member in class:__anon3216::LSRInstance
2427 findIVOperand(User::op_iterator OI, User::op_iterator OE, Loop *L, ScalarEvolution &SE) argument
2507 isProfitableIncrement(const SCEV *OperExpr, const SCEV *IncExpr, ScalarEvolution &SE) argument
2537 isProfitableChain(IVChain &Chain, SmallPtrSetImpl<Instruction*> &Users, ScalarEvolution &SE, const TargetTransformInfo &TTI) argument
3178 CollectSubexprs(const SCEV *S, const SCEVConstant *C, SmallVectorImpl<const SCEV *> &Ops, const Loop *L, ScalarEvolution &SE, unsigned Depth = 0) argument
4781 LSRInstance(Loop *L, IVUsers &IU, ScalarEvolution &SE, DominatorTree &DT, LoopInfo &LI, const TargetTransformInfo &TTI) argument
5004 auto &SE = getAnalysis<ScalarEvolutionWrapperPass>().getSE(); local
[all...]
H A DNaryReassociate.cpp179 ScalarEvolution *SE; member in class:__anon3230::NaryReassociate
216 SE = &getAnalysis<ScalarEvolutionWrapperPass>().getSE();
249 if (SE->isSCEVable(I->getType()) && isPotentiallyNaryReassociable(&*I)) {
250 const SCEV *OldSCEV = SE->getSCEV(&*I);
253 SE->forgetValue(&*I);
262 const SCEV *NewSCEV = SE->getSCEV(&*I);
407 IndexExprs.push_back(SE->getSCEV(*Index));
409 IndexExprs[I] = SE->getSCEV(LHS);
418 SE->getZeroExtendExpr(IndexExprs[I], GEP->getOperand(I)->getType());
420 const SCEV *CandidateExpr = SE
[all...]
/freebsd-11.0-release/crypto/heimdal/appl/telnet/telnetd/
H A Dtermstat.c60 IAC, SE);
68 IAC, SE);
/freebsd-11.0-release/contrib/llvm/tools/clang/lib/StaticAnalyzer/Checkers/
H A DVLASizeChecker.cpp96 const Expr *SE = VLA->getSizeExpr(); local
98 SVal sizeV = state->getSVal(SE, C.getLocationContext());
101 reportBug(VLA_Garbage, SE, state, C);
112 reportBug(VLA_Tainted, SE, nullptr, C);
123 reportBug(VLA_Zero, SE, stateZero, C);
137 QualType Ty = SE->getType();
148 reportBug(VLA_Negative, SE, state, C);
157 svalBuilder.evalCast(sizeD, SizeTy, SE->getType()).castAs<NonLoc>();
/freebsd-11.0-release/contrib/llvm/lib/CodeGen/
H A DEdgeBundles.cpp48 SE = MBB.succ_end(); SI != SE; ++SI)
85 SE = MBB.succ_end(); SI != SE; ++SI)
/freebsd-11.0-release/contrib/llvm/tools/clang/include/clang/StaticAnalyzer/Core/PathSensitive/
H A DSymbolManager.h89 symbol_iterator(const SymExpr *SE);
125 static inline bool classof(const SymExpr *SE) { argument
126 Kind k = SE->getKind();
155 static inline bool classof(const SymExpr *SE) { argument
156 return SE->getKind() == SymbolRegionValueKind;
199 static inline bool classof(const SymExpr *SE) { argument
200 return SE->getKind() == SymbolConjuredKind;
233 static inline bool classof(const SymExpr *SE) { argument
234 return SE->getKind() == SymbolDerivedKind;
264 static inline bool classof(const SymExpr *SE) { argument
309 classof(const SymExpr *SE) argument
345 classof(const SymExpr *SE) argument
367 classof(const SymExpr *SE) argument
403 classof(const SymExpr *SE) argument
438 classof(const SymExpr *SE) argument
472 classof(const SymExpr *SE) argument
681 operator <<(raw_ostream &os, const clang::ento::SymExpr *SE) argument
[all...]
/freebsd-11.0-release/contrib/llvm/lib/Target/PowerPC/
H A DPPCLoopDataPrefetch.cpp76 // FIXME: For some reason, preserving SE here breaks LSR (even if
88 ScalarEvolution *SE; member in class:__anon2983::PPCLoopDataPrefetch
108 SE = &getAnalysis<ScalarEvolutionWrapperPass>().getSE();
180 const SCEV *LSCEV = SE->getSCEV(PtrValue);
192 const SCEV *PtrDiff = SE->getMinusSCEV(LSCEVAddRec, K->second);
205 const SCEV *NextLSCEV = SE->getAddExpr(LSCEVAddRec, SE->getMulExpr(
206 SE->getConstant(LSCEVAddRec->getType(), ItersAhead),
207 LSCEVAddRec->getStepRecurrence(*SE)));
208 if (!isSafeToExpand(NextLSCEV, *SE))
[all...]

Completed in 243 milliseconds

1234567