Hoare12Hoare Logic, Part 1.2

Automation

Many of the proofs we have done so far with Hoare triples can be streamlined using the automation techniques that we introduced in the Auto chapter of Logical Foundations.
Recall that the auto tactic can be told to unfold definitions as part of its proof search. Let's give it that hint for the definitions and coercions we're using:
Hint Unfold assert_implies assertion_sub t_update : core.
Hint Unfold valid_hoare_triple : core.
Hint Unfold assert_of_Prop Aexp_of_nat Aexp_of_aexp : core.
Also recall that auto will search for a proof involving intros and apply. By default, the theorems that it will apply include any of the local hypotheses, as well as theorems in a core database.
The proof of hoare_consequence_pre, repeated below, looks like an opportune place for such automation, because all it does is unfold, intros, and apply. (It uses assumption, too, but that's just application of a hypothesis.)
Theorem hoare_consequence_pre' : (P P' Q : Assertion) c,
  {{P'}} c {{Q}}
  P ->> P'
  {{P}} c {{Q}}.
Proof.
  unfold valid_hoare_triple, "->>".
  intros P P' Q c Hhoare Himp st st' Heval Hpre.
  apply Hhoare with (st := st).
  - assumption.
  - apply Himp. assumption.
Qed.
Merely using auto, though, doesn't complete the proof.
Theorem hoare_consequence_pre'' : (P P' Q : Assertion) c,
  {{P'}} c {{Q}}
  P ->> P'
  {{P}} c {{Q}}.
Proof.
  auto. (* no progress *)
Abort.
The problem is the apply Hhoare with... part of the proof. Coq isn't able to figure out how to instantiate st without some help from us. Recall, though, that there are versions of many tactics that will use existential variables to make progress even when the regular versions of those tactics would get stuck.
Here, the eapply tactic will introduce an existential variable ?st as a placeholder for st, and eassumption will instantiate ?st with st when it discovers st in assumption Heval. By using eapply we are essentially telling Coq, "Be patient: The missing part is going to be filled in later in the proof."
Theorem hoare_consequence_pre''' : (P P' Q : Assertion) c,
  {{P'}} c {{Q}}
  P ->> P'
  {{P}} c {{Q}}.
Proof.
  unfold valid_hoare_triple, "->>".
  intros P P' Q c Hhoare Himp st st' Heval Hpre.
  eapply Hhoare.
  - eassumption.
  - apply Himp. assumption.
Qed.
The eauto tactic will use eapply as part of its proof search. So, the entire proof can actually be done in just one line.
Theorem hoare_consequence_pre'''' : (P P' Q : Assertion) c,
  {{P'}} c {{Q}}
  P ->> P'
  {{P}} c {{Q}}.
Proof.
  eauto.
Qed.
Of course, it's hard to predict that eauto suffices here without having gone through the original proof of hoare_consequence_pre to see the tactics it used. But now that we know eauto worked there, it's a good bet that it will also work for hoare_consequence_post.
Theorem hoare_consequence_post' : (P Q Q' : Assertion) c,
  {{P}} c {{Q'}}
  Q' ->> Q
  {{P}} c {{Q}}.
Proof.
  eauto.
Qed.
We can also use eapply to streamline a proof (hoare_asgn_example1), that we did earlier as an example of using the consequence rule:
Example hoare_asgn_example1' :
  {{True}} X := 1 {{X = 1}}.
Proof.
  eapply hoare_consequence_pre. (* no need to state an assertion *)
  - apply hoare_asgn.
  - unfold "->>", assertion_sub, t_update.
    intros st _. simpl. reflexivity.
Qed.
The final bullet of that proof also looks like a candidate for automation.
Example hoare_asgn_example1'' :
  {{True}} X := 1 {{X = 1}}.
Proof.
  eapply hoare_consequence_pre.
  - apply hoare_asgn.
  - auto.
Qed.
Now we have quite a nice proof script: it simply identifies the Hoare rules that need to be used and leaves the remaining low-level details up to Coq to figure out.
By now it might be apparent that the entire proof could be automated if we added hoare_consequence_pre and hoare_asgn to the hint database. We won't do that in this chapter, so that we can get a better understanding of when and how the Hoare rules are used. In the next chapter, Hoare2, we'll dive deeper into automating entire proofs of Hoare triples.
The other example of using consequence that we did earlier, hoare_asgn_example2, requires a little more work to automate. We can streamline the first line with eapply, but we can't just use auto for the final bullet, since it needs lia.
Example assertion_sub_example2' :
  {{X < 4}}
    X := X + 1
  {{X < 5}}.
Proof.
  eapply hoare_consequence_pre.
  - apply hoare_asgn.
  - auto. (* no progress *)
    unfold "->>", assertion_sub, t_update.
    intros st H. simpl in ×. lia.
Qed.
Let's introduce our own tactic to handle both that bullet and the bullet from example 1:
Ltac assertion_auto :=
  try auto; (* as in example 1, above *)
  try (unfold "->>", assertion_sub, t_update;
       intros; simpl in *; lia). (* as in example 2 *)

Example assertion_sub_example2'' :
  {{X < 4}}
    X := X + 1
  {{X < 5}}.
Proof.
  eapply hoare_consequence_pre.
  - apply hoare_asgn.
  - assertion_auto.
Qed.

Example hoare_asgn_example1''':
  {{True}} X := 1 {{X = 1}}.
Proof.
  eapply hoare_consequence_pre.
  - apply hoare_asgn.
  - assertion_auto.
Qed.
Again, we have quite a nice proof script. All the low-level details of proofs about assertions have been taken care of automatically. Of course, assertion_auto isn't able to prove everything we could possibly want to know about assertions -- there's no magic here! But it's good enough so far.

Exercise: 1 star, standard (hoare_asgn_examples_2)

Prove this triple. Try to make your proof script nicely automated by following the examples above.
Example assertion_sub_ex2' :
  {{ 0 3 3 5 }}
    X := 3
  {{ 0 X X 5 }}.
Proof.
  (* FILL IN HERE *) Admitted.

Sequencing + Assignment

Here's an example of a program involving both sequencing and assignment. Note the use of hoare_seq in conjunction with hoare_consequence_pre and the eapply tactic.
Example hoare_asgn_example3 : (a:aexp) (n:nat),
  {{a = n}}
    X := a;
    skip
  {{X = n}}.
Proof.
  intros a n. eapply hoare_seq.
  - (* right part of seq *)
    apply hoare_skip.
  - (* left part of seq *)
    eapply hoare_consequence_pre.
    + apply hoare_asgn.
    + assertion_auto.
Qed.
Informally, a nice way of displaying a proof using the sequencing rule is as a "decorated program" where the intermediate assertion Q is written between c1 and c2:
  {{ a = n }}
     X := a
              {{ X = n }}; <--- decoration for Q
     skip
  {{ X = n }}
We'll come back to the idea of decorated programs in much more detail in the next chapter.

Exercise: 2 stars, standard, especially useful (hoare_asgn_example4)

Translate this "decorated program" into a formal proof:
                   {{ True }} ->>
                   {{ 1 = 1 }}
    X := 1
                   {{ X = 1 }} ->>
                   {{ X = 1 ∧ 2 = 2 }};
    Y := 2
                   {{ X = 1 ∧ Y = 2 }}
Note the use of "->>" decorations, each marking a use of hoare_consequence_pre.
We've started you off by providing a use of hoare_seq that explicitly identifies X = 1 as the intermediate assertion.
Example hoare_asgn_example4 :
  {{ True }}
    X := 1;
    Y := 2
  {{ X = 1 Y = 2 }}.
Proof.
  eapply hoare_seq with (Q := (X = 1)%assertion).
  (* The annotation %assertion is needed to help Coq parse correctly. *)
  (* FILL IN HERE *) Admitted.

Exercise: 3 stars, standard, optional (swap_exercise)

Write an Imp program c that swaps the values of X and Y and show that it satisfies the following specification:
      {{XY}} c {{YX}} Your proof should not need to use unfold valid_hoare_triple.
Hints:
  • Remember that Imp commands need to be enclosed in <{...}> brackets.
  • Remember that the assignment rule works best when it's applied "back to front," from the postcondition to the precondition. So your proof will want to start at the end and work back to the beginning of your program.
  • Remember that eapply is your friend.)
Definition swap_program : com
  (* REPLACE THIS LINE WITH ":= _your_definition_ ." *). Admitted.

Theorem swap_exercise :
  {{X Y}}
    swap_program
  {{Y X}}.
Proof.
  (* FILL IN HERE *) Admitted.

Exercise: 4 stars, advanced, optional (invalid_triple)

Show that
    {{ a = n }} X := 3; Y := a {{ Y = n }} is not a valid Hoare triple for some choices of a and n.
Conceptual hint: Invent a particular a and n for which the triple in invalid, then use those to complete the proof.
Technical hint: Hypothesis H below begins a n, .... You'll want to instantiate that with the particular a and n you've invented. You can do that with assert and apply, but you may remember (from Tactics.v in Logical Foundations) that Coq offers an even easier tactic: specialize. If you write
       specialize H with (a := your_a) (n := your_n) the hypothesis will be instantiated on your_a and your_n.
Having chosen your a and n, proceed as follows:
  • Use the (assumed) validity of the given hoare triple to derive a state st' in which Y has some value y1
  • Use the evaluation rules (E_Seq and E_Asgn) to show that Y has a different value y2 in the same final state st'
  • Since y1 and y2 are both equal to st' Y, they are equal to each other. But we chose them to be different, so this is a contradiction, which finishes the proof.
Theorem invalid_triple : ¬ (a : aexp) (n : nat),
    {{ a = n }}
      X := 3; Y := a
    {{ Y = n }}.
Proof.
  unfold valid_hoare_triple.
  intros H.
  (* FILL IN HERE *) Admitted.

Conditionals

What sort of rule do we want for reasoning about conditional commands?
Certainly, if the same assertion Q holds after executing either of the branches, then it holds after the whole conditional. So we might be tempted to write:
{{P}} c1 {{Q}}
{{P}} c2 {{Q}}  

{{P}} if b then c1 else c2 {{Q}}
However, this is rather weak. For example, using this rule, we cannot show
     {{ True }}
       if X = 0
         then Y := 2
         else Y := X + 1
       end
     {{ XY }}
since the rule tells us nothing about the state in which the assignments take place in the "then" and "else" branches.
Fortunately, we can say something more precise. In the "then" branch, we know that the boolean expression b evaluates to true, and in the "else" branch, we know it evaluates to false. Making this information available in the premises of the rule gives us more information to work with when reasoning about the behavior of c1 and c2 (i.e., the reasons why they establish the postcondition Q).
{{P /\   b}} c1 {{Q}}
{{P /\ ~ b}} c2 {{Q}} (hoare_if)  

{{P}} if b then c1 else c2 end {{Q}}
To interpret this rule formally, we need to do a little work. Strictly speaking, the assertion we've written, P b, is the conjunction of an assertion and a boolean expression -- i.e., it doesn't typecheck. To fix this, we need a way of formally "lifting" any bexp b to an assertion. We'll write bassertion b for the assertion "the boolean expression b evaluates to true (in the given state)."
Definition bassertion b : Assertion :=
  fun st ⇒ (beval st b = true).

Coercion bassertion : bexp >-> Assertion.

Arguments bassertion /.
A useful fact about bassertion:
Lemma bexp_eval_false : b st,
  beval st b = false ¬ ((bassertion b) st).
Proof. congruence. Qed.

Hint Resolve bexp_eval_false : core.
We mentioned the congruence tactic in passing in Auto when building the find_rwd tactic. Like find_rwd, congruence is able to automatically find that both beval st b = false and beval st b = true are being assumed, notice the contradiction, and discriminate to complete the proof.
Now we can formalize the Hoare proof rule for conditionals and prove it correct.
Theorem hoare_if : P Q (b:bexp) c1 c2,
  {{ P b }} c1 {{Q}}
  {{ P ¬ b}} c2 {{Q}}
  {{P}} if b then c1 else c2 end {{Q}}.
That is (unwrapping the notations):
      Theorem hoare_if : P Q b c1 c2,
        {{fun stP stbassertion b st}} c1 {{Q}} →
        {{fun stP st ∧ ¬(bassertion b st)}} c2 {{Q}} →
        {{P}} if b then c1 else c2 end {{Q}}.
Proof.
  intros P Q b c1 c2 HTrue HFalse st st' HE HP.
  inversion HE; subst; eauto.
Qed.

Example

Here is a formal proof that the program we used to motivate the rule satisfies the specification we gave.
Example if_example :
  {{True}}
    if (X = 0)
      then Y := 2
      else Y := X + 1
    end
  {{X Y}}.
Proof.
  apply hoare_if.
  - (* Then *)
    eapply hoare_consequence_pre.
    + apply hoare_asgn.
    + assertion_auto. (* no progress *)
      unfold "->>", assertion_sub, t_update, bassertion.
      simpl. intros st [_ H]. apply eqb_eq in H.
      rewrite H. lia.
  - (* Else *)
    eapply hoare_consequence_pre.
    + apply hoare_asgn.
    + assertion_auto.
Qed.
As we did earlier, it would be nice to eliminate all the low-level proof script that isn't about the Hoare rules. Unfortunately, the assertion_auto tactic we wrote wasn't quite up to the job. Looking at the proof of if_example, we can see why. We had to unfold a definition (bassertion) and use a theorem (eqb_eq) that we didn't need in earlier proofs. So, let's add those into our tactic, and clean it up a little in the process.
Ltac assertion_auto' :=
  unfold "->>", assertion_sub, t_update, bassertion;
  intros; simpl in *;
  try rewriteeqb_eq in *; (* for equalities *)
  auto; try lia.
Now the proof is quite streamlined.
Example if_example'' :
  {{True}}
    if X = 0
      then Y := 2
      else Y := X + 1
    end
  {{X Y}}.
Proof.
  apply hoare_if.
  - eapply hoare_consequence_pre.
    + apply hoare_asgn.
    + assertion_auto'.
  - eapply hoare_consequence_pre.
    + apply hoare_asgn.
    + assertion_auto'.
Qed.
We can even shorten it a little bit more.
Example if_example''' :
  {{True}}
    if X = 0
      then Y := 2
      else Y := X + 1
    end
  {{X Y}}.
Proof.
  apply hoare_if; eapply hoare_consequence_pre;
    try apply hoare_asgn; try assertion_auto'.
Qed.
For later proofs, it will help to extend assertion_auto' to handle inequalities, too.
Ltac assertion_auto'' :=
  unfold "->>", assertion_sub, t_update, bassertion;
  intros; simpl in *;
  try rewriteeqb_eq in *;
  try rewriteleb_le in *; (* for inequalities *)
  auto; try lia.

Exercise: 2 stars, standard (if_minus_plus)

Prove the theorem below using hoare_if. Do not use unfold valid_hoare_triple. The assertion_auto'' tactic we just defined may be useful.
Theorem if_minus_plus :
  {{True}}
    if (X Y)
      then Z := Y - X
      else Y := X + Z
    end
  {{Y = X + Z}}.
Proof.
  (* FILL IN HERE *) Admitted.

Exercise: One-sided conditionals

In this exercise we consider extending Imp with "one-sided conditionals" of the form if1 b then c end. Here b is a boolean expression, and c is a command. If b evaluates to true, then command c is evaluated. If b evaluates to false, then if1 b then c end does nothing.
We recommend that you complete this exercise before attempting the ones that follow, as it should help solidify your understanding of the material.
The first step is to extend the syntax of commands and introduce the usual notations. (We've done this for you. We use a separate module to prevent polluting the global name space.)
Module If1.

Inductive com : Type :=
  | CSkip : com
  | CAsgn : string aexp com
  | CSeq : com com com
  | CIf : bexp com com com
  | CWhile : bexp com com
  | CIf1 : bexp com com.

Notation "'if1' x 'then' y 'end'" :=
         (CIf1 x y)
             (in custom com at level 0, x custom com at level 99).
Notation "'skip'" :=
         CSkip (in custom com at level 0).
Notation "x := y" :=
         (CAsgn x y)
            (in custom com at level 0, x constr at level 0,
             y at level 85, no associativity).
Notation "x ; y" :=
         (CSeq x y)
           (in custom com at level 90, right associativity).
Notation "'if' x 'then' y 'else' z 'end'" :=
         (CIf x y z)
           (in custom com at level 89, x at level 99,
            y at level 99, z at level 99).
Notation "'while' x 'do' y 'end'" :=
         (CWhile x y)
            (in custom com at level 89, x at level 99, y at level 99).

Exercise: 2 stars, standard, especially useful (if1_ceval)

Add two new evaluation rules to relation ceval, below, for if1. Let the rules for if guide you.

Inductive ceval : com state state Prop :=
  | E_Skip : st,
      st =[ skip ]=> st
  | E_Asgn : st a1 n x,
      aeval st a1 = n
      st =[ x := a1 ]=> (x !-> n ; st)
  | E_Seq : c1 c2 st st' st'',
      st =[ c1 ]=> st'
      st' =[ c2 ]=> st''
      st =[ c1 ; c2 ]=> st''
  | E_IfTrue : st st' b c1 c2,
      beval st b = true
      st =[ c1 ]=> st'
      st =[ if b then c1 else c2 end ]=> st'
  | E_IfFalse : st st' b c1 c2,
      beval st b = false
      st =[ c2 ]=> st'
      st =[ if b then c1 else c2 end ]=> st'
  | E_WhileFalse : b st c,
      beval st b = false
      st =[ while b do c end ]=> st
  | E_WhileTrue : st st' st'' b c,
      beval st b = true
      st =[ c ]=> st'
      st' =[ while b do c end ]=> st''
      st =[ while b do c end ]=> st''
(* FILL IN HERE *)

where "st '=[' c ']=>' st'" := (ceval c st st').

Hint Constructors ceval : core.
The following unit tests should be provable simply by eauto if you have defined the rules for if1 correctly.
Example if1true_test :
  empty_st =[ if1 X = 0 then X := 1 end ]=> (X !-> 1).
Proof. (* FILL IN HERE *) Admitted.

Example if1false_test :
  (X !-> 2) =[ if1 X = 0 then X := 1 end ]=> (X !-> 2).
Proof. (* FILL IN HERE *) Admitted.
Now we have to repeat the definition and notation of Hoare triples, so that they will use the updated com type.
Definition valid_hoare_triple
           (P : Assertion) (c : com) (Q : Assertion) : Prop :=
   st st',
       st =[ c ]=> st'
       P st
       Q st'.

Hint Unfold valid_hoare_triple : core.

Notation "{{ P }} c {{ Q }}" := (valid_hoare_triple P c Q)
                                  (at level 90, c custom com at level 99)
                                  : hoare_spec_scope.

Exercise: 2 stars, standard (hoare_if1)

Invent a Hoare logic proof rule for if1. State and prove a theorem named hoare_if1 that shows the validity of your rule. Use hoare_if as a guide. Try to invent a rule that is complete, meaning it can be used to prove the correctness of as many one-sided conditionals as possible. Also try to keep your rule compositional, meaning that any Imp command that appears in a premise should syntactically be a part of the command in the conclusion.
Hint: if you encounter difficulty getting Coq to parse part of your rule as an assertion, try manually indicating that it should be in the assertion scope. For example, if you want e to be parsed as an assertion, write it as (e)%assertion.
(* FILL IN HERE *)
For full credit, prove formally (hoare_if1_good) that your rule is precise enough to show the following Hoare triple is valid:
  {{ X + Y = Z }}
    if1 Y ≠ 0 then
      X := X + Y
    end
  {{ X = Z }}
(* Do not modify the following line: *)
Definition manual_grade_for_hoare_if1 : option (nat×string) := None.
Before the next exercise, we need to restate the Hoare rules of consequence (for preconditions) and assignment for the new com type.
Theorem hoare_consequence_pre : (P P' Q : Assertion) c,
  {{P'}} c {{Q}}
  P ->> P'
  {{P}} c {{Q}}.
Proof.
  eauto.
Qed.

Theorem hoare_asgn : Q X a,
  {{Q [X > a]}} (X := a) {{Q}}.
Proof.
  intros Q X a st st' Heval HQ.
  inversion Heval; subst.
  auto.
Qed.

Exercise: 2 stars, standard (hoare_if1_good)

Use your if1 rule to prove the following (valid) Hoare triple.
Hint: assertion_auto'' will once again get you most but not all the way to a completely automated proof. You can finish manually, or tweak the tactic further.
Hint: If you see a message like Unable to unify "Imp.ceval Imp.CSkip st st'" with..., it probably means you are using a definition or theorem e.g., hoare_skip from above this exercise without re-proving it for the new version of Imp with if1.
Lemma hoare_if1_good :
  {{ X + Y = Z }}
    if1 Y 0 then
      X := X + Y
    end
  {{ X = Z }}.
Proof. (* FILL IN HERE *) Admitted.
End If1.

While Loops

The Hoare rule for while loops is based on the idea of a command invariant (or just invariant): an assertion whose truth is guaranteed after executing a command, assuming it is true before.
That is, an assertion P is a command invariant of c if
      {{P}} c {{P}} holds. Note that the command invariant might temporarily become false in the middle of executing c, but by the end of c it must be restored.
As a first attempt at a while rule, we could try:

             {{P}} c {{P}}
      ---------------------------
      {{P} while b do c end {{P}}
That rule is valid: if P is a command invariant of c, as the premise requires, then no matter how many times the loop body executes, P is going to be true when the loop finally finishes.
But the rule also omits two crucial pieces of information. First, the loop terminates when b becomes false. So we can strengthen the postcondition in the conclusion:

              {{P}} c {{P}}
      ---------------------------------
      {{P} while b do c end {{P ∧ ¬b}}
Second, the loop body will be executed only if b is true. So we can also strengthen the precondition in the premise:

            {{Pb}} c {{P}}
      --------------------------------- (hoare_while)
      {{P} while b do c end {{P ∧ ¬b}}
That is the Hoare while rule. Note how it combines aspects of skip and conditionals:
  • If the loop body executes zero times, the rule is like skip in that the precondition survives to become (part of) the postcondition.
  • Like a conditional, we can assume guard b holds on entry to the subcommand.
Theorem hoare_while : P (b:bexp) c,
  {{P b}} c {{P}}
  {{P}} while b do c end {{P ¬ b}}.
Proof.
  intros P b c Hhoare st st' Heval HP.
  (* We proceed by induction on Heval, because, in the "keep looping" case,
     its hypotheses talk about the whole loop instead of just c. The
     remember is used to keep the original command in the hypotheses;
     otherwise, it would be lost in the induction. By using inversion
     we clear away all the cases except those involving while. *)

  remember <{while b do c end}> as original_command eqn:Horig.
  induction Heval;
    try (inversion Horig; subst; clear Horig);
    eauto.
Qed.
We call P a loop invariant of while b do c end if
      {{Pb}} c {{P}} is a valid Hoare triple.
This means that P will be true at the end of the loop body whenever the loop body executes. If P contradicts b, this holds trivially since the precondition is false.
For instance, X = 0 is a loop invariant of
      while X = 2 do X := 1 end since the program will never enter the loop.
The program
    while Y > 10 do Y := Y - 1; Z := Z + 1 end admits an interesting loop invariant:
    X = Y + Z Note that this doesn't contradict the loop guard but neither is it a command invariant of
    Y := Y - 1; Z := Z + 1 since, if X = 5, Y = 0 and Z = 5, running the command will set Y + Z to 6. The loop guard Y > 10 guarantees that this will not be the case. We will see many such loop invariants in the following chapter.
Example while_example :
  {{X 3}}
    while (X 2) do
      X := X + 1
    end
  {{X = 3}}.
Proof.
  eapply hoare_consequence_post.
  - apply hoare_while.
    eapply hoare_consequence_pre.
    + apply hoare_asgn.
    + assertion_auto''.
  - assertion_auto''.
Qed.
If the loop never terminates, any postcondition will work.
Theorem always_loop_hoare : Q,
  {{True}} while true do skip end {{Q}}.
Proof.
  intros Q.
  eapply hoare_consequence_post.
  - apply hoare_while. apply hoare_post_true. auto.
  - simpl. intros st [Hinv Hguard]. congruence.
Qed.
Of course, this result is not surprising if we remember that the definition of valid_hoare_triple asserts that the postcondition must hold only when the command terminates. If the command doesn't terminate, we can prove anything we like about the post-condition.
Hoare rules that specify what happens if commands terminate, without proving that they do, are said to describe a logic of partial correctness. It is also possible to give Hoare rules for total correctness, which additionally specifies that commands must terminate. Total correctness is out of the scope of this textbook.

Exercise: 3 stars, standard (hoare_add_loop)

Give a formal proof for the addition example from the lecture.
Hint: you might find lemmas negb_true_iff and leb_gt useful.
Example hoare_add_loop : (m n : nat),
  {{X = m Y = n}}
    while Y > 0
      do
        X := X + 1 ;
        Y := Y - 1
      end
  {{X = m + n}}.
Proof.
  (* FILL IN HERE *) Admitted.

Exercise: REPEAT

Exercise: 4 stars, advanced (hoare_repeat)

In this exercise, we'll add a new command to our language of commands: REPEAT c until b end. You will write the evaluation rule for REPEAT and add a new Hoare rule to the language for programs involving it. (You may recall that the evaluation rule is given in an example in the Auto chapter. Try to figure it out yourself here rather than peeking.)
Module RepeatExercise.

Inductive com : Type :=
  | CSkip : com
  | CAsgn : string aexp com
  | CSeq : com com com
  | CIf : bexp com com com
  | CWhile : bexp com com
  | CRepeat : com bexp com.
REPEAT behaves like while, except that the loop guard is checked after each execution of the body, with the loop repeating as long as the guard stays false. Because of this, the body will always execute at least once.
Notation "'repeat' e1 'until' b2 'end'" :=
          (CRepeat e1 b2)
              (in custom com at level 0,
               e1 custom com at level 99, b2 custom com at level 99).
Notation "'skip'" :=
         CSkip (in custom com at level 0).
Notation "x := y" :=
         (CAsgn x y)
            (in custom com at level 0, x constr at level 0,
             y at level 85, no associativity).
Notation "x ; y" :=
         (CSeq x y)
           (in custom com at level 90, right associativity).
Notation "'if' x 'then' y 'else' z 'end'" :=
         (CIf x y z)
           (in custom com at level 89, x at level 99,
            y at level 99, z at level 99).
Notation "'while' x 'do' y 'end'" :=
         (CWhile x y)
            (in custom com at level 89, x at level 99, y at level 99).
Add new rules for REPEAT to ceval below. You can use the rules for while as a guide, but remember that the body of a REPEAT should always execute at least once, and that the loop ends when the guard becomes true.
Inductive ceval : state com state Prop :=
  | E_Skip : st,
      st =[ skip ]=> st
  | E_Asgn : st a1 n x,
      aeval st a1 = n
      st =[ x := a1 ]=> (x !-> n ; st)
  | E_Seq : c1 c2 st st' st'',
      st =[ c1 ]=> st'
      st' =[ c2 ]=> st''
      st =[ c1 ; c2 ]=> st''
  | E_IfTrue : st st' b c1 c2,
      beval st b = true
      st =[ c1 ]=> st'
      st =[ if b then c1 else c2 end ]=> st'
  | E_IfFalse : st st' b c1 c2,
      beval st b = false
      st =[ c2 ]=> st'
      st =[ if b then c1 else c2 end ]=> st'
  | E_WhileFalse : b st c,
      beval st b = false
      st =[ while b do c end ]=> st
  | E_WhileTrue : st st' st'' b c,
      beval st b = true
      st =[ c ]=> st'
      st' =[ while b do c end ]=> st''
      st =[ while b do c end ]=> st''
(* FILL IN HERE *)

where "st '=[' c ']=>' st'" := (ceval st c st').
A couple of definitions from above, copied here so they use the new ceval.
Definition valid_hoare_triple (P : Assertion) (c : com) (Q : Assertion)
                        : Prop :=
   st st', st =[ c ]=> st' P st Q st'.

Notation "{{ P }} c {{ Q }}" :=
  (valid_hoare_triple P c Q) (at level 90, c custom com at level 99).
To make sure you've got the evaluation rules for repeat right, prove that ex1_repeat evaluates correctly.
Definition ex1_repeat :=
  <{ repeat
       X := 1;
       Y := Y + 1
     until (X = 1) end }>.

Theorem ex1_repeat_works :
  empty_st =[ ex1_repeat ]=> (Y !-> 1 ; X !-> 1).
Proof.
  (* FILL IN HERE *) Admitted.
Now state and prove a theorem, hoare_repeat, that expresses an appropriate proof rule for repeat commands. Use hoare_while as a model, and try to make your rule as precise as possible.
(* FILL IN HERE *)
For full credit, argue (informally) that your rule can be used to prove the following valid Hoare triple:
  {{ X > 0 }}
    repeat
      Y := X;
      X := X - 1
    until X = 0 end
  {{ X = 0 ∧ Y > 0 }}
End RepeatExercise.

(* Do not modify the following line: *)
Definition manual_grade_for_hoare_repeat : option (nat×string) := None.

Summary

So far, we've introduced Hoare Logic as a tool for reasoning about Imp programs. The rules of Hoare Logic are:
   (hoare_asgn)  

{{Q [X > a]}} X:=a {{Q}}
   (hoare_skip)  

{{ P }} skip {{ P }}
{{ P }} c1 {{ Q }}
{{ Q }} c2 {{ R }} (hoare_seq)  

{{ P }} c1;c2 {{ R }}
{{P /\   b}} c1 {{Q}}
{{P /\ ~ b}} c2 {{Q}} (hoare_if)  

{{P}} if b then c1 else c2 end {{Q}}
{{P /\ b}} c {{P}} (hoare_while)  

{{P}} while b do c end {{P /\ ~ b}}
{{P'}} c {{Q'}}
P ->> P'
Q' ->> Q (hoare_consequence)  

{{P}} c {{Q}}
Our task in this chapter has been to define the rules of Hoare logic, and prove that the definitions are sound. Having done so, we can now work within Hoare logic to prove that particular programs satisfy particular Hoare triples. In the next chapter, we'll see how Hoare logic is can be used to prove that more interesting programs satisfy interesting specifications of their behavior.
Crucially, we will do so without ever again unfolding the definition of Hoare triples -- i.e., we will take the rules of Hoare logic as a closed world for reasoning about programs.

Optional Additional Exercises

Havoc

In this exercise, we will derive proof rules for a HAVOC command, which is similar to the nondeterministic any expression from the the Imp chapter.
First, we enclose this work in a separate module, and recall the syntax and big-step semantics of Himp commands.
Module Himp.

Inductive com : Type :=
  | CSkip : com
  | CAsgn : string aexp com
  | CSeq : com com com
  | CIf : bexp com com com
  | CWhile : bexp com com
  | CHavoc : string com.

Notation "'havoc' l" := (CHavoc l)
                          (in custom com at level 60, l constr at level 0).
Notation "'skip'" :=
         CSkip (in custom com at level 0).
Notation "x := y" :=
         (CAsgn x y)
            (in custom com at level 0, x constr at level 0,
             y at level 85, no associativity).
Notation "x ; y" :=
         (CSeq x y)
           (in custom com at level 90, right associativity).
Notation "'if' x 'then' y 'else' z 'end'" :=
         (CIf x y z)
           (in custom com at level 89, x at level 99,
            y at level 99, z at level 99).
Notation "'while' x 'do' y 'end'" :=
         (CWhile x y)
            (in custom com at level 89, x at level 99, y at level 99).

Inductive ceval : com state state Prop :=
  | E_Skip : st,
      st =[ skip ]=> st
  | E_Asgn : st a1 n x,
      aeval st a1 = n
      st =[ x := a1 ]=> (x !-> n ; st)
  | E_Seq : c1 c2 st st' st'',
      st =[ c1 ]=> st'
      st' =[ c2 ]=> st''
      st =[ c1 ; c2 ]=> st''
  | E_IfTrue : st st' b c1 c2,
      beval st b = true
      st =[ c1 ]=> st'
      st =[ if b then c1 else c2 end ]=> st'
  | E_IfFalse : st st' b c1 c2,
      beval st b = false
      st =[ c2 ]=> st'
      st =[ if b then c1 else c2 end ]=> st'
  | E_WhileFalse : b st c,
      beval st b = false
      st =[ while b do c end ]=> st
  | E_WhileTrue : st st' st'' b c,
      beval st b = true
      st =[ c ]=> st'
      st' =[ while b do c end ]=> st''
      st =[ while b do c end ]=> st''
  | E_Havoc : st x n,
      st =[ havoc x ]=> (x !-> n ; st)

where "st '=[' c ']=>' st'" := (ceval c st st').

Hint Constructors ceval : core.
The definition of Hoare triples is exactly as before.
Definition valid_hoare_triple (P:Assertion) (c:com) (Q:Assertion) : Prop :=
   st st', st =[ c ]=> st' P st Q st'.

Hint Unfold valid_hoare_triple : core.

Notation "{{ P }} c {{ Q }}" := (valid_hoare_triple P c Q)
                                  (at level 90, c custom com at level 99)
                                  : hoare_spec_scope.
And the precondition consequence rule is exactly as before.
Theorem hoare_consequence_pre : (P P' Q : Assertion) c,
  {{P'}} c {{Q}}
  P ->> P'
  {{P}} c {{Q}}.
Proof. eauto. Qed.

Exercise: 3 stars, advanced, optional (hoare_havoc)

Complete the Hoare rule for HAVOC commands below by defining havoc_pre, and prove that the resulting rule is correct.
Definition havoc_pre (X : string) (Q : Assertion) (st : total_map nat) : Prop
  (* REPLACE THIS LINE WITH ":= _your_definition_ ." *). Admitted.

Theorem hoare_havoc : (Q : Assertion) (X : string),
  {{ havoc_pre X Q }} havoc X {{ Q }}.
Proof.
  (* FILL IN HERE *) Admitted.

Exercise: 3 stars, advanced, optional (havoc_post)

Complete the following proof without changing any of the provided commands. If you find that it can't be completed, your definition of havoc_pre is probably too strong. Find a way to relax it so that havoc_post can be proved.
Hint: the assertion_auto tactics we've built won't help you here. You need to proceed manually.
Theorem havoc_post : (P : Assertion) (X : string),
  {{ P }} havoc X {{ fun st (n:nat), P [X > n] st }}.
Proof.
  intros P X. eapply hoare_consequence_pre.
  - apply hoare_havoc.
  - (* FILL IN HERE *) Admitted.
End Himp.

Assert and Assume

Exercise: 4 stars, standard, optional (assert_vs_assume)

In this exercise, we will extend IMP with two commands, assert and assume. Both commands are ways to indicate that a certain assertion should hold any time this part of the program is reached. However they differ as follows:
  • If an assert statement fails, it causes the program to go into an error state and exit.
  • If an assume statement fails, the program fails to evaluate at all. In other words, the program gets stuck and has no final state.
The new set of commands is:
Module HoareAssertAssume.

Inductive com : Type :=
  | CSkip : com
  | CAsgn : string aexp com
  | CSeq : com com com
  | CIf : bexp com com com
  | CWhile : bexp com com
  | CAssert : bexp com
  | CAssume : bexp com.

Notation "'assert' l" := (CAssert l)
                           (in custom com at level 8, l custom com at level 0).
Notation "'assume' l" := (CAssume l)
                          (in custom com at level 8, l custom com at level 0).
Notation "'skip'" :=
         CSkip (in custom com at level 0).
Notation "x := y" :=
         (CAsgn x y)
            (in custom com at level 0, x constr at level 0,
             y at level 85, no associativity).
Notation "x ; y" :=
         (CSeq x y)
           (in custom com at level 90, right associativity).
Notation "'if' x 'then' y 'else' z 'end'" :=
         (CIf x y z)
           (in custom com at level 89, x at level 99,
            y at level 99, z at level 99).
Notation "'while' x 'do' y 'end'" :=
         (CWhile x y)
            (in custom com at level 89, x at level 99, y at level 99).
To define the behavior of assert and assume, we need to add notation for an error, which indicates that an assertion has failed. We modify the ceval relation, therefore, so that it relates a start state to either an end state or to error. The result type indicates the end value of a program, either a state or an error:
Inductive result : Type :=
  | RNormal : state result
  | RError : result.
Now we are ready to give you the ceval relation for the new language.
Inductive ceval : com state result Prop :=
  (* Old rules, several modified *)
  | E_Skip : st,
      st =[ skip ]=> RNormal st
  | E_Asgn : st a1 n x,
      aeval st a1 = n
      st =[ x := a1 ]=> RNormal (x !-> n ; st)
  | E_SeqNormal : c1 c2 st st' r,
      st =[ c1 ]=> RNormal st'
      st' =[ c2 ]=> r
      st =[ c1 ; c2 ]=> r
  | E_SeqError : c1 c2 st,
      st =[ c1 ]=> RError
      st =[ c1 ; c2 ]=> RError
  | E_IfTrue : st r b c1 c2,
      beval st b = true
      st =[ c1 ]=> r
      st =[ if b then c1 else c2 end ]=> r
  | E_IfFalse : st r b c1 c2,
      beval st b = false
      st =[ c2 ]=> r
      st =[ if b then c1 else c2 end ]=> r
  | E_WhileFalse : b st c,
      beval st b = false
      st =[ while b do c end ]=> RNormal st
  | E_WhileTrueNormal : st st' r b c,
      beval st b = true
      st =[ c ]=> RNormal st'
      st' =[ while b do c end ]=> r
      st =[ while b do c end ]=> r
  | E_WhileTrueError : st b c,
      beval st b = true
      st =[ c ]=> RError
      st =[ while b do c end ]=> RError
  (* Rules for Assert and Assume *)
  | E_AssertTrue : st b,
      beval st b = true
      st =[ assert b ]=> RNormal st
  | E_AssertFalse : st b,
      beval st b = false
      st =[ assert b ]=> RError
  | E_Assume : st b,
      beval st b = true
      st =[ assume b ]=> RNormal st

where "st '=[' c ']=>' r" := (ceval c st r).
We redefine hoare triples: Now, {{P}} c {{Q}} means that, whenever c is started in a state satisfying P, and terminates with result r, then r is not an error and the state of r satisfies Q.
Definition valid_hoare_triple
           (P : Assertion) (c : com) (Q : Assertion) : Prop :=
   st r,
     st =[ c ]=> r P st
     ( st', r = RNormal st' Q st').

Notation "{{ P }} c {{ Q }}" :=
  (valid_hoare_triple P c Q) (at level 90, c custom com at level 99)
  : hoare_spec_scope.
To test your understanding of this modification, give an example precondition and postcondition that are satisfied by the assume statement but not by the assert statement.
Theorem assert_assume_differ : (P:Assertion) b (Q:Assertion),
       ({{P}} assume b {{Q}})
   ¬ ({{P}} assert b {{Q}}).
(* FILL IN HERE *) Admitted.
Then prove that any triple for an assert also works when assert is replaced by assume.
Theorem assert_implies_assume : P b Q,
     ({{P}} assert b {{Q}})
   ({{P}} assume b {{Q}}).
Proof.
(* FILL IN HERE *) Admitted.
Next, here are proofs for the old hoare rules adapted to the new semantics. You don't need to do anything with these.
Theorem hoare_asgn : Q X a,
  {{Q [X > a]}} X := a {{Q}}.
Proof.
  unfold valid_hoare_triple.
  intros Q X a st st' HE HQ.
  inversion HE. subst.
   (X !-> aeval st a ; st). split; try reflexivity.
  assumption. Qed.

Theorem hoare_consequence_pre : (P P' Q : Assertion) c,
  {{P'}} c {{Q}}
  P ->> P'
  {{P}} c {{Q}}.
Proof.
  intros P P' Q c Hhoare Himp.
  intros st st' Hc HP. apply (Hhoare st st').
  - assumption.
  - apply Himp. assumption. Qed.

Theorem hoare_consequence_post : (P Q Q' : Assertion) c,
  {{P}} c {{Q'}}
  Q' ->> Q
  {{P}} c {{Q}}.
Proof.
  intros P Q Q' c Hhoare Himp.
  intros st r Hc HP.
  unfold valid_hoare_triple in Hhoare.
  assert ( st', r = RNormal st' Q' st').
  { apply (Hhoare st); assumption. }
  destruct H as [st' [Hr HQ'] ].
   st'. split; try assumption.
  apply Himp. assumption.
Qed.

Theorem hoare_seq : P Q R c1 c2,
  {{Q}} c2 {{R}}
  {{P}} c1 {{Q}}
  {{P}} c1;c2 {{R}}.
Proof.
  intros P Q R c1 c2 H1 H2 st r H12 Pre.
  inversion H12; subst.
  - eapply H1.
    + apply H6.
    + apply H2 in H3. apply H3 in Pre.
        destruct Pre as [st'0 [Heq HQ] ].
        inversion Heq; subst. assumption.
  - (* Find contradictory assumption *)
     apply H2 in H5. apply H5 in Pre.
     destruct Pre as [st' [C _] ].
     inversion C.
Qed.
Here are the other proof rules (sanity check)
Theorem hoare_skip : P,
     {{P}} skip {{P}}.
Proof.
  intros P st st' H HP. inversion H. subst.
  eexists. split.
  - reflexivity.
  - assumption.
Qed.

Theorem hoare_if : P Q (b:bexp) c1 c2,
  {{ P b}} c1 {{Q}}
  {{ P ¬ b}} c2 {{Q}}
  {{P}} if b then c1 else c2 end {{Q}}.
Proof.
  intros P Q b c1 c2 HTrue HFalse st st' HE HP.
  inversion HE; subst.
  - (* b is true *)
    apply (HTrue st st').
    + assumption.
    + split; assumption.
  - (* b is false *)
    apply (HFalse st st').
    + assumption.
    + split.
      × assumption.
      × apply bexp_eval_false. assumption.
Qed.

Theorem hoare_while : P (b:bexp) c,
  {{P b}} c {{P}}
  {{P}} while b do c end {{ P ¬b}}.
Proof.
  intros P b c Hhoare st st' He HP.
  remember <{while b do c end}> as wcom eqn:Heqwcom.
  induction He;
    try (inversion Heqwcom); subst; clear Heqwcom.
  - (* E_WhileFalse *)
    eexists. split.
    + reflexivity.
    + split; try assumption.
      apply bexp_eval_false. assumption.
  - (* E_WhileTrueNormal *)
    clear IHHe1.
    apply IHHe2.
    + reflexivity.
    + clear IHHe2 He2 r.
      unfold valid_hoare_triple in Hhoare.
      apply Hhoare in He1.
      × destruct He1 as [st1 [Heq Hst1] ].
        inversion Heq; subst.
        assumption.
      × split; assumption.
  - (* E_WhileTrueError *)
     exfalso. clear IHHe.
     unfold valid_hoare_triple in Hhoare.
     apply Hhoare in He.
     + destruct He as [st' [C _] ]. inversion C.
     + split; assumption.
Qed.
Finally, state Hoare rules for assert and assume and use them to prove a simple program correct. Name your rules hoare_assert and hoare_assume.
(* FILL IN HERE *)
Use your rules to prove the following triple.
Example assert_assume_example:
  {{True}}
    assume (X = 1);
    X := X + 1;
    assert (X = 2)
  {{True}}.
Proof.
(* FILL IN HERE *) Admitted.

End HoareAssertAssume.
(* 2025-06-16 19:18 *)