Hoare2Hoare Logic, Part II
Set Warnings "-notation-overridden,-parsing".
From Coq Require Import Strings.String.
From PLF Require Import Maps.
From Coq Require Import Bool.Bool.
From Coq Require Import Arith.Arith.
From Coq Require Import Arith.EqNat.
From Coq Require Import Arith.PeanoNat. Import Nat.
From Coq Require Import omega.Omega.
From PLF Require Import Hoare.
From PLF Require Import Imp.
Decorated Programs
X ::= m;;
Z ::= p;
WHILE ~(X = 0) DO
Z ::= Z - 1;;
X ::= X - 1
END
{{ True }}
X ::= m;;
Z ::= p;
WHILE ~(X = 0) DO
Z ::= Z - 1;;
X ::= X - 1
END
{{ Z = p - m }}
{{ True }} ->>
{{ m = m }}
X ::= m;;
{{ X = m }} ->>
{{ X = m ∧ p = p }}
Z ::= p;
{{ X = m ∧ Z = p }} ->>
{{ Z - X = p - m }}
WHILE ~(X = 0) DO
{{ Z - X = p - m ∧ X ≠ 0 }} ->>
{{ (Z - 1) - (X - 1) = p - m }}
Z ::= Z - 1;;
{{ Z - (X - 1) = p - m }}
X ::= X - 1
{{ Z - X = p - m }}
END
{{ Z - X = p - m ∧ ¬(X ≠ 0) }} ->>
{{ Z = p - m }}
- 如果 SKIP 的前置条件和后置条件相同,则它是局部一致的:
{{ P }} SKIP {{ P }}
- 我们说 c1 和 c2 的顺序组合是局部一致的(相对于断言 P 和 R),
如果 c1 是局部一致的(相对于断言 P 和 Q)并且
c2 是局部一致的(相对于断言 Q 和 R):
{{ P }} c1;; {{ Q }} c2 {{ R }}
- 如果赋值语句的前置条件是其后置条件的适当替换,则该赋值语句是局部一致的:
{{ P [X ⊢> a] }}
X ::= a
{{ P }}
- 我们说一个条件语句是局部一致的 (相对于断言 P 和 Q) ,
如果它的 "then" 和 "else" 两个分支顶部的断言恰好是 P ∧ b 和 P ∧ ¬b,
并且 "then" 分支是局部一致的 (相对于断言 P ∧ b 和 Q)
且 "else" 分支是局部一致的 (相对于断言 P ∧ ¬b 和 Q):
{{ P }}
TEST b THEN
{{ P ∧ b }}
c1
{{ Q }}
ELSE
{{ P ∧ ¬b }}
c2
{{ Q }}
FI
{{ Q }}
- 我们说一个前置条件为 P 的 while 循环是局部一致的,
如果它的后置条件是 P ∧ ¬b,
并且如果它循环体的前置条件和后置条件是 P ∧ b 和 P,
并且它的循环体是局部一致的:
{{ P }}
WHILE b DO
{{ P ∧ b }}
c1
{{ P }}
END
{{ P ∧ ¬b }}
- 由蕴含符号 ->> 分隔的一对断言是局部一致的,如果前者蕴含后者:
{{ P }} ->>
{{ P' }}
示例:使用加法和减法实现交换操作
X ::= X + Y;;
Y ::= X - Y;;
X ::= X - Y
(1) {{ X = m ∧ Y = n }} ->>
(2) {{ (X + Y) - ((X + Y) - Y) = n ∧ (X + Y) - Y = m }}
X ::= X + Y;;
(3) {{ X - (X - Y) = n ∧ X - Y = m }}
Y ::= X - Y;;
(4) {{ X - Y = n ∧ Y = m }}
X ::= X - Y
(5) {{ X = n ∧ Y = m }}
- 我们以未装饰的程序开始 (即: 所有不带数字编号的行).
- 我们添加规格说明 -- 即: 最外部的前置条件 (1) 和后置条件 (5). 在前置条件中, 我们使用参数 m 和 n 来记住变量 X 和 Y 的初始值, 以便我们可以在后置条件中引用它们.
- 我们机械地从后向前进行, 从 (5) 开始处理直到 (2). 在每一步中, 我们从赋值语句的后置条件获得它的前置条件, 方式是将被赋值的变量替换为赋值语句的右值. 例如, 我们通过替换 (5) 中的 X 为 X - Y 而获得 (4), 然后, 我们通过替换 (4) 中的 Y 为 X - Y 而获得 (3).
- 最终, 我们验证 (1) 逻辑上蕴含 (2) -- 即: 由 (1) 到 (2) 的步骤
是对 '后果法则 (law of consequence)' 的合法运用.
为此我们替换 X 为 m, Y 为 n 并计算如下:
(m + n) - ((m + n) - n) = n ∧ (m + n) - n = m
(m + n) - m = n ∧ m = m
n = n ∧ m = m
Example: Simple Conditionals
(1) {{True}}
TEST X ≤ Y THEN
(2) {{True ∧ X ≤ Y}} ->>
(3) {{(Y - X) + X = Y ∨ (Y - X) + Y = X}}
Z ::= Y - X
(4) {{Z + X = Y ∨ Z + Y = X}}
ELSE
(5) {{True ∧ ~(X ≤ Y) }} ->>
(6) {{(X - Y) + X = Y ∨ (X - Y) + Y = X}}
Z ::= X - Y
(7) {{Z + X = Y ∨ Z + Y = X}}
FI
(8) {{Z + X = Y ∨ Z + Y = X}}
- 我们从最外部的前置条件 (1) 和后置条件 (8) 开始.
- 我们依据 hoare_if 规则所描述的形式, 将后置条件 (8) 拷贝到 (4) 和 (7). 我们合取前置条件 (1) 与分支条件以得到 (2). 我们合取前置条件 (1) 与否定分支条件以得到 (5).
- 为了使用赋值规则得到 (3), 我们替换 (4) 中的 Z 为 Y - X. 为了得到 (6) 我们替换 (7) 中的 Z 为 X - Y.
- 最终, 我们验证 (2) 蕴含 (3) 并且 (5) 蕴含 (6). 这两个蕴含关系都关键地依赖分支条件中提到的 X 和 Y 的顺序. 比如, 如果我们知道 X ≤ Y 那么就能确保在 Y 中 减去 X 再加回 X 仍然得到 Y, 这正是合取式 (3) 的左边. 类似的, 知道 ¬ (X ≤ Y) 能确保在 X 中 减去 Y 再加回 Y 仍然得到 X, 这正是合取式 (6) 的右边. 请注意 n - m + m = n 并 _不是_ 对任意的自然数 n 和 m 总成立的 (比如: 3 - 5 + 5 = 5).
练习:2 星, standard (if_minus_plus_reloaded)
为以下程序填上合法的装饰:{{ True }}
TEST X ≤ Y THEN
{{ }} ->>
{{ }}
Z ::= Y - X
{{ }}
ELSE
{{ }} ->>
{{ }}
Y ::= X + Z
{{ }}
FI
{{ Y = X + Z }}
(* 请勿修改下面这一行: *)
Definition manual_grade_for_decorations_in_if_minus_plus_reloaded : option (nat×string) := None.
☐
Example: Reduce to Zero
(1) {{ True }}
WHILE ~(X = 0) DO
(2) {{ True ∧ X ≠ 0 }} ->>
(3) {{ True }}
X ::= X - 1
(4) {{ True }}
END
(5) {{ True ∧ ~(X ≠ 0) }} ->>
(6) {{ X = 0 }}
- Start with the outer precondition (1) and postcondition (6).
- Following the format dictated by the hoare_while rule, we copy (1) to (4). We conjoin (1) with the guard to obtain (2). The guard is a Boolean expression ~(X = 0), which for simplicity we express in assertion (2) as X ≠ 0. We also conjoin (1) with the negation of the guard to obtain (5). Note that, because the outer postcondition (6) does not syntactically match (5), we need a trivial use of the consequence rule from (5) to (6).
- Assertion (3) is the same as (4), because X does not appear in 4, so the substitution in the assignment rule is trivial.
- Finally, the implication between (2) and (3) is also trivial.
Definition reduce_to_zero' : com :=
WHILE ~(X = 0) DO
X ::= X - 1
END.
Theorem reduce_to_zero_correct' :
{{True}}
reduce_to_zero'
{{X = 0}}.
Proof.
unfold reduce_to_zero'.
(* First we need to transform the postcondition so
that hoare_while will apply. *)
eapply hoare_consequence_post.
apply hoare_while.
- (* Loop body preserves invariant *)
(* Need to massage precondition before hoare_asgn applies *)
eapply hoare_consequence_pre. apply hoare_asgn.
(* Proving trivial implication (2) ->> (3) *)
intros st [HT Hbp]. unfold assn_sub. constructor.
- (* Invariant and negated guard imply postcondition *)
intros st [Inv GuardFalse].
unfold bassn in GuardFalse. simpl in GuardFalse.
rewrite not_true_iff_false in GuardFalse.
rewrite negb_false_iff in GuardFalse.
apply eqb_eq in GuardFalse.
apply GuardFalse. Qed.
unfold reduce_to_zero'.
(* First we need to transform the postcondition so
that hoare_while will apply. *)
eapply hoare_consequence_post.
apply hoare_while.
- (* Loop body preserves invariant *)
(* Need to massage precondition before hoare_asgn applies *)
eapply hoare_consequence_pre. apply hoare_asgn.
(* Proving trivial implication (2) ->> (3) *)
intros st [HT Hbp]. unfold assn_sub. constructor.
- (* Invariant and negated guard imply postcondition *)
intros st [Inv GuardFalse].
unfold bassn in GuardFalse. simpl in GuardFalse.
rewrite not_true_iff_false in GuardFalse.
rewrite negb_false_iff in GuardFalse.
apply eqb_eq in GuardFalse.
apply GuardFalse. Qed.
Example: Division
X ::= m;;
Y ::= 0;;
WHILE n ≤ X DO
X ::= X - n;;
Y ::= Y + 1
END;
(1) {{ True }} ->>
(2) {{ n × 0 + m = m }}
X ::= m;;
(3) {{ n × 0 + X = m }}
Y ::= 0;;
(4) {{ n × Y + X = m }}
WHILE n ≤ X DO
(5) {{ n × Y + X = m ∧ n ≤ X }} ->>
(6) {{ n × (Y + 1) + (X - n) = m }}
X ::= X - n;;
(7) {{ n × (Y + 1) + X = m }}
Y ::= Y + 1
(8) {{ n × Y + X = m }}
END
(9) {{ n × Y + X = m ∧ ¬(n ≤ X) }} ->>
(10) {{ n × Y + X = m ∧ X < n }}
Finding Loop Invariants
Example: Slow Subtraction
{{ X = m ∧ Y = n }}
WHILE ~(X = 0) DO
Y ::= Y - 1;;
X ::= X - 1
END
{{ Y = n - m }}
(1) {{ X = m ∧ Y = n }} ->> (a)
(2) {{ Inv }}
WHILE ~(X = 0) DO
(3) {{ Inv ∧ X ≠ 0 }} ->> (c)
(4) {{ Inv [X ⊢> X-1] [Y ⊢> Y-1] }}
Y ::= Y - 1;;
(5) {{ Inv [X ⊢> X-1] }}
X ::= X - 1
(6) {{ Inv }}
END
(7) {{ Inv ∧ ¬(X ≠ 0) }} ->> (b)
(8) {{ Y = n - m }}
- (a) it must be weak enough to be implied by the loop's precondition, i.e., (1) must imply (2);
- (b) it must be strong enough to imply the program's postcondition, i.e., (7) must imply (8);
- (c) it must be preserved by each iteration of the loop (given that the loop guard evaluates to true), i.e., (3) must imply (4).
(1) {{ X = m ∧ Y = n }} ->> (a - OK)
(2) {{ True }}
WHILE ~(X = 0) DO
(3) {{ True ∧ X ≠ 0 }} ->> (c - OK)
(4) {{ True }}
Y ::= Y - 1;;
(5) {{ True }}
X ::= X - 1
(6) {{ True }}
END
(7) {{ True ∧ ~(X ≠ 0) }} ->> (b - WRONG!)
(8) {{ Y = n - m }}
(1) {{ X = m ∧ Y = n }} ->> (a - WRONG!)
(2) {{ Y = n - m }}
WHILE ~(X = 0) DO
(3) {{ Y = n - m ∧ X ≠ 0 }} ->> (c - WRONG!)
(4) {{ Y - 1 = n - m }}
Y ::= Y - 1;;
(5) {{ Y = n - m }}
X ::= X - 1
(6) {{ Y = n - m }}
END
(7) {{ Y = n - m ∧ ~(X ≠ 0) }} ->> (b - OK)
(8) {{ Y = n - m }}
(1) {{ X = m ∧ Y = n }} ->> (a - OK)
(2) {{ Y - X = n - m }}
WHILE ~(X = 0) DO
(3) {{ Y - X = n - m ∧ X ≠ 0 }} ->> (c - OK)
(4) {{ (Y - 1) - (X - 1) = n - m }}
Y ::= Y - 1;;
(5) {{ Y - (X - 1) = n - m }}
X ::= X - 1
(6) {{ Y - X = n - m }}
END
(7) {{ Y - X = n - m ∧ ~(X ≠ 0) }} ->> (b - OK)
(8) {{ Y = n - m }}
Exercise: Slow Assignment
练习:2 星, standard (slow_assignment)
A roundabout way of assigning a number currently stored in X to the variable Y is to start Y at 0, then decrement X until it hits 0, incrementing Y at each step. Here is a program that implements this idea:{{ X = m }}
Y ::= 0;;
WHILE ~(X = 0) DO
X ::= X - 1;;
Y ::= Y + 1
END
{{ Y = m }}
(* 请在此处解答 *)
(* 请勿修改下面这一行: *)
Definition manual_grade_for_decorations_in_slow_assignment : option (nat×string) := None.
☐
Exercise: Slow Addition
练习:3 星, standard, optional (add_slowly_decoration)
The following program adds the variable X into the variable Z by repeatedly decrementing X and incrementing Z.WHILE ~(X = 0) DO
Z ::= Z + 1;;
X ::= X - 1
END
(* 请在此处解答 *)
☐
Example: Parity
{{ X = m }}
WHILE 2 ≤ X DO
X ::= X - 2
END
{{ X = parity m }}
The postcondition does not hold at the beginning of the loop,
since m = parity m does not hold for an arbitrary m, so we
cannot use that as an invariant. To find an invariant that works,
let's think a bit about what this loop does. On each iteration it
decrements X by 2, which preserves the parity of X. So the
parity of X does not change, i.e., it is invariant. The initial
value of X is m, so the parity of X is always equal to the
parity of m. Using parity X = parity m as an invariant we
obtain the following decorated program:
{{ X = m }} ->> (a - OK)
{{ parity X = parity m }}
WHILE 2 ≤ X DO
{{ parity X = parity m ∧ 2 ≤ X }} ->> (c - OK)
{{ parity (X-2) = parity m }}
X ::= X - 2
{{ parity X = parity m }}
END
{{ parity X = parity m ∧ ~(2 ≤ X) }} ->> (b - OK)
{{ X = parity m }}
With this invariant, conditions (a), (b), and (c) are all
satisfied. For verifying (b), we observe that, when X < 2, we
have parity X = X (we can easily see this in the definition of
parity). For verifying (c), we observe that, when 2 ≤ X, we
have parity X = parity (X-2).
{{ X = m }} ->> (a - OK)
{{ parity X = parity m }}
WHILE 2 ≤ X DO
{{ parity X = parity m ∧ 2 ≤ X }} ->> (c - OK)
{{ parity (X-2) = parity m }}
X ::= X - 2
{{ parity X = parity m }}
END
{{ parity X = parity m ∧ ~(2 ≤ X) }} ->> (b - OK)
{{ X = parity m }}
练习:3 星, standard, optional (parity_formal)
Translate the above informal decorated program into a formal proof in Coq. Your proof should use the Hoare logic rules and should not unfold hoare_triple. Refer to reduce_to_zero for an example. You might find the following lemmas to be useful:Lemma parity_ge_2 : ∀ x,
2 ≤ x →
parity (x - 2) = parity x.
Proof.
induction x; intro. reflexivity.
destruct x. inversion H. inversion H1.
simpl. rewrite <- minus_n_O. reflexivity.
Qed.
induction x; intro. reflexivity.
destruct x. inversion H. inversion H1.
simpl. rewrite <- minus_n_O. reflexivity.
Qed.
Lemma parity_lt_2 : ∀ x,
¬ 2 ≤ x →
parity x = x.
Proof.
intros. induction x. reflexivity. destruct x. reflexivity.
exfalso. apply H. omega.
Qed.
intros. induction x. reflexivity. destruct x. reflexivity.
exfalso. apply H. omega.
Qed.
Theorem parity_correct : ∀ (m:nat),
{{ X = m }}
WHILE 2 ≤ X DO
X ::= X - 2
END
{{ X = parity m }}.
Proof.
(* 请在此处解答 *) Admitted.
☐
Example: Finding Square Roots
{{ X=m }}
Z ::= 0;;
WHILE (Z+1)*(Z+1) ≤ X DO
Z ::= Z+1
END
{{ Z×Z≤m ∧ m<(Z+1)*(Z+1) }}
(1) {{ X=m }} ->> (a - second conjunct of (2) WRONG!)
(2) {{ 0*0 ≤ m ∧ m<(0+1)*(0+1) }}
Z ::= 0;;
(3) {{ Z×Z ≤ m ∧ m<(Z+1)*(Z+1) }}
WHILE (Z+1)*(Z+1) ≤ X DO
(4) {{ Z×Z≤m ∧ (Z+1)*(Z+1)<=X }} ->> (c - WRONG!)
(5) {{ (Z+1)*(Z+1)<=m ∧ m<((Z+1)+1)*((Z+1)+1) }}
Z ::= Z+1
(6) {{ Z×Z≤m ∧ m<(Z+1)*(Z+1) }}
END
(7) {{ Z×Z≤m ∧ m<(Z+1)*(Z+1) ∧ ~((Z+1)*(Z+1)<=X) }} ->> (b - OK)
(8) {{ Z×Z≤m ∧ m<(Z+1)*(Z+1) }}
{{ X=m }} ->> (a - OK)
{{ X=m ∧ 0*0 ≤ m }}
Z ::= 0;
{{ X=m ∧ Z×Z ≤ m }}
WHILE (Z+1)*(Z+1) ≤ X DO
{{ X=m ∧ Z×Z≤m ∧ (Z+1)*(Z+1)<=X }} ->> (c - OK)
{{ X=m ∧ (Z+1)*(Z+1)<=m }}
Z ::= Z + 1
{{ X=m ∧ Z×Z≤m }}
END
{{ X=m ∧ Z×Z≤m ∧ ~((Z+1)*(Z+1)<=X) }} ->> (b - OK)
{{ Z×Z≤m ∧ m<(Z+1)*(Z+1) }}
Example: Squaring
{{ X = m }}
Y ::= 0;;
Z ::= 0;;
WHILE ~(Y = X) DO
Z ::= Z + X;;
Y ::= Y + 1
END
{{ Z = m×m }}
{{ X = m }} ->> (a - WRONG)
{{ 0 = m×m ∧ X = m }}
Y ::= 0;;
{{ 0 = m×m ∧ X = m }}
Z ::= 0;;
{{ Z = m×m ∧ X = m }}
WHILE ~(Y = X) DO
{{ Z = m×m ∧ X = m ∧ Y ≠ X }} ->> (c - WRONG)
{{ Z+X = m×m ∧ X = m }}
Z ::= Z + X;;
{{ Z = m×m ∧ X = m }}
Y ::= Y + 1
{{ Z = m×m ∧ X = m }}
END
{{ Z = m×m ∧ X = m ∧ ~(Y ≠ X) }} ->> (b - OK)
{{ Z = m×m }}
{{ X = m }} ->> (a - OK)
{{ 0 = 0*m ∧ X = m }}
Y ::= 0;;
{{ 0 = Y×m ∧ X = m }}
Z ::= 0;;
{{ Z = Y×m ∧ X = m }}
WHILE ~(Y = X) DO
{{ Z = Y×m ∧ X = m ∧ Y ≠ X }} ->> (c - OK)
{{ Z+X = (Y+1)*m ∧ X = m }}
Z ::= Z + X;
{{ Z = (Y+1)*m ∧ X = m }}
Y ::= Y + 1
{{ Z = Y×m ∧ X = m }}
END
{{ Z = Y×m ∧ X = m ∧ ~(Y ≠ X) }} ->> (b - OK)
{{ Z = m×m }}
Exercise: Factorial
练习:3 星, standard (factorial)
Recall that n! denotes the factorial of n (i.e., n! = 1*2*...*n). Here is an Imp program that calculates the factorial of the number initially stored in the variable X and puts it in the variable Y:{{ X = m }}
Y ::= 1 ;;
WHILE ~(X = 0)
DO
Y ::= Y × X ;;
X ::= X - 1
END
{{ Y = m! }}
{{ X = m }} ->>
{{ }}
Y ::= 1;;
{{ }}
WHILE ~(X = 0)
DO {{ }} ->>
{{ }}
Y ::= Y × X;;
{{ }}
X ::= X - 1
{{ }}
END
{{ }} ->>
{{ Y = m! }}
(* 请勿修改下面这一行: *)
Definition manual_grade_for_decorations_in_factorial : option (nat×string) := None.
☐
Exercise: Min
练习:3 星, standard (Min_Hoare)
Lemma lemma1 : ∀ x y,
(x<>0 ∧ y<>0) → min x y ≠ 0.
Lemma lemma2 : ∀ x y,
min (x-1) (y-1) = (min x y) - 1.
{{ True }} ->>
{{ }}
X ::= a;;
{{ }}
Y ::= b;;
{{ }}
Z ::= 0;;
{{ }}
WHILE ~(X = 0) && ~(Y = 0) DO
{{ }} ->>
{{ }}
X := X - 1;;
{{ }}
Y := Y - 1;;
{{ }}
Z := Z + 1
{{ }}
END
{{ }} ->>
{{ Z = min a b }}
(* 请勿修改下面这一行: *)
Definition manual_grade_for_decorations_in_Min_Hoare : option (nat×string) := None.
☐
练习:3 星, standard (two_loops)
Here is a very inefficient way of adding 3 numbers:X ::= 0;;
Y ::= 0;;
Z ::= c;;
WHILE ~(X = a) DO
X ::= X + 1;;
Z ::= Z + 1
END;;
WHILE ~(Y = b) DO
Y ::= Y + 1;;
Z ::= Z + 1
END
{{ True }} ->>
{{ }}
X ::= 0;;
{{ }}
Y ::= 0;;
{{ }}
Z ::= c;;
{{ }}
WHILE ~(X = a) DO
{{ }} ->>
{{ }}
X ::= X + 1;;
{{ }}
Z ::= Z + 1
{{ }}
END;;
{{ }} ->>
{{ }}
WHILE ~(Y = b) DO
{{ }} ->>
{{ }}
Y ::= Y + 1;;
{{ }}
Z ::= Z + 1
{{ }}
END
{{ }} ->>
{{ Z = a + b + c }}
(* 请勿修改下面这一行: *)
Definition manual_grade_for_decorations_in_two_loops : option (nat×string) := None.
☐
Exercise: Power Series
练习:4 星, standard, optional (dpow2_down)
Here is a program that computes the series: 1 + 2 + 2^2 + ... + 2^m = 2^(m+1) - 1X ::= 0;;
Y ::= 1;;
Z ::= 1;;
WHILE ~(X = m) DO
Z ::= 2 × Z;;
Y ::= Y + Z;;
X ::= X + 1
END
(* 请在此处解答 *)
☐
Weakest Preconditions (Optional)
{{ False }} X ::= Y + 1 {{ X ≤ 5 }}
{{ Y ≤ 4 ∧ Z = 0 }} X ::= Y + 1 {{ X ≤ 5 }}
{{ Y ≤ 4 }} X ::= Y + 1 {{ X ≤ 5 }}
That is, P is the weakest precondition of c for Q
if (a) P is a precondition for Q and c, and (b) P is the
weakest (easiest to satisfy) assertion that guarantees that
Q will hold after executing c.
1) {{ ? }} SKIP {{ X = 5 }}
2) {{ ? }} X ::= Y + Z {{ X = 5 }}
3) {{ ? }} X ::= Y {{ X = Y }}
4) {{ ? }}
TEST X = 0 THEN Y ::= Z + 1 ELSE Y ::= W + 2 FI
{{ Y = 5 }}
5) {{ ? }}
X ::= 5
{{ X = 0 }}
6) {{ ? }}
WHILE true DO X ::= 0 END
{{ X = 0 }}
练习:1 星, standard, optional (wp)
What are the weakest preconditions of the following commands for the following postconditions?1) {{ ? }} SKIP {{ X = 5 }}
2) {{ ? }} X ::= Y + Z {{ X = 5 }}
3) {{ ? }} X ::= Y {{ X = Y }}
4) {{ ? }}
TEST X = 0 THEN Y ::= Z + 1 ELSE Y ::= W + 2 FI
{{ Y = 5 }}
5) {{ ? }}
X ::= 5
{{ X = 0 }}
6) {{ ? }}
WHILE true DO X ::= 0 END
{{ X = 0 }}
(* 请在此处解答 *)
☐
☐
练习:3 星, advanced, optional (is_wp_formal)
Prove formally, using the definition of hoare_triple, that Y ≤ 4 is indeed the weakest precondition of X ::= Y + 1 with respect to postcondition X ≤ 5.练习:2 星, advanced, optional (hoare_asgn_weakest)
Show that the precondition in the rule hoare_asgn is in fact the weakest precondition.Theorem hoare_asgn_weakest : ∀ Q X a,
is_wp (Q [X ⊢> a]) (X ::= a) Q.
Proof.
(* 请在此处解答 *) Admitted.
☐
练习:2 星, advanced, optional (hoare_havoc_weakest)
Show that your havoc_pre rule from the himp_hoare exercise in the Hoare chapter returns the weakest precondition.
Module Himp2.
Import Himp.
Lemma hoare_havoc_weakest : ∀ (P Q : Assertion) (X : string),
{{ P }} HAVOC X {{ Q }} →
P ->> havoc_pre X Q.
Proof.
(* 请在此处解答 *) Admitted.
☐
Import Himp.
Lemma hoare_havoc_weakest : ∀ (P Q : Assertion) (X : string),
{{ P }} HAVOC X {{ Q }} →
P ->> havoc_pre X Q.
Proof.
(* 请在此处解答 *) Admitted.
☐
Formal Decorated Programs (Advanced)
Syntax
{{P}} ({{P}} SKIP {{P}}) ;; ({{P}} SKIP {{P}}) {{P}},
- The post-condition expected by each dcom d is embedded
in d.
- The pre-condition is supplied by the context.
Inductive dcom : Type :=
| DCSkip : Assertion → dcom
| DCSeq : dcom → dcom → dcom
| DCAsgn : string → aexp → Assertion → dcom
| DCIf : bexp → Assertion → dcom → Assertion → dcom
→ Assertion→ dcom
| DCWhile : bexp → Assertion → dcom → Assertion → dcom
| DCPre : Assertion → dcom → dcom
| DCPost : dcom → Assertion → dcom.
DCPre is used to provide the weakened precondition from
the rule of consequence. To provide the initial precondition
at the very top of the program, we use Decorated:
To avoid clashing with the existing Notation definitions for
ordinary commands, we introduce these notations in a special
scope called dcom_scope, and we Open this scope for the
remainder of the file.
Delimit Scope default with default.
Notation "'SKIP' {{ P }}"
:= (DCSkip P)
(at level 10) : dcom_scope.
Notation "l '::=' a {{ P }}"
:= (DCAsgn l a P)
(at level 60, a at next level) : dcom_scope.
Notation "'WHILE' b 'DO' {{ Pbody }} d 'END' {{ Ppost }}"
:= (DCWhile b Pbody d Ppost)
(at level 80, right associativity) : dcom_scope.
Notation "'TEST' b 'THEN' {{ P }} d 'ELSE' {{ P' }} d' 'FI' {{ Q }}"
:= (DCIf b P d P' d' Q)
(at level 80, right associativity) : dcom_scope.
Notation "'->>' {{ P }} d"
:= (DCPre P d)
(at level 90, right associativity) : dcom_scope.
Notation "d '->>' {{ P }}"
:= (DCPost d P)
(at level 80, right associativity) : dcom_scope.
Notation " d ;; d' "
:= (DCSeq d d')
(at level 80, right associativity) : dcom_scope.
Notation "{{ P }} d"
:= (Decorated P d)
(at level 90) : dcom_scope.
Delimit Scope dcom_scope with dcom.
Open Scope dcom_scope.
Example dec0 :=
SKIP {{ True }}.
Example dec1 :=
WHILE true DO {{ True }} SKIP {{ True }} END
{{ True }}.
(* Set Printing All. *)
Example dec_while : decorated :=
{{ True }}
WHILE ~(X = 0)
DO
{{ True ∧ (X ≠ 0) }}
X ::= X - 1
{{ True }}
END
{{ True ∧ X = 0}} ->>
{{ X = 0 }}.
Notation "'SKIP' {{ P }}"
:= (DCSkip P)
(at level 10) : dcom_scope.
Notation "l '::=' a {{ P }}"
:= (DCAsgn l a P)
(at level 60, a at next level) : dcom_scope.
Notation "'WHILE' b 'DO' {{ Pbody }} d 'END' {{ Ppost }}"
:= (DCWhile b Pbody d Ppost)
(at level 80, right associativity) : dcom_scope.
Notation "'TEST' b 'THEN' {{ P }} d 'ELSE' {{ P' }} d' 'FI' {{ Q }}"
:= (DCIf b P d P' d' Q)
(at level 80, right associativity) : dcom_scope.
Notation "'->>' {{ P }} d"
:= (DCPre P d)
(at level 90, right associativity) : dcom_scope.
Notation "d '->>' {{ P }}"
:= (DCPost d P)
(at level 80, right associativity) : dcom_scope.
Notation " d ;; d' "
:= (DCSeq d d')
(at level 80, right associativity) : dcom_scope.
Notation "{{ P }} d"
:= (Decorated P d)
(at level 90) : dcom_scope.
Delimit Scope dcom_scope with dcom.
Open Scope dcom_scope.
Example dec0 :=
SKIP {{ True }}.
Example dec1 :=
WHILE true DO {{ True }} SKIP {{ True }} END
{{ True }}.
(* Set Printing All. *)
Example dec_while : decorated :=
{{ True }}
WHILE ~(X = 0)
DO
{{ True ∧ (X ≠ 0) }}
X ::= X - 1
{{ True }}
END
{{ True ∧ X = 0}} ->>
{{ X = 0 }}.
It is easy to go from a dcom to a com by erasing all
annotations.
Fixpoint extract (d : dcom) : com :=
match d with
| DCSkip _ ⇒ SKIP
| DCSeq d1 d2 ⇒ (extract d1 ;; extract d2)
| DCAsgn X a _ ⇒ X ::= a
| DCIf b _ d1 _ d2 _ ⇒ TEST b THEN extract d1 ELSE extract d2 FI
| DCWhile b _ d _ ⇒ WHILE b DO extract d END
| DCPre _ d ⇒ extract d
| DCPost d _ ⇒ extract d
end.
Definition extract_dec (dec : decorated) : com :=
match dec with
| Decorated P d ⇒ extract d
end.
Print dec_while.
(*
dec_while =
{{fun _ : state => True}} (WHILE ~ X = 0
DO {{fun st : state => True /\ st X <> 0}}
X ::= X - 1 {{fun _ : state => True}}
END {{fun st : state => True /\ st X = 0}}) ->>
{{fun st : state => st X = 0}}
: decorated
*)
Compute (extract_dec dec_while).
(*
= (WHILE ~ "X"string - 1 END)*)
It is straightforward to extract the precondition and
postcondition from a decorated program.
Fixpoint post (d : dcom) : Assertion :=
match d with
| DCSkip P ⇒ P
| DCSeq d1 d2 ⇒ post d2
| DCAsgn X a Q ⇒ Q
| DCIf _ _ d1 _ d2 Q ⇒ Q
| DCWhile b Pbody c Ppost ⇒ Ppost
| DCPre _ d ⇒ post d
| DCPost c Q ⇒ Q
end.
Definition pre_dec (dec : decorated) : Assertion :=
match dec with
| Decorated P d ⇒ P
end.
Definition post_dec (dec : decorated) : Assertion :=
match dec with
| Decorated P d ⇒ post d
end.
Print dec_while.
(*
dec_while =
{{fun _ : state => True}} (WHILE ~ X = 0
DO {{fun st : state => True /\ st X <> 0}}
X ::= X - 1 {{fun _ : state => True}}
END {{fun st : state => True /\ st X = 0}}) ->>
{{fun st : state => st X = 0}}
: decorated
*)
Compute pre_dec dec_while.
(*
= fun _ : state => True
: Assertion
*)
Compute post_dec dec_while.
(*
= fun x : state => x "X"*)
We can express what it means for a decorated program to be
correct as follows:
Definition dec_correct (dec : decorated) :=
{{pre_dec dec}} (extract_dec dec) {{post_dec dec}}.
Example dec_while_triple_correct :
dec_correct dec_while
= {{ fun st ⇒ True }}
(WHILE ~(X = 0) DO X ::= X - 1 END)%imp
{{ fun st ⇒ st X = 0 }}.
Proof. reflexivity. Qed.
To check whether this Hoare triple is valid, we need a way to
extract the "proof obligations" from a decorated program. These
obligations are often called verification conditions, because
they are the facts that must be verified to see that the
decorations are logically consistent and thus constitute a proof
of correctness.
The function verification_conditions takes a dcom d together
with a precondition P and returns a proposition that, if it
can be proved, implies that the triple {{P}} (extract d) {{post d}}
is valid.
It does this by walking over d and generating a big
conjunction including all the "local checks" that we listed when
we described the informal rules for decorated programs. (Strictly
speaking, we need to massage the informal rules a little bit to
add some uses of the rule of consequence, but the correspondence
should be clear.)
Extracting Verification Conditions
Fixpoint verification_conditions (P : Assertion) (d : dcom) : Prop :=
match d with
| DCSkip Q ⇒
(P ->> Q)
| DCSeq d1 d2 ⇒
verification_conditions P d1
∧ verification_conditions (post d1) d2
| DCAsgn X a Q ⇒
(P ->> Q [X ⊢> a])
| DCIf b P1 d1 P2 d2 Q ⇒
((P ∧ b) ->> P1)%assertion
∧ ((P ∧ ¬ b) ->> P2)%assertion
∧ (post d1 ->> Q) ∧ (post d2 ->> Q)
∧ verification_conditions P1 d1
∧ verification_conditions P2 d2
| DCWhile b Pbody d Ppost ⇒
(* post d is the loop invariant and the initial
precondition *)
(P ->> post d)
∧ ((post d ∧ b) ->> Pbody)%assertion
∧ ((post d ∧ ¬ b) ->> Ppost)%assertion
∧ verification_conditions Pbody d
| DCPre P' d ⇒
(P ->> P') ∧ verification_conditions P' d
| DCPost d Q ⇒
verification_conditions P d ∧ (post d ->> Q)
end.
And now the key theorem, stating that verification_conditions
does its job correctly. Not surprisingly, we need to use each of
the Hoare Logic rules at some point in the proof.
Theorem verification_correct : ∀ d P,
verification_conditions P d → {{P}} (extract d) {{post d}}.
Proof.
induction d; intros P H; simpl in ×.
- (* Skip *)
eapply hoare_consequence_pre.
apply hoare_skip.
assumption.
- (* Seq *)
destruct H as [H1 H2].
eapply hoare_seq.
apply IHd2. apply H2.
apply IHd1. apply H1.
- (* Asgn *)
eapply hoare_consequence_pre.
apply hoare_asgn.
assumption.
- (* If *)
destruct H as [HPre1 [HPre2 [Hd1 [Hd2 [HThen HElse]]]]].
apply IHd1 in HThen. clear IHd1.
apply IHd2 in HElse. clear IHd2.
apply hoare_if.
+ eapply hoare_consequence_post with (Q':=post d1); eauto.
eapply hoare_consequence_pre; eauto.
+ eapply hoare_consequence_post with (Q':=post d2); eauto.
eapply hoare_consequence_pre; eauto.
- (* While *)
destruct H as [Hpre [Hbody1 [Hpost1 Hd]]].
eapply hoare_consequence_pre; eauto.
eapply hoare_consequence_post; eauto.
apply hoare_while.
eapply hoare_consequence_pre; eauto.
- (* Pre *)
destruct H as [HP Hd].
eapply hoare_consequence_pre. apply IHd. apply Hd. assumption.
- (* Post *)
destruct H as [Hd HQ].
eapply hoare_consequence_post. apply IHd. apply Hd. assumption.
Qed.
induction d; intros P H; simpl in ×.
- (* Skip *)
eapply hoare_consequence_pre.
apply hoare_skip.
assumption.
- (* Seq *)
destruct H as [H1 H2].
eapply hoare_seq.
apply IHd2. apply H2.
apply IHd1. apply H1.
- (* Asgn *)
eapply hoare_consequence_pre.
apply hoare_asgn.
assumption.
- (* If *)
destruct H as [HPre1 [HPre2 [Hd1 [Hd2 [HThen HElse]]]]].
apply IHd1 in HThen. clear IHd1.
apply IHd2 in HElse. clear IHd2.
apply hoare_if.
+ eapply hoare_consequence_post with (Q':=post d1); eauto.
eapply hoare_consequence_pre; eauto.
+ eapply hoare_consequence_post with (Q':=post d2); eauto.
eapply hoare_consequence_pre; eauto.
- (* While *)
destruct H as [Hpre [Hbody1 [Hpost1 Hd]]].
eapply hoare_consequence_pre; eauto.
eapply hoare_consequence_post; eauto.
apply hoare_while.
eapply hoare_consequence_pre; eauto.
- (* Pre *)
destruct H as [HP Hd].
eapply hoare_consequence_pre. apply IHd. apply Hd. assumption.
- (* Post *)
destruct H as [Hd HQ].
eapply hoare_consequence_post. apply IHd. apply Hd. assumption.
Qed.
Now that all the pieces are in place, we can verify an entire program.
Definition verification_conditions_dec (dec : decorated) : Prop :=
match dec with
| Decorated P d ⇒ verification_conditions P d
end.
Corollary verification_correct_dec : ∀ dec,
verification_conditions_dec dec → dec_correct dec.
Proof.
intros [P d]. apply verification_correct.
Qed.
The propositions generated by verification_conditions are fairly
big, and they contain many conjuncts that are essentially trivial.
===>
(((fun _ : state ⇒ True) ->> (fun _ : state ⇒ True)) ∧
((fun st : state ⇒ True ∧ bassn (~(X = 0)) st) ->>
(fun st : state ⇒ True ∧ st X ≠ 0)) ∧
((fun st : state ⇒ True ∧ ¬bassn (~(X = 0)) st) ->>
(fun st : state ⇒ True ∧ st X = 0)) ∧
(fun st : state ⇒ True ∧ st X ≠ 0) ->>
(fun _ : state ⇒ True) [X ⊢> X - 1]) ∧
(fun st : state ⇒ True ∧ st X = 0) ->>
(fun st : state ⇒ st X = 0)
Automation
Tactic Notation "verify" :=
apply verification_correct;
repeat split;
simpl; unfold assert_implies;
unfold ap in *; unfold ap2 in *; unfold bassn in *; unfold beval in *; unfold aeval in *;
unfold assn_sub; intros;
repeat (simpl in *;
rewrite t_update_eq ||
(try rewrite t_update_neq; [| (intro X; inversion X; fail)]));
simpl in *;
repeat match goal with [H : _ ∧ _ ⊢ _] ⇒ destruct H end;
repeat rewrite not_true_iff_false in *;
repeat rewrite not_false_iff_true in *;
repeat rewrite negb_true_iff in *;
repeat rewrite negb_false_iff in *;
repeat rewrite eqb_eq in *;
repeat rewrite eqb_neq in *;
repeat rewrite leb_iff in *;
repeat rewrite leb_iff_conv in *;
try subst;
simpl in *;
repeat
match goal with
[st : state ⊢ _] ⇒
match goal with
| [H : st _ = _ ⊢ _] ⇒ rewrite → H in *; clear H
| [H : _ = st _ ⊢ _] ⇒ rewrite <- H in *; clear H
end
end;
try eauto; try omega.
What's left after verify does its thing is "just the interesting
parts" of checking that the decorations are correct. For very
simple examples, verify sometimes even immediately solves the
goal (provided that the annotations are correct!).
Examples
Slow Subtraction
Example subtract_slowly_dec (m : nat) (p : nat) : decorated :=
{{ X = m ∧ Z = p }} ->>
{{ Z - X = p - m }}
WHILE ~(X = 0)
DO {{ Z - X = p - m ∧ X ≠ 0 }} ->>
{{ (Z - 1) - (X - 1) = p - m }}
Z ::= Z - 1
{{ Z - (X - 1) = p - m }} ;;
X ::= X - 1
{{ Z - X = p - m }}
END
{{ Z - X = p - m ∧ X = 0 }} ->>
{{ Z = p - m }}.
Theorem subtract_slowly_dec_correct : ∀ m p,
dec_correct (subtract_slowly_dec m p).
Proof. intros m p. verify. (* this grinds for a bit! *) Qed.
Definition swap : com :=
X ::= X + Y;;
Y ::= X - Y;;
X ::= X - Y.
Definition swap_dec (m n:nat) : decorated :=
{{ X = m ∧ Y = n}} ->>
{{ (X + Y) - ((X + Y) - Y) = n
∧ (X + Y) - Y = m }}
X ::= X + Y
{{ X - (X - Y) = n ∧ X - Y = m }};;
Y ::= X - Y
{{ X - Y = n ∧ Y = m }};;
X ::= X - Y
{{ X = n ∧ Y = m}}.
Theorem swap_correct : ∀ m n,
dec_correct (swap_dec m n).
Proof. intros; verify. Qed.
MRC hid some proofs here so as not to spoil earlier exercises.
Consider the pros and cons of this.
Division
Definition div_mod_dec (a b : nat) : decorated :=
{{ True }} ->>
{{ b × 0 + a = a }}
X ::= a
{{ b × 0 + X = a }};;
Y ::= 0
{{ b × Y + X = a }};;
WHILE b ≤ X DO
{{ b × Y + X = a ∧ b ≤ X }} ->>
{{ b × (Y + 1) + (X - b) = a }}
X ::= X - b
{{ b × (Y + 1) + X = a }};;
Y ::= Y + 1
{{ b × Y + X = a }}
END
{{ b × Y + X = a ∧ ~(b ≤ X) }} ->>
{{ b × Y + X = a ∧ (X < b) }}.
Theorem div_mod_dec_correct : ∀ a b,
dec_correct (div_mod_dec a b).
Proof. intros a b. verify.
rewrite mult_plus_distr_l. omega.
Qed.
There are actually several ways to phrase the loop invariant for
this program. Here is one natural one, which leads to a rather
long proof:
Inductive ev : nat → Prop :=
| ev_0 : ev O
| ev_SS : ∀ n : nat, ev n → ev (S (S n)).
Definition find_parity_dec (m:nat) : decorated :=
{{ X = m }} ->>
{{ X ≤ m ∧ ap ev (m - X) }}
WHILE 2 ≤ X DO
{{ (X ≤ m ∧ ap ev (m - X)) ∧ 2 ≤ X }} ->>
{{ X - 2 ≤ m ∧ ap ev (m - (X - 2)) }}
X ::= X - 2
{{ X ≤ m ∧ ap ev (m - X) }}
END
{{ (X ≤ m ∧ ap ev (m - X)) ∧ X < 2 }} ->>
{{ X = 0 ↔ ev m }}.
Lemma l1 : ∀ m n p,
p ≤ n →
n ≤ m →
m - (n - p) = m - n + p.
Proof. intros. omega. Qed.
Lemma l2 : ∀ m,
ev m →
ev (m + 2).
Proof. intros. rewrite plus_comm. simpl. constructor. assumption. Qed.
Lemma l3' : ∀ m,
ev m →
¬ev (S m).
Proof. induction m; intros H1 H2. inversion H2. apply IHm.
inversion H2; subst; assumption. assumption. Qed.
Lemma l3 : ∀ m,
1 ≤ m →
ev m →
ev (m - 1) →
False.
Proof. intros. apply l2 in H1.
assert (G : m - 1 + 2 = S m). clear H0 H1. omega.
rewrite G in H1. apply l3' in H0. apply H0. assumption. Qed.
Theorem find_parity_correct : ∀ m,
dec_correct (find_parity_dec m).
Proof.
intro m. verify;
(* simplification too aggressive ... reverting a bit *)
fold (2 <=? (st X)) in *;
try rewrite leb_iff in *;
try rewrite leb_iff_conv in *; eauto; try omega.
- (* invariant holds initially *)
rewrite minus_diag. constructor.
- (* invariant preserved *)
rewrite l1; try assumption.
apply l2; assumption.
- (* invariant strong enough to imply conclusion
(-> direction) *)
rewrite <- minus_n_O in H2. assumption.
- (* invariant strong enough to imply conclusion
(<- direction) *)
destruct (st X) as [| [| n]].
(* by H1 X can only be 0 or 1 *)
+ (* st X = 0 *)
reflexivity.
+ (* st X = 1 *)
apply l3 in H; try assumption. inversion H.
+ (* st X = 2 *)
clear H0 H2. (* omega confused otherwise *)
omega.
Qed.
Here is a more intuitive way of writing the invariant:
Definition find_parity_dec' (m:nat) : decorated :=
{{ X = m }} ->>
{{ ap ev X ↔ ev m }}
WHILE 2 ≤ X DO
{{ (ap ev X ↔ ev m) ∧ 2 ≤ X }} ->>
{{ ap ev (X - 2) ↔ ev m }}
X ::= X - 2
{{ ap ev X ↔ ev m }}
END
{{ (ap ev X ↔ ev m) ∧ ~(2 ≤ X) }} ->>
{{ X=0 ↔ ev m }}.
Lemma l4 : ∀ m,
2 ≤ m →
(ev (m - 2) ↔ ev m).
Proof.
induction m; intros. split; intro; constructor.
destruct m. inversion H. inversion H1. simpl in ×.
rewrite <- minus_n_O in ×. split; intro.
constructor. assumption.
inversion H0. assumption.
Qed.
Theorem find_parity_correct' : ∀ m,
dec_correct (find_parity_dec' m).
Proof.
intros m. verify;
(* simplification too aggressive ... reverting a bit *)
fold (2 <=? (st X)) in *;
try rewrite leb_iff in *;
try rewrite leb_iff_conv in *; intuition; eauto; try omega.
- (* invariant preserved (part 1) *)
rewrite l4 in H0; eauto.
- (* invariant preserved (part 2) *)
rewrite l4; eauto.
- (* invariant strong enough to imply conclusion
(-> direction) *)
apply H0. constructor.
- (* invariant strong enough to imply conclusion
(<- direction) *)
destruct (st X) as [| [| n]]. (* by H1 X can only be 0 or 1 *)
+ (* st X = 0 *)
reflexivity.
+ (* st X = 1 *)
inversion H.
+ (* st X = 2 *)
clear H0 H H3. (* omega confused otherwise *)
omega.
Qed.
Definition sqrt_dec (m:nat) : decorated :=
{{ X = m }} ->>
{{ X = m ∧ 0×0 ≤ m }}
Z ::= 0
{{ X = m ∧ Z×Z ≤ m }};;
WHILE (Z+1)*(Z+1) ≤ X DO
{{ (X = m ∧ Z×Z≤m)
∧ (Z + 1)*(Z + 1) ≤ X }} ->>
{{ X = m ∧ (Z+1)*(Z+1)≤m }}
Z ::= Z + 1
{{ X = m ∧ Z×Z≤m }}
END
{{ (X = m ∧ Z×Z≤m)
∧ ~((Z + 1)*(Z + 1) ≤ X) }} ->>
{{ Z×Z≤m ∧ m<(Z+1)*(Z+1) }}.
Theorem sqrt_correct : ∀ m,
dec_correct (sqrt_dec m).
Proof. intro m. verify. Qed.
Squaring
Definition square_dec (m : nat) : decorated :=
{{ X = m }}
Y ::= X
{{ X = m ∧ Y = m }};;
Z ::= 0
{{ X = m ∧ Y = m ∧ Z = 0}} ->>
{{ Z + X × Y = m × m }};;
WHILE ¬ (Y = 0) DO
{{ Z + X × Y = m × m ∧ Y ≠ 0 }} ->>
{{ (Z + X) + X × (Y - 1) = m × m }}
Z ::= Z + X
{{ Z + X × (Y - 1) = m × m }};;
Y ::= Y - 1
{{ Z + X × Y = m × m }}
END
{{ Z + X × Y = m × m ∧ Y = 0 }} ->>
{{ Z = m × m }}.
Theorem square_dec_correct : ∀ m,
dec_correct (square_dec m).
Proof.
intro n. verify.
- (* invariant preserved *)
destruct (st Y) as [| y'].
+ exfalso. auto.
+ simpl. rewrite <- minus_n_O.
assert (G : ∀ n m, n × S m = n + n × m). {
clear. intros. induction n. reflexivity. simpl.
rewrite IHn. omega. }
rewrite <- H. rewrite G. omega.
Qed.
Definition square_dec' (n : nat) : decorated :=
{{ True }}
X ::= n
{{ X = n }};;
Y ::= X
{{ X = n ∧ Y = n }};;
Z ::= 0
{{ X = n ∧ Y = n ∧ Z = 0 }} ->>
{{ Z = X × (X - Y)
∧ X = n ∧ Y ≤ X }};;
WHILE ~(Y = 0) DO
{{ (Z = X × (X - Y)
∧ X = n ∧ Y ≤ X)
∧ Y ≠ 0 }}
Z ::= Z + X
{{ Z = X × (X - (Y - 1))
∧ X = n ∧ Y ≤ X }};;
Y ::= Y - 1
{{ Z = X × (X - Y)
∧ X = n ∧ Y ≤ X }}
END
{{ (Z = X × (X - Y)
∧ X = n ∧ Y ≤ X)
∧ Y = 0 }} ->>
{{ Z = n × n }}.
Theorem square_dec'_correct : ∀ (n:nat),
dec_correct (square_dec' n).
Proof.
intro n. verify.
- (* invariant holds initially *)
rewrite minus_diag. omega.
- (* invariant preserved *) subst.
rewrite mult_minus_distr_l.
repeat rewrite mult_minus_distr_l. rewrite mult_1_r.
assert (G : ∀ n m p,
m ≤ n → p ≤ m → n - (m - p) = n - m + p).
intros. omega.
rewrite G. reflexivity. apply mult_le_compat_l. assumption.
destruct (st Y).
+ exfalso. auto.
+ clear. rewrite mult_succ_r. rewrite plus_comm.
apply le_plus_l.
- (* invariant + negation of guard imply
desired postcondition *)
rewrite <- minus_n_O. reflexivity.
Qed.
Definition square_simpler_dec (m : nat) : decorated :=
{{ X = m }} ->>
{{ 0 = 0×m ∧ X = m }}
Y ::= 0
{{ 0 = Y×m ∧ X = m }};;
Z ::= 0
{{ Z = Y×m ∧ X = m }};;
WHILE ~(Y = X) DO
{{ (Z = Y×m ∧ X = m)
∧ Y ≠ X }} ->>
{{ Z + X = (Y + 1)*m ∧ X = m }}
Z ::= Z + X
{{ Z = (Y + 1)*m ∧ X = m }};;
Y ::= Y + 1
{{ Z = Y×m ∧ X = m }}
END
{{ (Z = Y×m ∧ X = m) ∧ Y = X }} ->>
{{ Z = m×m }}.
Theorem square_simpler_dec_correct : ∀ m,
dec_correct (square_simpler_dec m).
Proof.
intro m. verify.
rewrite mult_plus_distr_r. omega.
Qed.
Fixpoint pow2 n :=
match n with
| 0 ⇒ 1
| S n' ⇒ 2 × (pow2 n')
end.
Definition dpow2_down (n : nat) :=
{{ True }} ->>
{{ 1 = (pow2 (0 + 1))-1 ∧ 1 = pow2 0 }}
X ::= 0
{{ 1 = (pow2 (0 + 1))-1 ∧ 1 = ap pow2 X }};;
Y ::= 1
{{ Y = (ap pow2 (X + 1))-1 ∧ 1 = ap pow2 X}};;
Z ::= 1
{{ Y = (ap pow2 (X + 1))-1 ∧ Z = ap pow2 X }};;
WHILE ~(X = n) DO
{{ (Y = (ap pow2 (X + 1))-1 ∧ Z = ap pow2 X)
∧ X ≠ n }} ->>
{{ Y + 2 × Z = (ap pow2 (X + 2))-1
∧ 2 × Z = ap pow2 (X + 1) }}
Z ::= 2 × Z
{{ Y + Z = (ap pow2 (X + 2))-1
∧ Z = ap pow2 (X + 1) }};;
Y ::= Y + Z
{{ Y = (ap pow2 (X + 2))-1
∧ Z = ap pow2 (X + 1) }};;
X ::= X + 1
{{ Y = (ap pow2 (X + 1))-1
∧ Z = ap pow2 X }}
END
{{ (Y = (ap pow2 (X + 1))-1 ∧ Z = ap pow2 X)
∧ X = n }} ->>
{{ Y = pow2 (n+1) - 1 }}.
Lemma pow2_plus_1 : ∀ n,
pow2 (n+1) = pow2 n + pow2 n.
Proof. induction n; simpl. reflexivity. omega. Qed.
Lemma pow2_le_1 : ∀ n, pow2 n ≥ 1.
Proof. induction n. simpl. constructor. simpl. omega. Qed.
Theorem dpow2_down_correct : ∀ n,
dec_correct (dpow2_down n).
Proof.
intro m. verify.
- (* 1 *)
rewrite pow2_plus_1. rewrite <- H0. reflexivity.
- (* 2 *)
rewrite <- plus_n_O.
rewrite <- pow2_plus_1. remember (st X) as n.
replace (pow2 (n + 1) - 1 + pow2 (n + 1))
with (pow2 (n + 1) + pow2 (n + 1) - 1) by omega.
rewrite <- pow2_plus_1.
replace (n + 1 + 1) with (n + 2) by omega.
reflexivity.
- (* 3 *)
rewrite <- plus_n_O. rewrite <- pow2_plus_1.
reflexivity.
- (* 4 *)
replace (st X + 1 + 1) with (st X + 2) by omega.
reflexivity.
Qed.
Further Exercises
练习:3 星, advanced (slow_assignment_dec)
In the slow_assignment exercise above, we saw a roundabout way of assigning a number currently stored in X to the variable Y: start Y at 0, then decrement X until it hits 0, incrementing Y at each step. Transform the informal decorated program your wrote for slow_assignment into a formal decorated program and prove its correctness. If all goes well, your correctness proof will need only intros and verify.{{ X = m ∧ 0 = 0 }}
Y ::= 0;;
{{ X = m ∧ Y = 0 }}
becomes
{{ fun st ⇒ st X = m ∧ 0 = 0 }}
Y ::= 0
{{ fun st ⇒ st X = m ∧ st Y = 0 }} ;;
Example slow_assignment_dec (m : nat) : decorated
(* 将本行替换成 ":= _你的_定义_ ." *). Admitted.
Theorem slow_assignment_dec_correct : ∀ m,
dec_correct (slow_assignment_dec m).
Proof. (* 请在此处解答 *) Admitted.
(* 请勿修改下面这一行: *)
Definition manual_grade_for_check_defn_of_slow_assignment_dec : option (nat×string) := None.
☐
练习:4 星, advanced (factorial_dec)
The factorial function is defined recursively in the Coq standard library in a way that is equivalent to the following:Fixpoint fact (n : nat) : nat :=
match n with
| O ⇒ 1
| S n' ⇒ n × (fact n')
end.
Using your solutions to factorial and slow_assignment_dec as a
guide, write a formal decorated program factorial_dec that
implements the factorial function, state a theorem named
factorial_dec_correct that says factorial_dec is correct, and
prove the theorem. If all goes well, verify will leave you with
just two subgoals, each of which requires establishing some
mathematical property of fact rather than proving anything about
your program.
Hint: when transforming a loop guard into a formal assertion, make
sure to express it with bassn.
(* 请在此处解答 *)
(* 请勿修改下面这一行: *)
Definition manual_grade_for_factorial_dec : option (nat×string) := None.
☐
练习:4 星, advanced, optional (fib_eqn)
The Fibonacci function is usually written like this:Fixpoint fib n :=
match n with
| 0 ⇒ 1
| 1 ⇒ 1
| _ ⇒ fib (pred n) + fib (pred (pred n))
end.
Fixpoint fib n :=
match n with
| 0 ⇒ 1
| S n' ⇒ match n' with
| 0 ⇒ 1
| S n'' ⇒ fib n' + fib n''
end
end.
Prove that fib satisfies the following equation:
练习:4 星, advanced, optional (fib)
The following Imp program leaves the value of fib n in the variable Y when it terminates:X ::= 1;;
Y ::= 1;;
Z ::= 1;;
WHILE ~(X = n + 1) DO
T ::= Z;;
Z ::= Z + Y;;
Y ::= T;;
X ::= X + 1
END
{{ True }} dfib {{ Y = fib n }}
Definition T : string := "T".
Definition dfib (n : nat) : decorated
(* 将本行替换成 ":= _你的_定义_ ." *). Admitted.
Theorem dfib_correct : ∀ n,
dec_correct (dfib n).
(* 请在此处解答 *) Admitted.
☐
Close Scope dcom_scope.
练习:5 星, advanced, optional (improve_dcom)
The formal decorated programs defined in this section are intended to look as similar as possible to the informal ones defined earlier in the chapter. If we drop this requirement, we can eliminate almost all annotations, just requiring final postconditions and loop invariants to be provided explicitly. Do this -- i.e., define a new version of dcom with as few annotations as possible and adapt the rest of the formal development leading up to the verification_correct theorem.(* 请在此处解答 *)
☐
练习:4 星, advanced, optional (implement_dcom)
Adapt the parser for Imp presented in chapter ImpParser of Logical Foundations to parse decorated commands (either ours or, even better, the ones you defined in the previous exercise).(* 请在此处解答 *)
☐
(* 2022-03-14 05:28:21 (UTC+00) *)