| author | wenzelm | 
| Fri, 29 Oct 2010 11:07:21 +0200 | |
| changeset 40253 | f99ec71de82d | 
| parent 39795 | 9e59b4c11039 | 
| child 43564 | 9864182c6bad | 
| permissions | -rw-r--r-- | 
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 1 | (*<*)theory Advanced imports Even uses "../../antiquote_setup.ML" begin(*>*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 2 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 3 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 4 | The premises of introduction rules may contain universal quantifiers and | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 5 | monotone functions. A universal quantifier lets the rule | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 6 | refer to any number of instances of | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 7 | the inductively defined set. A monotone function lets the rule refer | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 8 | to existing constructions (such as ``list of'') over the inductively defined | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 9 | set. The examples below show how to use the additional expressiveness | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 10 | and how to reason from the resulting definitions. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 11 | *} | 
| 10426 | 12 | |
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 13 | subsection{* Universal Quantifiers in Introduction Rules \label{sec:gterm-datatype} *}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 14 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 15 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 16 | \index{ground terms example|(}%
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 17 | \index{quantifiers!and inductive definitions|(}%
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 18 | As a running example, this section develops the theory of \textbf{ground
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 19 | terms}: terms constructed from constant and function | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 20 | symbols but not variables. To simplify matters further, we regard a | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 21 | constant as a function applied to the null argument list. Let us declare a | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 22 | datatype @{text gterm} for the type of ground  terms. It is a type constructor
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 23 | whose argument is a type of function symbols. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 24 | *} | 
| 10468 | 25 | |
| 26 | datatype 'f gterm = Apply 'f "'f gterm list" | |
| 27 | ||
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 28 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 29 | To try it out, we declare a datatype of some integer operations: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 30 | integer constants, the unary minus operator and the addition | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 31 | operator. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 32 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 33 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 34 | datatype integer_op = Number int | UnaryMinus | Plus | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 35 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 36 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 37 | Now the type @{typ "integer_op gterm"} denotes the ground 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 38 | terms built over those symbols. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 39 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 40 | The type constructor @{text gterm} can be generalized to a function 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 41 | over sets. It returns | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 42 | the set of ground terms that can be formed over a set @{text F} of function symbols. For
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 43 | example, we could consider the set of ground terms formed from the finite | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 44 | set @{text "{Number 2, UnaryMinus, Plus}"}.
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 45 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 46 | This concept is inductive. If we have a list @{text args} of ground terms 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 47 | over~@{text F} and a function symbol @{text f} in @{text F}, then we 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 48 | can apply @{text f} to @{text args} to obtain another ground term. 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 49 | The only difficulty is that the argument list may be of any length. Hitherto, | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 50 | each rule in an inductive definition referred to the inductively | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 51 | defined set a fixed number of times, typically once or twice. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 52 | A universal quantifier in the premise of the introduction rule | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 53 | expresses that every element of @{text args} belongs
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 54 | to our inductively defined set: is a ground term | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 55 | over~@{text F}.  The function @{term set} denotes the set of elements in a given 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 56 | list. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 57 | *} | 
| 10468 | 58 | |
| 23733 | 59 | inductive_set | 
| 60 | gterms :: "'f set \<Rightarrow> 'f gterm set" | |
| 61 | for F :: "'f set" | |
| 62 | where | |
| 10468 | 63 | step[intro!]: "\<lbrakk>\<forall>t \<in> set args. t \<in> gterms F; f \<in> F\<rbrakk> | 
| 64 | \<Longrightarrow> (Apply f args) \<in> gterms F" | |
| 65 | ||
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 66 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 67 | To demonstrate a proof from this definition, let us | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 68 | show that the function @{term gterms}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 69 | is \textbf{monotone}.  We shall need this concept shortly.
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 70 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 71 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 72 | lemma gterms_mono: "F\<subseteq>G \<Longrightarrow> gterms F \<subseteq> gterms G" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 73 | apply clarify | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 74 | apply (erule gterms.induct) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 75 | apply blast | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 76 | done | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 77 | (*<*) | 
| 10468 | 78 | lemma gterms_mono: "F\<subseteq>G \<Longrightarrow> gterms F \<subseteq> gterms G" | 
| 79 | apply clarify | |
| 80 | apply (erule gterms.induct) | |
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 81 | (*>*) | 
| 10882 | 82 | txt{*
 | 
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 83 | Intuitively, this theorem says that | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 84 | enlarging the set of function symbols enlarges the set of ground | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 85 | terms. The proof is a trivial rule induction. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 86 | First we use the @{text clarify} method to assume the existence of an element of
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 87 | @{term "gterms F"}.  (We could have used @{text "intro subsetI"}.)  We then
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 88 | apply rule induction. Here is the resulting subgoal: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 89 | @{subgoals[display,indent=0]}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 90 | The assumptions state that @{text f} belongs 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 91 | to~@{text F}, which is included in~@{text G}, and that every element of the list @{text args} is
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 92 | a ground term over~@{text G}.  The @{text blast} method finds this chain of reasoning easily.  
 | 
| 10468 | 93 | *} | 
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 94 | (*<*)oops(*>*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 95 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 96 | \begin{warn}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 97 | Why do we call this function @{text gterms} instead 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 98 | of @{text gterm}?  A constant may have the same name as a type.  However,
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 99 | name clashes could arise in the theorems that Isabelle generates. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 100 | Our choice of names keeps @{text gterms.induct} separate from 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 101 | @{text gterm.induct}.
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 102 | \end{warn}
 | 
| 10468 | 103 | |
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 104 | Call a term \textbf{well-formed} if each symbol occurring in it is applied
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 105 | to the correct number of arguments. (This number is called the symbol's | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 106 | \textbf{arity}.)  We can express well-formedness by
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 107 | generalizing the inductive definition of | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 108 | \isa{gterms}.
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 109 | Suppose we are given a function called @{text arity}, specifying the arities
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 110 | of all symbols.  In the inductive step, we have a list @{text args} of such
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 111 | terms and a function  symbol~@{text f}. If the length of the list matches the
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 112 | function's arity  then applying @{text f} to @{text args} yields a well-formed
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 113 | term. | 
| 10468 | 114 | *} | 
| 10426 | 115 | |
| 23733 | 116 | inductive_set | 
| 117 |   well_formed_gterm :: "('f \<Rightarrow> nat) \<Rightarrow> 'f gterm set"
 | |
| 118 | for arity :: "'f \<Rightarrow> nat" | |
| 119 | where | |
| 10468 | 120 | step[intro!]: "\<lbrakk>\<forall>t \<in> set args. t \<in> well_formed_gterm arity; | 
| 121 | length args = arity f\<rbrakk> | |
| 122 | \<Longrightarrow> (Apply f args) \<in> well_formed_gterm arity" | |
| 123 | ||
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 124 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 125 | The inductive definition neatly captures the reasoning above. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 126 | The universal quantification over the | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 127 | @{text set} of arguments expresses that all of them are well-formed.%
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 128 | \index{quantifiers!and inductive definitions|)}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 129 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 130 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 131 | subsection{* Alternative Definition Using a Monotone Function *}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 132 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 133 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 134 | \index{monotone functions!and inductive definitions|(}% 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 135 | An inductive definition may refer to the | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 136 | inductively defined set through an arbitrary monotone function. To | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 137 | demonstrate this powerful feature, let us | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 138 | change the inductive definition above, replacing the | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 139 | quantifier by a use of the function @{term lists}. This
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 140 | function, from the Isabelle theory of lists, is analogous to the | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 141 | function @{term gterms} declared above: if @{text A} is a set then
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 142 | @{term "lists A"} is the set of lists whose elements belong to
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 143 | @{term A}.  
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 144 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 145 | In the inductive definition of well-formed terms, examine the one | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 146 | introduction rule.  The first premise states that @{text args} belongs to
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 147 | the @{text lists} of well-formed terms.  This formulation is more
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 148 | direct, if more obscure, than using a universal quantifier. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 149 | *} | 
| 10426 | 150 | |
| 23733 | 151 | inductive_set | 
| 152 |   well_formed_gterm' :: "('f \<Rightarrow> nat) \<Rightarrow> 'f gterm set"
 | |
