src/Doc/Locales/Examples1.thy
author wenzelm
Wed, 26 Sep 2018 22:38:16 +0200
changeset 69074 787f3db8e313
parent 67399 eab6ce8368fa
child 69505 cc2d676d5395
permissions -rw-r--r--
tuned signature;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     1
theory Examples1
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     2
imports Examples
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     3
begin
57607
5ff0cf3f5f6f discontinued presumable workarounds for extra inter-theory space, which are obsolete since 0e5fa27d3293;
wenzelm
parents: 48985
diff changeset
     4
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
     5
section \<open>Use of Locales in Theories and Proofs
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
     6
  \label{sec:interpretation}\<close>
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
     7
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
     8
text \<open>
32983
a6914429005b Finished revisions of locales tutorial.
ballarin
parents: 32982
diff changeset
     9
  Locales can be interpreted in the contexts of theories and
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    10
  structured proofs.  These interpretations are dynamic, too.
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    11
  Conclusions of locales will be propagated to the current theory or
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    12
  the current proof context.%
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    13
\footnote{Strictly speaking, only interpretation in theories is
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    14
  dynamic since it is not possible to change locales or the locale
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    15
  hierarchy from within a proof.}
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    16
  The focus of this section is on
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    17
  interpretation in theories, but we will also encounter
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    18
  interpretations in proofs, in
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    19
  Section~\ref{sec:local-interpretation}.
30580
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 29293
diff changeset
    20
32982
40810d98f4c9 Changed part of the examples to int.
ballarin
parents: 32981
diff changeset
    21
  As an example, consider the type of integers @{typ int}.  The
67399
eab6ce8368fa ran isabelle update_op on all sources
nipkow
parents: 61701
diff changeset
    22
  relation @{term "(\<le>)"} is a total order over @{typ int}.  We start
eab6ce8368fa ran isabelle update_op on all sources
nipkow
parents: 61701
diff changeset
    23
  with the interpretation that @{term "(\<le>)"} is a partial order.  The
32983
a6914429005b Finished revisions of locales tutorial.
ballarin
parents: 32982
diff changeset
    24
  facilities of the interpretation command are explored gradually in
a6914429005b Finished revisions of locales tutorial.
ballarin
parents: 32982
diff changeset
    25
  three versions.
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    26
\<close>
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    27
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    28
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    29
subsection \<open>First Version: Replacement of Parameters Only
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    30
  \label{sec:po-first}\<close>
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    31
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    32
text \<open>
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    33
  The command \isakeyword{interpretation} is for the interpretation of
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    34
  locale in theories.  In the following example, the parameter of locale
