doc-src/Locales/Locales/Examples3.thy
author ballarin
Sat, 28 Mar 2009 22:14:21 +0100
changeset 30780 c3f1e8a9e0b5
parent 30751 36a255c2e428
child 30782 38e477e8524f
permissions -rw-r--r--
Default mode of qualifiers in locale commands.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     1
theory Examples3
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     2
imports Examples
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     3
begin
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     4
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     5
subsection {* Third Version: Local Interpretation *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     6
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     7
text {* In the above example, the fact that @{text \<le>} is a partial
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     8
  order for the natural numbers was used in the proof of the
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     9
  second goal.  In general, proofs of the equations may involve
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    10
  theorems implied by the fact the assumptions of the instantiated
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    11
  locale hold for the instantiating structure.  If these theorems have
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    12
  been shown abstractly in the locale they can be made available
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    13
  conveniently in the context through an auxiliary local interpretation (keyword
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    14
  \isakeyword{interpret}).  This interpretation is inside the proof of the global
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    15
  interpretation.  The third revision of the example illustrates this.  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    16
30780
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
    17
interpretation %visible nat: partial_order "op \<le> :: nat \<Rightarrow> nat \<Rightarrow> bool"
30580
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
    18
  where "partial_order.less op \<le> (x::nat) y = (x < y)"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    19
proof -
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    20
  show "partial_order (op \<le> :: nat \<Rightarrow> nat \<Rightarrow> bool)"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    21
    by unfold_locales auto
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
    22
  then interpret nat: partial_order "op \<le> :: [nat, nat] \<Rightarrow> bool" .
30580
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
    23
  show "partial_order.less op \<le> (x::nat) y = (x < y)"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    24
    unfolding nat.less_def by auto
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    25
qed
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    26
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    27
text {* The inner interpretation does not require an
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    28
  elaborate new proof, it is immediate from the preceeding fact and
30580
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
    29
  proved with ``.''.  Strict qualifiers are normally not necessary for
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
    30
  interpretations inside proofs, since these have only limited scope.
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
    31
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
    32
  The above interpretation enriches the local proof context by
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    33
  the very theorems also obtained in the interpretation from
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    34
  Section~\ref{sec:po-first}, and @{text nat.less_def} may directly be
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    35
  used to unfold the definition.  Theorems from the local
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    36
  interpretation disappear after leaving the proof context --- that
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    37
  is, after the closing \isakeyword{qed} --- and are
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    38
  then replaced by those with the desired substitutions of the strict
30580
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
    39
  order.  *}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    40
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    41
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    42
subsection {* Further Interpretations *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    43
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    44
text {* Further interpretations are necessary to reuse theorems from
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    45
  the other locales.  In @{text lattice} the operations @{text \<sqinter>} and
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    46
  @{text \<squnion>} are substituted by @{term "min :: nat \<Rightarrow> nat \<Rightarrow> nat"} and
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    47
  @{term "max :: nat \<Rightarrow> nat \<Rightarrow> nat"}.  The entire proof for the
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    48
  interpretation is reproduced in order to give an example of a more
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    49
  elaborate interpretation proof.  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    50
30780
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
    51
interpretation %visible nat: lattice "op \<le> :: nat \<Rightarrow> nat \<Rightarrow> bool"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    52
  where "lattice.meet op \<le> (x::nat) y = min x y"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    53
    and "lattice.join op \<le> (x::nat) y = max x y"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    54
proof -
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    55
  show "lattice (op \<le> :: nat \<Rightarrow> nat \<Rightarrow> bool)"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    56
    txt {* We have already shown that this is a partial order, *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    57
    apply unfold_locales
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    58
    txt {* hence only the lattice axioms remain to be shown: @{subgoals
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    59
      [display]}  After unfolding @{text is_inf} and @{text is_sup}, *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    60
    apply (unfold nat.is_inf_def nat.is_sup_def)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    61
    txt {* the goals become @{subgoals [display]} which can be solved
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    62
      by Presburger arithmetic. *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    63
    by arith+
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    64
  txt {* In order to show the equations, we put ourselves in a
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    65
    situation where the lattice theorems can be used in a convenient way. *}
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
    66
  then interpret nat: lattice "op \<le> :: nat \<Rightarrow> nat \<Rightarrow> bool" .
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    67
  show "lattice.meet op \<le> (x::nat) y = min x y"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    68
    by (bestsimp simp: nat.meet_def nat.is_inf_def)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    69
  show "lattice.join op \<le> (x::nat) y = max x y"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    70
    by (bestsimp simp: nat.join_def nat.is_sup_def)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    71
qed
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    72
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    73
text {* That the relation @{text \<le>} is a total order completes this
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    74
  sequence of interpretations. *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    75
30780
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
    76
interpretation %visible nat: total_order "op \<le> :: nat \<Rightarrow> nat \<Rightarrow> bool"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    77
  by unfold_locales arith
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    78
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    79
text {* Theorems that are available in the theory at this point are shown in
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    80
  Table~\ref{tab:nat-lattice}.
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    81
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    82
\begin{table}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    83
\hrule
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    84
\vspace{2ex}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    85
\begin{center}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    86
\begin{tabular}{l}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    87
  @{thm [source] nat.less_def} from locale @{text partial_order}: \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    88
  \quad @{thm nat.less_def} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    89
  @{thm [source] nat.meet_left} from locale @{text lattice}: \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    90
  \quad @{thm nat.meet_left} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    91
  @{thm [source] nat.join_distr} from locale @{text distrib_lattice}: \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    92
  \quad @{thm nat.join_distr} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    93
  @{thm [source] nat.less_total} from locale @{text total_order}: \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    94
  \quad @{thm nat.less_total}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    95
\end{tabular}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    96
\end{center}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    97
\hrule
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    98
\caption{Interpreted theorems for @{text \<le>} on the natural numbers.}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    99
\label{tab:nat-lattice}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   100
\end{table}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   101
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   102
  Note that since the locale hierarchy reflects that total orders are
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   103
  distributive lattices, an explicit interpretation of distributive
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   104
  lattices for the order relation on natural numbers is not neccessary.
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   105
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   106
  Why not push this idea further and just give the last interpretation
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   107
  as a single interpretation instead of the sequence of three?  The
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   108
  reasons for this are twofold:
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   109
\begin{itemize}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   110
\item
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   111
  Often it is easier to work in an incremental fashion, because later
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   112
  interpretations require theorems provided by earlier
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   113
  interpretations.
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   114
\item
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   115
  Assume that a definition is made in some locale $l_1$, and that $l_2$
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   116
  imports $l_1$.  Let an equation for the definition be
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   117
  proved in an interpretation of $l_2$.  The equation will be unfolded
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   118
  in interpretations of theorems added to $l_2$ or below in the import
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   119
  hierarchy, but not for theorems added above $l_2$.
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   120
  Hence, an equation interpreting a definition should always be given in
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   121
  an interpretation of the locale where the definition is made, not in
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   122
  an interpretation of a locale further down the hierarchy.
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   123
\end{itemize}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   124
  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   125
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   126
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   127
subsection {* Lattice @{text "dvd"} on @{typ nat} *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   128
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   129
text {* Divisibility on the natural numbers is a distributive lattice
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   130
  but not a total order.  Interpretation again proceeds
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   131
  incrementally. *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   132
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   133
interpretation nat_dvd: partial_order "op dvd :: nat \<Rightarrow> nat \<Rightarrow> bool"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   134
  where "partial_order.less op dvd (x::nat) y = (x dvd y \<and> x \<noteq> y)"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   135
proof -
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   136
  show "partial_order (op dvd :: nat \<Rightarrow> nat \<Rightarrow> bool)"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   137
    by unfold_locales (auto simp: dvd_def)
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   138
  then interpret nat_dvd: partial_order "op dvd :: nat \<Rightarrow> nat \<Rightarrow> bool" .
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   139
  show "partial_order.less op dvd (x::nat) y = (x dvd y \<and> x \<noteq> y)"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   140
    apply (unfold nat_dvd.less_def)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   141
    apply auto
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   142
    done
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   143
qed
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   144
30580
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
   145
text {* Note that in Isabelle/HOL there is no symbol for strict
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
   146
  divisibility.  Instead, interpretation substitutes @{term "x dvd y \<and>
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
   147
  x \<noteq> y"}.  *}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   148
30780
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
   149
interpretation nat_dvd: lattice "op dvd :: nat \<Rightarrow> nat \<Rightarrow> bool"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   150
  where nat_dvd_meet_eq:
27595
3ac9e3cd1fa3 curried gcd
haftmann
parents: 27503
diff changeset
   151
      "lattice.meet op dvd = gcd"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   152
    and nat_dvd_join_eq:
27595
3ac9e3cd1fa3 curried gcd
haftmann
parents: 27503
diff changeset
   153
      "lattice.join op dvd = lcm"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   154
proof -
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   155
  show "lattice (op dvd :: nat \<Rightarrow> nat \<Rightarrow> bool)"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   156
    apply unfold_locales
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   157
    apply (unfold nat_dvd.is_inf_def nat_dvd.is_sup_def)
27595
3ac9e3cd1fa3 curried gcd
haftmann
parents: 27503
diff changeset
   158
    apply (rule_tac x = "gcd x y" in exI)
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   159
    apply auto [1]
27595
3ac9e3cd1fa3 curried gcd
haftmann
parents: 27503
diff changeset
   160
    apply (rule_tac x = "lcm x y" in exI)
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   161
    apply (auto intro: lcm_dvd1 lcm_dvd2 lcm_least)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   162
    done
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   163
  then interpret nat_dvd: lattice "op dvd :: nat \<Rightarrow> nat \<Rightarrow> bool" .
27595
3ac9e3cd1fa3 curried gcd
haftmann
parents: 27503
diff changeset
   164
  show "lattice.meet op dvd = gcd"
3ac9e3cd1fa3 curried gcd
haftmann
parents: 27503
diff changeset
   165
    apply (auto simp add: expand_fun_eq)
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   166
    apply (unfold nat_dvd.meet_def)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   167
    apply (rule the_equality)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   168
    apply (unfold nat_dvd.is_inf_def)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   169
    by auto
27595
3ac9e3cd1fa3 curried gcd
haftmann
parents: 27503
diff changeset
   170
  show "lattice.join op dvd = lcm"
3ac9e3cd1fa3 curried gcd
haftmann
parents: 27503
diff changeset
   171
    apply (auto simp add: expand_fun_eq)
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   172
    apply (unfold nat_dvd.join_def)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   173
    apply (rule the_equality)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   174
    apply (unfold nat_dvd.is_sup_def)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   175
    by (auto intro: lcm_dvd1 lcm_dvd2 lcm_least)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   176
qed
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   177
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   178
text {* Equations @{thm [source] nat_dvd_meet_eq} and @{thm [source]
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   179
  nat_dvd_join_eq} are named since they are handy in the proof of
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   180
  the subsequent interpretation. *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   181
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   182
(*
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   183
definition
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   184
  is_lcm :: "nat \<Rightarrow> nat \<Rightarrow> nat \<Rightarrow> bool" where
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   185
  "is_lcm p m n \<longleftrightarrow> m dvd p \<and> n dvd p \<and>
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   186
    (\<forall>d. m dvd d \<longrightarrow> n dvd d \<longrightarrow> p dvd d)"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   187
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   188
lemma is_gcd: "is_lcm (lcm (m, n)) m n"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   189
  by (simp add: is_lcm_def lcm_least)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   190
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   191
lemma gcd_lcm_distr_lemma:
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   192
  "[| is_gcd g1 x l1; is_lcm l1 y z; is_gcd g2 x y; is_gcd g3 x z |] ==> is_lcm g1 g2 g3"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   193
apply (unfold is_gcd_def is_lcm_def dvd_def)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   194
apply (clarsimp simp: mult_ac)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   195
apply (blast intro: mult_is_0)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   196
thm mult_is_0 [THEN iffD1]
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   197
*)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   198
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   199
lemma %invisible gcd_lcm_distr:
27595
3ac9e3cd1fa3 curried gcd
haftmann
parents: 27503
diff changeset
   200
  "gcd x (lcm y z) = lcm (gcd x y) (gcd x z)" sorry
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   201
30780
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
   202
interpretation %visible nat_dvd:
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   203
  distrib_lattice "op dvd :: nat \<Rightarrow> nat \<Rightarrow> bool"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   204
  apply unfold_locales
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   205
  txt {* @{subgoals [display]} *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   206
  apply (unfold nat_dvd_meet_eq nat_dvd_join_eq)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   207
  txt {* @{subgoals [display]} *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   208
  apply (rule gcd_lcm_distr) done
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   209
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   210
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   211
text {* Theorems that are available in the theory after these
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   212
  interpretations are shown in Table~\ref{tab:nat-dvd-lattice}.
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   213
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   214
\begin{table}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   215
\hrule
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   216
\vspace{2ex}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   217
\begin{center}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   218
\begin{tabular}{l}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   219
  @{thm [source] nat_dvd.less_def} from locale @{text partial_order}: \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   220
  \quad @{thm nat_dvd.less_def} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   221
  @{thm [source] nat_dvd.meet_left} from locale @{text lattice}: \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   222
  \quad @{thm nat_dvd.meet_left} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   223
  @{thm [source] nat_dvd.join_distr} from locale @{text distrib_lattice}: \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   224
  \quad @{thm nat_dvd.join_distr} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   225
\end{tabular}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   226
\end{center}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   227
\hrule
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   228
\caption{Interpreted theorems for @{text dvd} on the natural numbers.}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   229
\label{tab:nat-dvd-lattice}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   230
\end{table}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   231
  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   232
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   233
text {*
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   234
  The full syntax of the interpretation commands is shown in
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   235
  Table~\ref{tab:commands}.  The grammar refers to
30580
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
   236
  \textit{expression}, which stands for a \emph{locale} expression.
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 30393
diff changeset
   237
  Locale expressions are discussed in the following section.
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   238
  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   239
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   240
27077
f64166dd92f0 moved labels into actual sections;
wenzelm
parents: 27075
diff changeset
   241
section {* Locale Expressions \label{sec:expressions} *}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   242
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   243
text {*
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   244
  A map @{term \<phi>} between partial orders @{text \<sqsubseteq>} and @{text \<preceq>}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   245
  is called order preserving if @{text "x \<sqsubseteq> y"} implies @{text "\<phi> x \<preceq>
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   246
  \<phi> y"}.  This situation is more complex than those encountered so
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   247
  far: it involves two partial orders, and it is desirable to use the
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   248
  existing locale for both.
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   249
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   250
  Inspecting the grammar of locale commands in
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   251
  Table~\ref{tab:commands} reveals that the import of a locale can be
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   252
  more than just a single locale.  In general, the import is a
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   253
  \emph{locale expression}.  These enable to combine locales
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   254
  and instantiate parameters.  A locale expression is a sequence of
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   255
  locale \emph{instances} followed by an optional \isakeyword{for}
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   256
  clause.  Each instance consists of a locale reference, which may be
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   257
  preceded by a qualifer and succeeded by instantiations of the
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   258
  parameters of that locale.  Instantiations may be either positional
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   259
  or through explicit parameter argument pairs.
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   260
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   261
  Using a locale expression, a locale for order
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   262
  preserving maps can be declared in the following way.  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   263
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   264
  locale order_preserving =
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   265
    le: partial_order le + le': partial_order le'
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   266
      for le (infixl "\<sqsubseteq>" 50) and le' (infixl "\<preceq>" 50) +
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   267
    fixes \<phi> :: "'a \<Rightarrow> 'b"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   268
    assumes hom_le: "x \<sqsubseteq> y \<Longrightarrow> \<phi> x \<preceq> \<phi> y"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   269
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   270
text {* The second and third line contain the expression --- two
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   271
  instances of the partial order locale with instantiations @{text le}
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   272
  and @{text le'}, respectively.  The \isakeyword{for} clause consists
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   273
  of parameter declarations and is similar to the context element
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   274
  \isakeyword{fixes}.  The notable difference is that the
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   275
  \isakeyword{for} clause is part of the expression, and only
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   276
  parameters defined in the expression may occur in its instances.
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   277
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   278
  Instances are \emph{morphisms} on locales.  Their effect on the
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   279
  parameters is naturally lifted to terms, propositions and theorems,
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   280
  and thus to the assumptions and conclusions of a locale.  The
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   281
  assumption of a locale expression is the conjunction of the
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   282
  assumptions of the instances.  The conclusions of a sequence of
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   283
  instances are obtained by appending the conclusions of the
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   284
  instances in the order of the sequence.
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   285
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   286
  The qualifiers in the expression are already a familiar concept from
30780
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
   287
  the \isakeyword{interpretation} command
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
   288
  (Section~\ref{sec:po-first}).  Here, they serve to distinguish names
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
   289
  (in particular theorem names) for the two partial orders within the
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
   290
  locale.  Qualifiers in the \isakeyword{locale} command (and in
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
   291
  \isakeyword{sublocale}) default to optional --- that is, they need
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
   292
  not occur in references to the qualified names.  Here are examples
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
   293
  of theorems in locale @{text order_preserving}: *}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   294
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   295
context %invisible order_preserving begin
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   296
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   297
text {*
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   298
  @{thm [source] le.less_le_trans}: @{thm le.less_le_trans}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   299
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   300
  @{thm [source] hom_le}: @{thm hom_le}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   301
  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   302
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   303
text {* The theorems for the partial order @{text \<preceq>}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   304
  are qualified by @{text le'}.  For example, @{thm [source]
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   305
  le'.less_le_trans}: @{thm [display, indent=2] le'.less_le_trans} *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   306
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   307
end %invisible
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   308
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   309
text {* This example reveals that there is no infix syntax for the strict
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   310
  version of @{text \<preceq>}!  This can be declared through an abbreviation.
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   311
  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   312
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   313
  abbreviation (in order_preserving)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   314
    less' (infixl "\<prec>" 50) where "less' \<equiv> partial_order.less le'"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   315
30393
aa6f42252bf6 replaced old locale option by proper "text (in locale)";
wenzelm
parents: 29568
diff changeset
   316
text (in order_preserving) {* Now the theorem is displayed nicely as
aa6f42252bf6 replaced old locale option by proper "text (in locale)";
wenzelm
parents: 29568
diff changeset
   317
  @{thm le'.less_le_trans}.  *}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   318
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   319
text {* Qualifiers not only apply to theorem names, but also to names
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   320
  introduced by definitions and abbreviations.  In locale
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   321
  @{text partial_order} the full name of the strict order of @{text \<sqsubseteq>} is
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   322
  @{text le.less} and therefore @{text le'.less} is the full name of
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   323
  the strict order of @{text \<preceq>}.  Hence, the equation in the
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   324
  abbreviation above could have been also written as @{text "less' \<equiv>
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   325
  le'.less"}. *}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   326
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   327
text {* Readers may find the declaration of locale @{text
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   328
  order_preserving} a little awkward, because the declaration and
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   329
  concrete syntax for @{text le} from @{text partial_order} are
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   330
  repeated in the declaration of @{text order_preserving}.  Locale
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   331
  expressions provide a convenient short hand for this.  A parameter
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   332
  in an instance is \emph{untouched} if no instantiation term is
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   333
  provided for it.  In positional instantiations, a parameter position
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   334
  may be skipped with an underscore, and it is allowed to give fewer
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   335
  instantiation terms than the instantiated locale's number of
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   336
  parameters.  In named instantiations, instantiation pairs for
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   337
  certain parameters may simply be omitted.  Untouched parameters are
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   338
  declared by the locale expression and with their concrete syntax by
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   339
  implicitly adding them to the beginning of the \isakeyword{for}
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   340
  clause.
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   341
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   342
  The following locales illustrate this.  A map @{text \<phi>} is a
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   343
  lattice homomorphism if it preserves meet and join. *}
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   344
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   345
  locale lattice_hom =
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   346
    le: lattice + le': lattice le' for le' (infixl "\<preceq>" 50) +
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   347
    fixes \<phi>
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   348
    assumes hom_meet:
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   349
	"\<phi> (x \<sqinter> y) = le'.meet (\<phi> x) (\<phi> y)"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   350
      and hom_join:
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   351
	"\<phi> (x \<squnion> y) = le'.join (\<phi> x) (\<phi> y)"
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   352
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   353
  abbreviation (in lattice_hom)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   354
    meet' (infixl "\<sqinter>''" 50) where "meet' \<equiv> le'.meet"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   355
  abbreviation (in lattice_hom)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   356
    join' (infixl "\<squnion>''" 50) where "join' \<equiv> le'.join"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   357
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   358
text {* A homomorphism is an endomorphism if both orders coincide. *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   359
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   360
  locale lattice_end = lattice_hom _ le
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   361
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   362
text {* In this declaration, the first parameter of @{text
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   363
  lattice_hom}, @{text le}, is untouched and then used to instantiate
30780
c3f1e8a9e0b5 Default mode of qualifiers in locale commands.
ballarin
parents: 30751
diff changeset
   364
  the second parameter.  Its concrete syntax is preserved. *}
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   365
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   366
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   367
text {* The inheritance diagram of the situation we have now is shown
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   368
  in Figure~\ref{fig:hom}, where the dashed line depicts an
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   369
  interpretation which is introduced below.  Renamings are
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   370
  indicated by $\sqsubseteq \mapsto \preceq$ etc.  The expression
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   371
  imported by @{text lattice_end} identifies the first and second
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   372
  parameter of @{text lattice_hom}.  By looking at the inheritance diagram it would seem
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   373
  that two identical copies of each of the locales @{text
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   374
  partial_order} and @{text lattice} are imported.  This is not the
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   375
  case!  Inheritance paths with identical morphisms are detected and
27503
a019d6568a3c fix typo
huffman
parents: 27081
diff changeset
   376
  the conclusions of the respective locales appear only once.
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   377
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   378
\begin{figure}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   379
\hrule \vspace{2ex}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   380
\begin{center}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   381
\begin{tikzpicture}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   382
  \node (o) at (0,0) {@{text partial_order}};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   383
  \node (oh) at (1.5,-2) {@{text order_preserving}};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   384
  \node (oh1) at (1.5,-0.7) {$\scriptscriptstyle \sqsubseteq \mapsto \sqsubseteq$};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   385
  \node (oh2) at (0,-1.3) {$\scriptscriptstyle \sqsubseteq \mapsto \preceq$};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   386
  \node (l) at (-1.5,-2) {@{text lattice}};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   387
  \node (lh) at (0,-4) {@{text lattice_hom}};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   388
  \node (lh1) at (0,-2.7) {$\scriptscriptstyle \sqsubseteq \mapsto \sqsubseteq$};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   389
  \node (lh2) at (-1.5,-3.3) {$\scriptscriptstyle \sqsubseteq \mapsto \preceq$};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   390
  \node (le) at (0,-6) {@{text lattice_end}};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   391
  \node (le1) at (0,-4.8)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   392
    [anchor=west]{$\scriptscriptstyle \sqsubseteq \mapsto \sqsubseteq$};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   393
  \node (le2) at (0,-5.2)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   394
    [anchor=west]{$\scriptscriptstyle \preceq \mapsto \sqsubseteq$};
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   395
  \draw (o) -- (l);
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   396
  \draw[dashed] (oh) -- (lh);
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   397
  \draw (lh) -- (le);
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   398
  \draw (o) .. controls (oh1.south west) .. (oh);
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   399
  \draw (o) .. controls (oh2.north east) .. (oh);
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   400
  \draw (l) .. controls (lh1.south west) .. (lh);
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   401
  \draw (l) .. controls (lh2.north east) .. (lh);
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   402
\end{tikzpicture}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   403
\end{center}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   404
\hrule
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   405
\caption{Hierarchy of Homomorphism Locales.}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   406
\label{fig:hom}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   407
\end{figure}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   408
  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   409
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   410
text {* It can be shown easily that a lattice homomorphism is order
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   411
  preserving.  As the final example of this section, a locale
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   412
  interpretation is used to assert this: *}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   413
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   414
  sublocale lattice_hom \<subseteq> order_preserving proof unfold_locales
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   415
    fix x y
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   416
    assume "x \<sqsubseteq> y"
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   417
    then have "y = (x \<squnion> y)" by (simp add: le.join_connection)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   418
    then have "\<phi> y = (\<phi> x \<squnion>' \<phi> y)" by (simp add: hom_join [symmetric])
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   419
    then show "\<phi> x \<preceq> \<phi> y" by (simp add: le'.join_connection)
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   420
  qed
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   421
30393
aa6f42252bf6 replaced old locale option by proper "text (in locale)";
wenzelm
parents: 29568
diff changeset
   422
text (in lattice_hom) {*
aa6f42252bf6 replaced old locale option by proper "text (in locale)";
wenzelm
parents: 29568
diff changeset
   423
  Theorems and other declarations --- syntax, in particular --- from
aa6f42252bf6 replaced old locale option by proper "text (in locale)";
wenzelm
parents: 29568
diff changeset
   424
  the locale @{text order_preserving} are now active in @{text
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   425
  lattice_hom}, for example
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   426
30393
aa6f42252bf6 replaced old locale option by proper "text (in locale)";
wenzelm
parents: 29568
diff changeset
   427
  @{thm [source] le'.less_le_trans}:
aa6f42252bf6 replaced old locale option by proper "text (in locale)";
wenzelm
parents: 29568
diff changeset
   428
  @{thm le'.less_le_trans}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   429
  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   430
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   431
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   432
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   433
section {* Further Reading *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   434
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   435
text {* More information on locales and their interpretation is
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   436
  available.  For the locale hierarchy of import and interpretation
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   437
  dependencies see \cite{Ballarin2006a}; interpretations in theories
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   438
  and proofs are covered in \cite{Ballarin2006b}.  In the latter, we
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   439
  show how interpretation in proofs enables to reason about families
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   440
  of algebraic structures, which cannot be expressed with locales
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   441
  directly.
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   442
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   443
  Haftmann and Wenzel \cite{HaftmannWenzel2007} overcome a restriction
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   444
  of axiomatic type classes through a combination with locale
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   445
  interpretation.  The result is a Haskell-style class system with a
30750
3779e2158dad Update explanation of locale expressions to locale reimplementation.
ballarin
parents: 30580
diff changeset
   446
  facility to generate ML and Haskell code.  Classes are sufficient for
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   447
  simple specifications with a single type parameter.  The locales for
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   448
  orders and lattices presented in this tutorial fall into this
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   449
  category.  Order preserving maps, homomorphisms and vector spaces,
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   450
  on the other hand, do not.
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   451
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   452
  The original work of Kamm\"uller on locales \cite{KammullerEtAl1999}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   453
  may be of interest from a historical perspective.  The mathematical
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   454
  background on orders and lattices is taken from Jacobson's textbook
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   455
  on algebra \cite[Chapter~8]{Jacobson1985}.
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   456
  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   457
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   458
text {*
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   459
\begin{table}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   460
\hrule
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   461
\vspace{2ex}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   462
\begin{center}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   463
\begin{tabular}{l>$c<$l}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   464
  \multicolumn{3}{l}{Miscellaneous} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   465
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   466
  \textit{attr-name} & ::=
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   467
  & \textit{name} $|$ \textit{attribute} $|$
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   468
    \textit{name} \textit{attribute} \\
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   469
  \textit{qualifier} & ::=
30751
36a255c2e428 Corrections to locale syntax.
ballarin
parents: 30750
diff changeset
   470
  & \textit{name} [``\textbf{?}'' $|$ ``\textbf{!}''] \\[2ex]
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   471
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   472
  \multicolumn{3}{l}{Context Elements} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   473
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   474
  \textit{fixes} & ::=
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   475
  & \textit{name} [ ``\textbf{::}'' \textit{type} ]
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   476
    [ ``\textbf{(}'' \textbf{structure} ``\textbf{)}'' $|$
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   477
    \textit{mixfix} ] \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   478
\begin{comment}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   479
  \textit{constrains} & ::=
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   480
  & \textit{name} ``\textbf{::}'' \textit{type} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   481
\end{comment}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   482
  \textit{assumes} & ::=
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   483
  & [ \textit{attr-name} ``\textbf{:}'' ] \textit{proposition} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   484
\begin{comment}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   485
  \textit{defines} & ::=
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   486
  & [ \textit{attr-name} ``\textbf{:}'' ] \textit{proposition} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   487
  \textit{notes} & ::=
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   488
  & [ \textit{attr-name} ``\textbf{=}'' ]
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   489
    ( \textit{qualified-name} [ \textit{attribute} ] )$^+$ \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   490
\end{comment}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   491
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   492
  \textit{element} & ::=
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   493
  & \textbf{fixes} \textit{fixes} ( \textbf{and} \textit{fixes} )$^*$ \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   494
\begin{comment}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   495
  & |
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   496
  & \textbf{constrains} \textit{constrains}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   497
    ( \textbf{and} \textit{constrains} )$^*$ \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   498
\end{comment}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   499
  & |
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   500
  & \textbf{assumes} \textit{assumes} ( \textbf{and} \textit{assumes} )$^*$ \\[2ex]
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   501
%\begin{comment}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   502
%  & |
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   503
%  & \textbf{defines} \textit{defines} ( \textbf{and} \textit{defines} )$^*$ \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   504
%  & |
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   505
%  & \textbf{notes} \textit{notes} ( \textbf{and} \textit{notes} )$^*$ \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   506
%\end{comment}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   507
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   508
  \multicolumn{3}{l}{Locale Expressions} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   509
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   510
  \textit{pos-insts} & ::=
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   511
  & ( \textit{term} $|$ ``\textbf{\_}'' )$^*$ \\
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   512
  \textit{named-insts} & ::=
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   513
  & \textbf{where} \textit{name} ``\textbf{=}'' \textit{term}
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   514
  ( \textbf{and} \textit{name} ``\textbf{=}'' \textit{term} )$^*$ \\
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   515
  \textit{instance} & ::=
30751
36a255c2e428 Corrections to locale syntax.
ballarin
parents: 30750
diff changeset
   516
  & [ \textit{qualifier} ``\textbf{:}'' ]
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   517
    \textit{qualified-name} ( \textit{pos-insts} $|$ \textit{named-inst} ) \\
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   518
  \textit{expression}  & ::= 
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   519
  & \textit{instance} ( ``\textbf{+}'' \textit{instance} )$^*$
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   520
    [ \textbf{for} \textit{fixes} ( \textbf{and} \textit{fixes} )$^*$ ] \\[2ex]
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   521
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   522
  \multicolumn{3}{l}{Declaration of Locales} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   523
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   524
  \textit{locale} & ::=
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   525
  & \textit{element}$^+$ \\
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   526
  & | & \textit{expression} [ ``\textbf{+}'' \textit{element}$^+$ ] \\
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   527
  \textit{toplevel} & ::=
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   528
  & \textbf{locale} \textit{name} [ ``\textbf{=}''
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   529
    \textit{locale} ] \\[2ex]
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   530
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   531
  \multicolumn{3}{l}{Interpretation} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   532
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   533
  \textit{equation} & ::= & [ \textit{attr-name} ``\textbf{:}'' ]
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   534
    \textit{prop} \\
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   535
  \textit{equations} & ::= &  \textbf{where} \textit{equation} ( \textbf{and}
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   536
    \textit{equation} )$^*$  \\
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   537
  \textit{toplevel} & ::=
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   538
  & \textbf{sublocale} \textit{name} ( ``$<$'' $|$
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   539
    ``$\subseteq$'' ) \textit{expression} \textit{proof} \\
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   540
  & |
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   541
  & \textbf{interpretation}
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   542
    \textit{expression} [ \textit{equations} ] \textit{proof} \\
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   543
  & |
29566
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   544
  & \textbf{interpret}
937baa077df2 Fixed tutorial to compile with new locales; grammar of new locale commands.
ballarin
parents: 27595
diff changeset
   545
    \textit{expression} \textit{proof} \\[2ex]
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   546
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   547
  \multicolumn{3}{l}{Diagnostics} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   548
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   549
  \textit{toplevel} & ::=
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   550
  & \textbf{print\_locale} [ ``\textbf{!}'' ] \textit{locale} \\
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   551
  & | & \textbf{print\_locales} 
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   552
\end{tabular}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   553
\end{center}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   554
\hrule
29567
286c01be90cb Merged, overriding earlier fix.
ballarin
parents: 29293 29566
diff changeset
   555
\caption{Syntax of Locale Commands (abridged).}
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   556
\label{tab:commands}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   557
\end{table}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   558
  *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   559
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   560
text {* \textbf{Acknowledgements.}  Alexander Krauss, Tobias Nipkow,
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   561
  Christian Sternagel and Makarius Wenzel have made useful comments on
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   562
  a draft of this document. *}
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   563
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
   564
end