| 153 | for arity :: "'f \<Rightarrow> nat" | |
| 154 | where | |
| 10468 | 155 | step[intro!]: "\<lbrakk>args \<in> lists (well_formed_gterm' arity); | 
| 156 | length args = arity f\<rbrakk> | |
| 157 | \<Longrightarrow> (Apply f args) \<in> well_formed_gterm' arity" | |
| 158 | monos lists_mono | |
| 159 | ||
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 160 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 161 | We cite the theorem @{text lists_mono} to justify 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 162 | using the function @{term lists}.%
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 163 | \footnote{This particular theorem is installed by default already, but we
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 164 | include the \isakeyword{monos} declaration in order to illustrate its syntax.}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 165 | @{named_thms [display,indent=0] lists_mono [no_vars] (lists_mono)}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 166 | Why must the function be monotone? An inductive definition describes | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 167 | an iterative construction: each element of the set is constructed by a | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 168 | finite number of introduction rule applications. For example, the | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 169 | elements of \isa{even} are constructed by finitely many applications of
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 170 | the rules | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 171 | @{thm [display,indent=0] even.intros [no_vars]}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 172 | All references to a set in its | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 173 | inductive definition must be positive. Applications of an | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 174 | introduction rule cannot invalidate previous applications, allowing the | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 175 | construction process to converge. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 176 | The following pair of rules do not constitute an inductive definition: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 177 | \begin{trivlist}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 178 | \item @{term "0 \<in> even"}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 179 | \item @{term "n \<notin> even \<Longrightarrow> (Suc n) \<in> even"}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 180 | \end{trivlist}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 181 | Showing that 4 is even using these rules requires showing that 3 is not | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 182 | even. It is far from trivial to show that this set of rules | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 183 | characterizes the even numbers. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 184 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 185 | Even with its use of the function \isa{lists}, the premise of our
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 186 | introduction rule is positive: | 
| 32891 | 187 | @{thm [display,indent=0] (prem 1) step [no_vars]}
 | 
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 188 | To apply the rule we construct a list @{term args} of previously
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 189 | constructed well-formed terms. We obtain a | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 190 | new term, @{term "Apply f args"}.  Because @{term lists} is monotone,
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 191 | applications of the rule remain valid as new terms are constructed. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 192 | Further lists of well-formed | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 193 | terms become available and none are taken away.% | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 194 | \index{monotone functions!and inductive definitions|)} 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 195 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 196 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 197 | subsection{* A Proof of Equivalence *}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 198 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 199 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 200 | We naturally hope that these two inductive definitions of ``well-formed'' | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 201 | coincide. The equality can be proved by separate inclusions in | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 202 | each direction. Each is a trivial rule induction. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 203 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 204 | |
| 10468 | 205 | lemma "well_formed_gterm arity \<subseteq> well_formed_gterm' arity" | 
| 206 | apply clarify | |
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 207 | apply (erule well_formed_gterm.induct) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 208 | apply auto | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 209 | done | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 210 | (*<*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 211 | lemma "well_formed_gterm arity \<subseteq> well_formed_gterm' arity" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 212 | apply clarify | 
| 10468 | 213 | apply (erule well_formed_gterm.induct) | 
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 214 | (*>*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 215 | txt {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 216 | The @{text clarify} method gives
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 217 | us an element of @{term "well_formed_gterm arity"} on which to perform 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 218 | induction. The resulting subgoal can be proved automatically: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 219 | @{subgoals[display,indent=0]}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 220 | This proof resembles the one given in | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 221 | {\S}\ref{sec:gterm-datatype} above, especially in the form of the
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 222 | induction hypothesis. Next, we consider the opposite inclusion: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 223 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 224 | (*<*)oops(*>*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 225 | lemma "well_formed_gterm' arity \<subseteq> well_formed_gterm arity" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 226 | apply clarify | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 227 | apply (erule well_formed_gterm'.induct) | 
| 10468 | 228 | apply auto | 
| 229 | done | |
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 230 | (*<*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 231 | lemma "well_formed_gterm' arity \<subseteq> well_formed_gterm arity" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 232 | apply clarify | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 233 | apply (erule well_formed_gterm'.induct) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 234 | (*>*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 235 | txt {*
 | 
| 27167 | 236 | The proof script is virtually identical, | 
| 237 | but the subgoal after applying induction may be surprising: | |
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 238 | @{subgoals[display,indent=0,margin=65]}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 239 | The induction hypothesis contains an application of @{term lists}.  Using a
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 240 | monotone function in the inductive definition always has this effect. The | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 241 | subgoal may look uninviting, but fortunately | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 242 | @{term lists} distributes over intersection:
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 243 | @{named_thms [display,indent=0] lists_Int_eq [no_vars] (lists_Int_eq)}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 244 | Thanks to this default simplification rule, the induction hypothesis | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 245 | is quickly replaced by its two parts: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 246 | \begin{trivlist}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 247 | \item @{term "args \<in> lists (well_formed_gterm' arity)"}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 248 | \item @{term "args \<in> lists (well_formed_gterm arity)"}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 249 | \end{trivlist}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 250 | Invoking the rule @{text well_formed_gterm.step} completes the proof.  The
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 251 | call to @{text auto} does all this work.
 | 
| 10468 | 252 | |
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 253 | This example is typical of how monotone functions | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 254 | \index{monotone functions} can be used.  In particular, many of them
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 255 | distribute over intersection. Monotonicity implies one direction of | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 256 | this set equality; we have this theorem: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 257 | @{named_thms [display,indent=0] mono_Int [no_vars] (mono_Int)}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 258 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 259 | (*<*)oops(*>*) | 
| 10426 | 260 | |
| 10370 | 261 | |
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 262 | subsection{* Another Example of Rule Inversion *}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 263 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 264 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 265 | \index{rule inversion|(}%
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 266 | Does @{term gterms} distribute over intersection?  We have proved that this
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 267 | function is monotone, so @{text mono_Int} gives one of the inclusions.  The
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 268 | opposite inclusion asserts that if @{term t} is a ground term over both of the
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 269 | sets | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 270 | @{term F} and~@{term G} then it is also a ground term over their intersection,
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 271 | @{term "F \<inter> G"}.
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 272 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 273 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 274 | lemma gterms_IntI: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 275 | "t \<in> gterms F \<Longrightarrow> t \<in> gterms G \<longrightarrow> t \<in> gterms (F\<inter>G)" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 276 | (*<*)oops(*>*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 277 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 278 | Attempting this proof, we get the assumption | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 279 | @{term "Apply f args \<in> gterms G"}, which cannot be broken down. 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 280 | It looks like a job for rule inversion:\cmmdx{inductive\protect\_cases}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 281 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 282 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 283 | inductive_cases gterm_Apply_elim [elim!]: "Apply f args \<in> gterms F" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 284 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 285 | text {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 286 | Here is the result. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 287 | @{named_thms [display,indent=0,margin=50] gterm_Apply_elim [no_vars] (gterm_Apply_elim)}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 288 | This rule replaces an assumption about @{term "Apply f args"} by 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 289 | assumptions about @{term f} and~@{term args}.  
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 290 | No cases are discarded (there was only one to begin | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 291 | with) but the rule applies specifically to the pattern @{term "Apply f args"}.
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 292 | It can be applied repeatedly as an elimination rule without looping, so we | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 293 | have given the @{text "elim!"} attribute. 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 294 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 295 | Now we can prove the other half of that distributive law. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 296 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 297 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 298 | lemma gterms_IntI [rule_format, intro!]: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 299 | "t \<in> gterms F \<Longrightarrow> t \<in> gterms G \<longrightarrow> t \<in> gterms (F\<inter>G)" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 300 | apply (erule gterms.induct) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 301 | apply blast | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 302 | done | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 303 | (*<*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 304 | lemma "t \<in> gterms F \<Longrightarrow> t \<in> gterms G \<longrightarrow> t \<in> gterms (F\<inter>G)" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 305 | apply (erule gterms.induct) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 306 | (*>*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 307 | txt {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 308 | The proof begins with rule induction over the definition of | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 309 | @{term gterms}, which leaves a single subgoal:  
 | 
| 10882 | 310 | @{subgoals[display,indent=0,margin=65]}
 | 
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 311 | To prove this, we assume @{term "Apply f args \<in> gterms G"}.  Rule inversion,
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 312 | in the form of @{text gterm_Apply_elim}, infers
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 313 | that every element of @{term args} belongs to 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 314 | @{term "gterms G"}; hence (by the induction hypothesis) it belongs
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 315 | to @{term "gterms (F \<inter> G)"}.  Rule inversion also yields
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 316 | @{term "f \<in> G"} and hence @{term "f \<in> F \<inter> G"}. 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 317 | All of this reasoning is done by @{text blast}.
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 318 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 319 | \smallskip | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 320 | Our distributive law is a trivial consequence of previously-proved results: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 321 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 322 | (*<*)oops(*>*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 323 | lemma gterms_Int_eq [simp]: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 324 | "gterms (F \<inter> G) = gterms F \<inter> gterms G" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 325 | by (blast intro!: mono_Int monoI gterms_mono) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 326 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 327 | text_raw {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 328 | \index{rule inversion|)}%
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 329 | \index{ground terms example|)}
 | 
| 10370 | 330 | |
| 331 | ||
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 332 | \begin{isamarkuptext}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 333 | \begin{exercise}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 334 | A function mapping function symbols to their | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 335 | types is called a \textbf{signature}.  Given a type 
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 336 | ranging over type symbols, we can represent a function's type by a | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 337 | list of argument types paired with the result type. | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 338 | Complete this inductive definition: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 339 | \begin{isabelle}
 | 
| 10468 | 340 | *} | 
| 341 | ||
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 342 | inductive_set | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 343 |   well_typed_gterm :: "('f \<Rightarrow> 't list * 't) \<Rightarrow> ('f gterm * 't)set"
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 344 | for sig :: "'f \<Rightarrow> 't list * 't" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 345 | (*<*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 346 | where | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 347 | step[intro!]: | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 348 | "\<lbrakk>\<forall>pair \<in> set args. pair \<in> well_typed_gterm sig; | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 349 | sig f = (map snd args, rtype)\<rbrakk> | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 350 | \<Longrightarrow> (Apply f (map fst args), rtype) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 351 | \<in> well_typed_gterm sig" | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 352 | (*>*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 353 | text_raw {*
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 354 | \end{isabelle}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 355 | \end{exercise}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 356 | \end{isamarkuptext}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 357 | *} | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 358 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 359 | (*<*) | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 360 | |
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 361 | text{*the following declaration isn't actually used*}
 | 
| 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 362 | primrec | 
| 39795 | 363 | integer_arity :: "integer_op \<Rightarrow> nat" | 
| 364 | where | |
| 365 | "integer_arity (Number n) = 0" | |
| 366 | | "integer_arity UnaryMinus = 1" | |
| 367 | | "integer_arity Plus = 2" | |
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 368 | |
| 10468 | 369 | text{* the rest isn't used: too complicated.  OK for an exercise though.*}
 | 
| 370 | ||
| 23733 | 371 | inductive_set | 
| 372 | integer_signature :: "(integer_op * (unit list * unit)) set" | |
| 373 | where | |
| 374 | Number: "(Number n, ([], ())) \<in> integer_signature" | |
| 375 | | UnaryMinus: "(UnaryMinus, ([()], ())) \<in> integer_signature" | |
| 376 | | Plus: "(Plus, ([(),()], ())) \<in> integer_signature" | |
| 10468 | 377 | |
| 23733 | 378 | inductive_set | 
| 379 |   well_typed_gterm' :: "('f \<Rightarrow> 't list * 't) \<Rightarrow> ('f gterm * 't)set"
 | |
| 380 | for sig :: "'f \<Rightarrow> 't list * 't" | |
| 381 | where | |
| 10468 | 382 | step[intro!]: | 
| 383 | "\<lbrakk>args \<in> lists(well_typed_gterm' sig); | |
| 384 | sig f = (map snd args, rtype)\<rbrakk> | |
| 385 | \<Longrightarrow> (Apply f (map fst args), rtype) | |
| 386 | \<in> well_typed_gterm' sig" | |
| 10370 | 387 | monos lists_mono | 
| 388 | ||
| 389 | ||
| 10468 | 390 | lemma "well_typed_gterm sig \<subseteq> well_typed_gterm' sig" | 
| 10370 | 391 | apply clarify | 
| 10468 | 392 | apply (erule well_typed_gterm.induct) | 
| 10370 | 393 | apply auto | 
| 394 | done | |
| 395 | ||
| 10468 | 396 | lemma "well_typed_gterm' sig \<subseteq> well_typed_gterm sig" | 
| 10370 | 397 | apply clarify | 
| 10468 | 398 | apply (erule well_typed_gterm'.induct) | 
| 10370 | 399 | apply auto | 
| 400 | done | |
| 401 | ||
| 10468 | 402 | |
| 10370 | 403 | end | 
| 23842 
9d87177f1f89
LaTeX code is now generated directly from theory file.
 berghofe parents: 
23733diff
changeset | 404 | (*>*) |