src/Doc/Prog_Prove/Types_and_funs.thy
author wenzelm
Tue, 31 Mar 2015 22:31:05 +0200
changeset 59886 e0dc738eb08c
parent 58860 fee7cfa69c50
child 64862 2baa926a958d
permissions -rw-r--r--
support for explicit scope of private entries;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
     1
(*<*)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
     2
theory Types_and_funs
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
     3
imports Main
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
     4
begin
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
     5
(*>*)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
     6
text{*
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
     7
\vspace{-5ex}
52361
7d5ad23b8245 all headings in upper case
nipkow
parents: 52045
diff changeset
     8
\section{Type and Function Definitions}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
     9
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    10
Type synonyms are abbreviations for existing types, for example
58521
nipkow
parents: 58519
diff changeset
    11
\index{string@@{text string}}*}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    12
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    13
type_synonym string = "char list"
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    14
58521
nipkow
parents: 58519
diff changeset
    15
text{*
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    16
Type synonyms are expanded after parsing and are not present in internal representation and output. They are mere conveniences for the reader.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    17
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    18
\subsection{Datatypes}
51465
c5c466706549 add label for referencing in semantics book
kleing
parents: 51393
diff changeset
    19
\label{sec:datatypes}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    20
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    21
The general form of a datatype definition looks like this:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    22
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    23
\begin{tabular}{@ {}rclcll}
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
    24
\indexed{\isacom{datatype}}{datatype} @{text "('a\<^sub>1,\<dots>,'a\<^sub>n)t"}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    25
     & = & $C_1 \ @{text"\""}\tau_{1,1}@{text"\""} \dots @{text"\""}\tau_{1,n_1}@{text"\""}$ \\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    26
     & $|$ & \dots \\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    27
     & $|$ & $C_k \ @{text"\""}\tau_{k,1}@{text"\""} \dots @{text"\""}\tau_{k,n_k}@{text"\""}$
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    28
\end{tabular}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    29
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    30
It introduces the constructors \
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
    31
$C_i :: \tau_{i,1}\Rightarrow \cdots \Rightarrow \tau_{i,n_i} \Rightarrow$~@{text "('a\<^sub>1,\<dots>,'a\<^sub>n)t"} \ and expresses that any value of this type is built from these constructors in a unique manner. Uniqueness is implied by the following
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    32
properties of the constructors:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    33
\begin{itemize}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    34
\item \emph{Distinctness:} $C_i\ \ldots \neq C_j\ \dots$ \quad if $i \neq j$
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    35
\item \emph{Injectivity:}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    36
\begin{tabular}[t]{l}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    37
 $(C_i \ x_1 \dots x_{n_i} = C_i \ y_1 \dots y_{n_i}) =$\\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    38
 $(x_1 = y_1 \land \dots \land x_{n_i} = y_{n_i})$
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    39
\end{tabular}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    40
\end{itemize}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    41
The fact that any value of the datatype is built from the constructors implies
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
    42
the \concept{structural induction}\index{induction} rule: to show
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
    43
$P~x$ for all $x$ of type @{text "('a\<^sub>1,\<dots>,'a\<^sub>n)t"},
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    44
one needs to show $P(C_i\ x_1 \dots x_{n_i})$ (for each $i$) assuming
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
    45
$P(x_j)$ for all $j$ where $\tau_{i,j} =$~@{text "('a\<^sub>1,\<dots>,'a\<^sub>n)t"}.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    46
Distinctness and injectivity are applied automatically by @{text auto}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    47
and other proof methods. Induction must be applied explicitly.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    48
58605
nipkow
parents: 58602
diff changeset
    49
Like in functional programming languages, datatype values can be taken apart
nipkow
parents: 58602
diff changeset
    50
with case expressions\index{case expression}\index{case expression@@{text "case ... of"}}, for example
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    51
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    52
\noquotes{@{term[source] "(case xs of [] \<Rightarrow> 0 | x # _ \<Rightarrow> Suc x)"}}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    53
\end{quote}
58605
nipkow
parents: 58602
diff changeset
    54
Case expressions must be enclosed in parentheses.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    55
58605
nipkow
parents: 58602
diff changeset
    56
As an example of a datatype beyond @{typ nat} and @{text list}, consider binary trees:
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    57
*}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    58
47306
56d72c923281 made sure that " is shown in tutorial text
nipkow
parents: 47269
diff changeset
    59
