semantics and verification of software
play

Semantics and Verification of Software Summer Semester 2019 Lecture - PowerPoint PPT Presentation

Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness) Thomas Noll Software Modeling and Verification Group RWTH Aachen University


  1. Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness) Thomas Noll Software Modeling and Verification Group RWTH Aachen University https://moves.rwth-aachen.de/teaching/ss-19/sv-sw/

  2. Recap: Hoare Logic Hoare Logic Goal: syntactic derivation of valid partial correctness properties. Here A [ x �→ a ] denotes the syntactic replacement of every occurrence of x by a in A . Tony Hoare (* 1934) Definition (Hoare Logic) The Hoare rules are given by (skip) { A } skip { A } (asgn) { A [ x �→ a ] } x := a { A } (seq) { A } c 1 { C } { C } c 2 { B } (if) { A ∧ b } c 1 { B } { A ∧ ¬ b } c 2 { B } { A } c 1 ; c 2 { B } { A } if b then c 1 else c 2 end { B } = ( B ′ ⇒ B ) = ( A ⇒ A ′ ) { A ′ } c { B ′ } { A ∧ b } c { A } (cons) | | (while) { A } while b do c end { A ∧ ¬ b } { A } c { B } A partial correctness property is provable (notation: ⊢ { A } c { B } ) if it is derivable by the Hoare rules. In (while), A is called a (loop) invariant. 3 of 22 Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness)

  3. Recap: Hoare Logic Soundness of Hoare Logic Theorem (Soundness of Hoare Logic) For every partial correctness property { A } c { B } , ⊢ { A } c { B } ⇒ | = { A } c { B } . Proof. Let ⊢ { A } c { B } . By induction over the structure of the corresponding proof tree we = I A , C � c � σ = ⊥ or C � c � σ | = I B show that, for every σ ∈ Σ and I ∈ Int such that σ | (on the board). 4 of 22 Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness)

  4. Incompleteness of Hoare Logic Incompleteness of Hoare Logic I Soundness: only valid partial correctness properties are provable � Completeness: all valid partial correctness properties are systematically derivable � Theorem 11.1 (G¨ odel’s Incompleteness Theorem) The set of all valid assertions { A ∈ Assn | | = A } is not recursively enumerable, i.e., there exists no proof system for Assn in which all valid assertions are systematically derivable. Proof. Kurt G¨ odel see [Winskel 1996, p. 110 ff] (1906–1978) 6 of 22 Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness)

  5. Incompleteness of Hoare Logic Incompleteness of Hoare Logic II Corollary 11.2 There is no proof system in which all valid partial correctness properties can be enumerated. Proof. Given A ∈ Assn , | = A is obviously equivalent to { true } skip { A } . Thus the enumerability of all valid partial correctness properties would imply the enumerability of all valid assertions. Remark: alternative proof (using computability theory): { true } c { false } is valid iff c does not terminate on any input state. But the set of all non-terminating WHILE statements is not enumerable. 7 of 22 Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness)

  6. Relative Completeness of Hoare Logic Relative Completeness of Hoare Logic I • We will see: actual reason of incompleteness is rule = ( B ′ ⇒ B ) = ( A ⇒ A ′ ) { A ′ } c { B ′ } (cons) | | { A } c { B } since it is based on the validity of implications within Assn • The other language constructs are “enumerable” • Therefore: separation of proof system (Hoare Logic) and assertion language ( Assn ) • One can show: if an “oracle” is available which decides whether a given assertion is valid, then all valid partial correctness properties can be systematically derived ⇒ “Relative completeness” 9 of 22 Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness)

  7. Relative Completeness of Hoare Logic Relative Completeness of Hoare Logic II Theorem 11.3 (Cook’s Completeness Theorem) Hoare Logic is relatively complete, i.e., for every partial correctness property { A } c { B } : | = { A } c { B } ⇒ ⊢ { A } c { B } . Stephen A. Cook (* 1939) Thus: if we know that a partial correctness property is valid, then we know that there is a corresponding proof. The proof uses the following concept: assume that, e.g., { A } c 1 ; c 2 { B } has to be derived. This requires an intermediate assertion C ∈ Assn such that { A } c 1 { C } and { C } c 2 { B } . How to find it? 10 of 22 Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness)

  8. Relative Completeness of Hoare Logic Weakest Liberal Preconditions I Definition 11.4 (Weakest liberal precondition) Given c ∈ Cmd and S ⊆ Σ , the weakest (liberal) precondition of S with respect to c collects all states σ such that running c in σ does not terminate or yields a state in S : wlp � c � S := { σ ∈ Σ | C � c � σ ∈ S ∪ {⊥}} . Corollary 11.5 For every c ∈ Cmd, A , B ∈ Assn, and I ∈ Int: = I { A } c { B } ⇐ ⇒ A I ⊆ wlp � c � B I 1. | 0 = wlp � c � B I for every I ∈ Int, then | 2. If A 0 ∈ Assn such that A I = { A } c { B } ⇐ ⇒ | = ( A ⇒ A 0 ) Remarks: • Corollary 11.5 justifies the notion of weakest precondition: it is entailed by every precondition A that makes { A } c { B } valid. • In the following, we do not distinguish between sets of program states (such as S or A I ) and predicates on program states (such as B � b � ). 11 of 22 Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness)

  9. Relative Completeness of Hoare Logic Weakest Liberal Preconditions II Lemma 11.6 (Weakest liberal precondition transformer) Weakest liberal preconditions wlp � . � . : Cmd × 2 Σ → 2 Σ can be computed as follows: wlp � skip � S = S wlp � x := a � S = { σ ∈ Σ | σ [ x �→ A � a � σ ] ∈ S } wlp � c 1 ; c 2 � S = wlp � c 1 � ( wlp � c 2 � S ) wlp � if b then c 1 else c 2 end � S = ( B � b � ∩ wlp � c 1 � S ) ∪ ( B � ¬ b � ∩ wlp � c 2 � S ) wlp � while b do c end � S = FIX (Ψ) where FIX (Ψ) denotes the greatest fixpoint (w.r.t. ( 2 Σ , ⊆ ) ) of Ψ : 2 Σ → 2 Σ : T �→ ( B � b � ∩ wlp � c � T ) ∪ ( B � ¬ b � ∩ S ) Remark: FIX (Ψ) of a continuous function Ψ on lattice ( 2 Σ , ⊆ ) can be computed by fixpoint iteration (see following slide) Proof. omitted 12 of 22 Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness)

  10. Relative Completeness of Hoare Logic Weakest Liberal Preconditions III Example 11.7 Using Lemma 11.6, we want to determine the weakest liberal precondition for c 0 � �� � { ? } while x � = 0 ∧ x � = 1 do { x = 1 } x := x-2 end � �� � c i.e., wlp � c � S for S := B � x = 1 � . • wlp � c � S = FIX (Ψ) for Ψ( T ) = ( B � x � = 0 ∧ x � = 1 � ∩ wlp � c 0 � T ) ∪ ( B � x ∈ { 0 , 1 } � ∩ S ) � �� � • wlp � c 0 � T = { σ ∈ Σ | σ [ x �→ σ ( x ) − 2 ] ∈ T } = S • Fixpoint iteration (with initial value � ∅ = Σ ): Ψ(Σ) = ( B � x � = 0 ∧ x � = 1 � ∩ wlp � c 0 � Σ) ∪ S = B � x � = 0 � Ψ 2 (Σ) = ( B � x � = 0 ∧ x � = 1 � ∩ wlp � c 0 � ( B � x � = 0 � )) ∪ S = B � x � = 0 ∧ x � = 2 � Ψ 3 (Σ) = ( B � x � = 0 ∧ x � = 1 � ∩ wlp � c 0 � ( B � x � = 0 ∧ x � = 2 � )) ∪ S = B � x � = 0 ∧ x � = 2 ∧ x � = 4 � . . . ⇒ FIX (Ψ) = � n ∈ N Ψ n (Σ) = { σ ∈ Σ | σ ( x ) ∈ Z < 0 ∪ { 1 , 3 , 5 , . . . }} 13 of 22 Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness)

  11. Relative Completeness of Hoare Logic Weakest Liberal Preconditions IV Definition 11.8 (Expressivity of assertion languages) An assertion language Assn is called expressive if it allows to “syntactify” weakest preconditions, that is, for every c ∈ Cmd and B ∈ Assn , there exists A c , B ∈ Assn c , B = wlp � c � B I for every I ∈ Int . such that A I Theorem 11.9 (Expressivity of Assn ) Assn is expressive. Proof (idea; see (Winskel 1996, p. 103 ff) for details). Given c ∈ Cmd and B ∈ Assn , construct A c , B ∈ Assn with = I A c , B ⇐ = I B (for every σ ∈ Σ , I ∈ Int ). For example: σ | ⇒ C � c � σ | A x := a , B := B [ x �→ a ] A skip , B := B A c 1 ; c 2 , B := A c 1 , A c 2 , B . . . (for while : “G¨ odelisation” of sequences of intermediate states) 14 of 22 Semantics and Verification of Software Summer Semester 2019 Lecture 11: Axiomatic Semantics of WHILE III (Completeness & Total Correctness)

Download Presentation
Download Policy: The content available on the website is offered to you 'AS IS' for your personal information and use only. It cannot be commercialized, licensed, or distributed on other websites without prior consent from the author. To download a presentation, simply click this link. If you encounter any difficulties during the download process, it's possible that the publisher has removed the file from their server.

Recommend


More recommend