1 / 48

TexPoint fonts used in EMF. Read the TexPoint manual before you delete this box.: A A

Art of Invariant Generation applied to. Symbolic Bound Computation. Part 2. Sumit Gulwani (Microsoft Research, Redmond, USA). Oregon Summer School July 2009. TexPoint fonts used in EMF. Read the TexPoint manual before you delete this box.: A A. Art of Invariant Generation.

airlia
Download Presentation

TexPoint fonts used in EMF. Read the TexPoint manual before you delete this box.: A A

An Image/Link below is provided (as is) to download presentation Download Policy: Content on the Website is provided to you AS IS for your information and personal use and may not be sold / licensed / shared on other websites without getting consent from its author. Content is provided to you AS IS for your information and personal use only. Download presentation by click this link. While downloading, if for some reason you are not able to download a presentation, the publisher may have deleted the file from their server. During download, if you can't get a presentation, the file might be deleted by the publisher.

E N D

Presentation Transcript


  1. Art of Invariant Generation applied to Symbolic Bound Computation Part 2 SumitGulwani (Microsoft Research, Redmond, USA) Oregon Summer School July 2009 TexPoint fonts used in EMF. Read the TexPoint manual before you delete this box.: AA

  2. Art of Invariant Generation • Program Transformations • Reduce need for sophisticated invariant generation. • E.g., control-flow refinement, loop-flattening/peeling, non-standard cut-points, quantitative attributes instrumentation. • Colorful Logic • Language of Invariants • E.g., arithmetic, uninterpreted fns, lists/arrays • Fixpoint Brush • Automatic generation of invariants in some shade of logic, e.g., conjunctive/k-disjunctive/predicate abstraction. • E.g., Iterative, Constraint-based, Proof Rules

  3. Logic • To validate correctness of loop-free programs, or programs annotated with loop invariants, decision procedures are enough. • Provided the logic is closed under WP. <Pre, S, Post> is valid iff Pre ) WP(S, Post) is valid iff Pre Æ:WP(S,Post) is unsatisfiable • To validate correctness of programs with loops, we need to automatically discover loop invariants using fixpoint computation techniques. • This requires algorithms that are more sophisticated than decision procedures.

  4. Fixpoint Brush We will briefly study fixpoint techniques for discovering loop invariants in conjunctive fragments of various logics. • Iterative • Forward • Backward • Constraint-based • Proof-rules

  5. Iterative Forward: Examples Start with Precondition and propagate facts forward using Existential elimination operator until fixpoint. • Data-flow analysis • Join at merge points • Finite abstract domains • Abstract Interpretation • Join at merge points • Widening for infinite height abstract domains. • Model Checking • Analyze all paths precisely without join at merge points. • Finite abstractions (e.g., boolean abstraction) required • Counterexample guided abstraction refinement • BDD based data-structures for efficiency

  6. Key Operators needed by Iterative Forward Fixpoint checking: Decision Procedure. DecideT() = Yes, iff is satisfiable Transfer Function for Assignment Node: Existential Quantifier Elimination Eliminate(, V) = strongest Á’ such that V 2Vars(Á’) Transfer Function for Merge Node: Join Join(1 , 2) = strongest  s.t. 1) and 2) Eliminate and Join are usually harder than Decide.

  7. Difference Constraints • Abstract element: • conjunction of xi-xj·cij • can be represented using matrix M, where M[i][j]=cij • Decide(M): • M’ := Saturate(M); • Declare unsatiff9i: M’[i][i] < 0 • Join(M1, M2): • M’1 := Saturate(M1); M’2 := Saturate(M2); • Let M3 be s.t. M3[i][j] = Max { M’1[i][j], M’2[i][j] } • return M3

  8. Difference Constraints • Eliminate(M, xi): • M’ := Saturate(M); • Let M1 be s.t. M1[j][k] = 1 (if j=i or k=i) = M’[j][k] otherwise • return M1 • Widen(M1, M2): • M’1 := Saturate(M1); M’2 := Saturate(M2); • Let M3 be s.t. M3[i][j] = M1[i][j] (if M1[i][j] = M2[i][j])) = 1 (otherwise) • return M3

  9. Example: Abstract Interpretation using Difference Constraints true y := 0; z := 2; y=0, z=2 ? y=0 Æ z=2 ? 0·y·1 Æ z=y+2 0·y·2 Æ z=y+2 0·y Æ z=y+2 0·y<51 Æ z=y+2 1·y·2 Æ z=y+2 1·y<51 Æ z=y+2 y=1 Æ z=3 ? y < 50 y=50 Æ z=y+2 False True Assert (z=52) y=0 Æ z=2 0·y·1 Æ z=y+2 0·y<50 Æ z=y+2 ? y++; z++;

  10. Uninterpreted Functions • Abstract element: • conjunction of e1=e2, where e := y | F(e1,e2) • can be represented using EDAGs • Decide(G): • G’ := Saturate(G); • Declare unsatiff G contains e1  e2 and G’ has e1, e2 in the same congruence class. • Eliminate(G, y): • G’ := Saturate(G); • Erase y; (might need to delete some dangling expressions) • return G’

  11. Uninterpreted Functions • Join(G1, G2): • G’1 := Saturate(G1); G’2 := Saturate(G2); • G := Intersect(G’1, G’2); • return G; For each node n = <U, F(ni,n’i)> in G’1 and node m = <V, F(mj,m’j)> in G’2, G contains a node [n,m] = <U Å V, F([ni, mj],[n’i,m’j])>

  12. y1, F y1, F y1, F y2, F y2, F y2, F F F F F F F y3,y4 y5 y6 y7 y6,y7 y3 y4,y5 y7 y6 y4,y5 y3 Uninterpreted Functions: Example of Join G1 G2 G = Join(G1,G2)

  13. Recap: Combinationof Decision Procedures • Decide(E12): • <E1, E2> := Purify&Saturate(E12); • Return DecideT1(E1) ÆDecideT2(E2);

  14. Combination: Join Algorithm (1st attempt) • JoinT12(L12, R12): • <L1, L2> := Purify&Saturate(L12); <R1, R2> := Purify&Saturate(R12); • A1:= JoinT1(L1, R1); A2 := JoinT2(L2, R2); • Return A1ÆA2;

  15. Combination: Join Algorithm • JoinT12(L12, R12): • <L1, L2> := Purify&Saturate(L12); <R1, R2> := Purify&Saturate(R12); • DL := Æ {vi=<vi,vj> | vi2Vars(L1ÆL2), vj2Vars(R1ÆR2) }; DR := Æ {vj=<vi,vj> | vi2Vars(L1ÆL2), vj2Vars(R1ÆR2) }; • L’1 := L1Æ DL; R’1 := R1Æ DR; L’2 := L2Æ DL; R’2 := R2Æ DR; • A1 := JoinT1(L’1, R’1); A2 := JoinT2(L’2, R’2); • V := Vars(A1ÆA2) – Program Variables; A12 := EliminateT12(A1ÆA2, V); • Return A12;

  16. Combination: Example of Join Algorithm z=a-1 Æ y=F(a) z=b-1 Æ y=F(b) Joinuf+la z=a-1 a=ha,bi y=F(a) a=ha,bi z=b-1 b=ha,bi y=F(b) b=ha,bi Joinuf Joinla ha,bi=1+z y=F(ha,bi) { ha,bi } Eliminateuf+la y=F(1+z)

  17. Combination: Existential Quantifier Elimination • ElimintateT12(E12, V): • <E1, E2> := Purify&Saturate(E12); • <D, Defs> := DefSaturate(E1, E2, V [ Temp Variables); • V’ := V [ Temp Variables – D; E’1 := EliminateT1(E1, V’); E’2 := EliminateT2(E2, V’); • E := (E’1Æ E’2) [Defs(y)/y]; • Return E; DefSaturate(E1, E2, U) returns the set of all variables D that have definitions Defs in terms of variables not in U as implied by E1Æ E2.

  18. c  z-1 a F(z-1) Combination: Example of Existential Elimination a·b·y Æ z=c+1 Æ a=F2(b) Æ c=F(b) { a, b, c } Eliminateuf+la a·b·y Æ z=c+1 a=F2(b) Æ c=F(b) Defuf Defla { b } Eliminatela Eliminateuf c  z-1 a F(z-1) a · y Æ z=c+1 a = F(c) Substitute F(z-1) · y

  19. Example: Abstract Interpretation over Combined Domain true class List { List next; } x, y; N(z) = 0, if z = null = 1 + N(z.next) y := x; i := 0; y=x, i=0 ? 0·i·2, N(x)=N(y)+i 0·i, N(x)=N(y)+i 0·i·1 N(x)=N(y)+i 1·i·2, N(x)=N(y)+i ? y=x, i=0 1·i, N(x)=N(y)+i y=x.next, i=1, xnull N(x)=N(x.next)+1 ? ynull False True 0·i·1, y  null N(x)=N(y)+i 0·i, y  null N(x)=N(y)+i 0·i Æ N(x)=i ? y=x, i=0, ynull i := i+1; y := y.next;

  20. Iterative Forward: References • Uninterpreted Functions • A Polynomial-Time Algorithm for Global Value Numbering; Gulwani, Necula; SAS ‘04 • Linear Arithmetic + Uninterpreted Functions • Combining Abstract Interpreters; Gulwani, Tiwari; PLDI ’06 • Theory of Arrays/Lists • Quantified Abstract Domains • Lifting Abstract Interpreters to Quantified Logical Domains; Gulwani, McCloskey, Tiwari; POPL ‘08 • Discovering Properties about Arrays in Simple Programs; Halbwachs, Péron; PLDI ‘08 • Shape Analysis • Parametric Shape Analysis via 3-Valued Logic; Sagiv, Reps, Wilhelm; POPL ‘99, TOPLAS ‘02

  21. Iterative Forward: References • Theory of Arrays/Lists • Combination of Shape Analysis + Arithmetic • A Combination Framework for tracking partition sizes; Gulwani, Lev-Ami, Sagiv; POPL ’09 • Non-linear Arithmetic • User-defined axioms + Expression Abstraction • A Numerical Abstract Domain Based on Expression Abstraction and Max Operator with Application in Timing Analysis; Gulavani, Gulwani; CAV ’08 • Polynomial Equalities • An Abstract Interpretation Approach for Automatic Generation of Polynomial Invariants; Rodriguez-Carbonell, Kapur; SAS ‘04

  22. Fixpoint Brush • Iterative • Forward • Backward • Constraint-based • Proof-rules

  23. Iterative Backward • Comparison with Iterative Forward • Positives: Can compute preconditions, Goal-directed • Negatives: Requires assertions or template assertions. • Transfer Function for Assignment Node is easier. • Substitution takes role of existential elimination. • Transfer Function for Conditional Node is challenging. • Requires abductive reasoning/under-approximations. • Abduct(,g) = weakest ’ s.t. ’Æg)  • Case-split reasoning as opposed to Saturation based, and hence typically not closed under conjunctions. • Optimally weak solutions for negative unknowns as opposed to optimally strong solutions for positive unknowns.

  24. Iterative Backward: References Program Verification using Templates over Predicate Abstraction; Srivastava, Gulwani; PLDI ‘09 Assertion Checking Unified; Gulwani, Tiwari; VMCAI ‘07 Computing Procedure Summaries for Interprocedural Analysis; Gulwani, Tiwari; ESOP ‘07

  25. Fixpoint Brush • Iterative • Forward • Backward • Constraint-based • Proof-rules

  26. Constraint-based Invariant Generation Pre while (c) S Post Base Case Precision Inductive Case Pre ) I I Æ:c ) Post (I Æ c)[S] ) I VCGen I 8X 9 I Verification Constraint (Second-order) • Key Idea: Reduce the second-order verification constraint to a first-ordersatisfiability constraint that can be solved using off-the-shelf SAT/SMT solvers • Choose a template for I (specific color/shade in some logic). • Convert 8 into 9. Goal-directed invariant generation for verification of a Hoare triple (Pre, Program, Post)

  27. Key Idea in reducing 8 to 9 for various Domains Trick for converting 8 to 9 is known for following domains: • Linear Arithmetic • Farkas Lemma • Linear Arithmetic + Uninterpreted Fns. • Farkas Lemma + Ackerman’s Reduction • Non-linear Arithmetic • Grobner Basis • Predicate Abstraction • Boolean indicator variables + Cover Algorithm (Abduction) • Quantified Predicate Abstraction • Boolean indicator variables + More general Abduction

  28. Constraint-based Invariant Generation: References • Linear Arithmetic • Constraint-based Linear-relations analysis; Sankaranarayanan, Sipma, Manna; SAS ’04 • Program analysis as constraint solving; Gulwani, Srivastava, Venkatesan; PLDI ‘08 • Linear Arithmetic + Uninterpreted Fns. • Invariant synthesis for combined theories; Beyer, Henzinger, Majumdar, Rybalchenko; VMCAI ‘07 • Non-linear Arithmetic • Non-linear loop invariant generation using Gröbner bases; Sankaranarayanan, Sipma, Manna; POPL ’04 • Predicate Abstraction • Constraint-based invariant inference over predicate abstraction; Gulwani, Srivastava, Venkatesan; VMCAI ’09 • Quantified Predicate Abstraction • Program verification using templates over predicate abstraction; Srivastava, Gulwani; PLDI ‘09

  29. Constraint-based Invariant Generation • Linear Arithmetic • Linear Arithmetic + Uninterpreted Fns. • Non-linear Arithmetic • Predicate Abstraction • Quantified Predicate Abstraction

  30. Farkas Lemma 8X Æk(ek¸0) ) e¸0 iff 9k¸0 8X (e ´ + kkek) Example Let’s find Farkas witness ,1,2 for the implication x¸2 Æ y¸3 ) 2x+y¸6 9,1,2¸0 s.t. 8x,y [2x+y-6 ´ +1(x-2) + 2(y-3)] Equating coefficients of x,y and constant terms, we get: 2=1Æ 1=2Æ -6=-21-32 which implies =1, 1=2, 2=1.

  31. Solving 2nd order constraints using Farkas Lemma 9I 8X 1(I,X) • Second-order to First-order • Assume I has some form, e.g., j ajxj¸ 0 • 9I 8X 1(I,X) translates to 9aj8X 2(aj,X) • First-order to “only existentially quantified” • Farkas Lemma helps translate 8 to 9 • 8X (Æk(ek¸0) ) e¸0) iff9k¸0 8X (e ´ + kkek) • Eliminate X from polynomial equality by equating coefficients. • 9aj8X 2(aj,X) translates to 9aj9¸k3(aj,¸k) • “only existentially quantified” to SAT • Bit-vector modeling for integer variables

  32. Example [n=1 Æ m=1] x := 0; y := 0; while (x < 100) x := x+n; y := y+m; [y ¸ 100] n=m=1 Æ x=y=0 ) I I Æ x¸100 ) y¸100 I Æ x<100 ) I[xÃx+n, yÃy+m] VCGen I Invariant Template Satisfying Solution Loop Invariant a0 + a1x + a2y + a3n + a4m ¸ 0 b0 + b1x + b2y + b3n + b4m ¸ 0 c0 + c1x + c2y + c3n + c4m ¸ 0 y ¸ x m ¸1 n · 1 a2=b0=c4=1, a1=b3=c0=-1 a2=b2=1, a1=b1=-1 y ¸ x m ¸ n a0 + a1x + a2y + a3n + a4m ¸ 0 b0 + b1x + b2y + b3n + b4m ¸ 0 UNSAT Invalid triple or Imprecise Template a0 + a1x + a2y + a3n + a4m ¸ 0

  33. Constraint-based Invariant Generation • Linear Arithmetic • Linear Arithmetic + Uninterpreted Fns. • Non-linear Arithmetic • Predicate Abstraction • Quantified Predicate Abstraction

  34. Solving 2nd order constraints using Boolean Indicator Variables + Cover Algorithm 9I 8X 1(I,X) • Second-order to First-order (Boolean indicator variables) • Assume I has the form P1Ç P2, where P1, P2µ P Let bi,jdenote presence of pj2P in Pi Then, I can be written as (Æj b1,j)pj) Ç (Æj b2,j)pj) 9I 8X 1(I,X) translates to 9bi,j 8X 2(bi,j,X) • Can generalize to k disjuncts • First-order to “only existentially quantified” • Cover Algorithm helps translate 8 to 9 • 9bi,j8X 2(bi,j,X) translates to SAT formula 9bi,j 3(bi,j)

  35. Example [m > 0] x := 0; y := 0; while (x < m) x := x+1; y := y+1; [y=m] VCGen m>0 ) I[xÃ0, yÃ0] I Æ x¸m) y=m I Æ x<m ) I[xÃx+1, yÃy+1] I x·y, x¸y, x<y x·m, x¸m, x<m y·m, y¸m, y<m Suppose P = and k = 1 Then, I has the form P1, where P1µ P m>0 ) P1[xÃ0, yÃ0] (1) P1Æ x¸m) y=m (2) P1Æ x<m ) P1[xÃx+1, yÃy+1] (3)

  36. Example (1) m>0 ) P1 [xÃ0, yÃ0] x·y, x¸y, x<y x·m, x¸m, x<m y·m, y¸m, y<m 0·0, 0¸0, 0<0 0·m, 0¸m, 0<m 0·m, 0¸m, 0<m xÃ0, yÃ0 Hence, (1) ´ P1 doesn’t contain x<y, x¸m, y¸m ´:bx¸mÆ:bx<y Æ:by¸m (2) P1Æ x¸m) y=m (i) y·mÆy¸m (ii) x<m (iii) x·yÆy·m There are 3 maximally-weak choices for P1 (computed using Predicate Cover Algorithm) Hence, (2) ´ P1 contains at least one of above combinations ´ (bx<m) Ç (by·mÆ by¸m)Ç (bx·yÆby·m)

  37. Example (1) :bx¸mÆ:bx<y Æ:by¸m Obtained from solving local/small SMT queries (2) (bx<m)Ç (by·mÆby¸m)Ç (bx·yÆby·m) (3) (by·m) (by<mÇby·x))Æ:bx<mÆ:by<m SAT Solver by·x , by·m, bx·y: true rest: false [m > 0] x := 0; y := 0; while (x < m) x := x+1; y := y+1; [y=m] I I: (y=xÆy·m)

  38. Bonus Material Where can we go? Going beyond Invariant Generation with Constraint-based techniques…

  39. Example: Bresenham’s Line Drawing Algorithm [0<Y·X] v1:=2Y-X; y:=0; x:=0; while (x · X) out[x] := y; if (v1<0) v1:=v1+2Y; else v1:=v1+2(Y-X); y++; return out; [8k (0·k·X ) |out[k]–(Y/X)k| · ½)] Postcondition: The best fit line shouldn’t deviate more than half a pixel from the real line, i.e., |y – (Y/X)x| · 1/2

  40. Transition System Representation [0<Y·X] v1:=2Y-X; y:=0; x:=0; while (x·X) v1<0: out’=Update(out,x,y) Æv’1=v1+2Y Æ y’=y Æ x’=x+1 v1¸0: out’=Update(out,x,y) Æv1=v1+2(Y-X) Æ y’=y+1Æ x’=x+1 [8k (0·k·X ) |out[k]–(Y/X)k| · ½)] [Pre] sentry; while (gloop) gbody1: sbody1; gbody2: sbody2; [Post] Or, equivalently, Where, gbody1: v1<0 gbody2: v1¸0 gloop: x·X sentry: v1’=2Y-X Æ y’=0 Æ x’=0 sbody1: out’=Update(out,x,y) Æv’1=v1+2Y Æ x’=x+1 Æ y’=y • sbody2: out’=Update(out,x,y) Æv’1=v1+2(Y-X) Æ x’=x+1 Æ y’=y+1

  41. Verification Constraint Generation & Solution PreÆsentry) I’ I ÆgloopÆgbody1Æsbody1) I’ I ÆgloopÆgbody2Æsbody2) I’ • I Æ:gloop) Post Verification Constraint: Given Pre, Post, gloop, gbody1, gbody2, sbody1, sbody2, we can find solution for I using constraint-based techniques. 0<Y·X Æv1=2(x+1)Y-(2y+1)X Æ2(Y-X)·v1·2Y Æ8k(0·k·x ) |out[k]–(Y/X)k| · ½) I:

  42. The Surprise! PreÆsentry) I’ I ÆgloopÆgbody1Æsbody1) I’ I ÆgloopÆgbody2Æsbody2) I’ • I Æ:gloop) Post Verification Constraint: • What if we treat each g and s as unknowns like I? • We get a solution that has gbody1 = gbody2 = false. • This doesn’t correspond to a valid transition system. • We can fix this by encoding gbody1Çgbody2 = true. • We now get a solution that has gloop = true. • This corresponds to a non-terminating loop. • We can fix this by encoding existence of a ranking function. • We now discover each g and s along with I. • We have gone from Invariant Synthesis to Program Synthesis.

  43. Fixpoint Brush • Iterative • Forward • Backward • Constraint-based • Proof-rules

  44. Proof Rules while (cond(X)) ¼: X’ := F(X); Bounding Loop Iterations If (cond(X) Æ X’=F(X)) ) (e>0 Æ e[X’/X]·e-1), Then Bound(¼)·e Candidate expressions for e: Look inside Cond(X). Bounding values of monotonically increasing variables If (cond(X) Æ X’=F(X)) )y’·y+c), Then yout·yin + c£Bound(¼) Candidate constants for c: 1, 2

  45. Recurrence Solving Techniques vs. Our Fixpoint Brush Recurrence Solving Techniques vs. Our Fixpoint Brush Undergraduate Textbook on Algorithms by Cormen, Leiserson, Rivest, Stein describes 3 fundamental methods for recurrence solving: Example of a recurrence: T(n)=T(n-1)+2n Æ T(0)=0 • Iteration Method • Expands/unfolds the recurrence relation • Similar to Iterative approach • Substitution Method • Assumes a template for a closed-form • Similar to Constraint-based approach • Masters Theorem • Provides a cook-book solution for T(n)=aT(n/b)+f(n) • Similar to Proof-Rules approach

  46. Fixpoint Brush • Iterative • Forward • Backward • Constraint-based • Proof-rules • Learning • Iterative, but w/o monotonic increase or decrease. • Distance to fixed-point decreases in each iteration.

  47. Learning: References • Program Verification as Probabilistic Inference; Gulwani, Jojic; POPL ’07 • Learning Regular Sets from Queries and Counterexamples; Angluin; Information and Computing ‘87 • Learning Synthesis of interface specifications for Java classes; Alur, Madhusudan, Nam; POPL ‘05. • Learning meets verification; Leucker; FMCO ‘06 • May/Must Analyses? • Game-theoretic Analyses?

  48. Fixpoint Brush: Summary • Iterative • Forward • Join, Existential Elimination • Backward • Abduct • Constraint-based • Exotic; Works well for small code-fragments • 8 to 9 • Proof-rules • Scalable • Requires understanding design patterns • Learning

More Related