datatype 'a tree = Tip | Node  "'a tree"  'a  "'a tree"
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    60
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    61
text{* with a mirror function: *}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    62
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    63
fun mirror :: "'a tree \<Rightarrow> 'a tree" where
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    64
"mirror Tip = Tip" |
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    65
"mirror (Node l a r) = Node (mirror r) a (mirror l)"
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    66
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    67
text{* The following lemma illustrates induction: *}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    68
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    69
lemma "mirror(mirror t) = t"
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    70
apply(induction t)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    71
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    72
txt{* yields
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    73
@{subgoals[display]}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    74
The induction step contains two induction hypotheses, one for each subtree.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    75
An application of @{text auto} finishes the proof.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    76
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    77
A very simple but also very useful datatype is the predefined
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
    78
@{datatype[display] option}\index{option@@{text option}}\index{None@@{const None}}\index{Some@@{const Some}}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    79
Its sole purpose is to add a new element @{const None} to an existing
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    80
type @{typ 'a}. To make sure that @{const None} is distinct from all the
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    81
elements of @{typ 'a}, you wrap them up in @{const Some} and call
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    82
the new type @{typ"'a option"}. A typical application is a lookup function
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    83
on a list of key-value pairs, often called an association list:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    84
*}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    85
(*<*)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    86
apply auto
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    87
done
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    88
(*>*)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    89
fun lookup :: "('a * 'b) list \<Rightarrow> 'a \<Rightarrow> 'b option" where
47306
56d72c923281 made sure that " is shown in tutorial text
nipkow
parents: 47269
diff changeset
    90
"lookup [] x = None" |
56d72c923281 made sure that " is shown in tutorial text
nipkow
parents: 47269
diff changeset
    91
"lookup ((a,b) # ps) x = (if a = x then Some b else lookup ps x)"
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    92
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
    93
text{*
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
    94
Note that @{text"\<tau>\<^sub>1 * \<tau>\<^sub>2"} is the type of pairs, also written @{text"\<tau>\<^sub>1 \<times> \<tau>\<^sub>2"}.
51393
df0f306f030f added pairs
nipkow
parents: 48985
diff changeset
    95
Pairs can be taken apart either by pattern matching (as above) or with the
57804
nipkow
parents: 56989
diff changeset
    96
projection functions @{const fst} and @{const snd}: @{thm fst_conv[of x y]} and @{thm snd_conv[of x y]}.
nipkow
parents: 56989
diff changeset
    97
Tuples are simulated by pairs nested to the right: @{term"(a,b,c)"}
nipkow
parents: 56989
diff changeset
    98
is short for @{text"(a, (b, c))"} and @{text "\<tau>\<^sub>1 \<times> \<tau>\<^sub>2 \<times> \<tau>\<^sub>3"} is short for
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
    99
@{text "\<tau>\<^sub>1 \<times> (\<tau>\<^sub>2 \<times> \<tau>\<^sub>3)"}.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   100
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   101
\subsection{Definitions}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   102
56989
nipkow
parents: 56451
diff changeset
   103
Non-recursive functions can be defined as in the following example:
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
   104
\index{definition@\isacom{definition}}*}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   105
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   106
definition sq :: "nat \<Rightarrow> nat" where
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   107
"sq n = n * n"
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   108
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   109
text{* Such definitions do not allow pattern matching but only
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
   110
@{text"f x\<^sub>1 \<dots> x\<^sub>n = t"}, where @{text f} does not occur in @{text t}.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   111
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   112
\subsection{Abbreviations}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   113
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   114
Abbreviations are similar to definitions:
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
   115
\index{abbreviation@\isacom{abbreviation}}*}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   116
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   117
abbreviation sq' :: "nat \<Rightarrow> nat" where
52045
nipkow
parents: 51465
diff changeset
   118
"sq' n \<equiv> n * n"
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   119
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   120
text{* The key difference is that @{const sq'} is only syntactic sugar:
58521
nipkow
parents: 58519
diff changeset
   121
after parsing, @{term"sq' t"} is replaced by \mbox{@{term"t*t"}};
52045
nipkow
parents: 51465
diff changeset
   122
before printing, every occurrence of @{term"u*u"} is replaced by
nipkow
parents: 51465
diff changeset
   123
\mbox{@{term"sq' u"}}.  Internally, @{const sq'} does not exist.
nipkow
parents: 51465
diff changeset
   124
This is the
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   125
advantage of abbreviations over definitions: definitions need to be expanded
52045
nipkow
parents: 51465
diff changeset
   126
explicitly (\autoref{sec:rewr-defs}) whereas abbreviations are already
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   127
expanded upon parsing. However, abbreviations should be introduced sparingly:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   128
if abused, they can lead to a confusing discrepancy between the internal and
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   129
external view of a term.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   130
52045
nipkow
parents: 51465
diff changeset
   131
The ASCII representation of @{text"\<equiv>"} is \texttt{==} or \xsymbol{equiv}.
nipkow
parents: 51465
diff changeset
   132
52361
7d5ad23b8245 all headings in upper case
nipkow
parents: 52045
diff changeset
   133
\subsection{Recursive Functions}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   134
\label{sec:recursive-funs}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   135
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
   136
Recursive functions are defined with \indexed{\isacom{fun}}{fun} by pattern matching
56989
nipkow
parents: 56451
diff changeset
   137
over datatype constructors. The order of equations matters, as in
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   138
functional programming languages. However, all HOL functions must be
58602
ab56811d76c6 tuned spaces
nipkow
parents: 58521
diff changeset
   139
total. This simplifies the logic --- terms are always defined --- but means
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   140
that recursive functions must terminate. Otherwise one could define a
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   141
function @{prop"f n = f n + (1::nat)"} and conclude \mbox{@{prop"(0::nat) = 1"}} by
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   142
subtracting @{term"f n"} on both sides.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   143
47711
c1cca2a052e4 doc update
nipkow
parents: 47306
diff changeset
   144
Isabelle's automatic termination checker requires that the arguments of
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   145
recursive calls on the right-hand side must be strictly smaller than the
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   146
arguments on the left-hand side. In the simplest case, this means that one
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   147
fixed argument position decreases in size with each recursive call. The size
58504
nipkow
parents: 58502
diff changeset
   148
is measured as the number of constructors (excluding 0-ary ones, e.g., @{text
47711
c1cca2a052e4 doc update
nipkow
parents: 47306
diff changeset
   149
Nil}). Lexicographic combinations are also recognized. In more complicated
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   150
situations, the user may have to prove termination by hand. For details
58620
7435b6a3f72e more antiquotations;
wenzelm
parents: 58605
diff changeset
   151
see~@{cite Krauss}.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   152
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   153
Functions defined with \isacom{fun} come with their own induction schema
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   154
that mirrors the recursion schema and is derived from the termination
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   155
order. For example,
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   156
*}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   157
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   158
fun div2 :: "nat \<Rightarrow> nat" where
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   159
"div2 0 = 0" |
54136
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   160
"div2 (Suc 0) = 0" |
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   161
"div2 (Suc(Suc n)) = Suc(div2 n)"
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   162
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   163
text{* does not just define @{const div2} but also proves a
47711
c1cca2a052e4 doc update
nipkow
parents: 47306
diff changeset
   164
customized induction rule:
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   165
\[
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   166
\inferrule{
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   167
\mbox{@{thm (prem 1) div2.induct}}\\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   168
\mbox{@{thm (prem 2) div2.induct}}\\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   169
\mbox{@{thm (prem 3) div2.induct}}}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   170
{\mbox{@{thm (concl) div2.induct[of _ "m"]}}}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   171
\]
47711
c1cca2a052e4 doc update
nipkow
parents: 47306
diff changeset
   172
This customized induction rule can simplify inductive proofs. For example,
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   173
*}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   174
54571
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   175
lemma "div2(n) = n div 2"
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   176
apply(induction n rule: div2.induct)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   177
54571
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   178
txt{* (where the infix @{text div} is the predefined division operation)
56989
nipkow
parents: 56451
diff changeset
   179
yields the subgoals
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   180
@{subgoals[display,margin=65]}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   181
An application of @{text auto} finishes the proof.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   182
Had we used ordinary structural induction on @{text n},
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   183
the proof would have needed an additional
47711
c1cca2a052e4 doc update
nipkow
parents: 47306
diff changeset
   184
case analysis in the induction step.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   185
54571
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   186
This example leads to the following induction heuristic:
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   187
\begin{quote}
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   188
\emph{Let @{text f} be a recursive function.
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   189
If the definition of @{text f} is more complicated
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   190
than having one equation for each constructor of some datatype,
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
   191
then properties of @{text f} are best proved via @{text "f.induct"}.\index{inductionrule@@{text".induct"}}}
54571
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   192
\end{quote}
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   193
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   194
The general case is often called \concept{computation induction},
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   195
because the induction follows the (terminating!) computation.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   196
For every defining equation
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   197
\begin{quote}
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
   198
@{text "f(e) = \<dots> f(r\<^sub>1) \<dots> f(r\<^sub>k) \<dots>"}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   199
\end{quote}
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
   200
where @{text"f(r\<^sub>i)"}, @{text"i=1\<dots>k"}, are all the recursive calls,
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   201
the induction rule @{text"f.induct"} contains one premise of the form
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   202
\begin{quote}
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
   203
@{text"P(r\<^sub>1) \<Longrightarrow> \<dots> \<Longrightarrow> P(r\<^sub>k) \<Longrightarrow> P(e)"}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   204
\end{quote}
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
   205
If @{text "f :: \<tau>\<^sub>1 \<Rightarrow> \<dots> \<Rightarrow> \<tau>\<^sub>n \<Rightarrow> \<tau>"} then @{text"f.induct"} is applied like this:
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   206
\begin{quote}
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
   207
\isacom{apply}@{text"(induction x\<^sub>1 \<dots> x\<^sub>n rule: f.induct)"}\index{inductionrule@@{text"induction ... rule:"}}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   208
\end{quote}
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
   209
where typically there is a call @{text"f x\<^sub>1 \<dots> x\<^sub>n"} in the goal.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   210
But note that the induction rule does not mention @{text f} at all,
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   211
except in its name, and is applicable independently of @{text f}.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   212
54136
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   213
54436
nipkow
parents: 54195
diff changeset
   214
\subsection*{Exercises}
54136
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   215
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   216
\begin{exercise}
54194
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   217
Starting from the type @{text "'a tree"} defined in the text, define
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   218
a function @{text "contents ::"} @{typ "'a tree \<Rightarrow> 'a list"}
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   219
that collects all values in a tree in a list, in any order,
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   220
without removing duplicates.
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   221
Then define a function @{text "treesum ::"} @{typ "nat tree \<Rightarrow> nat"}
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   222
that sums up all values in a tree of natural numbers
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   223
and prove @{prop "treesum t = listsum(contents t)"}.
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   224
\end{exercise}
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   225
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   226
\begin{exercise}
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   227
Define a new type @{text "'a tree2"} of binary trees where values are also
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   228
stored in the leaves of the tree.  Also reformulate the
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   229
@{const mirror} function accordingly. Define two functions
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   230
@{text "pre_order"} and @{text "post_order"} of type @{text "'a tree2 \<Rightarrow> 'a list"}
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   231
that traverse a tree and collect all stored values in the respective order in
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   232
a list. Prove @{prop "pre_order (mirror t) = rev (post_order t)"}.
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   233
\end{exercise}
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   234
12c9ad3142be added exercises
nipkow
parents: 54136
diff changeset
   235
\begin{exercise}
54571
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   236
Define a function @{text "intersperse ::"} @{typ "'a \<Rightarrow> 'a list \<Rightarrow> 'a list"}
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   237
such that @{text "intersperse a [x\<^sub>1, ..., x\<^sub>n] = [x\<^sub>1, a, x\<^sub>2, a, ..., a, x\<^sub>n]"}.
be1186cb03ce replaced bad example
nipkow
parents: 54467
diff changeset
   238
Now prove that @{prop "map f (intersperse a xs) = intersperse (f a) (map f xs)"}.
54136
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   239
\end{exercise}
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   240
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   241
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
   242
\section{Induction Heuristics}\index{induction heuristics}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   243
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   244
We have already noted that theorems about recursive functions are proved by
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   245
induction. In case the function has more than one argument, we have followed
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   246
the following heuristic in the proofs about the append function:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   247
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   248
\emph{Perform induction on argument number $i$\\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   249
 if the function is defined by recursion on argument number $i$.}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   250
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   251
The key heuristic, and the main point of this section, is to
58502
nipkow
parents: 58486
diff changeset
   252
\emph{generalize the goal before induction}.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   253
The reason is simple: if the goal is
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   254
too specific, the induction hypothesis is too weak to allow the induction
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   255
step to go through. Let us illustrate the idea with an example.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   256
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   257
Function @{const rev} has quadratic worst-case running time
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   258
because it calls append for each element of the list and
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   259
append is linear in its first argument.  A linear time version of
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   260
@{const rev} requires an extra argument where the result is accumulated
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   261
gradually, using only~@{text"#"}:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   262
*}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   263
(*<*)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   264
apply auto
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   265
done
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   266
(*>*)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   267
fun itrev :: "'a list \<Rightarrow> 'a list \<Rightarrow> 'a list" where
47711
c1cca2a052e4 doc update
nipkow
parents: 47306
diff changeset
   268
"itrev []        ys = ys" |
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   269
"itrev (x#xs) ys = itrev xs (x#ys)"
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   270
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   271
text{* The behaviour of @{const itrev} is simple: it reverses
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   272
its first argument by stacking its elements onto the second argument,
47711
c1cca2a052e4 doc update
nipkow
parents: 47306
diff changeset
   273
and it returns that second argument when the first one becomes
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   274
empty. Note that @{const itrev} is tail-recursive: it can be
56989
nipkow
parents: 56451
diff changeset
   275
compiled into a loop; no stack is necessary for executing it.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   276
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   277
Naturally, we would like to show that @{const itrev} does indeed reverse
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   278
its first argument provided the second one is empty:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   279
*}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   280
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   281
lemma "itrev xs [] = rev xs"
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   282
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   283
txt{* There is no choice as to the induction variable:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   284
*}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   285
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   286
apply(induction xs)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   287
apply(auto)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   288
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   289
txt{*
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   290
Unfortunately, this attempt does not prove
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   291
the induction step:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   292
@{subgoals[display,margin=70]}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   293
The induction hypothesis is too weak.  The fixed
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   294
argument,~@{term"[]"}, prevents it from rewriting the conclusion.  
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   295
This example suggests a heuristic:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   296
\begin{quote}
58502
nipkow
parents: 58486
diff changeset
   297
\emph{Generalize goals for induction by replacing constants by variables.}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   298
\end{quote}
58519
nipkow
parents: 58504
diff changeset
   299
Of course one cannot do this naively: @{prop"itrev xs ys = rev xs"} is
58502
nipkow
parents: 58486
diff changeset
   300
just not true.  The correct generalization is
58860
fee7cfa69c50 eliminated spurious semicolons;
wenzelm
parents: 58620
diff changeset
   301
*}
fee7cfa69c50 eliminated spurious semicolons;
wenzelm
parents: 58620
diff changeset
   302
(*<*)oops(*>*)
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   303
lemma "itrev xs ys = rev xs @ ys"
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   304
(*<*)apply(induction xs, auto)(*>*)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   305
txt{*
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   306
If @{text ys} is replaced by @{term"[]"}, the right-hand side simplifies to
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   307
@{term"rev xs"}, as required.
58502
nipkow
parents: 58486
diff changeset
   308
In this instance it was easy to guess the right generalization.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   309
Other situations can require a good deal of creativity.  
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   310
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   311
Although we now have two variables, only @{text xs} is suitable for
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   312
induction, and we repeat our proof attempt. Unfortunately, we are still
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   313
not there:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   314
@{subgoals[display,margin=65]}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   315
The induction hypothesis is still too weak, but this time it takes no
58502
nipkow
parents: 58486
diff changeset
   316
intuition to generalize: the problem is that the @{text ys}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   317
in the induction hypothesis is fixed,
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   318
but the induction hypothesis needs to be applied with
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   319
@{term"a # ys"} instead of @{text ys}. Hence we prove the theorem
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   320
for all @{text ys} instead of a fixed one. We can instruct induction
58502
nipkow
parents: 58486
diff changeset
   321
to perform this generalization for us by adding @{text "arbitrary: ys"}\index{arbitrary@@{text"arbitrary:"}}.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   322
*}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   323
(*<*)oops
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   324
lemma "itrev xs ys = rev xs @ ys"
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   325
(*>*)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   326
apply(induction xs arbitrary: ys)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   327
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   328
txt{* The induction hypothesis in the induction step is now universally quantified over @{text ys}:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   329
@{subgoals[display,margin=65]}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   330
Thus the proof succeeds:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   331
*}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   332
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   333
apply auto
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   334
done
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   335
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   336
text{*
58502
nipkow
parents: 58486
diff changeset
   337
This leads to another heuristic for generalization:
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   338
\begin{quote}
58502
nipkow
parents: 58486
diff changeset
   339
\emph{Generalize induction by generalizing all free
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   340
variables\\ {\em(except the induction variable itself)}.}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   341
\end{quote}
58502
nipkow
parents: 58486
diff changeset
   342
Generalization is best performed with @{text"arbitrary: y\<^sub>1 \<dots> y\<^sub>k"}. 
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   343
This heuristic prevents trivial failures like the one above.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   344
However, it should not be applied blindly.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   345
It is not always required, and the additional quantifiers can complicate
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   346
matters in some cases. The variables that need to be quantified are typically
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   347
those that change in recursive calls.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   348
54136
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   349
54436
nipkow
parents: 54195
diff changeset
   350
\subsection*{Exercises}
54136
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   351
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   352
\begin{exercise}
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   353
Write a tail-recursive variant of the @{text add} function on @{typ nat}:
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   354
@{term "itadd :: nat \<Rightarrow> nat \<Rightarrow> nat"}.
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   355
Tail-recursive means that in the recursive case, @{text itadd} needs to call
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   356
itself directly: \mbox{@{term"itadd (Suc m) n"}} @{text"= itadd \<dots>"}.
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   357
Prove @{prop "itadd m n = add m n"}.
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   358
\end{exercise}
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   359
c206cb2a3afe more exercises
nipkow
parents: 53015
diff changeset
   360
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   361
\section{Simplification}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   362
55317
834a84553e02 started index
nipkow
parents: 54605
diff changeset
   363
So far we have talked a lot about simplifying terms without explaining the concept.
834a84553e02 started index
nipkow
parents: 54605
diff changeset
   364
\conceptidx{Simplification}{simplification} means
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   365
\begin{itemize}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   366
\item using equations $l = r$ from left to right (only),
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   367
\item as long as possible.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   368
\end{itemize}
47711
c1cca2a052e4 doc update
nipkow
parents: 47306
diff changeset
   369
To emphasize the directionality, equations that have been given the
55317
834a84553e02 started index
nipkow
parents: 54605
diff changeset
   370
@{text"simp"} attribute are called \conceptidx{simplification rules}{simplification rule}.
834a84553e02 started index
nipkow
parents: 54605
diff changeset
   371
Logically, they are still symmetric, but proofs by
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   372
simplification use them only in the left-to-right direction.  The proof tool
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   373
that performs simplifications is called the \concept{simplifier}. It is the
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   374
basis of @{text auto} and other related proof methods.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   375
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   376
The idea of simplification is best explained by an example. Given the
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   377
simplification rules
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   378
\[
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   379
\begin{array}{rcl@ {\quad}l}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   380
@{term"0 + n::nat"} &@{text"="}& @{text n} & (1) \\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   381
@{term"(Suc m) + n"} &@{text"="}& @{term"Suc (m + n)"} & (2) \\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   382
@{text"(Suc m \<le> Suc n)"} &@{text"="}& @{text"(m \<le> n)"} & (3)\\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   383
@{text"(0 \<le> m)"} &@{text"="}& @{const True} & (4)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   384
\end{array}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   385
\]
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   386
the formula @{prop"0 + Suc 0 \<le> Suc 0 + x"} is simplified to @{const True}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   387
as follows:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   388
\[
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   389
\begin{array}{r@ {}c@ {}l@ {\quad}l}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   390
@{text"(0 + Suc 0"} & \leq & @{text"Suc 0 + x)"}  & \stackrel{(1)}{=} \\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   391
@{text"(Suc 0"}     & \leq & @{text"Suc 0 + x)"}  & \stackrel{(2)}{=} \\
57817
nipkow
parents: 57804
diff changeset
   392
@{text"(Suc 0"}     & \leq & @{text"Suc (0 + x))"} & \stackrel{(3)}{=} \\
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   393
@{text"(0"}         & \leq & @{text"0 + x)"}      & \stackrel{(4)}{=} \\[1ex]
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   394
 & @{const True}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   395
\end{array}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   396
\]
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   397
Simplification is often also called \concept{rewriting}
55317
834a84553e02 started index
nipkow
parents: 54605
diff changeset
   398
and simplification rules \conceptidx{rewrite rules}{rewrite rule}.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   399
52361
7d5ad23b8245 all headings in upper case
nipkow
parents: 52045
diff changeset
   400
\subsection{Simplification Rules}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   401
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   402
The attribute @{text"simp"} declares theorems to be simplification rules,
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   403
which the simplifier will use automatically. In addition,
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   404
\isacom{datatype} and \isacom{fun} commands implicitly declare some
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   405
simplification rules: \isacom{datatype} the distinctness and injectivity
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   406
rules, \isacom{fun} the defining equations. Definitions are not declared
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   407
as simplification rules automatically! Nearly any theorem can become a
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   408
simplification rule. The simplifier will try to transform it into an
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   409
equation. For example, the theorem @{prop"\<not> P"} is turned into @{prop"P = False"}.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   410
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   411
Only equations that really simplify, like @{prop"rev (rev xs) = xs"} and
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   412
@{prop"xs @ [] = xs"}, should be declared as simplification
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   413
rules. Equations that may be counterproductive as simplification rules
58521
nipkow
parents: 58519
diff changeset
   414
should only be used in specific proof steps (see \autoref{sec:simp} below).
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   415
Distributivity laws, for example, alter the structure of terms
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   416
and can produce an exponential blow-up.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   417
52361
7d5ad23b8245 all headings in upper case
nipkow
parents: 52045
diff changeset
   418
\subsection{Conditional Simplification Rules}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   419
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   420
Simplification rules can be conditional.  Before applying such a rule, the
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   421
simplifier will first try to prove the preconditions, again by
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   422
simplification. For example, given the simplification rules
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   423
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   424
@{prop"p(0::nat) = True"}\\
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   425
@{prop"p(x) \<Longrightarrow> f(x) = g(x)"},
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   426
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   427
the term @{term"f(0::nat)"} simplifies to @{term"g(0::nat)"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   428
but @{term"f(1::nat)"} does not simplify because @{prop"p(1::nat)"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   429
is not provable.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   430
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   431
\subsection{Termination}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   432
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   433
Simplification can run forever, for example if both @{prop"f x = g x"} and
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   434
@{prop"g(x) = f(x)"} are simplification rules. It is the user's
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   435
responsibility not to include simplification rules that can lead to
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   436
nontermination, either on their own or in combination with other
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   437
simplification rules. The right-hand side of a simplification rule should
58602
ab56811d76c6 tuned spaces
nipkow
parents: 58521
diff changeset
   438
always be ``simpler'' than the left-hand side --- in some sense. But since
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   439
termination is undecidable, such a check cannot be automated completely
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   440
and Isabelle makes little attempt to detect nontermination.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   441
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   442
When conditional simplification rules are applied, their preconditions are
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   443
proved first. Hence all preconditions need to be
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   444
simpler than the left-hand side of the conclusion. For example
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   445
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   446
@{prop "n < m \<Longrightarrow> (n < Suc m) = True"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   447
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   448
is suitable as a simplification rule: both @{prop"n<m"} and @{const True}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   449
are simpler than \mbox{@{prop"n < Suc m"}}. But
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   450
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   451
@{prop "Suc n < m \<Longrightarrow> (n < m) = True"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   452
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   453
leads to nontermination: when trying to rewrite @{prop"n<m"} to @{const True}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   454
one first has to prove \mbox{@{prop"Suc n < m"}}, which can be rewritten to @{const True} provided @{prop"Suc(Suc n) < m"}, \emph{ad infinitum}.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   455
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
   456
\subsection{The \indexed{@{text simp}}{simp} Proof Method}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   457
\label{sec:simp}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   458
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   459
So far we have only used the proof method @{text auto}.  Method @{text simp}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   460
is the key component of @{text auto}, but @{text auto} can do much more. In
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   461
some cases, @{text auto} is overeager and modifies the proof state too much.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   462
In such cases the more predictable @{text simp} method should be used.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   463
Given a goal
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   464
\begin{quote}
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
   465
@{text"1. \<lbrakk> P\<^sub>1; \<dots>; P\<^sub>m \<rbrakk> \<Longrightarrow> C"}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   466
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   467
the command
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   468
\begin{quote}
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
   469
\isacom{apply}@{text"(simp add: th\<^sub>1 \<dots> th\<^sub>n)"}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   470
\end{quote}
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
   471
simplifies the assumptions @{text "P\<^sub>i"} and the conclusion @{text C} using
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   472
\begin{itemize}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   473
\item all simplification rules, including the ones coming from \isacom{datatype} and \isacom{fun},
53015
a1119cf551e8 standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
wenzelm
parents: 52718
diff changeset
   474
\item the additional lemmas @{text"th\<^sub>1 \<dots> th\<^sub>n"}, and
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   475
\item the assumptions.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   476
\end{itemize}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   477
In addition to or instead of @{text add} there is also @{text del} for removing
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   478
simplification rules temporarily. Both are optional. Method @{text auto}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   479
can be modified similarly:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   480
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   481
\isacom{apply}@{text"(auto simp add: \<dots> simp del: \<dots>)"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   482
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   483
Here the modifiers are @{text"simp add"} and @{text"simp del"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   484
instead of just @{text add} and @{text del} because @{text auto}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   485
does not just perform simplification.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   486
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   487
Note that @{text simp} acts only on subgoal 1, @{text auto} acts on all
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   488
subgoals. There is also @{text simp_all}, which applies @{text simp} to
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   489
all subgoals.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   490
56989
nipkow
parents: 56451
diff changeset
   491
\subsection{Rewriting with Definitions}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   492
\label{sec:rewr-defs}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   493
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   494
Definitions introduced by the command \isacom{definition}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   495
can also be used as simplification rules,
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   496
but by default they are not: the simplifier does not expand them
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   497
automatically. Definitions are intended for introducing abstract concepts and
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   498
not merely as abbreviations. Of course, we need to expand the definition
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   499
initially, but once we have proved enough abstract properties of the new
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   500
constant, we can forget its original definition. This style makes proofs more
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   501
robust: if the definition has to be changed, only the proofs of the abstract
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   502
properties will be affected.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   503
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   504
The definition of a function @{text f} is a theorem named @{text f_def}
58605
nipkow
parents: 58602
diff changeset
   505
and can be added to a call of @{text simp} like any other theorem:
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   506
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   507
\isacom{apply}@{text"(simp add: f_def)"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   508
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   509
In particular, let-expressions can be unfolded by
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   510
making @{thm[source] Let_def} a simplification rule.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   511
52361
7d5ad23b8245 all headings in upper case
nipkow
parents: 52045
diff changeset
   512
\subsection{Case Splitting With @{text simp}}
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   513
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   514
Goals containing if-expressions are automatically split into two cases by
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   515
@{text simp} using the rule
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   516
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   517
@{prop"P(if A then s else t) = ((A \<longrightarrow> P(s)) \<and> (~A \<longrightarrow> P(t)))"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   518
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   519
For example, @{text simp} can prove
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   520
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   521
@{prop"(A \<and> B) = (if A then B else False)"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   522
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   523
because both @{prop"A \<longrightarrow> (A & B) = B"} and @{prop"~A \<longrightarrow> (A & B) = False"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   524
simplify to @{const True}.
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   525
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   526
We can split case-expressions similarly. For @{text nat} the rule looks like this:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   527
@{prop[display,margin=65,indent=4]"P(case e of 0 \<Rightarrow> a | Suc n \<Rightarrow> b n) = ((e = 0 \<longrightarrow> P a) & (ALL n. e = Suc n \<longrightarrow> P(b n)))"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   528
Case expressions are not split automatically by @{text simp}, but @{text simp}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   529
can be instructed to do so:
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   530
\begin{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   531
\isacom{apply}@{text"(simp split: nat.split)"}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   532
\end{quote}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   533
splits all case-expressions over natural numbers. For an arbitrary
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
   534
datatype @{text t} it is @{text "t.split"}\index{split@@{text".split"}} instead of @{thm[source] nat.split}.
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   535
Method @{text auto} can be modified in exactly the same way.
55348
366718f2ff85 indexed document
nipkow
parents: 55318
diff changeset
   536
The modifier \indexed{@{text "split:"}}{split} can be followed by multiple names.
54605
nipkow
parents: 54571
diff changeset
   537
Splitting if or case-expressions in the assumptions requires 
nipkow
parents: 54571
diff changeset
   538
@{text "split: if_splits"} or @{text "split: t.splits"}.
52593
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   539
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   540
54436
nipkow
parents: 54195
diff changeset
   541
\subsection*{Exercises}
52593
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   542
54195
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   543
\exercise\label{exe:tree0}
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   544
Define a datatype @{text tree0} of binary tree skeletons which do not store
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   545
any information, neither in the inner nodes nor in the leaves.
54467
663a927fdc88 comments by Sean Seefried
nipkow
parents: 54436
diff changeset
   546
Define a function @{text "nodes :: tree0 \<Rightarrow> nat"} that counts the number of
54195
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   547
all nodes (inner nodes and leaves) in such a tree.
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   548
Consider the following recursive function:
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   549
*}
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   550
(*<*)
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   551
datatype tree0 = Tip | Node tree0 tree0
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   552
(*>*)
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   553
fun explode :: "nat \<Rightarrow> tree0 \<Rightarrow> tree0" where
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   554
"explode 0 t = t" |
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   555
"explode (Suc n) t = explode n (Node t t)"
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   556
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   557
text {*
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   558
Find an equation expressing the size of a tree after exploding it
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   559
(\noquotes{@{term [source] "nodes (explode n t)"}}) as a function
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   560
of @{term "nodes t"} and @{text n}. Prove your equation.
56989
nipkow
parents: 56451
diff changeset
   561
You may use the usual arithmetic operators, including the exponentiation
54195
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   562
operator ``@{text"^"}''. For example, \noquotes{@{prop [source] "2 ^ 2 = 4"}}.
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   563
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   564
Hint: simplifying with the list of theorems @{thm[source] algebra_simps}
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   565
takes care of common algebraic properties of the arithmetic operators.
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   566
\endexercise
1e685123926d more exercises
nipkow
parents: 54194
diff changeset
   567
52593
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   568
\exercise
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   569
Define arithmetic expressions in one variable over integers (type @{typ int})
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   570
as a data type:
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   571
*}
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   572
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   573
datatype exp = Var | Const int | Add exp exp | Mult exp exp
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   574
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   575
text{*
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   576
Define a function \noquotes{@{term [source]"eval :: exp \<Rightarrow> int \<Rightarrow> int"}}
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   577
such that @{term"eval e x"} evaluates @{text e} at the value
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   578
@{text x}.
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   579
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   580
A polynomial can be represented as a list of coefficients, starting with
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   581
the constant. For example, @{term "[4, 2, -1, 3::int]"} represents the
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   582
polynomial $4 + 2x - x^2 + 3x^3$.
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   583
Define a function \noquotes{@{term [source] "evalp :: int list \<Rightarrow> int \<Rightarrow> int"}}
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   584
that evaluates a polynomial at the given value.
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   585
Define a function \noquotes{@{term[source] "coeffs :: exp \<Rightarrow> int list"}}
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   586
that transforms an expression into a polynomial. This may require auxiliary
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   587
functions. Prove that @{text coeffs} preserves the value of the expression:
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   588
\mbox{@{prop"evalp (coeffs e) x = eval e x"}.}
54467
663a927fdc88 comments by Sean Seefried
nipkow
parents: 54436
diff changeset
   589
Hint: consider the hint in Exercise~\ref{exe:tree0}.
52593
aedf7b01c6e4 added exercises
nipkow
parents: 52361
diff changeset
   590
\endexercise
47269
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   591
*}
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   592
(*<*)
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   593
end
29aa0c071875 New manual Programming and Proving in Isabelle/HOL
nipkow
parents:
diff changeset
   594
(*>*)