doc-src/Classes/Thy/Classes.thy
author haftmann
Mon, 22 Feb 2010 17:02:39 +0100
changeset 35282 8fd9d555d04d
parent 31931 0b1d807b1c2d
child 37706 c63649d8d75b
permissions -rw-r--r--
dropped references to old axclass from documentation
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
     1
theory Classes
28565
haftmann
parents: 28540
diff changeset
     2
imports Main Setup
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
     3
begin
75b56e51fade initial draft
haftmann
parents:
diff changeset
     4
75b56e51fade initial draft
haftmann
parents:
diff changeset
     5
section {* Introduction *}
75b56e51fade initial draft
haftmann
parents:
diff changeset
     6
75b56e51fade initial draft
haftmann
parents:
diff changeset
     7
text {*
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
     8
  Type classes were introduced by Wadler and Blott \cite{wadler89how}
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
     9
  into the Haskell language to allow for a reasonable implementation
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    10
  of overloading\footnote{throughout this tutorial, we are referring
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    11
  to classical Haskell 1.0 type classes, not considering
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    12
  later additions in expressiveness}.
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    13
  As a canonical example, a polymorphic equality function
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    14
  @{text "eq \<Colon> \<alpha> \<Rightarrow> \<alpha> \<Rightarrow> bool"} which is overloaded on different
22550
c5039bee2602 updated
haftmann
parents: 22479
diff changeset
    15
  types for @{text "\<alpha>"}, which is achieved by splitting introduction
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    16
  of the @{text eq} function from its overloaded definitions by means
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    17
  of @{text class} and @{text instance} declarations:
30227
853abb4853cc tuned manuals
haftmann
parents: 30226
diff changeset
    18
  \footnote{syntax here is a kind of isabellized Haskell}
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    19
28565
haftmann
parents: 28540
diff changeset
    20
  \begin{quote}
haftmann
parents: 28540
diff changeset
    21
30227
853abb4853cc tuned manuals
haftmann
parents: 30226
diff changeset
    22
  \noindent@{text "class eq where"} \\
28565
haftmann
parents: 28540
diff changeset
    23
  \hspace*{2ex}@{text "eq \<Colon> \<alpha> \<Rightarrow> \<alpha> \<Rightarrow> bool"}
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
    24
28565
haftmann
parents: 28540
diff changeset
    25
  \medskip\noindent@{text "instance nat \<Colon> eq where"} \\
haftmann
parents: 28540
diff changeset
    26
  \hspace*{2ex}@{text "eq 0 0 = True"} \\
haftmann
parents: 28540
diff changeset
    27
  \hspace*{2ex}@{text "eq 0 _ = False"} \\
haftmann
parents: 28540
diff changeset
    28
  \hspace*{2ex}@{text "eq _ 0 = False"} \\
haftmann
parents: 28540
diff changeset
    29
  \hspace*{2ex}@{text "eq (Suc n) (Suc m) = eq n m"}
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    30
28948
1860f016886d fixed typo
haftmann
parents: 28947
diff changeset
    31
  \medskip\noindent@{text "instance (\<alpha>\<Colon>eq, \<beta>\<Colon>eq) pair \<Colon> eq where"} \\
28565
haftmann
parents: 28540
diff changeset
    32
  \hspace*{2ex}@{text "eq (x1, y1) (x2, y2) = eq x1 x2 \<and> eq y1 y2"}
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
    33
28565
haftmann
parents: 28540
diff changeset
    34
  \medskip\noindent@{text "class ord extends eq where"} \\
haftmann
parents: 28540
diff changeset
    35
  \hspace*{2ex}@{text "less_eq \<Colon> \<alpha> \<Rightarrow> \<alpha> \<Rightarrow> bool"} \\
haftmann
parents: 28540
diff changeset
    36
  \hspace*{2ex}@{text "less \<Colon> \<alpha> \<Rightarrow> \<alpha> \<Rightarrow> bool"}
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    37
28565
haftmann
parents: 28540
diff changeset
    38
  \end{quote}
haftmann
parents: 28540
diff changeset
    39
haftmann
parents: 28540
diff changeset
    40
  \noindent Type variables are annotated with (finitely many) classes;
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    41
  these annotations are assertions that a particular polymorphic type
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    42
  provides definitions for overloaded functions.
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    43
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    44
  Indeed, type classes not only allow for simple overloading
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    45
  but form a generic calculus, an instance of order-sorted
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
    46
  algebra \cite{nipkow-sorts93,Nipkow-Prehofer:1993,Wenzel:1997:TPHOL}.
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
    47
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
    48
  From a software engineering point of view, type classes
28540
haftmann
parents: 27505
diff changeset
    49
  roughly correspond to interfaces in object-oriented languages like Java;
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    50
  so, it is naturally desirable that type classes do not only
24991
c6f5cc939c29 added subclass command
haftmann
parents: 24628
diff changeset
    51
  provide functions (class parameters) but also state specifications
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    52
  implementations must obey.  For example, the @{text "class eq"}
22550
c5039bee2602 updated
haftmann
parents: 22479
diff changeset
    53
  above could be given the following specification, demanding that
c5039bee2602 updated
haftmann
parents: 22479
diff changeset
    54
  @{text "class eq"} is an equivalence relation obeying reflexivity,
c5039bee2602 updated
haftmann
parents: 22479
diff changeset
    55
  symmetry and transitivity:
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    56
28565
haftmann
parents: 28540
diff changeset
    57
  \begin{quote}
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    58
28565
haftmann
parents: 28540
diff changeset
    59
  \noindent@{text "class eq where"} \\
haftmann
parents: 28540
diff changeset
    60
  \hspace*{2ex}@{text "eq \<Colon> \<alpha> \<Rightarrow> \<alpha> \<Rightarrow> bool"} \\
haftmann
parents: 28540
diff changeset
    61
  @{text "satisfying"} \\
haftmann
parents: 28540
diff changeset
    62
  \hspace*{2ex}@{text "refl: eq x x"} \\
haftmann
parents: 28540
diff changeset
    63
  \hspace*{2ex}@{text "sym: eq x y \<longleftrightarrow> eq x y"} \\
haftmann
parents: 28540
diff changeset
    64
  \hspace*{2ex}@{text "trans: eq x y \<and> eq y z \<longrightarrow> eq x z"}
haftmann
parents: 28540
diff changeset
    65
haftmann
parents: 28540
diff changeset
    66
  \end{quote}
haftmann
parents: 28540
diff changeset
    67
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
    68
  \noindent From a theoretical point of view, type classes are lightweight
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
    69
  modules; Haskell type classes may be emulated by
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    70
  SML functors \cite{classes_modules}. 
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    71
  Isabelle/Isar offers a discipline of type classes which brings
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    72
  all those aspects together:
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    73
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    74
  \begin{enumerate}
24991
c6f5cc939c29 added subclass command
haftmann
parents: 24628
diff changeset
    75
    \item specifying abstract parameters together with
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    76
       corresponding specifications,
28540
haftmann
parents: 27505
diff changeset
    77
    \item instantiating those abstract parameters by a particular
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    78
       type
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    79
    \item in connection with a ``less ad-hoc'' approach to overloading,
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
    80
    \item with a direct link to the Isabelle module system:
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
    81
      locales \cite{kammueller-locales}.
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    82
  \end{enumerate}
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    83
22550
c5039bee2602 updated
haftmann
parents: 22479
diff changeset
    84
  \noindent Isar type classes also directly support code generation
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
    85
  in a Haskell like fashion. Internally, they are mapped to more primitive 
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
    86
  Isabelle concepts \cite{Haftmann-Wenzel:2006:classes}.
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    87
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    88
  This tutorial demonstrates common elements of structured specifications
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    89
  and abstract reasoning with type classes by the algebraic hierarchy of
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
    90
  semigroups, monoids and groups.  Our background theory is that of
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
    91
  Isabelle/HOL \cite{isa-tutorial}, for which some
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    92
  familiarity is assumed.
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
    93
*}
75b56e51fade initial draft
haftmann
parents:
diff changeset
    94
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
    95