67399
eab6ce8368fa ran isabelle update_op on all sources
nipkow
parents: 61701
diff changeset
    35
  @{text partial_order} is replaced by @{term "(\<le>) :: int \<Rightarrow> int \<Rightarrow>
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    36
  bool"} and the locale instance is interpreted in the current
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    37
  theory.\<close>
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    38
67399
eab6ce8368fa ran isabelle update_op on all sources
nipkow
parents: 61701
diff changeset
    39
  interpretation %visible int: partial_order "(\<le>) :: int \<Rightarrow> int \<Rightarrow> bool"
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    40
txt \<open>\normalsize
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    41
  The argument of the command is a simple \emph{locale expression}
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    42
  consisting of the name of the interpreted locale, which is
32982
40810d98f4c9 Changed part of the examples to int.
ballarin
parents: 32981
diff changeset
    43
  preceded by the qualifier @{text "int:"} and succeeded by a
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    44
  white-space-separated list of terms, which provide a full
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    45
  instantiation of the locale parameters.  The parameters are referred
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    46
  to by order of declaration, which is also the order in which
32983
a6914429005b Finished revisions of locales tutorial.
ballarin
parents: 32982
diff changeset
    47
  \isakeyword{print\_locale} outputs them.  The locale has only a
a6914429005b Finished revisions of locales tutorial.
ballarin
parents: 32982
diff changeset
    48
  single parameter, hence the list of instantiation terms is a
a6914429005b Finished revisions of locales tutorial.
ballarin
parents: 32982
diff changeset
    49
  singleton.
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    50
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    51
  The command creates the goal
30580
cc5a55d7a5be Updated chapters 1-5 to locale reimplementation.
ballarin
parents: 29293
diff changeset
    52
  @{subgoals [display]} which can be shown easily:
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    53
\<close>
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    54
    by unfold_locales auto
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    55
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    56
text \<open>The effect of the command is that instances of all
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    57
  conclusions of the locale are available in the theory, where names
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    58
  are prefixed by the qualifier.  For example, transitivity for @{typ
32982
40810d98f4c9 Changed part of the examples to int.
ballarin
parents: 32981
diff changeset
    59
  int} is named @{thm [source] int.trans} and is the following
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    60
  theorem:
32982
40810d98f4c9 Changed part of the examples to int.
ballarin
parents: 32981
diff changeset
    61
  @{thm [display, indent=2] int.trans}
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    62
  It is not possible to reference this theorem simply as @{text
32983
a6914429005b Finished revisions of locales tutorial.
ballarin
parents: 32982
diff changeset
    63
  trans}.  This prevents unwanted hiding of existing theorems of the
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    64
  theory by an interpretation.\<close>
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    65
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    66
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    67
subsection \<open>Second Version: Replacement of Definitions\<close>
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    68
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    69
text \<open>Not only does the above interpretation qualify theorem names.
32982
40810d98f4c9 Changed part of the examples to int.
ballarin
parents: 32981
diff changeset
    70
  The prefix @{text int} is applied to all names introduced in locale
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    71
  conclusions including names introduced in definitions.  The
32983
a6914429005b Finished revisions of locales tutorial.
ballarin
parents: 32982
diff changeset
    72
  qualified name @{text int.less} is short for
67399
eab6ce8368fa ran isabelle update_op on all sources
nipkow
parents: 61701
diff changeset
    73
  the interpretation of the definition, which is @{text "partial_order.less (\<le>)"}.
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    74
  Qualified name and expanded form may be used almost
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    75
  interchangeably.%
67399
eab6ce8368fa ran isabelle update_op on all sources
nipkow
parents: 61701
diff changeset
    76
\footnote{Since @{term "(\<le>)"} is polymorphic, for @{text "partial_order.less (\<le>)"} a
32982
40810d98f4c9 Changed part of the examples to int.
ballarin
parents: 32981
diff changeset
    77
  more general type will be inferred than for @{text int.less} which
40810d98f4c9 Changed part of the examples to int.
ballarin
parents: 32981
diff changeset
    78
  is over type @{typ int}.}
61701
e89cfc004f18 Refine the supression of abbreviations for morphisms that are not identities.
ballarin
parents: 61566
diff changeset
    79
  The former is preferred on output, as for example in the theorem
32982
40810d98f4c9 Changed part of the examples to int.
ballarin
parents: 32981
diff changeset
    80
  @{thm [source] int.less_le_trans}: @{thm [display, indent=2]
40810d98f4c9 Changed part of the examples to int.
ballarin
parents: 32981
diff changeset
    81
  int.less_le_trans}
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    82
  Both notations for the strict order are not satisfactory.  The
67399
eab6ce8368fa ran isabelle update_op on all sources
nipkow
parents: 61701
diff changeset
    83
  constant @{term "(<)"} is the strict order for @{typ int}.
32981
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    84
  In order to allow for the desired replacement, interpretation
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    85
  accepts \emph{equations} in addition to the parameter instantiation.
0114e04a0d64 Save current state of locales tutorial.
ballarin
parents: 30826
diff changeset
    86
  These follow the locale expression and are indicated with the
61566
c3d6e570ccef Keyword 'rewrites' identifies rewrite morphisms.
ballarin
parents: 61419
diff changeset
    87
  keyword \isakeyword{rewrites}.  This is the revised interpretation:
61419
3c3f8b182e4b isabelle update_cartouches;
wenzelm
parents: 57607
diff changeset
    88
\<close>
27063
d1d35284542f New version covering interpretation.
ballarin
parents:
diff changeset
    89
end