OperationalSemantics chapter done

This commit is contained in:
Adam Chlipala 2016-02-28 14:50:20 -05:00
parent f5685818a2
commit bf825fea8b
2 changed files with 97 additions and 60 deletions

View file

@ -590,96 +590,97 @@ Proof.
assumption. assumption.
Qed. Qed.
Lemma manually_proved_invariant' : Lemma manually_proved_invariant' : forall n,
invariantFor (trsys_of ($0 $+ ("n", 0) $+ ("a", 0)) (while "n" loop "a" <- "a" + "n";; "n" <- "n" - 2 done)) isEven n
-> invariantFor (trsys_of ($0 $+ ("n", n) $+ ("a", 0)) (while "n" loop "a" <- "a" + "n";; "n" <- "n" - 2 done))
(fun s => all_programs (snd s) (fun s => all_programs (snd s)
/\ exists n a, fst s $? "n" = Some n /\ exists n a, fst s $? "n" = Some n
/\ fst s $? "a" = Some a /\ fst s $? "a" = Some a
/\ isEven n /\ isEven n
/\ isEven a). /\ isEven a).
Proof. Proof.
simplify.
apply invariant_induction; simplify. apply invariant_induction; simplify.
first_order. first_order.
unfold all_programs. unfold all_programs.
subst; simplify; equality. subst; simplify; equality.
subst; simplify. subst; simplify.
exists 0, 0. exists n, 0.
propositional. propositional.
constructor. constructor.
constructor.
invert H. invert H0.
invert H2. invert H3.
invert H. invert H0.
invert H2.
invert H3. invert H3.
invert H4. invert H4.
invert H5.
(* Note our use here of [invert] to break down hypotheses with [exists] and (* Note our use here of [invert] to break down hypotheses with [exists] and
* [/\]. *) * [/\]. *)
invert H0; simplify. invert H1; simplify.
unfold all_programs in *; simplify; propositional; try equality. unfold all_programs in *; simplify; propositional; try equality.
invert H1; simplify. invert H2; simplify.
rewrite H. rewrite H0.
exists (x - 2), x0; propositional. exists (x - 2), x0; propositional.
apply isEven_minus2; assumption. apply isEven_minus2; assumption.
unfold all_programs in *; simplify; propositional; try equality. unfold all_programs in *; simplify; propositional; try equality.
invert H1. invert H2.
invert H4; equality. invert H5; equality.
invert H1. invert H2.
invert H4. invert H5.
rewrite H, H2; simplify. rewrite H0, H3; simplify.
eexists; eexists. eexists; eexists.
propositional; try eassumption. propositional; try eassumption.
apply isEven_plus; assumption. apply isEven_plus; assumption.
invert H0.
invert H4.
invert H0.
invert H4.
invert H0.
invert H4.
invert H1. invert H1.
invert H5.
invert H1.
invert H5.
invert H1.
invert H5.
invert H2.
equality. equality.
invert H0.
invert H4.
invert H1. invert H1.
rewrite H, H2; simplify. invert H5.
invert H2.
rewrite H0, H3; simplify.
eexists; eexists; propositional; try eassumption. eexists; eexists; propositional; try eassumption.
apply isEven_plus; assumption. apply isEven_plus; assumption.
invert H1. invert H2.
invert H4. invert H5.
invert H1. invert H2.
equality. equality.
invert H1. invert H2.
invert H4. invert H5.
invert H1. invert H2.
eexists; eexists; propositional; eassumption. eexists; eexists; propositional; eassumption.
invert H0. invert H1.
invert H4. invert H5.
equality. equality.
invert H0. invert H1.
invert H4. invert H5.
rewrite H; simplify. rewrite H0; simplify.
do 2 eexists; propositional; try eassumption. do 2 eexists; propositional; try eassumption.
apply isEven_minus2; assumption. apply isEven_minus2; assumption.
invert H1. invert H2.
invert H4. invert H5.
invert H1. invert H2.
invert H4. invert H5.
unfold all_programs in *; simplify; propositional; try equality. unfold all_programs in *; simplify; propositional; try equality.
invert H0.
do 2 eexists; propositional; try eassumption.
invert H1. invert H1.
do 2 eexists; propositional; try eassumption. do 2 eexists; propositional; try eassumption.
invert H2.
do 2 eexists; propositional; try eassumption.
unfold all_programs in *; simplify; propositional; equality. unfold all_programs in *; simplify; propositional; equality.
unfold all_programs in *; simplify; propositional; equality. unfold all_programs in *; simplify; propositional; equality.
unfold all_programs in *; simplify; propositional; try equality. unfold all_programs in *; simplify; propositional; try equality.
invert H0. invert H1.
do 2 eexists; propositional; try eassumption. do 2 eexists; propositional; try eassumption.
unfold all_programs in *; simplify; propositional; try equality. unfold all_programs in *; simplify; propositional; try equality.
invert H0. invert H1.
do 2 eexists; propositional; try eassumption. do 2 eexists; propositional; try eassumption.
Qed. Qed.
@ -687,15 +688,16 @@ Qed.
Hint Constructors isEven. Hint Constructors isEven.
Hint Resolve isEven_minus2 isEven_plus. Hint Resolve isEven_minus2 isEven_plus.
Lemma manually_proved_invariant'_snazzy : Lemma manually_proved_invariant'_snazzy : forall n,
invariantFor (trsys_of ($0 $+ ("n", 0) $+ ("a", 0)) (while "n" loop "a" <- "a" + "n";; "n" <- "n" - 2 done)) isEven n
-> invariantFor (trsys_of ($0 $+ ("n", n) $+ ("a", 0)) (while "n" loop "a" <- "a" + "n";; "n" <- "n" - 2 done))
(fun s => all_programs (snd s) (fun s => all_programs (snd s)
/\ exists n a, fst s $? "n" = Some n /\ exists n a, fst s $? "n" = Some n
/\ fst s $? "a" = Some a /\ fst s $? "a" = Some a
/\ isEven n /\ isEven n
/\ isEven a). /\ isEven a).
Proof. Proof.
apply invariant_induction; simplify; unfold all_programs in *; first_order; subst; simplify; simplify; apply invariant_induction; simplify; unfold all_programs in *; first_order; subst; simplify;
try match goal with try match goal with
| [ H : step _ _ |- _ ] => invert H; simplify | [ H : step _ _ |- _ ] => invert H; simplify
end; end;
@ -707,12 +709,14 @@ Proof.
end; simplify); equality || eauto 7. end; simplify); equality || eauto 7.
Qed. Qed.
Theorem manually_proved_invariant : Theorem manually_proved_invariant : forall n,
invariantFor (trsys_of ($0 $+ ("n", 0) $+ ("a", 0)) (while "n" loop "a" <- "a" + "n";; "n" <- "n" - 2 done)) isEven n
-> invariantFor (trsys_of ($0 $+ ("n", n) $+ ("a", 0)) (while "n" loop "a" <- "a" + "n";; "n" <- "n" - 2 done))
(fun s => exists a, fst s $? "a" = Some a /\ isEven a). (fun s => exists a, fst s $? "a" = Some a /\ isEven a).
Proof. Proof.
simplify.
eapply invariant_weaken. eapply invariant_weaken.
apply manually_proved_invariant'. apply manually_proved_invariant'; assumption.
first_order. first_order.
Qed. Qed.