section {* A simple algebra example \label{sec:example} *}
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
    96
75b56e51fade initial draft
haftmann
parents:
diff changeset
    97
subsection {* Class definition *}
75b56e51fade initial draft
haftmann
parents:
diff changeset
    98
75b56e51fade initial draft
haftmann
parents:
diff changeset
    99
text {*
75b56e51fade initial draft
haftmann
parents:
diff changeset
   100
  Depending on an arbitrary type @{text "\<alpha>"}, class @{text
28565
haftmann
parents: 28540
diff changeset
   101
  "semigroup"} introduces a binary operator @{text "(\<otimes>)"} that is
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   102
  assumed to be associative:
75b56e51fade initial draft
haftmann
parents:
diff changeset
   103
*}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   104
29705
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   105
class %quote semigroup =
28565
haftmann
parents: 28540
diff changeset
   106
  fixes mult :: "\<alpha> \<Rightarrow> \<alpha> \<Rightarrow> \<alpha>"    (infixl "\<otimes>" 70)
haftmann
parents: 28540
diff changeset
   107
  assumes assoc: "(x \<otimes> y) \<otimes> z = x \<otimes> (y \<otimes> z)"
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   108
75b56e51fade initial draft
haftmann
parents:
diff changeset
   109
text {*
28565
haftmann
parents: 28540
diff changeset
   110
  \noindent This @{command class} specification consists of two
haftmann
parents: 28540
diff changeset
   111
  parts: the \qn{operational} part names the class parameter
haftmann
parents: 28540
diff changeset
   112
  (@{element "fixes"}), the \qn{logical} part specifies properties on them
haftmann
parents: 28540
diff changeset
   113
  (@{element "assumes"}).  The local @{element "fixes"} and
haftmann
parents: 28540
diff changeset
   114
  @{element "assumes"} are lifted to the theory toplevel,
haftmann
parents: 28540
diff changeset
   115
  yielding the global
24991
c6f5cc939c29 added subclass command
haftmann
parents: 24628
diff changeset
   116
  parameter @{term [source] "mult \<Colon> \<alpha>\<Colon>semigroup \<Rightarrow> \<alpha> \<Rightarrow> \<alpha>"} and the
28565
haftmann
parents: 28540
diff changeset
   117
  global theorem @{fact "semigroup.assoc:"}~@{prop [source] "\<And>x y
22479
de15ea8fb348 updated code generation sections
haftmann
parents: 22473
diff changeset
   118
  z \<Colon> \<alpha>\<Colon>semigroup. (x \<otimes> y) \<otimes> z = x \<otimes> (y \<otimes> z)"}.
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   119
*}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   120
75b56e51fade initial draft
haftmann
parents:
diff changeset
   121
75b56e51fade initial draft
haftmann
parents:
diff changeset
   122
subsection {* Class instantiation \label{sec:class_inst} *}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   123
75b56e51fade initial draft
haftmann
parents:
diff changeset
   124
text {*
28565
haftmann
parents: 28540
diff changeset
   125
  The concrete type @{typ int} is made a @{class semigroup}
24991
c6f5cc939c29 added subclass command
haftmann
parents: 24628
diff changeset
   126
  instance by providing a suitable definition for the class parameter
28565
haftmann
parents: 28540
diff changeset
   127
  @{text "(\<otimes>)"} and a proof for the specification of @{fact assoc}.
haftmann
parents: 28540
diff changeset
   128
  This is accomplished by the @{command instantiation} target:
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   129
*}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   130
28565
haftmann
parents: 28540
diff changeset
   131
instantiation %quote int :: semigroup
haftmann
parents: 28540
diff changeset
   132
begin
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   133
28565
haftmann
parents: 28540
diff changeset
   134
definition %quote
haftmann
parents: 28540
diff changeset
   135
  mult_int_def: "i \<otimes> j = i + (j\<Colon>int)"
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   136
28565
haftmann
parents: 28540
diff changeset
   137
instance %quote proof
haftmann
parents: 28540
diff changeset
   138
  fix i j k :: int have "(i + j) + k = i + (j + k)" by simp
haftmann
parents: 28540
diff changeset
   139
  then show "(i \<otimes> j) \<otimes> k = i \<otimes> (j \<otimes> k)"
28566
haftmann
parents: 28565
diff changeset
   140
    unfolding mult_int_def .
28565
haftmann
parents: 28540
diff changeset
   141
qed
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   142
28565
haftmann
parents: 28540
diff changeset
   143
end %quote
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   144
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   145
text {*
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   146
  \noindent @{command instantiation} defines class parameters
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   147
  at a particular instance using common specification tools (here,
28565
haftmann
parents: 28540
diff changeset
   148
  @{command definition}).  The concluding @{command instance}
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   149
  opens a proof that the given parameters actually conform
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   150
  to the class specification.  Note that the first proof step
28565
haftmann
parents: 28540
diff changeset
   151
  is the @{method default} method,
haftmann
parents: 28540
diff changeset
   152
  which for such instance proofs maps to the @{method intro_classes} method.
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   153
  This reduces an instance judgement to the relevant primitive
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   154
  proof goals; typically it is the first method applied
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   155
  in an instantiation proof.
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   156
28565
haftmann
parents: 28540
diff changeset
   157
  From now on, the type-checker will consider @{typ int}
haftmann
parents: 28540
diff changeset
   158
  as a @{class semigroup} automatically, i.e.\ any general results
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   159
  are immediately available on concrete instances.
28565
haftmann
parents: 28540
diff changeset
   160
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   161
  \medskip Another instance of @{class semigroup} yields the natural numbers:
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   162
*}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   163
28565
haftmann
parents: 28540
diff changeset
   164
instantiation %quote nat :: semigroup
haftmann
parents: 28540
diff changeset
   165
begin
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   166
28565
haftmann
parents: 28540
diff changeset
   167
primrec %quote mult_nat where
haftmann
parents: 28540
diff changeset
   168
  "(0\<Colon>nat) \<otimes> n = n"
haftmann
parents: 28540
diff changeset
   169
  | "Suc m \<otimes> n = Suc (m \<otimes> n)"
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   170
28565
haftmann
parents: 28540
diff changeset
   171
instance %quote proof
haftmann
parents: 28540
diff changeset
   172
  fix m n q :: nat 
haftmann
parents: 28540
diff changeset
   173
  show "m \<otimes> n \<otimes> q = m \<otimes> (n \<otimes> q)"
haftmann
parents: 28540
diff changeset
   174
    by (induct m) auto
haftmann
parents: 28540
diff changeset
   175
qed
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   176
28565
haftmann
parents: 28540
diff changeset
   177
end %quote
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   178
25871
45753d56d935 some more primrec
haftmann
parents: 25868
diff changeset
   179
text {*
45753d56d935 some more primrec
haftmann
parents: 25868
diff changeset
   180
  \noindent Note the occurence of the name @{text mult_nat}
45753d56d935 some more primrec
haftmann
parents: 25868
diff changeset
   181
  in the primrec declaration;  by default, the local name of
31675
6c95ec0394f1 fixed grammar
haftmann
parents: 31255
diff changeset
   182
  a class operation @{text f} to be instantiated on type constructor
6c95ec0394f1 fixed grammar
haftmann
parents: 31255
diff changeset
   183
  @{text \<kappa>} is mangled as @{text f_\<kappa>}.  In case of uncertainty,
28565
haftmann
parents: 28540
diff changeset
   184
  these names may be inspected using the @{command "print_context"} command
25871
45753d56d935 some more primrec
haftmann
parents: 25868
diff changeset
   185
  or the corresponding ProofGeneral button.
45753d56d935 some more primrec
haftmann
parents: 25868
diff changeset
   186
*}
45753d56d935 some more primrec
haftmann
parents: 25868
diff changeset
   187
25247
haftmann
parents: 25200
diff changeset
   188
subsection {* Lifting and parametric types *}
haftmann
parents: 25200
diff changeset
   189
haftmann
parents: 25200
diff changeset
   190
text {*
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   191
  Overloaded definitions given at a class instantiation
25247
haftmann
parents: 25200
diff changeset
   192
  may include recursion over the syntactic structure of types.
haftmann
parents: 25200
diff changeset
   193
  As a canonical example, we model product semigroups
haftmann
parents: 25200
diff changeset
   194
  using our simple algebra:
haftmann
parents: 25200
diff changeset
   195
*}
haftmann
parents: 25200
diff changeset
   196
28565
haftmann
parents: 28540
diff changeset
   197
instantiation %quote * :: (semigroup, semigroup) semigroup
haftmann
parents: 28540
diff changeset
   198
begin
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   199
28565
haftmann
parents: 28540
diff changeset
   200
definition %quote
31931
0b1d807b1c2d restored subscripts
haftmann
parents: 31691
diff changeset
   201
  mult_prod_def: "p\<^isub>1 \<otimes> p\<^isub>2 = (fst p\<^isub>1 \<otimes> fst p\<^isub>2, snd p\<^isub>1 \<otimes> snd p\<^isub>2)"
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   202
28565
haftmann
parents: 28540
diff changeset
   203
instance %quote proof
31931
0b1d807b1c2d restored subscripts
haftmann
parents: 31691
diff changeset
   204
  fix p\<^isub>1 p\<^isub>2 p\<^isub>3 :: "\<alpha>\<Colon>semigroup \<times> \<beta>\<Colon>semigroup"
0b1d807b1c2d restored subscripts
haftmann
parents: 31691
diff changeset
   205
  show "p\<^isub>1 \<otimes> p\<^isub>2 \<otimes> p\<^isub>3 = p\<^isub>1 \<otimes> (p\<^isub>2 \<otimes> p\<^isub>3)"
28566
haftmann
parents: 28565
diff changeset
   206
    unfolding mult_prod_def by (simp add: assoc)
28565
haftmann
parents: 28540
diff changeset
   207
qed      
25247
haftmann
parents: 25200
diff changeset
   208
28565
haftmann
parents: 28540
diff changeset
   209
end %quote
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   210
25247
haftmann
parents: 25200
diff changeset
   211
text {*
31675
6c95ec0394f1 fixed grammar
haftmann
parents: 31255
diff changeset
   212
  \noindent Associativity of product semigroups is established using
28565
haftmann
parents: 28540
diff changeset
   213
  the definition of @{text "(\<otimes>)"} on products and the hypothetical
27505
ddd1e71adbfc fix more typos
huffman
parents: 27504
diff changeset
   214
  associativity of the type components;  these hypotheses
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   215
  are legitimate due to the @{class semigroup} constraints imposed
28565
haftmann
parents: 28540
diff changeset
   216
  on the type components by the @{command instance} proposition.
25247
haftmann
parents: 25200
diff changeset
   217
  Indeed, this pattern often occurs with parametric types
haftmann
parents: 25200
diff changeset
   218
  and type classes.
haftmann
parents: 25200
diff changeset
   219
*}
haftmann
parents: 25200
diff changeset
   220
haftmann
parents: 25200
diff changeset
   221
haftmann
parents: 25200
diff changeset
   222
subsection {* Subclassing *}
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   223
75b56e51fade initial draft
haftmann
parents:
diff changeset
   224
text {*
28565
haftmann
parents: 28540
diff changeset
   225
  We define a subclass @{text monoidl} (a semigroup with a left-hand neutral)
haftmann
parents: 28540
diff changeset
   226
  by extending @{class semigroup}
haftmann
parents: 28540
diff changeset
   227
  with one additional parameter @{text neutral} together
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   228
  with its characteristic property:
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   229
*}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   230
28565
haftmann
parents: 28540
diff changeset
   231
class %quote monoidl = semigroup +
haftmann
parents: 28540
diff changeset
   232
  fixes neutral :: "\<alpha>" ("\<one>")
haftmann
parents: 28540
diff changeset
   233
  assumes neutl: "\<one> \<otimes> x = x"
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   234
75b56e51fade initial draft
haftmann
parents:
diff changeset
   235
text {*
25247
haftmann
parents: 25200
diff changeset
   236
  \noindent Again, we prove some instances, by
24991
c6f5cc939c29 added subclass command
haftmann
parents: 24628
diff changeset
   237
  providing suitable parameter definitions and proofs for the
27505
ddd1e71adbfc fix more typos
huffman
parents: 27504
diff changeset
   238
  additional specifications.  Observe that instantiations
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   239
  for types with the same arity may be simultaneous:
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   240
*}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   241
28566
haftmann
parents: 28565
diff changeset
   242
instantiation %quote nat and int :: monoidl
haftmann
parents: 28565
diff changeset
   243
begin
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   244
28566
haftmann
parents: 28565
diff changeset
   245
definition %quote
haftmann
parents: 28565
diff changeset
   246
  neutral_nat_def: "\<one> = (0\<Colon>nat)"
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   247
28566
haftmann
parents: 28565
diff changeset
   248
definition %quote
haftmann
parents: 28565
diff changeset
   249
  neutral_int_def: "\<one> = (0\<Colon>int)"
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   250
28566
haftmann
parents: 28565
diff changeset
   251
instance %quote proof
haftmann
parents: 28565
diff changeset
   252
  fix n :: nat
haftmann
parents: 28565
diff changeset
   253
  show "\<one> \<otimes> n = n"
haftmann
parents: 28565
diff changeset
   254
    unfolding neutral_nat_def by simp
haftmann
parents: 28565
diff changeset
   255
next
haftmann
parents: 28565
diff changeset
   256
  fix k :: int
haftmann
parents: 28565
diff changeset
   257
  show "\<one> \<otimes> k = k"
haftmann
parents: 28565
diff changeset
   258
    unfolding neutral_int_def mult_int_def by simp
haftmann
parents: 28565
diff changeset
   259
qed
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   260
28566
haftmann
parents: 28565
diff changeset
   261
end %quote
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   262
28566
haftmann
parents: 28565
diff changeset
   263
instantiation %quote * :: (monoidl, monoidl) monoidl
haftmann
parents: 28565
diff changeset
   264
begin
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   265
28566
haftmann
parents: 28565
diff changeset
   266
definition %quote
haftmann
parents: 28565
diff changeset
   267
  neutral_prod_def: "\<one> = (\<one>, \<one>)"
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   268
28566
haftmann
parents: 28565
diff changeset
   269
instance %quote proof
haftmann
parents: 28565
diff changeset
   270
  fix p :: "\<alpha>\<Colon>monoidl \<times> \<beta>\<Colon>monoidl"
haftmann
parents: 28565
diff changeset
   271
  show "\<one> \<otimes> p = p"
haftmann
parents: 28565
diff changeset
   272
    unfolding neutral_prod_def mult_prod_def by (simp add: neutl)
haftmann
parents: 28565
diff changeset
   273
qed
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   274
28566
haftmann
parents: 28565
diff changeset
   275
end %quote
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   276
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   277
text {*
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   278
  \noindent Fully-fledged monoids are modelled by another subclass,
24991
c6f5cc939c29 added subclass command
haftmann
parents: 24628
diff changeset
   279
  which does not add new parameters but tightens the specification:
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   280
*}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   281
28566
haftmann
parents: 28565
diff changeset
   282
class %quote monoid = monoidl +
haftmann
parents: 28565
diff changeset
   283
  assumes neutr: "x \<otimes> \<one> = x"
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   284
28566
haftmann
parents: 28565
diff changeset
   285
instantiation %quote nat and int :: monoid 
haftmann
parents: 28565
diff changeset
   286
begin
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   287
28566
haftmann
parents: 28565
diff changeset
   288
instance %quote proof
haftmann
parents: 28565
diff changeset
   289
  fix n :: nat
haftmann
parents: 28565
diff changeset
   290
  show "n \<otimes> \<one> = n"
haftmann
parents: 28565
diff changeset
   291
    unfolding neutral_nat_def by (induct n) simp_all
haftmann
parents: 28565
diff changeset
   292
next
haftmann
parents: 28565
diff changeset
   293
  fix k :: int
haftmann
parents: 28565
diff changeset
   294
  show "k \<otimes> \<one> = k"
haftmann
parents: 28565
diff changeset
   295
    unfolding neutral_int_def mult_int_def by simp
haftmann
parents: 28565
diff changeset
   296
qed
25247
haftmann
parents: 25200
diff changeset
   297
28566
haftmann
parents: 28565
diff changeset
   298
end %quote
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   299
28566
haftmann
parents: 28565
diff changeset
   300
instantiation %quote * :: (monoid, monoid) monoid
haftmann
parents: 28565
diff changeset
   301
begin
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   302
28566
haftmann
parents: 28565
diff changeset
   303
instance %quote proof 
haftmann
parents: 28565
diff changeset
   304
  fix p :: "\<alpha>\<Colon>monoid \<times> \<beta>\<Colon>monoid"
haftmann
parents: 28565
diff changeset
   305
  show "p \<otimes> \<one> = p"
haftmann
parents: 28565
diff changeset
   306
    unfolding neutral_prod_def mult_prod_def by (simp add: neutr)
haftmann
parents: 28565
diff changeset
   307
qed
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   308
28566
haftmann
parents: 28565
diff changeset
   309
end %quote
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   310
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   311
text {*
28565
haftmann
parents: 28540
diff changeset
   312
  \noindent To finish our small algebra example, we add a @{text group} class
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   313
  with a corresponding instance:
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   314
*}
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   315
28566
haftmann
parents: 28565
diff changeset
   316
class %quote group = monoidl +
haftmann
parents: 28565
diff changeset
   317
  fixes inverse :: "\<alpha> \<Rightarrow> \<alpha>"    ("(_\<div>)" [1000] 999)
haftmann
parents: 28565
diff changeset
   318
  assumes invl: "x\<div> \<otimes> x = \<one>"
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   319
28566
haftmann
parents: 28565
diff changeset
   320
instantiation %quote int :: group
haftmann
parents: 28565
diff changeset
   321
begin
haftmann
parents: 28565
diff changeset
   322
haftmann
parents: 28565
diff changeset
   323
definition %quote
haftmann
parents: 28565
diff changeset
   324
  inverse_int_def: "i\<div> = - (i\<Colon>int)"
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   325
28566
haftmann
parents: 28565
diff changeset
   326
instance %quote proof
haftmann
parents: 28565
diff changeset
   327
  fix i :: int
haftmann
parents: 28565
diff changeset
   328
  have "-i + i = 0" by simp
haftmann
parents: 28565
diff changeset
   329
  then show "i\<div> \<otimes> i = \<one>"
haftmann
parents: 28565
diff changeset
   330
    unfolding mult_int_def neutral_int_def inverse_int_def .
haftmann
parents: 28565
diff changeset
   331
qed
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   332
28566
haftmann
parents: 28565
diff changeset
   333
end %quote
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   334
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   335
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   336
section {* Type classes as locales *}
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   337
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   338
subsection {* A look behind the scenes *}
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   339
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   340
text {*
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   341
  The example above gives an impression how Isar type classes work
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   342
  in practice.  As stated in the introduction, classes also provide
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   343
  a link to Isar's locale system.  Indeed, the logical core of a class
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   344
  is nothing other than a locale:
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   345
*}
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   346
29705
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   347
class %quote idem =
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   348
  fixes f :: "\<alpha> \<Rightarrow> \<alpha>"
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   349
  assumes idem: "f (f x) = f x"
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   350
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   351
text {*
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   352
  \noindent essentially introduces the locale
30227
853abb4853cc tuned manuals
haftmann
parents: 30226
diff changeset
   353
*} (*<*)setup %invisible {* Sign.add_path "foo" *}
853abb4853cc tuned manuals
haftmann
parents: 30226
diff changeset
   354
(*>*)
28566
haftmann
parents: 28565
diff changeset
   355
locale %quote idem =
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   356
  fixes f :: "\<alpha> \<Rightarrow> \<alpha>"
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   357
  assumes idem: "f (f x) = f x"
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   358
22550
c5039bee2602 updated
haftmann
parents: 22479
diff changeset
   359
text {* \noindent together with corresponding constant(s): *}
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   360
28566
haftmann
parents: 28565
diff changeset
   361
consts %quote f :: "\<alpha> \<Rightarrow> \<alpha>"
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   362
22550
c5039bee2602 updated
haftmann
parents: 22479
diff changeset
   363
text {*
c5039bee2602 updated
haftmann
parents: 22479
diff changeset
   364
  \noindent The connection to the type system is done by means
35282
8fd9d555d04d dropped references to old axclass from documentation
haftmann
parents: 31931
diff changeset
   365
  of a primitive type class
30227
853abb4853cc tuned manuals
haftmann
parents: 30226
diff changeset
   366
*} (*<*)setup %invisible {* Sign.add_path "foo" *}
853abb4853cc tuned manuals
haftmann
parents: 30226
diff changeset
   367
(*>*)
35282
8fd9d555d04d dropped references to old axclass from documentation
haftmann
parents: 31931
diff changeset
   368
classes %quote idem < type
8fd9d555d04d dropped references to old axclass from documentation
haftmann
parents: 31931
diff changeset
   369
(*<*)axiomatization where idem: "f (f (x::\<alpha>\<Colon>idem)) = f x"
8fd9d555d04d dropped references to old axclass from documentation
haftmann
parents: 31931
diff changeset
   370
setup %invisible {* Sign.parent_path *}(*>*)
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   371
22550
c5039bee2602 updated
haftmann
parents: 22479
diff changeset
   372
text {* \noindent together with a corresponding interpretation: *}
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   373
29513
363f17dee9ca adapted to changes in class package
haftmann
parents: 29294
diff changeset
   374
interpretation %quote idem_class:
29294
6cd3ac4708d2 crude adaption to intermediate class/locale version;
wenzelm
parents: 28948
diff changeset
   375
  idem "f \<Colon> (\<alpha>\<Colon>idem) \<Rightarrow> \<alpha>"
35282
8fd9d555d04d dropped references to old axclass from documentation
haftmann
parents: 31931
diff changeset
   376
(*<*)proof qed (rule idem)(*>*)
28565
haftmann
parents: 28540
diff changeset
   377
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   378
text {*
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   379
  \noindent This gives you the full power of the Isabelle module system;
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   380
  conclusions in locale @{text idem} are implicitly propagated
22479
de15ea8fb348 updated code generation sections
haftmann
parents: 22473
diff changeset
   381
  to class @{text idem}.
30227
853abb4853cc tuned manuals
haftmann
parents: 30226
diff changeset
   382
*} (*<*)setup %invisible {* Sign.parent_path *}
853abb4853cc tuned manuals
haftmann
parents: 30226
diff changeset
   383
(*>*)
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   384
subsection {* Abstract reasoning *}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   385
75b56e51fade initial draft
haftmann
parents:
diff changeset
   386
text {*
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   387
  Isabelle locales enable reasoning at a general level, while results
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   388
  are implicitly transferred to all instances.  For example, we can
75b56e51fade initial draft
haftmann
parents:
diff changeset
   389
  now establish the @{text "left_cancel"} lemma for groups, which
25247
haftmann
parents: 25200
diff changeset
   390
  states that the function @{text "(x \<otimes>)"} is injective:
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   391
*}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   392
28566
haftmann
parents: 28565
diff changeset
   393
lemma %quote (in group) left_cancel: "x \<otimes> y = x \<otimes> z \<longleftrightarrow> y = z"
haftmann
parents: 28565
diff changeset
   394
proof
haftmann
parents: 28565
diff changeset
   395
  assume "x \<otimes> y = x \<otimes> z"
haftmann
parents: 28565
diff changeset
   396
  then have "x\<div> \<otimes> (x \<otimes> y) = x\<div> \<otimes> (x \<otimes> z)" by simp
haftmann
parents: 28565
diff changeset
   397
  then have "(x\<div> \<otimes> x) \<otimes> y = (x\<div> \<otimes> x) \<otimes> z" using assoc by simp
haftmann
parents: 28565
diff changeset
   398
  then show "y = z" using neutl and invl by simp
haftmann
parents: 28565
diff changeset
   399
next
haftmann
parents: 28565
diff changeset
   400
  assume "y = z"
haftmann
parents: 28565
diff changeset
   401
  then show "x \<otimes> y = x \<otimes> z" by simp
haftmann
parents: 28565
diff changeset
   402
qed
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   403
75b56e51fade initial draft
haftmann
parents:
diff changeset
   404
text {*
28565
haftmann
parents: 28540
diff changeset
   405
  \noindent Here the \qt{@{keyword "in"} @{class group}} target specification
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   406
  indicates that the result is recorded within that context for later
28565
haftmann
parents: 28540
diff changeset
   407
  use.  This local theorem is also lifted to the global one @{fact
22479
de15ea8fb348 updated code generation sections
haftmann
parents: 22473
diff changeset
   408
  "group.left_cancel:"} @{prop [source] "\<And>x y z \<Colon> \<alpha>\<Colon>group. x \<otimes> y = x \<otimes>
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   409
  z \<longleftrightarrow> y = z"}.  Since type @{text "int"} has been made an instance of
75b56e51fade initial draft
haftmann
parents:
diff changeset
   410
  @{text "group"} before, we may refer to that fact as well: @{prop
22479
de15ea8fb348 updated code generation sections
haftmann
parents: 22473
diff changeset
   411
  [source] "\<And>x y z \<Colon> int. x \<otimes> y = x \<otimes> z \<longleftrightarrow> y = z"}.
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   412
*}
75b56e51fade initial draft
haftmann
parents:
diff changeset
   413
75b56e51fade initial draft
haftmann
parents:
diff changeset
   414
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   415
subsection {* Derived definitions *}
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   416
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   417
text {*
35282
8fd9d555d04d dropped references to old axclass from documentation
haftmann
parents: 31931
diff changeset
   418
  Isabelle locales are targets which support local definitions:
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   419
*}
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   420
28566
haftmann
parents: 28565
diff changeset
   421
primrec %quote (in monoid) pow_nat :: "nat \<Rightarrow> \<alpha> \<Rightarrow> \<alpha>" where
haftmann
parents: 28565
diff changeset
   422
  "pow_nat 0 x = \<one>"
haftmann
parents: 28565
diff changeset
   423
  | "pow_nat (Suc n) x = x \<otimes> pow_nat n x"
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   424
75b56e51fade initial draft
haftmann
parents:
diff changeset
   425
text {*
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   426
  \noindent If the locale @{text group} is also a class, this local
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   427
  definition is propagated onto a global definition of
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   428
  @{term [source] "pow_nat \<Colon> nat \<Rightarrow> \<alpha>\<Colon>monoid \<Rightarrow> \<alpha>\<Colon>monoid"}
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   429
  with corresponding theorems
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   430
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   431
  @{thm pow_nat.simps [no_vars]}.
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   432
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   433
  \noindent As you can see from this example, for local
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   434
  definitions you may use any specification tool
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   435
  which works together with locales, such as Krauss's recursive function package
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   436
  \cite{krauss2006}.
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   437
*}
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   438
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   439
25247
haftmann
parents: 25200
diff changeset
   440
subsection {* A functor analogy *}
haftmann
parents: 25200
diff changeset
   441
haftmann
parents: 25200
diff changeset
   442
text {*
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   443
  We introduced Isar classes by analogy to type classes in
25247
haftmann
parents: 25200
diff changeset
   444
  functional programming;  if we reconsider this in the
haftmann
parents: 25200
diff changeset
   445
  context of what has been said about type classes and locales,
haftmann
parents: 25200
diff changeset
   446
  we can drive this analogy further by stating that type
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   447
  classes essentially correspond to functors that have
25247
haftmann
parents: 25200
diff changeset
   448
  a canonical interpretation as type classes.
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   449
  There is also the possibility of other interpretations.
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   450
  For example, @{text list}s also form a monoid with
28565
haftmann
parents: 28540
diff changeset
   451
  @{text append} and @{term "[]"} as operations, but it
25247
haftmann
parents: 25200
diff changeset
   452
  seems inappropriate to apply to lists
27505
ddd1e71adbfc fix more typos
huffman
parents: 27504
diff changeset
   453
  the same operations as for genuinely algebraic types.
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   454
  In such a case, we can simply make a particular interpretation
25247
haftmann
parents: 25200
diff changeset
   455
  of monoids for lists:
haftmann
parents: 25200
diff changeset
   456
*}
haftmann
parents: 25200
diff changeset
   457
30729
461ee3e49ad3 interpretation/interpret: prefixes are mandatory by default;
wenzelm
parents: 30227
diff changeset
   458
interpretation %quote list_monoid: monoid append "[]"
28947
ac1a14b5a085 unfold_locales is default method - no need for explicit references
haftmann
parents: 28566
diff changeset
   459
  proof qed auto
25247
haftmann
parents: 25200
diff changeset
   460
haftmann
parents: 25200
diff changeset
   461
text {*
haftmann
parents: 25200
diff changeset
   462
  \noindent This enables us to apply facts on monoids
haftmann
parents: 25200
diff changeset
   463
  to lists, e.g. @{thm list_monoid.neutl [no_vars]}.
haftmann
parents: 25200
diff changeset
   464
haftmann
parents: 25200
diff changeset
   465
  When using this interpretation pattern, it may also
haftmann
parents: 25200
diff changeset
   466
  be appropriate to map derived definitions accordingly:
haftmann
parents: 25200
diff changeset
   467
*}
haftmann
parents: 25200
diff changeset
   468
28566
haftmann
parents: 28565
diff changeset
   469
primrec %quote replicate :: "nat \<Rightarrow> \<alpha> list \<Rightarrow> \<alpha> list" where
haftmann
parents: 28565
diff changeset
   470
  "replicate 0 _ = []"
haftmann
parents: 28565
diff changeset
   471
  | "replicate (Suc n) xs = xs @ replicate n xs"
25247
haftmann
parents: 25200
diff changeset
   472
30729
461ee3e49ad3 interpretation/interpret: prefixes are mandatory by default;
wenzelm
parents: 30227
diff changeset
   473
interpretation %quote list_monoid: monoid append "[]" where
28566
haftmann
parents: 28565
diff changeset
   474
  "monoid.pow_nat append [] = replicate"
haftmann
parents: 28565
diff changeset
   475
proof -
29513
363f17dee9ca adapted to changes in class package
haftmann
parents: 29294
diff changeset
   476
  interpret monoid append "[]" ..
28566
haftmann
parents: 28565
diff changeset
   477
  show "monoid.pow_nat append [] = replicate"
haftmann
parents: 28565
diff changeset
   478
  proof
haftmann
parents: 28565
diff changeset
   479
    fix n
haftmann
parents: 28565
diff changeset
   480
    show "monoid.pow_nat append [] n = replicate n"
haftmann
parents: 28565
diff changeset
   481
      by (induct n) auto
haftmann
parents: 28565
diff changeset
   482
  qed
haftmann
parents: 28565
diff changeset
   483
qed intro_locales
25247
haftmann
parents: 25200
diff changeset
   484
31255
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   485
text {*
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   486
  \noindent This pattern is also helpful to reuse abstract
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   487
  specifications on the \emph{same} type.  For example, think of a
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   488
  class @{text preorder}; for type @{typ nat}, there are at least two
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   489
  possible instances: the natural order or the order induced by the
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   490
  divides relation.  But only one of these instances can be used for
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   491
  @{command instantiation}; using the locale behind the class @{text
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   492
  preorder}, it is still possible to utilise the same abstract
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   493
  specification again using @{command interpretation}.
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   494
*}
25247
haftmann
parents: 25200
diff changeset
   495
24991
c6f5cc939c29 added subclass command
haftmann
parents: 24628
diff changeset
   496
subsection {* Additional subclass relations *}
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   497
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   498
text {*
31255
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   499
  Any @{text "group"} is also a @{text "monoid"}; this can be made
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   500
  explicit by claiming an additional subclass relation, together with
0f8cb37bcafd clarified benefit of interpretation
haftmann
parents: 30729
diff changeset
   501
  a proof of the logical difference:
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   502
*}
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   503
28566
haftmann
parents: 28565
diff changeset
   504
subclass %quote (in group) monoid
28947
ac1a14b5a085 unfold_locales is default method - no need for explicit references
haftmann
parents: 28566
diff changeset
   505
proof
28566
haftmann
parents: 28565
diff changeset
   506
  fix x
haftmann
parents: 28565
diff changeset
   507
  from invl have "x\<div> \<otimes> x = \<one>" by simp
haftmann
parents: 28565
diff changeset
   508
  with assoc [symmetric] neutl invl have "x\<div> \<otimes> (x \<otimes> \<one>) = x\<div> \<otimes> x" by simp
haftmann
parents: 28565
diff changeset
   509
  with left_cancel show "x \<otimes> \<one> = x" by simp
haftmann
parents: 28565
diff changeset
   510
qed
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   511
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   512
text {*
30227
853abb4853cc tuned manuals
haftmann
parents: 30226
diff changeset
   513
  The logical proof is carried out on the locale level.
28947
ac1a14b5a085 unfold_locales is default method - no need for explicit references
haftmann
parents: 28566
diff changeset
   514
  Afterwards it is propagated
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   515
  to the type system, making @{text group} an instance of
25247
haftmann
parents: 25200
diff changeset
   516
  @{text monoid} by adding an additional edge
haftmann
parents: 25200
diff changeset
   517
  to the graph of subclass relations
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   518
  (\figref{fig:subclass}).
25247
haftmann
parents: 25200
diff changeset
   519
haftmann
parents: 25200
diff changeset
   520
  \begin{figure}[htbp]
haftmann
parents: 25200
diff changeset
   521
   \begin{center}
haftmann
parents: 25200
diff changeset
   522
     \small
haftmann
parents: 25200
diff changeset
   523
     \unitlength 0.6mm
haftmann
parents: 25200
diff changeset
   524
     \begin{picture}(40,60)(0,0)
haftmann
parents: 25200
diff changeset
   525
       \put(20,60){\makebox(0,0){@{text semigroup}}}
haftmann
parents: 25200
diff changeset
   526
       \put(20,40){\makebox(0,0){@{text monoidl}}}
haftmann
parents: 25200
diff changeset
   527
       \put(00,20){\makebox(0,0){@{text monoid}}}
haftmann
parents: 25200
diff changeset
   528
       \put(40,00){\makebox(0,0){@{text group}}}
haftmann
parents: 25200
diff changeset
   529
       \put(20,55){\vector(0,-1){10}}
haftmann
parents: 25200
diff changeset
   530
       \put(15,35){\vector(-1,-1){10}}
haftmann
parents: 25200
diff changeset
   531
       \put(25,35){\vector(1,-3){10}}
haftmann
parents: 25200
diff changeset
   532
     \end{picture}
haftmann
parents: 25200
diff changeset
   533
     \hspace{8em}
haftmann
parents: 25200
diff changeset
   534
     \begin{picture}(40,60)(0,0)
haftmann
parents: 25200
diff changeset
   535
       \put(20,60){\makebox(0,0){@{text semigroup}}}
haftmann
parents: 25200
diff changeset
   536
       \put(20,40){\makebox(0,0){@{text monoidl}}}
haftmann
parents: 25200
diff changeset
   537
       \put(00,20){\makebox(0,0){@{text monoid}}}
haftmann
parents: 25200
diff changeset
   538
       \put(40,00){\makebox(0,0){@{text group}}}
haftmann
parents: 25200
diff changeset
   539
       \put(20,55){\vector(0,-1){10}}
haftmann
parents: 25200
diff changeset
   540
       \put(15,35){\vector(-1,-1){10}}
haftmann
parents: 25200
diff changeset
   541
       \put(05,15){\vector(3,-1){30}}
haftmann
parents: 25200
diff changeset
   542
     \end{picture}
haftmann
parents: 25200
diff changeset
   543
     \caption{Subclass relationship of monoids and groups:
haftmann
parents: 25200
diff changeset
   544
        before and after establishing the relationship
30134
c2640140b951 fixed typo
haftmann
parents: 29705
diff changeset
   545
        @{text "group \<subseteq> monoid"};  transitive edges are left out.}
25247
haftmann
parents: 25200
diff changeset
   546
     \label{fig:subclass}
haftmann
parents: 25200
diff changeset
   547
   \end{center}
haftmann
parents: 25200
diff changeset
   548
  \end{figure}
30227
853abb4853cc tuned manuals
haftmann
parents: 30226
diff changeset
   549
25247
haftmann
parents: 25200
diff changeset
   550
  For illustration, a derived definition
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   551
  in @{text group} using @{text pow_nat}
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   552
*}
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   553
28565
haftmann
parents: 28540
diff changeset
   554
definition %quote (in group) pow_int :: "int \<Rightarrow> \<alpha> \<Rightarrow> \<alpha>" where
haftmann
parents: 28540
diff changeset
   555
  "pow_int k x = (if k >= 0
haftmann
parents: 28540
diff changeset
   556
    then pow_nat (nat k) x
haftmann
parents: 28540
diff changeset
   557
    else (pow_nat (nat (- k)) x)\<div>)"
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   558
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   559
text {*
25247
haftmann
parents: 25200
diff changeset
   560
  \noindent yields the global definition of
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   561
  @{term [source] "pow_int \<Colon> int \<Rightarrow> \<alpha>\<Colon>group \<Rightarrow> \<alpha>\<Colon>group"}
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   562
  with the corresponding theorem @{thm pow_int_def [no_vars]}.
24991
c6f5cc939c29 added subclass command
haftmann
parents: 24628
diff changeset
   563
*}
23956
48494ccfabaf updated
haftmann
parents: 22845
diff changeset
   564
25868
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   565
subsection {* A note on syntax *}
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   566
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   567
text {*
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   568
  As a convenience, class context syntax allows references
27505
ddd1e71adbfc fix more typos
huffman
parents: 27504
diff changeset
   569
  to local class operations and their global counterparts
25868
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   570
  uniformly;  type inference resolves ambiguities.  For example:
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   571
*}
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   572
28565
haftmann
parents: 28540
diff changeset
   573
context %quote semigroup
25868
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   574
begin
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   575
28565
haftmann
parents: 28540
diff changeset
   576
term %quote "x \<otimes> y" -- {* example 1 *}
haftmann
parents: 28540
diff changeset
   577
term %quote "(x\<Colon>nat) \<otimes> y" -- {* example 2 *}
25868
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   578
28566
haftmann
parents: 28565
diff changeset
   579
end  %quote
25868
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   580
28565
haftmann
parents: 28540
diff changeset
   581
term %quote "x \<otimes> y" -- {* example 3 *}
25868
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   582
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   583
text {*
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   584
  \noindent Here in example 1, the term refers to the local class operation
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   585
  @{text "mult [\<alpha>]"}, whereas in example 2 the type constraint
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   586
  enforces the global class operation @{text "mult [nat]"}.
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   587
  In the global context in example 3, the reference is
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   588
  to the polymorphic global class operation @{text "mult [?\<alpha> \<Colon> semigroup]"}.
97c6787099bc a note on syntax
haftmann
parents: 25533
diff changeset
   589
*}
22347
ddbf185a3be0 continued
haftmann
parents: 22317
diff changeset
   590
29705
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   591
section {* Further issues *}
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   592
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   593
subsection {* Type classes and code generation *}
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   594
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   595
text {*
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   596
  Turning back to the first motivation for type classes,
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   597
  namely overloading, it is obvious that overloading
28565
haftmann
parents: 28540
diff changeset
   598
  stemming from @{command class} statements and
haftmann
parents: 28540
diff changeset
   599
  @{command instantiation}
25533
0140cc7b26ad added something about instantiation target
haftmann
parents: 25369
diff changeset
   600
  targets naturally maps to Haskell type classes.
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   601
  The code generator framework \cite{isabelle-codegen} 
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   602
  takes this into account.  If the target language (e.g.~SML)
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   603
  lacks type classes, then they
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   604
  are implemented by an explicit dictionary construction.
28540
haftmann
parents: 27505
diff changeset
   605
  As example, let's go back to the power function:
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   606
*}
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   607
28565
haftmann
parents: 28540
diff changeset
   608
definition %quote example :: int where
haftmann
parents: 28540
diff changeset
   609
  "example = pow_int 10 (-2)"
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   610
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   611
text {*
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   612
  \noindent This maps to Haskell as follows:
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   613
*}
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   614
28565
haftmann
parents: 28540
diff changeset
   615
text %quote {*@{code_stmts example (Haskell)}*}
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   616
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   617
text {*
31691
7d50527dc008 Polishing the English
paulson
parents: 31675
diff changeset
   618
  \noindent The code in SML has explicit dictionary passing:
22317
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   619
*}
b550d2c6ca90 continued class tutorial
haftmann
parents: 20946
diff changeset
   620
28565
haftmann
parents: 28540
diff changeset
   621
text %quote {*@{code_stmts example (SML)}*}
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   622
29705
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   623
subsection {* Inspecting the type class universe *}
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   624
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   625
text {*
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   626
  To facilitate orientation in complex subclass structures,
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   627
  two diagnostics commands are provided:
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   628
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   629
  \begin{description}
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   630
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   631
    \item[@{command "print_classes"}] print a list of all classes
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   632
      together with associated operations etc.
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   633
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   634
    \item[@{command "class_deps"}] visualizes the subclass relation
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   635
      between all classes as a Hasse diagram.
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   636
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   637
  \end{description}
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   638
*}
a1ecdd8cf81c updated class documentation
haftmann
parents: 29513
diff changeset
   639
20946
75b56e51fade initial draft
haftmann
parents:
diff changeset
   640
end