View file

@ -1319,7 +1319,7 @@ $$\begin{array}{rrcl}
\newcommand{\bigstep}[2]{#1 \Downarrow #2} \newcommand{\bigstep}[2]{#1 \Downarrow #2}
\emph{Big-step operational semantics}\index{big-step operational semantics} explains what it means to run a program to completion. \emph{Big-step operational semantics}\index{big-step operational semantics} explains what it means to run a program to completion.
For our example relation, we will define a relation written $\bigstep{(v, c)}{v'}$, for ``command $c$, run with variable valuation $v$, terminates, modifying the valuation to $v'$.'' For our example language, we define a relation written $\bigstep{(v, c)}{v'}$, for ``command $c$, run with variable valuation $v$, terminates, modifying the valuation to $v'$.''
This relation is fairly straightforward to define with inference rules. This relation is fairly straightforward to define with inference rules.
\encoding \encoding
@ -1499,20 +1499,20 @@ Different theorems are easier to prove with different semantics, so it is helpfu
\subsection{Transition Systems from Small-Step Semantics} \subsection{Transition Systems from Small-Step Semantics}
The small-step semantics is a natural fit with our working definition of transition systems. The small-step semantics is a natural fit with our working definition of transition systems.
We can define a transition system from any valuation and command, where $\mathbb V$ is the set of valuations and $\mathbb C$ the set of commands, by $\mathbb T(v, c) = \angled{\mathbb V \times \mathbb C, {(v, c)}, \to}$. We can define a transition system from any valuation and command, where $\mathbb V$ is the set of valuations and $\mathbb C$ the set of commands, by $\mathbb T(v, c) = \angled{\mathbb V \times \mathbb C, \{(v, c)\}, \to}$.
Now we bring to bear all of our machinery about invariants and their proof methods. Now we bring to bear all of our machinery about invariants and their proof methods.
For instance, consider program $P = \while{\mathtt{n}}{\assign{\mathtt{a}}{\mathtt{a} + \mathtt{n}}; \assign{\mathtt{n}}{\mathtt{n} - 2}}$. For instance, consider program $P = \while{\mathtt{n}}{\assign{\mathtt{a}}{\mathtt{a} + \mathtt{n}}; \assign{\mathtt{n}}{\mathtt{n} - 2}}$.
\invariants \invariants
\begin{theorem} \begin{theorem}
For $\mathbb T(\mupd{\mupd{\mempty}{\mathtt{n}}{0}}{\mathtt{a}}{0}, P)$, it is an invariant that the valuation maps variable $\mathtt{a}$ to an even number. Given even $n$, for $\mathbb T(\mupd{\mupd{\mempty}{\mathtt{n}}{n}}{\mathtt{a}}{0}, P)$, it is an invariant that the valuation maps variable $\mathtt{a}$ to an even number.
\end{theorem} \end{theorem}
\begin{proof} \begin{proof}
First, we strengthen the invariant. First, we strengthen the invariant.
We compute the set $\overline{P}$ of all commands that can be reached from $P$ by stepping the small-step semantics. We compute the set $\overline{P}$ of all commands that can be reached from $P$ by stepping the small-step semantics.
This set is finite, even though the set of \emph{reachable valuations} is infinite. This set is finite, even though the set of \emph{reachable valuations} is infinite, considering all potential $n$ values.
Our strengthened invariant is $I(v, c) = c \in \overline{P} \land (\exists n. \; \msel{v}{\mathtt{n}} = n \land \textrm{even}(n)) \land (\exists a. \; \msel{v}{\mathtt{a}} = a \land \textrm{even}(a))$. Our strengthened invariant is $I(v, c) = c \in \overline{P} \land (\exists n. \; \msel{v}{\mathtt{n}} = n \land \textrm{even}(n)) \land (\exists a. \; \msel{v}{\mathtt{a}} = a \land \textrm{even}(a))$.
In other words, we strengthen by adding the constraints that (1) we do not stray from the expected set of reachable commands and (2) variable \texttt{n} also remains even. In other words, we strengthen by adding the constraints that (1) we do not stray from the expected set of reachable commands and (2) variable \texttt{n} also remains even.
@ -1523,16 +1523,15 @@ For instance, consider program $P = \while{\mathtt{n}}{\assign{\mathtt{a}}{\math
\section{Contextual Small-Step Semantics} \section{Contextual Small-Step Semantics}
The reader may have noticed some tedium in certain rules of the small-step semantics, like this one. The reader may have noticed some tedium in certain rules of the small-step semantics, like this one.
$$\infer{\bigstep{(v, c_1; c_2)}{v_2}}{ $$\infer{\smallstep{(v, c_1; c_2)}{(v', c'_1; c_2)}}{
\bigstep{(v, c_1)}{v_1} \smallstep{(v, c_1)}{(v', c'_1)}
& \bigstep{(v_1, c_2)}{v_2}
}$$ }$$
This rule is an example of a \emph{congruence rule}\index{congruence rule}, which shows how to take a step and \emph{lift} it into a step within a larger command, whose other subcommands are unaffected. This rule is an example of a \emph{congruence rule}\index{congruence rule}, which shows how to take a step and \emph{lift} it into a step within a larger command, whose other subcommands are unaffected.
Complex languages can require many congruence rules, and yet we feel like we should be able to avoid repeating all this boilerplate logic somehow. Complex languages can require many congruence rules, and yet we feel like we should be able to avoid repeating all this boilerplate logic somehow.
A common way to do so is switching to \emph{contextual small-step semantics}\index{contextual small-step semantics}. A common way to do so is switching to \emph{contextual small-step semantics}\index{contextual small-step semantics}.
We illustrate with our running example language. We illustrate with our running example language.
The first step is to define a set of \emph{evaluation contexts}\index{evaluation contexts}, which formalize the spots within a larger command where interesting steps are enabled. The first step is to define a set of \emph{evaluation contexts}\index{evaluation contexts}, which formalize the spots within a larger command where steps are enabled.
\encoding \encoding
$$\begin{array}{rrcl} $$\begin{array}{rrcl}
\textrm{Evaluation contexts} & C &::=& \Box \mid C; c \textrm{Evaluation contexts} & C &::=& \Box \mid C; c
@ -1593,7 +1592,7 @@ Let's revisit last section's example, to see contextual semantics in action, esp
\to_\mathsf{c} & (\mupd{\mupd{\mempty}{\mathtt{input}}{2}}{\mathtt{output}}{2}, (\skipe; \assign{\mathtt{input}}{\mathtt{input} - 1}); \mathtt{factorial\_loop}) \\ \to_\mathsf{c} & (\mupd{\mupd{\mempty}{\mathtt{input}}{2}}{\mathtt{output}}{2}, (\skipe; \assign{\mathtt{input}}{\mathtt{input} - 1}); \mathtt{factorial\_loop}) \\
= & (\mupd{\mupd{\mempty}{\mathtt{input}}{2}}{\mathtt{output}}{2}, \plug{(\Box; \mathtt{factorial\_loop})}{\skipe; \assign{\mathtt{input}}{\mathtt{input} - 1})} \\ = & (\mupd{\mupd{\mempty}{\mathtt{input}}{2}}{\mathtt{output}}{2}, \plug{(\Box; \mathtt{factorial\_loop})}{\skipe; \assign{\mathtt{input}}{\mathtt{input} - 1})} \\
\to_\mathsf{c} & (\mupd{\mupd{\mempty}{\mathtt{input}}{2}}{\mathtt{output}}{2}, \assign{\mathtt{input}}{\mathtt{input} - 1}; \mathtt{factorial\_loop}) \\ \to_\mathsf{c} & (\mupd{\mupd{\mempty}{\mathtt{input}}{2}}{\mathtt{output}}{2}, \assign{\mathtt{input}}{\mathtt{input} - 1}; \mathtt{factorial\_loop}) \\
= & (\mupd{\mupd{\mempty}{\mathtt{input}}{2}}{\mathtt{output}}{2}, \plug{\Box; \mathtt{factorial\_loop}}{\assign{\mathtt{input}}{\mathtt{input} - 1}}) \\ = & (\mupd{\mupd{\mempty}{\mathtt{input}}{2}}{\mathtt{output}}{2}, \plug{(\Box; \mathtt{factorial\_loop})}{\assign{\mathtt{input}}{\mathtt{input} - 1}}) \\
\to_\mathsf{c} & (\mupd{\mupd{\mempty}{\mathtt{input}}{1}}{\mathtt{output}}{2}, \skipe; \mathtt{factorial\_loop}) \\ \to_\mathsf{c} & (\mupd{\mupd{\mempty}{\mathtt{input}}{1}}{\mathtt{output}}{2}, \skipe; \mathtt{factorial\_loop}) \\
= & (\mupd{\mupd{\mempty}{\mathtt{input}}{1}}{\mathtt{output}}{2}, \plug{\Box}{\skipe; \mathtt{factorial\_loop}}) \\ = & (\mupd{\mupd{\mempty}{\mathtt{input}}{1}}{\mathtt{output}}{2}, \plug{\Box}{\skipe; \mathtt{factorial\_loop}}) \\
\to^*_\mathsf{c} & \ldots \\ \to^*_\mathsf{c} & \ldots \\
@ -1642,7 +1641,6 @@ This new semantics formulation is equivalent to the other two, as we establish n
\subsection{Evaluation Contexts Pay Off: Adding Concurrency} \subsection{Evaluation Contexts Pay Off: Adding Concurrency}
To showcase the convenience of contextual semantics, let's extend our example language with a simple construct for running two commands in parallel\index{parallel composition of threads}, implicitly extending the definition of plugging accordingly. To showcase the convenience of contextual semantics, let's extend our example language with a simple construct for running two commands in parallel\index{parallel composition of threads}, implicitly extending the definition of plugging accordingly.
$$\begin{array}{rrcl} $$\begin{array}{rrcl}
\textrm{Commands} & c &::=& \ldots \mid c || c \textrm{Commands} & c &::=& \ldots \mid c || c
\end{array}$$ \end{array}$$
@ -1663,6 +1661,41 @@ In fact, in the accompanying Coq code, literally the same proof scripts establis
It's not often that concurrency comes for free in a rigorous proof! It's not often that concurrency comes for free in a rigorous proof!
\section{Determinism}
Our last extension with parallelism introduced intentional nondeterminism in the semantics: a single starting state can step to multiple different next states.
However, the three semantics for the original language are deterministic, and we can prove it.
\begin{theorem}
If $\bigstep{(v, c)}{v_1}$ and $\bigstep{(v, c)}{v_2}$, then $v_1 = v_2$.
\end{theorem}
\begin{proof}
By induction on the derivation of $\bigstep{(v, c)}{v_1}$ and inversion on the derivation of $\bigstep{(v, c)}{v_2}$.
\end{proof}
\begin{theorem}
If $\smallstep{(v, c)}{(v_1, c_1)}$ and $\smallstep{(v, c)}{(v_2, c_2)}$, then $v_1 = v_2$ and $c_1 = c_2$.
\end{theorem}
\begin{proof}
By induction on the derivation of $\smallstep{(v, c)}{(v_1, c_1)}$ and inversion on the derivation of $\smallstep{(v, c)}{(v_2, c_2)}$.
\end{proof}
\begin{theorem}
If $\smallstepc{(v, c)}{(v_1, c_1)}$ and $\smallstepc{(v, c)}{(v_2, c_2)}$, then $v_1 = v_2$ and $c_1 = c_2$.
\end{theorem}
\begin{proof}
Follows from the last theorem and the equivalence we proved between $\to$ and $\to_\mathsf{c}$.
\end{proof}
We'll stop, for now, in our tour of useful properties of operational semantics.
All of the rest of the book is based on small-step semantics, with or without evaluation contexts.
As we study new kinds of programming languages, we will see how to model them operationally.
Almost every new proof technique is phrased as an approach to establishing invariants of transition systems based on small-step semantics.
%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%% %%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%%
\appendix \appendix