doc-src/IsarRef/Thy/Proof.thy
author Walther Neuper <neuper@ist.tugraz.at>
Thu, 12 Aug 2010 15:03:34 +0200
branchisac-from-Isabelle2009-2
changeset 37913 20e3616b2d9c
parent 37465 dfca6c4cd1e8
child 40516 9ffbc25e1606
permissions -rw-r--r--
prepare reactivation of isac-update-Isa09-2
wenzelm@26869
     1
theory Proof
wenzelm@26869
     2
imports Main
wenzelm@26869
     3
begin
wenzelm@26869
     4
wenzelm@30070
     5
chapter {* Proofs \label{ch:proofs} *}
wenzelm@26869
     6
wenzelm@26870
     7
text {*
wenzelm@26870
     8
  Proof commands perform transitions of Isar/VM machine
wenzelm@26870
     9
  configurations, which are block-structured, consisting of a stack of
wenzelm@26870
    10
  nodes with three main components: logical proof context, current
wenzelm@30067
    11
  facts, and open goals.  Isar/VM transitions are typed according to
wenzelm@30067
    12
  the following three different modes of operation:
wenzelm@26870
    13
wenzelm@28760
    14
  \begin{description}
wenzelm@26870
    15
wenzelm@28760
    16
  \item @{text "proof(prove)"} means that a new goal has just been
wenzelm@26870
    17
  stated that is now to be \emph{proven}; the next command may refine
wenzelm@26870
    18
  it by some proof method, and enter a sub-proof to establish the
wenzelm@26870
    19
  actual result.
wenzelm@26870
    20
wenzelm@28760
    21
  \item @{text "proof(state)"} is like a nested theory mode: the
wenzelm@26870
    22
  context may be augmented by \emph{stating} additional assumptions,
wenzelm@26870
    23
  intermediate results etc.
wenzelm@26870
    24
wenzelm@28760
    25
  \item @{text "proof(chain)"} is intermediate between @{text
wenzelm@26870
    26
  "proof(state)"} and @{text "proof(prove)"}: existing facts (i.e.\
wenzelm@26870
    27
  the contents of the special ``@{fact_ref this}'' register) have been
wenzelm@26870
    28
  just picked up in order to be used when refining the goal claimed
wenzelm@26870
    29
  next.
wenzelm@26870
    30
wenzelm@28760
    31
  \end{description}
wenzelm@26870
    32
wenzelm@30067
    33
  The proof mode indicator may be understood as an instruction to the
wenzelm@30067
    34
  writer, telling what kind of operation may be performed next.  The
wenzelm@30067
    35
  corresponding typings of proof commands restricts the shape of
wenzelm@30067
    36
  well-formed proof texts to particular command sequences.  So dynamic
wenzelm@30067
    37
  arrangements of commands eventually turn out as static texts of a
wenzelm@30067
    38
  certain structure.
wenzelm@30067
    39
wenzelm@30067
    40
  \Appref{ap:refcard} gives a simplified grammar of the (extensible)
wenzelm@30067
    41
  language emerging that way from the different types of proof
wenzelm@30067
    42
  commands.  The main ideas of the overall Isar framework are
wenzelm@30067
    43
  explained in \chref{ch:isar-framework}.
wenzelm@26870
    44
*}
wenzelm@26870
    45
wenzelm@26870
    46
wenzelm@28755
    47
section {* Proof structure *}
wenzelm@28755
    48
wenzelm@36366
    49
subsection {* Example proofs *}
wenzelm@36366
    50
wenzelm@36366
    51
text {*
wenzelm@36366
    52
  \begin{matharray}{rcl}
wenzelm@36366
    53
    @{command_def "example_proof"} & : & @{text "local_theory \<rightarrow> proof(state)"} \\
wenzelm@36366
    54
  \end{matharray}
wenzelm@36366
    55
wenzelm@36366
    56
  \begin{description}
wenzelm@36366
    57
wenzelm@36366
    58
  \item @{command "example_proof"} opens an empty proof body.  This
wenzelm@36366
    59
  allows to experiment with Isar, without producing any persistent
wenzelm@36366
    60
  result.
wenzelm@36366
    61
wenzelm@36366
    62
  Structurally, this is like a vacous @{command "lemma"} statement
wenzelm@36366
    63
  followed by ``@{command "proof"}~@{text "-"}'', which means the
wenzelm@36366
    64
  example proof may be closed by a regular @{command "qed"}, or
wenzelm@36366
    65
  discontinued by @{command "oops"}.
wenzelm@36366
    66
wenzelm@36366
    67
  \end{description}
wenzelm@36366
    68
*}
wenzelm@36366
    69
wenzelm@36366
    70
wenzelm@28755
    71
subsection {* Blocks *}
wenzelm@28755
    72
wenzelm@28755
    73
text {*
wenzelm@28755
    74
  \begin{matharray}{rcl}
wenzelm@28761
    75
    @{command_def "next"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28761
    76
    @{command_def "{"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28761
    77
    @{command_def "}"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28755
    78
  \end{matharray}
wenzelm@28755
    79
wenzelm@28755
    80
  While Isar is inherently block-structured, opening and closing
wenzelm@28755
    81
  blocks is mostly handled rather casually, with little explicit
wenzelm@28755
    82
  user-intervention.  Any local goal statement automatically opens
wenzelm@28755
    83
  \emph{two} internal blocks, which are closed again when concluding
wenzelm@28755
    84
  the sub-proof (by @{command "qed"} etc.).  Sections of different
wenzelm@28755
    85
  context within a sub-proof may be switched via @{command "next"},
wenzelm@28755
    86
  which is just a single block-close followed by block-open again.
wenzelm@28755
    87
  The effect of @{command "next"} is to reset the local proof context;
wenzelm@28755
    88
  there is no goal focus involved here!
wenzelm@28755
    89
wenzelm@28755
    90
  For slightly more advanced applications, there are explicit block
wenzelm@28755
    91
  parentheses as well.  These typically achieve a stronger forward
wenzelm@28755
    92
  style of reasoning.
wenzelm@28755
    93
wenzelm@28760
    94
  \begin{description}
wenzelm@28755
    95
wenzelm@28760
    96
  \item @{command "next"} switches to a fresh block within a
wenzelm@28755
    97
  sub-proof, resetting the local context to the initial one.
wenzelm@28755
    98
wenzelm@28760
    99
  \item @{command "{"} and @{command "}"} explicitly open and close
wenzelm@28755
   100
  blocks.  Any current facts pass through ``@{command "{"}''
wenzelm@28755
   101
  unchanged, while ``@{command "}"}'' causes any result to be
wenzelm@28755
   102
  \emph{exported} into the enclosing context.  Thus fixed variables
wenzelm@28755
   103
  are generalized, assumptions discharged, and local definitions
wenzelm@28755
   104
  unfolded (cf.\ \secref{sec:proof-context}).  There is no difference
wenzelm@28755
   105
  of @{command "assume"} and @{command "presume"} in this mode of
wenzelm@28755
   106
  forward reasoning --- in contrast to plain backward reasoning with
wenzelm@28755
   107
  the result exported at @{command "show"} time.
wenzelm@28755
   108
wenzelm@28760
   109
  \end{description}
wenzelm@28755
   110
*}
wenzelm@28755
   111
wenzelm@28755
   112
wenzelm@28755
   113
subsection {* Omitting proofs *}
wenzelm@28755
   114
wenzelm@28755
   115
text {*
wenzelm@28755
   116
  \begin{matharray}{rcl}
wenzelm@28761
   117
    @{command_def "oops"} & : & @{text "proof \<rightarrow> local_theory | theory"} \\
wenzelm@28755
   118
  \end{matharray}
wenzelm@28755
   119
wenzelm@28755
   120
  The @{command "oops"} command discontinues the current proof
wenzelm@28755
   121
  attempt, while considering the partial proof text as properly
wenzelm@28755
   122
  processed.  This is conceptually quite different from ``faking''
wenzelm@28755
   123
  actual proofs via @{command_ref "sorry"} (see
wenzelm@28755
   124
  \secref{sec:proof-steps}): @{command "oops"} does not observe the
wenzelm@28755
   125
  proof structure at all, but goes back right to the theory level.
wenzelm@28755
   126
  Furthermore, @{command "oops"} does not produce any result theorem
wenzelm@28755
   127
  --- there is no intended claim to be able to complete the proof
wenzelm@28755
   128
  anyhow.
wenzelm@28755
   129
wenzelm@28755
   130
  A typical application of @{command "oops"} is to explain Isar proofs
wenzelm@28755
   131
  \emph{within} the system itself, in conjunction with the document
wenzelm@28838
   132
  preparation tools of Isabelle described in \chref{ch:document-prep}.
wenzelm@28755
   133
  Thus partial or even wrong proof attempts can be discussed in a
wenzelm@28755
   134
  logically sound manner.  Note that the Isabelle {\LaTeX} macros can
wenzelm@28755
   135
  be easily adapted to print something like ``@{text "\<dots>"}'' instead of
wenzelm@28755
   136
  the keyword ``@{command "oops"}''.
wenzelm@28755
   137
wenzelm@28755
   138
  \medskip The @{command "oops"} command is undo-able, unlike
wenzelm@28755
   139
  @{command_ref "kill"} (see \secref{sec:history}).  The effect is to
wenzelm@28755
   140
  get back to the theory just before the opening of the proof.
wenzelm@28755
   141
*}
wenzelm@28755
   142
wenzelm@28755
   143
wenzelm@28754
   144
section {* Statements *}
wenzelm@28754
   145
wenzelm@28754
   146
subsection {* Context elements \label{sec:proof-context} *}
wenzelm@26870
   147
wenzelm@26870
   148
text {*
wenzelm@26870
   149
  \begin{matharray}{rcl}
wenzelm@28761
   150
    @{command_def "fix"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28761
   151
    @{command_def "assume"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28761
   152
    @{command_def "presume"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28761
   153
    @{command_def "def"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@26870
   154
  \end{matharray}
wenzelm@26870
   155
wenzelm@26870
   156
  The logical proof context consists of fixed variables and
wenzelm@26870
   157
  assumptions.  The former closely correspond to Skolem constants, or
wenzelm@26870
   158
  meta-level universal quantification as provided by the Isabelle/Pure
wenzelm@26870
   159
  logical framework.  Introducing some \emph{arbitrary, but fixed}
wenzelm@26870
   160
  variable via ``@{command "fix"}~@{text x}'' results in a local value
wenzelm@26870
   161
  that may be used in the subsequent proof as any other variable or
wenzelm@26870
   162
  constant.  Furthermore, any result @{text "\<turnstile> \<phi>[x]"} exported from
wenzelm@26870
   163
  the context will be universally closed wrt.\ @{text x} at the
wenzelm@26870
   164
  outermost level: @{text "\<turnstile> \<And>x. \<phi>[x]"} (this is expressed in normal
wenzelm@26870
   165
  form using Isabelle's meta-variables).
wenzelm@26870
   166
wenzelm@26870
   167
  Similarly, introducing some assumption @{text \<chi>} has two effects.
wenzelm@26870
   168
  On the one hand, a local theorem is created that may be used as a
wenzelm@26870
   169
  fact in subsequent proof steps.  On the other hand, any result
wenzelm@26870
   170
  @{text "\<chi> \<turnstile> \<phi>"} exported from the context becomes conditional wrt.\
wenzelm@26870
   171
  the assumption: @{text "\<turnstile> \<chi> \<Longrightarrow> \<phi>"}.  Thus, solving an enclosing goal
wenzelm@26870
   172
  using such a result would basically introduce a new subgoal stemming
wenzelm@26870
   173
  from the assumption.  How this situation is handled depends on the
wenzelm@26870
   174
  version of assumption command used: while @{command "assume"}
wenzelm@26870
   175
  insists on solving the subgoal by unification with some premise of
wenzelm@26870
   176
  the goal, @{command "presume"} leaves the subgoal unchanged in order
wenzelm@26870
   177
  to be proved later by the user.
wenzelm@26870
   178
wenzelm@26870
   179
  Local definitions, introduced by ``@{command "def"}~@{text "x \<equiv>
wenzelm@26870
   180
  t"}'', are achieved by combining ``@{command "fix"}~@{text x}'' with
wenzelm@26870
   181
  another version of assumption that causes any hypothetical equation
wenzelm@26870
   182
  @{text "x \<equiv> t"} to be eliminated by the reflexivity rule.  Thus,
wenzelm@26870
   183
  exporting some result @{text "x \<equiv> t \<turnstile> \<phi>[x]"} yields @{text "\<turnstile>
wenzelm@26870
   184
  \<phi>[t]"}.
wenzelm@26870
   185
wenzelm@26870
   186
  \begin{rail}
wenzelm@26870
   187
    'fix' (vars + 'and')
wenzelm@26870
   188
    ;
wenzelm@26870
   189
    ('assume' | 'presume') (props + 'and')
wenzelm@26870
   190
    ;
wenzelm@26870
   191
    'def' (def + 'and')
wenzelm@26870
   192
    ;
wenzelm@26870
   193
    def: thmdecl? \\ name ('==' | equiv) term termpat?
wenzelm@26870
   194
    ;
wenzelm@26870
   195
  \end{rail}
wenzelm@26870
   196
wenzelm@28760
   197
  \begin{description}
wenzelm@26870
   198
  
wenzelm@28760
   199
  \item @{command "fix"}~@{text x} introduces a local variable @{text
wenzelm@28760
   200
  x} that is \emph{arbitrary, but fixed.}
wenzelm@26870
   201
  
wenzelm@28760
   202
  \item @{command "assume"}~@{text "a: \<phi>"} and @{command
wenzelm@28760
   203
  "presume"}~@{text "a: \<phi>"} introduce a local fact @{text "\<phi> \<turnstile> \<phi>"} by
wenzelm@26870
   204
  assumption.  Subsequent results applied to an enclosing goal (e.g.\
wenzelm@26870
   205
  by @{command_ref "show"}) are handled as follows: @{command
wenzelm@26870
   206
  "assume"} expects to be able to unify with existing premises in the
wenzelm@26870
   207
  goal, while @{command "presume"} leaves @{text \<phi>} as new subgoals.
wenzelm@26870
   208
  
wenzelm@26870
   209
  Several lists of assumptions may be given (separated by
wenzelm@26870
   210
  @{keyword_ref "and"}; the resulting list of current facts consists
wenzelm@26870
   211
  of all of these concatenated.
wenzelm@26870
   212
  
wenzelm@28760
   213
  \item @{command "def"}~@{text "x \<equiv> t"} introduces a local
wenzelm@26870
   214
  (non-polymorphic) definition.  In results exported from the context,
wenzelm@26870
   215
  @{text x} is replaced by @{text t}.  Basically, ``@{command
wenzelm@26870
   216
  "def"}~@{text "x \<equiv> t"}'' abbreviates ``@{command "fix"}~@{text
wenzelm@26870
   217
  x}~@{command "assume"}~@{text "x \<equiv> t"}'', with the resulting
wenzelm@26870
   218
  hypothetical equation solved by reflexivity.
wenzelm@26870
   219
  
wenzelm@26870
   220
  The default name for the definitional equation is @{text x_def}.
wenzelm@26870
   221
  Several simultaneous definitions may be given at the same time.
wenzelm@26870
   222
wenzelm@28760
   223
  \end{description}
wenzelm@26870
   224
wenzelm@26870
   225
  The special name @{fact_ref prems} refers to all assumptions of the
wenzelm@26870
   226
  current context as a list of theorems.  This feature should be used
wenzelm@26870
   227
  with great care!  It is better avoided in final proof texts.
wenzelm@26870
   228
*}
wenzelm@26870
   229
wenzelm@26870
   230
wenzelm@28754
   231
subsection {* Term abbreviations \label{sec:term-abbrev} *}
wenzelm@28754
   232
wenzelm@28754
   233
text {*
wenzelm@28754
   234
  \begin{matharray}{rcl}
wenzelm@28761
   235
    @{command_def "let"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28754
   236
    @{keyword_def "is"} & : & syntax \\
wenzelm@28754
   237
  \end{matharray}
wenzelm@28754
   238
wenzelm@28754
   239
  Abbreviations may be either bound by explicit @{command
wenzelm@28754
   240
  "let"}~@{text "p \<equiv> t"} statements, or by annotating assumptions or
wenzelm@28754
   241
  goal statements with a list of patterns ``@{text "(\<IS> p\<^sub>1 \<dots>
wenzelm@28754
   242
  p\<^sub>n)"}''.  In both cases, higher-order matching is invoked to
wenzelm@28754
   243
  bind extra-logical term variables, which may be either named
wenzelm@28754
   244
  schematic variables of the form @{text ?x}, or nameless dummies
wenzelm@28754
   245
  ``@{variable _}'' (underscore). Note that in the @{command "let"}
wenzelm@28754
   246
  form the patterns occur on the left-hand side, while the @{keyword
wenzelm@28754
   247
  "is"} patterns are in postfix position.
wenzelm@28754
   248
wenzelm@28754
   249
  Polymorphism of term bindings is handled in Hindley-Milner style,
wenzelm@28754
   250
  similar to ML.  Type variables referring to local assumptions or
wenzelm@28754
   251
  open goal statements are \emph{fixed}, while those of finished
wenzelm@28754
   252
  results or bound by @{command "let"} may occur in \emph{arbitrary}
wenzelm@28754
   253
  instances later.  Even though actual polymorphism should be rarely
wenzelm@28754
   254
  used in practice, this mechanism is essential to achieve proper
wenzelm@28754
   255
  incremental type-inference, as the user proceeds to build up the
wenzelm@28754
   256
  Isar proof text from left to right.
wenzelm@28754
   257
wenzelm@28754
   258
  \medskip Term abbreviations are quite different from local
wenzelm@28754
   259
  definitions as introduced via @{command "def"} (see
wenzelm@28754
   260
  \secref{sec:proof-context}).  The latter are visible within the
wenzelm@28754
   261
  logic as actual equations, while abbreviations disappear during the
wenzelm@28754
   262
  input process just after type checking.  Also note that @{command
wenzelm@28754
   263
  "def"} does not support polymorphism.
wenzelm@28754
   264
wenzelm@28754
   265
  \begin{rail}
wenzelm@28754
   266
    'let' ((term + 'and') '=' term + 'and')
wenzelm@28754
   267
    ;  
wenzelm@28754
   268
  \end{rail}
wenzelm@28754
   269
wenzelm@28754
   270
  The syntax of @{keyword "is"} patterns follows \railnonterm{termpat}
wenzelm@28754
   271
  or \railnonterm{proppat} (see \secref{sec:term-decls}).
wenzelm@28754
   272
wenzelm@28760
   273
  \begin{description}
wenzelm@28754
   274
wenzelm@28760
   275
  \item @{command "let"}~@{text "p\<^sub>1 = t\<^sub>1 \<AND> \<dots> p\<^sub>n = t\<^sub>n"} binds any
wenzelm@28760
   276
  text variables in patterns @{text "p\<^sub>1, \<dots>, p\<^sub>n"} by simultaneous
wenzelm@28760
   277
  higher-order matching against terms @{text "t\<^sub>1, \<dots>, t\<^sub>n"}.
wenzelm@28754
   278
wenzelm@28760
   279
  \item @{text "(\<IS> p\<^sub>1 \<dots> p\<^sub>n)"} resembles @{command "let"}, but
wenzelm@28760
   280
  matches @{text "p\<^sub>1, \<dots>, p\<^sub>n"} against the preceding statement.  Also
wenzelm@28760
   281
  note that @{keyword "is"} is not a separate command, but part of
wenzelm@28760
   282
  others (such as @{command "assume"}, @{command "have"} etc.).
wenzelm@28754
   283
wenzelm@28760
   284
  \end{description}
wenzelm@28754
   285
wenzelm@28754
   286
  Some \emph{implicit} term abbreviations\index{term abbreviations}
wenzelm@28754
   287
  for goals and facts are available as well.  For any open goal,
wenzelm@28754
   288
  @{variable_ref thesis} refers to its object-level statement,
wenzelm@28754
   289
  abstracted over any meta-level parameters (if present).  Likewise,
wenzelm@28754
   290
  @{variable_ref this} is bound for fact statements resulting from
wenzelm@28754
   291
  assumptions or finished goals.  In case @{variable this} refers to
wenzelm@28754
   292
  an object-logic statement that is an application @{text "f t"}, then
wenzelm@28754
   293
  @{text t} is bound to the special text variable ``@{variable "\<dots>"}''
wenzelm@28754
   294
  (three dots).  The canonical application of this convenience are
wenzelm@28754
   295
  calculational proofs (see \secref{sec:calculation}).
wenzelm@28754
   296
*}
wenzelm@28754
   297
wenzelm@28754
   298
wenzelm@28754
   299
subsection {* Facts and forward chaining *}
wenzelm@26870
   300
wenzelm@26870
   301
text {*
wenzelm@26870
   302
  \begin{matharray}{rcl}
wenzelm@28761
   303
    @{command_def "note"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28761
   304
    @{command_def "then"} & : & @{text "proof(state) \<rightarrow> proof(chain)"} \\
wenzelm@28761
   305
    @{command_def "from"} & : & @{text "proof(state) \<rightarrow> proof(chain)"} \\
wenzelm@28761
   306
    @{command_def "with"} & : & @{text "proof(state) \<rightarrow> proof(chain)"} \\
wenzelm@28761
   307
    @{command_def "using"} & : & @{text "proof(prove) \<rightarrow> proof(prove)"} \\
wenzelm@28761
   308
    @{command_def "unfolding"} & : & @{text "proof(prove) \<rightarrow> proof(prove)"} \\
wenzelm@26870
   309
  \end{matharray}
wenzelm@26870
   310
wenzelm@26870
   311
  New facts are established either by assumption or proof of local
wenzelm@26870
   312
  statements.  Any fact will usually be involved in further proofs,
wenzelm@26870
   313
  either as explicit arguments of proof methods, or when forward
wenzelm@26870
   314
  chaining towards the next goal via @{command "then"} (and variants);
wenzelm@26870
   315
  @{command "from"} and @{command "with"} are composite forms
wenzelm@26870
   316
  involving @{command "note"}.  The @{command "using"} elements
wenzelm@26870
   317
  augments the collection of used facts \emph{after} a goal has been
wenzelm@26870
   318
  stated.  Note that the special theorem name @{fact_ref this} refers
wenzelm@26870
   319
  to the most recently established facts, but only \emph{before}
wenzelm@26870
   320
  issuing a follow-up claim.
wenzelm@26870
   321
wenzelm@26870
   322
  \begin{rail}
wenzelm@26870
   323
    'note' (thmdef? thmrefs + 'and')
wenzelm@26870
   324
    ;
wenzelm@26870
   325
    ('from' | 'with' | 'using' | 'unfolding') (thmrefs + 'and')
wenzelm@26870
   326
    ;
wenzelm@26870
   327
  \end{rail}
wenzelm@26870
   328
wenzelm@28760
   329
  \begin{description}
wenzelm@26870
   330
wenzelm@28760
   331
  \item @{command "note"}~@{text "a = b\<^sub>1 \<dots> b\<^sub>n"} recalls existing facts
wenzelm@28760
   332
  @{text "b\<^sub>1, \<dots>, b\<^sub>n"}, binding the result as @{text a}.  Note that
wenzelm@28760
   333
  attributes may be involved as well, both on the left and right hand
wenzelm@28760
   334
  sides.
wenzelm@26870
   335
wenzelm@28760
   336
  \item @{command "then"} indicates forward chaining by the current
wenzelm@26870
   337
  facts in order to establish the goal to be claimed next.  The
wenzelm@26870
   338
  initial proof method invoked to refine that will be offered the
wenzelm@26870
   339
  facts to do ``anything appropriate'' (see also
wenzelm@26870
   340
  \secref{sec:proof-steps}).  For example, method @{method_ref rule}
wenzelm@26870
   341
  (see \secref{sec:pure-meth-att}) would typically do an elimination
wenzelm@26870
   342
  rather than an introduction.  Automatic methods usually insert the
wenzelm@26870
   343
  facts into the goal state before operation.  This provides a simple
wenzelm@26870
   344
  scheme to control relevance of facts in automated proof search.
wenzelm@26870
   345
  
wenzelm@28760
   346
  \item @{command "from"}~@{text b} abbreviates ``@{command
wenzelm@26870
   347
  "note"}~@{text b}~@{command "then"}''; thus @{command "then"} is
wenzelm@26870
   348
  equivalent to ``@{command "from"}~@{text this}''.
wenzelm@26870
   349
  
wenzelm@28760
   350
  \item @{command "with"}~@{text "b\<^sub>1 \<dots> b\<^sub>n"} abbreviates ``@{command
wenzelm@28760
   351
  "from"}~@{text "b\<^sub>1 \<dots> b\<^sub>n \<AND> this"}''; thus the forward chaining
wenzelm@28760
   352
  is from earlier facts together with the current ones.
wenzelm@26870
   353
  
wenzelm@28760
   354
  \item @{command "using"}~@{text "b\<^sub>1 \<dots> b\<^sub>n"} augments the facts being
wenzelm@28760
   355
  currently indicated for use by a subsequent refinement step (such as
wenzelm@28760
   356
  @{command_ref "apply"} or @{command_ref "proof"}).
wenzelm@26870
   357
  
wenzelm@28760
   358
  \item @{command "unfolding"}~@{text "b\<^sub>1 \<dots> b\<^sub>n"} is structurally
wenzelm@28760
   359
  similar to @{command "using"}, but unfolds definitional equations
wenzelm@28760
   360
  @{text "b\<^sub>1, \<dots> b\<^sub>n"} throughout the goal state and facts.
wenzelm@26870
   361
wenzelm@28760
   362
  \end{description}
wenzelm@26870
   363
wenzelm@26870
   364
  Forward chaining with an empty list of theorems is the same as not
wenzelm@26870
   365
  chaining at all.  Thus ``@{command "from"}~@{text nothing}'' has no
wenzelm@26870
   366
  effect apart from entering @{text "prove(chain)"} mode, since
wenzelm@26870
   367
  @{fact_ref nothing} is bound to the empty list of theorems.
wenzelm@26870
   368
wenzelm@26870
   369
  Basic proof methods (such as @{method_ref rule}) expect multiple
wenzelm@26870
   370
  facts to be given in their proper order, corresponding to a prefix
wenzelm@26870
   371
  of the premises of the rule involved.  Note that positions may be
wenzelm@26870
   372
  easily skipped using something like @{command "from"}~@{text "_
wenzelm@26870
   373
  \<AND> a \<AND> b"}, for example.  This involves the trivial rule
wenzelm@26870
   374
  @{text "PROP \<psi> \<Longrightarrow> PROP \<psi>"}, which is bound in Isabelle/Pure as
wenzelm@26870
   375
  ``@{fact_ref "_"}'' (underscore).
wenzelm@26870
   376
wenzelm@26870
   377
  Automated methods (such as @{method simp} or @{method auto}) just
wenzelm@26870
   378
  insert any given facts before their usual operation.  Depending on
wenzelm@26870
   379
  the kind of procedure involved, the order of facts is less
wenzelm@26870
   380
  significant here.
wenzelm@26870
   381
*}
wenzelm@26870
   382
wenzelm@26870
   383
wenzelm@28754
   384
subsection {* Goals \label{sec:goals} *}
wenzelm@26870
   385
wenzelm@26870
   386
text {*
wenzelm@26870
   387
  \begin{matharray}{rcl}
wenzelm@28761
   388
    @{command_def "lemma"} & : & @{text "local_theory \<rightarrow> proof(prove)"} \\
wenzelm@28761
   389
    @{command_def "theorem"} & : & @{text "local_theory \<rightarrow> proof(prove)"} \\
wenzelm@28761
   390
    @{command_def "corollary"} & : & @{text "local_theory \<rightarrow> proof(prove)"} \\
wenzelm@36320
   391
    @{command_def "schematic_lemma"} & : & @{text "local_theory \<rightarrow> proof(prove)"} \\
wenzelm@36320
   392
    @{command_def "schematic_theorem"} & : & @{text "local_theory \<rightarrow> proof(prove)"} \\
wenzelm@36320
   393
    @{command_def "schematic_corollary"} & : & @{text "local_theory \<rightarrow> proof(prove)"} \\
wenzelm@28761
   394
    @{command_def "have"} & : & @{text "proof(state) | proof(chain) \<rightarrow> proof(prove)"} \\
wenzelm@28761
   395
    @{command_def "show"} & : & @{text "proof(state) | proof(chain) \<rightarrow> proof(prove)"} \\
wenzelm@28761
   396
    @{command_def "hence"} & : & @{text "proof(state) \<rightarrow> proof(prove)"} \\
wenzelm@28761
   397
    @{command_def "thus"} & : & @{text "proof(state) \<rightarrow> proof(prove)"} \\
wenzelm@28761
   398
    @{command_def "print_statement"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
wenzelm@26870
   399
  \end{matharray}
wenzelm@26870
   400
wenzelm@26870
   401
  From a theory context, proof mode is entered by an initial goal
wenzelm@26870
   402
  command such as @{command "lemma"}, @{command "theorem"}, or
wenzelm@26870
   403
  @{command "corollary"}.  Within a proof, new claims may be
wenzelm@26870
   404
  introduced locally as well; four variants are available here to
wenzelm@26870
   405
  indicate whether forward chaining of facts should be performed
wenzelm@26870
   406
  initially (via @{command_ref "then"}), and whether the final result
wenzelm@26870
   407
  is meant to solve some pending goal.
wenzelm@26870
   408
wenzelm@26870
   409
  Goals may consist of multiple statements, resulting in a list of
wenzelm@26870
   410
  facts eventually.  A pending multi-goal is internally represented as
wenzelm@28856
   411
  a meta-level conjunction (@{text "&&&"}), which is usually
wenzelm@26870
   412
  split into the corresponding number of sub-goals prior to an initial
wenzelm@26870
   413
  method application, via @{command_ref "proof"}
wenzelm@26870
   414
  (\secref{sec:proof-steps}) or @{command_ref "apply"}
wenzelm@26870
   415
  (\secref{sec:tactic-commands}).  The @{method_ref induct} method
wenzelm@26870
   416
  covered in \secref{sec:cases-induct} acts on multiple claims
wenzelm@26870
   417
  simultaneously.
wenzelm@26870
   418
wenzelm@26870
   419
  Claims at the theory level may be either in short or long form.  A
wenzelm@26870
   420
  short goal merely consists of several simultaneous propositions
wenzelm@26870
   421
  (often just one).  A long goal includes an explicit context
wenzelm@26870
   422
  specification for the subsequent conclusion, involving local
wenzelm@26870
   423
  parameters and assumptions.  Here the role of each part of the
wenzelm@26870
   424
  statement is explicitly marked by separate keywords (see also
wenzelm@26870
   425
  \secref{sec:locale}); the local assumptions being introduced here
wenzelm@26870
   426
  are available as @{fact_ref assms} in the proof.  Moreover, there
wenzelm@26870
   427
  are two kinds of conclusions: @{element_def "shows"} states several
wenzelm@26870
   428
  simultaneous propositions (essentially a big conjunction), while
wenzelm@26870
   429
  @{element_def "obtains"} claims several simultaneous simultaneous
wenzelm@26870
   430
  contexts of (essentially a big disjunction of eliminated parameters
wenzelm@26870
   431
  and assumptions, cf.\ \secref{sec:obtain}).
wenzelm@26870
   432
wenzelm@26870
   433
  \begin{rail}
wenzelm@36320
   434
    ('lemma' | 'theorem' | 'corollary' |
wenzelm@36320
   435
     'schematic\_lemma' | 'schematic\_theorem' | 'schematic\_corollary') target? (goal | longgoal)
wenzelm@26870
   436
    ;
wenzelm@26870
   437
    ('have' | 'show' | 'hence' | 'thus') goal
wenzelm@26870
   438
    ;
wenzelm@26870
   439
    'print\_statement' modes? thmrefs
wenzelm@26870
   440
    ;
wenzelm@26870
   441
  
wenzelm@26870
   442
    goal: (props + 'and')
wenzelm@26870
   443
    ;
wenzelm@26870
   444
    longgoal: thmdecl? (contextelem *) conclusion
wenzelm@26870
   445
    ;
wenzelm@26870
   446
    conclusion: 'shows' goal | 'obtains' (parname? case + '|')
wenzelm@26870
   447
    ;
wenzelm@26870
   448
    case: (vars + 'and') 'where' (props + 'and')
wenzelm@26870
   449
    ;
wenzelm@26870
   450
  \end{rail}
wenzelm@26870
   451
wenzelm@28760
   452
  \begin{description}
wenzelm@26870
   453
  
wenzelm@28760
   454
  \item @{command "lemma"}~@{text "a: \<phi>"} enters proof mode with
wenzelm@26870
   455
  @{text \<phi>} as main goal, eventually resulting in some fact @{text "\<turnstile>
wenzelm@26870
   456
  \<phi>"} to be put back into the target context.  An additional
wenzelm@26870
   457
  \railnonterm{context} specification may build up an initial proof
wenzelm@26870
   458
  context for the subsequent claim; this includes local definitions
wenzelm@26870
   459
  and syntax as well, see the definition of @{syntax contextelem} in
wenzelm@26870
   460
  \secref{sec:locale}.
wenzelm@26870
   461
  
wenzelm@28760
   462
  \item @{command "theorem"}~@{text "a: \<phi>"} and @{command
wenzelm@28760
   463
  "corollary"}~@{text "a: \<phi>"} are essentially the same as @{command
wenzelm@26870
   464
  "lemma"}~@{text "a: \<phi>"}, but the facts are internally marked as
wenzelm@26870
   465
  being of a different kind.  This discrimination acts like a formal
wenzelm@26870
   466
  comment.
wenzelm@36320
   467
wenzelm@36320
   468
  \item @{command "schematic_lemma"}, @{command "schematic_theorem"},
wenzelm@36320
   469
  @{command "schematic_corollary"} are similar to @{command "lemma"},
wenzelm@36320
   470
  @{command "theorem"}, @{command "corollary"}, respectively but allow
wenzelm@36320
   471
  the statement to contain unbound schematic variables.
wenzelm@36320
   472
wenzelm@36320
   473
  Under normal circumstances, an Isar proof text needs to specify
wenzelm@36320
   474
  claims explicitly.  Schematic goals are more like goals in Prolog,
wenzelm@36320
   475
  where certain results are synthesized in the course of reasoning.
wenzelm@36320
   476
  With schematic statements, the inherent compositionality of Isar
wenzelm@36320
   477
  proofs is lost, which also impacts performance, because proof
wenzelm@36320
   478
  checking is forced into sequential mode.
wenzelm@26870
   479
  
wenzelm@28760
   480
  \item @{command "have"}~@{text "a: \<phi>"} claims a local goal,
wenzelm@26870
   481
  eventually resulting in a fact within the current logical context.
wenzelm@26870
   482
  This operation is completely independent of any pending sub-goals of
wenzelm@26870
   483
  an enclosing goal statements, so @{command "have"} may be freely
wenzelm@26870
   484
  used for experimental exploration of potential results within a
wenzelm@26870
   485
  proof body.
wenzelm@26870
   486
  
wenzelm@28760
   487
  \item @{command "show"}~@{text "a: \<phi>"} is like @{command
wenzelm@26870
   488
  "have"}~@{text "a: \<phi>"} plus a second stage to refine some pending
wenzelm@26870
   489
  sub-goal for each one of the finished result, after having been
wenzelm@26870
   490
  exported into the corresponding context (at the head of the
wenzelm@26870
   491
  sub-proof of this @{command "show"} command).
wenzelm@26870
   492
  
wenzelm@26870
   493
  To accommodate interactive debugging, resulting rules are printed
wenzelm@26870
   494
  before being applied internally.  Even more, interactive execution
wenzelm@26870
   495
  of @{command "show"} predicts potential failure and displays the
wenzelm@26870
   496
  resulting error as a warning beforehand.  Watch out for the
wenzelm@26870
   497
  following message:
wenzelm@26870
   498
wenzelm@26870
   499
  %FIXME proper antiquitation
wenzelm@26870
   500
  \begin{ttbox}
wenzelm@26870
   501
  Problem! Local statement will fail to solve any pending goal
wenzelm@26870
   502
  \end{ttbox}
wenzelm@26870
   503
  
wenzelm@28760
   504
  \item @{command "hence"} abbreviates ``@{command "then"}~@{command
wenzelm@26870
   505
  "have"}'', i.e.\ claims a local goal to be proven by forward
wenzelm@26870
   506
  chaining the current facts.  Note that @{command "hence"} is also
wenzelm@26870
   507
  equivalent to ``@{command "from"}~@{text this}~@{command "have"}''.
wenzelm@26870
   508
  
wenzelm@28760
   509
  \item @{command "thus"} abbreviates ``@{command "then"}~@{command
wenzelm@26870
   510
  "show"}''.  Note that @{command "thus"} is also equivalent to
wenzelm@26870
   511
  ``@{command "from"}~@{text this}~@{command "show"}''.
wenzelm@26870
   512
  
wenzelm@28760
   513
  \item @{command "print_statement"}~@{text a} prints facts from the
wenzelm@26870
   514
  current theory or proof context in long statement form, according to
wenzelm@26870
   515
  the syntax for @{command "lemma"} given above.
wenzelm@26870
   516
wenzelm@28760
   517
  \end{description}
wenzelm@26870
   518
wenzelm@26870
   519
  Any goal statement causes some term abbreviations (such as
wenzelm@26870
   520
  @{variable_ref "?thesis"}) to be bound automatically, see also
wenzelm@26922
   521
  \secref{sec:term-abbrev}.
wenzelm@26870
   522
wenzelm@26870
   523
  The optional case names of @{element_ref "obtains"} have a twofold
wenzelm@26870
   524
  meaning: (1) during the of this claim they refer to the the local
wenzelm@26870
   525
  context introductions, (2) the resulting rule is annotated
wenzelm@26870
   526
  accordingly to support symbolic case splits when used with the
wenzelm@27116
   527
  @{method_ref cases} method (cf.\ \secref{sec:cases-induct}).
wenzelm@26870
   528
*}
wenzelm@26870
   529
wenzelm@26870
   530
wenzelm@28754
   531
section {* Refinement steps *}
wenzelm@28754
   532
wenzelm@28754
   533
subsection {* Proof method expressions \label{sec:proof-meth} *}
wenzelm@28754
   534
wenzelm@28754
   535
text {*
wenzelm@28754
   536
  Proof methods are either basic ones, or expressions composed of
wenzelm@28754
   537
  methods via ``@{verbatim ","}'' (sequential composition),
wenzelm@28754
   538
  ``@{verbatim "|"}'' (alternative choices), ``@{verbatim "?"}'' 
wenzelm@28754
   539
  (try), ``@{verbatim "+"}'' (repeat at least once), ``@{verbatim
wenzelm@28754
   540
  "["}@{text n}@{verbatim "]"}'' (restriction to first @{text n}
wenzelm@28754
   541
  sub-goals, with default @{text "n = 1"}).  In practice, proof
wenzelm@28754
   542
  methods are usually just a comma separated list of
wenzelm@28754
   543
  \railqtok{nameref}~\railnonterm{args} specifications.  Note that
wenzelm@28754
   544
  parentheses may be dropped for single method specifications (with no
wenzelm@28754
   545
  arguments).
wenzelm@28754
   546
wenzelm@28754
   547
  \indexouternonterm{method}
wenzelm@28754
   548
  \begin{rail}
wenzelm@28754
   549
    method: (nameref | '(' methods ')') (() | '?' | '+' | '[' nat? ']')
wenzelm@28754
   550
    ;
wenzelm@28754
   551
    methods: (nameref args | method) + (',' | '|')
wenzelm@28754
   552
    ;
wenzelm@28754
   553
  \end{rail}
wenzelm@28754
   554
wenzelm@28754
   555
  Proper Isar proof methods do \emph{not} admit arbitrary goal
wenzelm@28754
   556
  addressing, but refer either to the first sub-goal or all sub-goals
wenzelm@28754
   557
  uniformly.  The goal restriction operator ``@{text "[n]"}''
wenzelm@28754
   558
  evaluates a method expression within a sandbox consisting of the
wenzelm@28754
   559
  first @{text n} sub-goals (which need to exist).  For example, the
wenzelm@28754
   560
  method ``@{text "simp_all[3]"}'' simplifies the first three
wenzelm@28754
   561
  sub-goals, while ``@{text "(rule foo, simp_all)[]"}'' simplifies all
wenzelm@28754
   562
  new goals that emerge from applying rule @{text "foo"} to the
wenzelm@28754
   563
  originally first one.
wenzelm@28754
   564
wenzelm@28754
   565
  Improper methods, notably tactic emulations, offer a separate
wenzelm@28754
   566
  low-level goal addressing scheme as explicit argument to the
wenzelm@28754
   567
  individual tactic being involved.  Here ``@{text "[!]"}'' refers to
wenzelm@28754
   568
  all goals, and ``@{text "[n-]"}'' to all goals starting from @{text
wenzelm@28754
   569
  "n"}.
wenzelm@28754
   570
wenzelm@28754
   571
  \indexouternonterm{goalspec}
wenzelm@28754
   572
  \begin{rail}
wenzelm@28754
   573
    goalspec: '[' (nat '-' nat | nat '-' | nat | '!' ) ']'
wenzelm@28754
   574
    ;
wenzelm@28754
   575
  \end{rail}
wenzelm@28754
   576
*}
wenzelm@28754
   577
wenzelm@28754
   578
wenzelm@28754
   579
subsection {* Initial and terminal proof steps \label{sec:proof-steps} *}
wenzelm@26870
   580
wenzelm@26870
   581
text {*
wenzelm@26870
   582
  \begin{matharray}{rcl}
wenzelm@28761
   583
    @{command_def "proof"} & : & @{text "proof(prove) \<rightarrow> proof(state)"} \\
wenzelm@28761
   584
    @{command_def "qed"} & : & @{text "proof(state) \<rightarrow> proof(state) | local_theory | theory"} \\
wenzelm@28761
   585
    @{command_def "by"} & : & @{text "proof(prove) \<rightarrow> proof(state) | local_theory | theory"} \\
wenzelm@28761
   586
    @{command_def ".."} & : & @{text "proof(prove) \<rightarrow> proof(state) | local_theory | theory"} \\
wenzelm@28761
   587
    @{command_def "."} & : & @{text "proof(prove) \<rightarrow> proof(state) | local_theory | theory"} \\
wenzelm@28761
   588
    @{command_def "sorry"} & : & @{text "proof(prove) \<rightarrow> proof(state) | local_theory | theory"} \\
wenzelm@26870
   589
  \end{matharray}
wenzelm@26870
   590
wenzelm@26870
   591
  Arbitrary goal refinement via tactics is considered harmful.
wenzelm@26870
   592
  Structured proof composition in Isar admits proof methods to be
wenzelm@26870
   593
  invoked in two places only.
wenzelm@26870
   594
wenzelm@26870
   595
  \begin{enumerate}
wenzelm@26870
   596
wenzelm@26870
   597
  \item An \emph{initial} refinement step @{command_ref
wenzelm@26870
   598
  "proof"}~@{text "m\<^sub>1"} reduces a newly stated goal to a number
wenzelm@26870
   599
  of sub-goals that are to be solved later.  Facts are passed to
wenzelm@26870
   600
  @{text "m\<^sub>1"} for forward chaining, if so indicated by @{text
wenzelm@26870
   601
  "proof(chain)"} mode.
wenzelm@26870
   602
  
wenzelm@26870
   603
  \item A \emph{terminal} conclusion step @{command_ref "qed"}~@{text
wenzelm@26870
   604
  "m\<^sub>2"} is intended to solve remaining goals.  No facts are
wenzelm@26870
   605
  passed to @{text "m\<^sub>2"}.
wenzelm@26870
   606
wenzelm@26870
   607
  \end{enumerate}
wenzelm@26870
   608
wenzelm@26870
   609
  The only other (proper) way to affect pending goals in a proof body
wenzelm@26870
   610
  is by @{command_ref "show"}, which involves an explicit statement of
wenzelm@26870
   611
  what is to be solved eventually.  Thus we avoid the fundamental
wenzelm@26870
   612
  problem of unstructured tactic scripts that consist of numerous
wenzelm@26870
   613
  consecutive goal transformations, with invisible effects.
wenzelm@26870
   614
wenzelm@26870
   615
  \medskip As a general rule of thumb for good proof style, initial
wenzelm@26870
   616
  proof methods should either solve the goal completely, or constitute
wenzelm@26870
   617
  some well-understood reduction to new sub-goals.  Arbitrary
wenzelm@26870
   618
  automatic proof tools that are prone leave a large number of badly
wenzelm@26870
   619
  structured sub-goals are no help in continuing the proof document in
wenzelm@26870
   620
  an intelligible manner.
wenzelm@26870
   621
wenzelm@26870
   622
  Unless given explicitly by the user, the default initial method is
wenzelm@26870
   623
  ``@{method_ref rule}'', which applies a single standard elimination
wenzelm@26870
   624
  or introduction rule according to the topmost symbol involved.
wenzelm@26870
   625
  There is no separate default terminal method.  Any remaining goals
wenzelm@26870
   626
  are always solved by assumption in the very last step.
wenzelm@26870
   627
wenzelm@26870
   628
  \begin{rail}
wenzelm@26870
   629
    'proof' method?
wenzelm@26870
   630
    ;
wenzelm@26870
   631
    'qed' method?
wenzelm@26870
   632
    ;
wenzelm@26870
   633
    'by' method method?
wenzelm@26870
   634
    ;
wenzelm@26870
   635
    ('.' | '..' | 'sorry')
wenzelm@26870
   636
    ;
wenzelm@26870
   637
  \end{rail}
wenzelm@26870
   638
wenzelm@28760
   639
  \begin{description}
wenzelm@26870
   640
  
wenzelm@28760
   641
  \item @{command "proof"}~@{text "m\<^sub>1"} refines the goal by proof
wenzelm@28760
   642
  method @{text "m\<^sub>1"}; facts for forward chaining are passed if so
wenzelm@28760
   643
  indicated by @{text "proof(chain)"} mode.
wenzelm@26870
   644
  
wenzelm@28760
   645
  \item @{command "qed"}~@{text "m\<^sub>2"} refines any remaining goals by
wenzelm@28760
   646
  proof method @{text "m\<^sub>2"} and concludes the sub-proof by assumption.
wenzelm@28760
   647
  If the goal had been @{text "show"} (or @{text "thus"}), some
wenzelm@28760
   648
  pending sub-goal is solved as well by the rule resulting from the
wenzelm@28760
   649
  result \emph{exported} into the enclosing goal context.  Thus @{text
wenzelm@28760
   650
  "qed"} may fail for two reasons: either @{text "m\<^sub>2"} fails, or the
wenzelm@28760
   651
  resulting rule does not fit to any pending goal\footnote{This
wenzelm@28760
   652
  includes any additional ``strong'' assumptions as introduced by
wenzelm@28760
   653
  @{command "assume"}.} of the enclosing context.  Debugging such a
wenzelm@28760
   654
  situation might involve temporarily changing @{command "show"} into
wenzelm@28760
   655
  @{command "have"}, or weakening the local context by replacing
wenzelm@28760
   656
  occurrences of @{command "assume"} by @{command "presume"}.
wenzelm@26870
   657
  
wenzelm@28760
   658
  \item @{command "by"}~@{text "m\<^sub>1 m\<^sub>2"} is a \emph{terminal
wenzelm@28760
   659
  proof}\index{proof!terminal}; it abbreviates @{command
wenzelm@28760
   660
  "proof"}~@{text "m\<^sub>1"}~@{text "qed"}~@{text "m\<^sub>2"}, but with
wenzelm@28760
   661
  backtracking across both methods.  Debugging an unsuccessful
wenzelm@28760
   662
  @{command "by"}~@{text "m\<^sub>1 m\<^sub>2"} command can be done by expanding its
wenzelm@28760
   663
  definition; in many cases @{command "proof"}~@{text "m\<^sub>1"} (or even
wenzelm@28760
   664
  @{text "apply"}~@{text "m\<^sub>1"}) is already sufficient to see the
wenzelm@26870
   665
  problem.
wenzelm@26870
   666
wenzelm@28760
   667
  \item ``@{command ".."}'' is a \emph{default
wenzelm@26870
   668
  proof}\index{proof!default}; it abbreviates @{command "by"}~@{text
wenzelm@26870
   669
  "rule"}.
wenzelm@26870
   670
wenzelm@28760
   671
  \item ``@{command "."}'' is a \emph{trivial
wenzelm@26870
   672
  proof}\index{proof!trivial}; it abbreviates @{command "by"}~@{text
wenzelm@26870
   673
  "this"}.
wenzelm@26870
   674
  
wenzelm@28760
   675
  \item @{command "sorry"} is a \emph{fake proof}\index{proof!fake}
wenzelm@26870
   676
  pretending to solve the pending claim without further ado.  This
wenzelm@26870
   677
  only works in interactive development, or if the @{ML
wenzelm@26870
   678
  quick_and_dirty} flag is enabled (in ML).  Facts emerging from fake
wenzelm@26870
   679
  proofs are not the real thing.  Internally, each theorem container
wenzelm@26870
   680
  is tainted by an oracle invocation, which is indicated as ``@{text
wenzelm@26870
   681
  "[!]"}'' in the printed result.
wenzelm@26870
   682
  
wenzelm@26870
   683
  The most important application of @{command "sorry"} is to support
wenzelm@26870
   684
  experimentation and top-down proof development.
wenzelm@26870
   685
wenzelm@28760
   686
  \end{description}
wenzelm@26870
   687
*}
wenzelm@26870
   688
wenzelm@26870
   689
wenzelm@28754
   690
subsection {* Fundamental methods and attributes \label{sec:pure-meth-att} *}
wenzelm@26870
   691
wenzelm@26870
   692
text {*
wenzelm@26870
   693
  The following proof methods and attributes refer to basic logical
wenzelm@26870
   694
  operations of Isar.  Further methods and attributes are provided by
wenzelm@26870
   695
  several generic and object-logic specific tools and packages (see
wenzelm@26870
   696
  \chref{ch:gen-tools} and \chref{ch:hol}).
wenzelm@26870
   697
wenzelm@26870
   698
  \begin{matharray}{rcl}
wenzelm@28761
   699
    @{method_def "-"} & : & @{text method} \\
wenzelm@28761
   700
    @{method_def "fact"} & : & @{text method} \\
wenzelm@28761
   701
    @{method_def "assumption"} & : & @{text method} \\
wenzelm@28761
   702
    @{method_def "this"} & : & @{text method} \\
wenzelm@28761
   703
    @{method_def "rule"} & : & @{text method} \\
wenzelm@28761
   704
    @{attribute_def (Pure) "intro"} & : & @{text attribute} \\
wenzelm@28761
   705
    @{attribute_def (Pure) "elim"} & : & @{text attribute} \\
wenzelm@28761
   706
    @{attribute_def (Pure) "dest"} & : & @{text attribute} \\
wenzelm@28761
   707
    @{attribute_def "rule"} & : & @{text attribute} \\[0.5ex]
wenzelm@28761
   708
    @{attribute_def "OF"} & : & @{text attribute} \\
wenzelm@28761
   709
    @{attribute_def "of"} & : & @{text attribute} \\
wenzelm@28761
   710
    @{attribute_def "where"} & : & @{text attribute} \\
wenzelm@26870
   711
  \end{matharray}
wenzelm@26870
   712
wenzelm@26870
   713
  \begin{rail}
wenzelm@26870
   714
    'fact' thmrefs?
wenzelm@26870
   715
    ;
wenzelm@26870
   716
    'rule' thmrefs?
wenzelm@26870
   717
    ;
wenzelm@26870
   718
    rulemod: ('intro' | 'elim' | 'dest') ((('!' | () | '?') nat?) | 'del') ':' thmrefs
wenzelm@26870
   719
    ;
wenzelm@26870
   720
    ('intro' | 'elim' | 'dest') ('!' | () | '?') nat?
wenzelm@26870
   721
    ;
wenzelm@26870
   722
    'rule' 'del'
wenzelm@26870
   723
    ;
wenzelm@26870
   724
    'OF' thmrefs
wenzelm@26870
   725
    ;
wenzelm@26870
   726
    'of' insts ('concl' ':' insts)?
wenzelm@26870
   727
    ;
wenzelm@26870
   728
    'where' ((name | var | typefree | typevar) '=' (type | term) * 'and')
wenzelm@26870
   729
    ;
wenzelm@26870
   730
  \end{rail}
wenzelm@26870
   731
wenzelm@28760
   732
  \begin{description}
wenzelm@26870
   733
  
wenzelm@28760
   734
  \item ``@{method "-"}'' (minus) does nothing but insert the forward
wenzelm@28760
   735
  chaining facts as premises into the goal.  Note that command
wenzelm@26870
   736
  @{command_ref "proof"} without any method actually performs a single
wenzelm@26870
   737
  reduction step using the @{method_ref rule} method; thus a plain
wenzelm@26870
   738
  \emph{do-nothing} proof step would be ``@{command "proof"}~@{text
wenzelm@26870
   739
  "-"}'' rather than @{command "proof"} alone.
wenzelm@26870
   740
  
wenzelm@28760
   741
  \item @{method "fact"}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} composes some fact from
wenzelm@28760
   742
  @{text "a\<^sub>1, \<dots>, a\<^sub>n"} (or implicitly from the current proof context)
wenzelm@28760
   743
  modulo unification of schematic type and term variables.  The rule
wenzelm@28760
   744
  structure is not taken into account, i.e.\ meta-level implication is
wenzelm@28760
   745
  considered atomic.  This is the same principle underlying literal
wenzelm@28760
   746
  facts (cf.\ \secref{sec:syn-att}): ``@{command "have"}~@{text
wenzelm@28760
   747
  "\<phi>"}~@{command "by"}~@{text fact}'' is equivalent to ``@{command
wenzelm@28760
   748
  "note"}~@{verbatim "`"}@{text \<phi>}@{verbatim "`"}'' provided that
wenzelm@28760
   749
  @{text "\<turnstile> \<phi>"} is an instance of some known @{text "\<turnstile> \<phi>"} in the
wenzelm@28760
   750
  proof context.
wenzelm@26870
   751
  
wenzelm@28760
   752
  \item @{method assumption} solves some goal by a single assumption
wenzelm@26870
   753
  step.  All given facts are guaranteed to participate in the
wenzelm@26870
   754
  refinement; this means there may be only 0 or 1 in the first place.
wenzelm@26870
   755
  Recall that @{command "qed"} (\secref{sec:proof-steps}) already
wenzelm@26870
   756
  concludes any remaining sub-goals by assumption, so structured
wenzelm@26870
   757
  proofs usually need not quote the @{method assumption} method at
wenzelm@26870
   758
  all.
wenzelm@26870
   759
  
wenzelm@28760
   760
  \item @{method this} applies all of the current facts directly as
wenzelm@26870
   761
  rules.  Recall that ``@{command "."}'' (dot) abbreviates ``@{command
wenzelm@26870
   762
  "by"}~@{text this}''.
wenzelm@26870
   763
  
wenzelm@28760
   764
  \item @{method rule}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} applies some rule given as
wenzelm@28760
   765
  argument in backward manner; facts are used to reduce the rule
wenzelm@28760
   766
  before applying it to the goal.  Thus @{method rule} without facts
wenzelm@28760
   767
  is plain introduction, while with facts it becomes elimination.
wenzelm@26870
   768
  
wenzelm@26870
   769
  When no arguments are given, the @{method rule} method tries to pick
wenzelm@26870
   770
  appropriate rules automatically, as declared in the current context
wenzelm@26901
   771
  using the @{attribute (Pure) intro}, @{attribute (Pure) elim},
wenzelm@26901
   772
  @{attribute (Pure) dest} attributes (see below).  This is the
wenzelm@26901
   773
  default behavior of @{command "proof"} and ``@{command ".."}'' 
wenzelm@26901
   774
  (double-dot) steps (see \secref{sec:proof-steps}).
wenzelm@26870
   775
  
wenzelm@28760
   776
  \item @{attribute (Pure) intro}, @{attribute (Pure) elim}, and
wenzelm@28760
   777
  @{attribute (Pure) dest} declare introduction, elimination, and
wenzelm@30169
   778
  destruct rules, to be used with method @{method rule}, and similar
wenzelm@30169
   779
  tools.  Note that the latter will ignore rules declared with
wenzelm@30169
   780
  ``@{text "?"}'', while ``@{text "!"}''  are used most aggressively.
wenzelm@26870
   781
  
wenzelm@26870
   782
  The classical reasoner (see \secref{sec:classical}) introduces its
wenzelm@26870
   783
  own variants of these attributes; use qualified names to access the
wenzelm@26901
   784
  present versions of Isabelle/Pure, i.e.\ @{attribute (Pure)
wenzelm@26901
   785
  "Pure.intro"}.
wenzelm@26870
   786
  
wenzelm@28760
   787
  \item @{attribute rule}~@{text del} undeclares introduction,
wenzelm@26870
   788
  elimination, or destruct rules.
wenzelm@26870
   789
  
wenzelm@30462
   790
  \item @{attribute OF}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} applies some
wenzelm@30462
   791
  theorem to all of the given rules @{text "a\<^sub>1, \<dots>, a\<^sub>n"}
wenzelm@30462
   792
  (in parallel).  This corresponds to the @{ML "op MRS"} operation in
wenzelm@30462
   793
  ML, but note the reversed order.  Positions may be effectively
wenzelm@30462
   794
  skipped by including ``@{text _}'' (underscore) as argument.
wenzelm@26870
   795
  
wenzelm@28760
   796
  \item @{attribute of}~@{text "t\<^sub>1 \<dots> t\<^sub>n"} performs positional
wenzelm@28760
   797
  instantiation of term variables.  The terms @{text "t\<^sub>1, \<dots>, t\<^sub>n"} are
wenzelm@28760
   798
  substituted for any schematic variables occurring in a theorem from
wenzelm@28760
   799
  left to right; ``@{text _}'' (underscore) indicates to skip a
wenzelm@28760
   800
  position.  Arguments following a ``@{text "concl:"}'' specification
wenzelm@28760
   801
  refer to positions of the conclusion of a rule.
wenzelm@26870
   802
  
wenzelm@28760
   803
  \item @{attribute "where"}~@{text "x\<^sub>1 = t\<^sub>1 \<AND> \<dots> x\<^sub>n = t\<^sub>n"}
wenzelm@28760
   804
  performs named instantiation of schematic type and term variables
wenzelm@28760
   805
  occurring in a theorem.  Schematic variables have to be specified on
wenzelm@28760
   806
  the left-hand side (e.g.\ @{text "?x1.3"}).  The question mark may
wenzelm@28760
   807
  be omitted if the variable name is a plain identifier without index.
wenzelm@28760
   808
  As type instantiations are inferred from term instantiations,
wenzelm@28760
   809
  explicit type instantiations are seldom necessary.
wenzelm@26870
   810
wenzelm@28760
   811
  \end{description}
wenzelm@26870
   812
*}
wenzelm@26870
   813
wenzelm@26870
   814
wenzelm@28754
   815
subsection {* Emulating tactic scripts \label{sec:tactic-commands} *}
wenzelm@26870
   816
wenzelm@26870
   817
text {*
wenzelm@26870
   818
  The Isar provides separate commands to accommodate tactic-style
wenzelm@26870
   819
  proof scripts within the same system.  While being outside the
wenzelm@26870
   820
  orthodox Isar proof language, these might come in handy for
wenzelm@26870
   821
  interactive exploration and debugging, or even actual tactical proof
wenzelm@26870
   822
  within new-style theories (to benefit from document preparation, for
wenzelm@26870
   823
  example).  See also \secref{sec:tactics} for actual tactics, that
wenzelm@26870
   824
  have been encapsulated as proof methods.  Proper proof methods may
wenzelm@26870
   825
  be used in scripts, too.
wenzelm@26870
   826
wenzelm@26870
   827
  \begin{matharray}{rcl}
wenzelm@28761
   828
    @{command_def "apply"}@{text "\<^sup>*"} & : & @{text "proof(prove) \<rightarrow> proof(prove)"} \\
wenzelm@28761
   829
    @{command_def "apply_end"}@{text "\<^sup>*"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28761
   830
    @{command_def "done"}@{text "\<^sup>*"} & : & @{text "proof(prove) \<rightarrow> proof(state) | local_theory | theory"} \\
wenzelm@28761
   831
    @{command_def "defer"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow> proof"} \\
wenzelm@28761
   832
    @{command_def "prefer"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow> proof"} \\
wenzelm@28761
   833
    @{command_def "back"}@{text "\<^sup>*"} & : & @{text "proof \<rightarrow> proof"} \\
wenzelm@26870
   834
  \end{matharray}
wenzelm@26870
   835
wenzelm@26870
   836
  \begin{rail}
wenzelm@26870
   837
    ( 'apply' | 'apply\_end' ) method
wenzelm@26870
   838
    ;
wenzelm@26870
   839
    'defer' nat?
wenzelm@26870
   840
    ;
wenzelm@26870
   841
    'prefer' nat
wenzelm@26870
   842
    ;
wenzelm@26870
   843
  \end{rail}
wenzelm@26870
   844
wenzelm@28760
   845
  \begin{description}
wenzelm@26870
   846
wenzelm@28760
   847
  \item @{command "apply"}~@{text m} applies proof method @{text m} in
wenzelm@28760
   848
  initial position, but unlike @{command "proof"} it retains ``@{text
wenzelm@28760
   849
  "proof(prove)"}'' mode.  Thus consecutive method applications may be
wenzelm@28760
   850
  given just as in tactic scripts.
wenzelm@26870
   851
  
wenzelm@26870
   852
  Facts are passed to @{text m} as indicated by the goal's
wenzelm@26870
   853
  forward-chain mode, and are \emph{consumed} afterwards.  Thus any
wenzelm@26870
   854
  further @{command "apply"} command would always work in a purely
wenzelm@26870
   855
  backward manner.
wenzelm@26870
   856
  
wenzelm@28760
   857
  \item @{command "apply_end"}~@{text "m"} applies proof method @{text
wenzelm@28760
   858
  m} as if in terminal position.  Basically, this simulates a
wenzelm@26870
   859
  multi-step tactic script for @{command "qed"}, but may be given
wenzelm@26870
   860
  anywhere within the proof body.
wenzelm@26870
   861
  
wenzelm@26894
   862
  No facts are passed to @{text m} here.  Furthermore, the static
wenzelm@26870
   863
  context is that of the enclosing goal (as for actual @{command
wenzelm@26870
   864
  "qed"}).  Thus the proof method may not refer to any assumptions
wenzelm@26870
   865
  introduced in the current body, for example.
wenzelm@26870
   866
  
wenzelm@28760
   867
  \item @{command "done"} completes a proof script, provided that the
wenzelm@28760
   868
  current goal state is solved completely.  Note that actual
wenzelm@26870
   869
  structured proof commands (e.g.\ ``@{command "."}'' or @{command
wenzelm@26870
   870
  "sorry"}) may be used to conclude proof scripts as well.
wenzelm@26870
   871
wenzelm@28760
   872
  \item @{command "defer"}~@{text n} and @{command "prefer"}~@{text n}
wenzelm@28760
   873
  shuffle the list of pending goals: @{command "defer"} puts off
wenzelm@26870
   874
  sub-goal @{text n} to the end of the list (@{text "n = 1"} by
wenzelm@26870
   875
  default), while @{command "prefer"} brings sub-goal @{text n} to the
wenzelm@26870
   876
  front.
wenzelm@26870
   877
  
wenzelm@28760
   878
  \item @{command "back"} does back-tracking over the result sequence
wenzelm@28760
   879
  of the latest proof command.  Basically, any proof command may
wenzelm@28760
   880
  return multiple results.
wenzelm@26870
   881
  
wenzelm@28760
   882
  \end{description}
wenzelm@26870
   883
wenzelm@26870
   884
  Any proper Isar proof method may be used with tactic script commands
wenzelm@26870
   885
  such as @{command "apply"}.  A few additional emulations of actual
wenzelm@26870
   886
  tactics are provided as well; these would be never used in actual
wenzelm@26870
   887
  structured proofs, of course.
wenzelm@26870
   888
*}
wenzelm@26870
   889
wenzelm@26870
   890
wenzelm@28757
   891
subsection {* Defining proof methods *}
wenzelm@28757
   892
wenzelm@28757
   893
text {*
wenzelm@28757
   894
  \begin{matharray}{rcl}
wenzelm@28761
   895
    @{command_def "method_setup"} & : & @{text "theory \<rightarrow> theory"} \\
wenzelm@28757
   896
  \end{matharray}
wenzelm@28757
   897
wenzelm@28757
   898
  \begin{rail}
wenzelm@28757
   899
    'method\_setup' name '=' text text
wenzelm@28757
   900
    ;
wenzelm@28757
   901
  \end{rail}
wenzelm@28757
   902
wenzelm@28760
   903
  \begin{description}
wenzelm@28757
   904
wenzelm@28760
   905
  \item @{command "method_setup"}~@{text "name = text description"}
wenzelm@28757
   906
  defines a proof method in the current theory.  The given @{text
wenzelm@30547
   907
  "text"} has to be an ML expression of type
wenzelm@30547
   908
  @{ML_type "(Proof.context -> Proof.method) context_parser"}, cf.\
wenzelm@30547
   909
  basic parsers defined in structure @{ML_struct Args} and @{ML_struct
wenzelm@30547
   910
  Attrib}.  There are also combinators like @{ML METHOD} and @{ML
wenzelm@30547
   911
  SIMPLE_METHOD} to turn certain tactic forms into official proof
wenzelm@30547
   912
  methods; the primed versions refer to tactics with explicit goal
wenzelm@30547
   913
  addressing.
wenzelm@28757
   914
wenzelm@30547
   915
  Here are some example method definitions:
wenzelm@28757
   916
wenzelm@28760
   917
  \end{description}
wenzelm@28757
   918
*}
wenzelm@28757
   919
wenzelm@30547
   920
    method_setup my_method1 = {*
wenzelm@30547
   921
      Scan.succeed (K (SIMPLE_METHOD' (fn i: int => no_tac)))
wenzelm@30547
   922
    *}  "my first method (without any arguments)"
wenzelm@30547
   923
wenzelm@30547
   924
    method_setup my_method2 = {*
wenzelm@30547
   925
      Scan.succeed (fn ctxt: Proof.context =>
wenzelm@30547
   926
        SIMPLE_METHOD' (fn i: int => no_tac))
wenzelm@30547
   927
    *}  "my second method (with context)"
wenzelm@30547
   928
wenzelm@30547
   929
    method_setup my_method3 = {*
wenzelm@30547
   930
      Attrib.thms >> (fn thms: thm list => fn ctxt: Proof.context =>
wenzelm@30547
   931
        SIMPLE_METHOD' (fn i: int => no_tac))
wenzelm@30547
   932
    *}  "my third method (with theorem arguments and context)"
wenzelm@30547
   933
wenzelm@28757
   934
wenzelm@26870
   935
section {* Generalized elimination \label{sec:obtain} *}
wenzelm@26870
   936
wenzelm@26870
   937
text {*
wenzelm@26870
   938
  \begin{matharray}{rcl}
wenzelm@28761
   939
    @{command_def "obtain"} & : & @{text "proof(state) | proof(chain) \<rightarrow> proof(prove)"} \\
wenzelm@28761
   940
    @{command_def "guess"}@{text "\<^sup>*"} & : & @{text "proof(state) | proof(chain) \<rightarrow> proof(prove)"} \\
wenzelm@26870
   941
  \end{matharray}
wenzelm@26870
   942
wenzelm@26870
   943
  Generalized elimination means that additional elements with certain
wenzelm@26870
   944
  properties may be introduced in the current context, by virtue of a
wenzelm@26870
   945
  locally proven ``soundness statement''.  Technically speaking, the
wenzelm@26870
   946
  @{command "obtain"} language element is like a declaration of
wenzelm@26870
   947
  @{command "fix"} and @{command "assume"} (see also see
wenzelm@26870
   948
  \secref{sec:proof-context}), together with a soundness proof of its
wenzelm@26870
   949
  additional claim.  According to the nature of existential reasoning,
wenzelm@26870
   950
  assumptions get eliminated from any result exported from the context
wenzelm@26870
   951
  later, provided that the corresponding parameters do \emph{not}
wenzelm@26870
   952
  occur in the conclusion.
wenzelm@26870
   953
wenzelm@26870
   954
  \begin{rail}
wenzelm@26870
   955
    'obtain' parname? (vars + 'and') 'where' (props + 'and')
wenzelm@26870
   956
    ;
wenzelm@26870
   957
    'guess' (vars + 'and')
wenzelm@26870
   958
    ;
wenzelm@26870
   959
  \end{rail}
wenzelm@26870
   960
wenzelm@26870
   961
  The derived Isar command @{command "obtain"} is defined as follows
wenzelm@26870
   962
  (where @{text "b\<^sub>1, \<dots>, b\<^sub>k"} shall refer to (optional)
wenzelm@26870
   963
  facts indicated for forward chaining).
wenzelm@26870
   964
  \begin{matharray}{l}
wenzelm@26870
   965
    @{text "\<langle>using b\<^sub>1 \<dots> b\<^sub>k\<rangle>"}~~@{command "obtain"}~@{text "x\<^sub>1 \<dots> x\<^sub>m \<WHERE> a: \<phi>\<^sub>1 \<dots> \<phi>\<^sub>n  \<langle>proof\<rangle> \<equiv>"} \\[1ex]
wenzelm@26870
   966
    \quad @{command "have"}~@{text "\<And>thesis. (\<And>x\<^sub>1 \<dots> x\<^sub>m. \<phi>\<^sub>1 \<Longrightarrow> \<dots> \<phi>\<^sub>n \<Longrightarrow> thesis) \<Longrightarrow> thesis"} \\
wenzelm@30049
   967
    \quad @{command "proof"}~@{method succeed} \\
wenzelm@26870
   968
    \qquad @{command "fix"}~@{text thesis} \\
wenzelm@26870
   969
    \qquad @{command "assume"}~@{text "that [Pure.intro?]: \<And>x\<^sub>1 \<dots> x\<^sub>m. \<phi>\<^sub>1 \<Longrightarrow> \<dots> \<phi>\<^sub>n \<Longrightarrow> thesis"} \\
wenzelm@26870
   970
    \qquad @{command "then"}~@{command "show"}~@{text thesis} \\
wenzelm@26870
   971
    \quad\qquad @{command "apply"}~@{text -} \\
wenzelm@26870
   972
    \quad\qquad @{command "using"}~@{text "b\<^sub>1 \<dots> b\<^sub>k  \<langle>proof\<rangle>"} \\
wenzelm@26870
   973
    \quad @{command "qed"} \\
wenzelm@26870
   974
    \quad @{command "fix"}~@{text "x\<^sub>1 \<dots> x\<^sub>m"}~@{command "assume"}@{text "\<^sup>* a: \<phi>\<^sub>1 \<dots> \<phi>\<^sub>n"} \\
wenzelm@26870
   975
  \end{matharray}
wenzelm@26870
   976
wenzelm@26870
   977
  Typically, the soundness proof is relatively straight-forward, often
wenzelm@26870
   978
  just by canonical automated tools such as ``@{command "by"}~@{text
wenzelm@26870
   979
  simp}'' or ``@{command "by"}~@{text blast}''.  Accordingly, the
wenzelm@26870
   980
  ``@{text that}'' reduction above is declared as simplification and
wenzelm@26870
   981
  introduction rule.
wenzelm@26870
   982
wenzelm@26870
   983
  In a sense, @{command "obtain"} represents at the level of Isar
wenzelm@26870
   984
  proofs what would be meta-logical existential quantifiers and
wenzelm@26870
   985
  conjunctions.  This concept has a broad range of useful
wenzelm@26870
   986
  applications, ranging from plain elimination (or introduction) of
wenzelm@26870
   987
  object-level existential and conjunctions, to elimination over
wenzelm@26870
   988
  results of symbolic evaluation of recursive definitions, for
wenzelm@26870
   989
  example.  Also note that @{command "obtain"} without parameters acts
wenzelm@26870
   990
  much like @{command "have"}, where the result is treated as a
wenzelm@26870
   991
  genuine assumption.
wenzelm@26870
   992
wenzelm@26870
   993
  An alternative name to be used instead of ``@{text that}'' above may
wenzelm@26870
   994
  be given in parentheses.
wenzelm@26870
   995
wenzelm@26870
   996
  \medskip The improper variant @{command "guess"} is similar to
wenzelm@26870
   997
  @{command "obtain"}, but derives the obtained statement from the
wenzelm@26870
   998
  course of reasoning!  The proof starts with a fixed goal @{text
wenzelm@26870
   999
  thesis}.  The subsequent proof may refine this to anything of the
wenzelm@26870
  1000
  form like @{text "\<And>x\<^sub>1 \<dots> x\<^sub>m. \<phi>\<^sub>1 \<Longrightarrow> \<dots>
wenzelm@26870
  1001
  \<phi>\<^sub>n \<Longrightarrow> thesis"}, but must not introduce new subgoals.  The
wenzelm@26870
  1002
  final goal state is then used as reduction rule for the obtain
wenzelm@26870
  1003
  scheme described above.  Obtained parameters @{text "x\<^sub>1, \<dots>,
wenzelm@26870
  1004
  x\<^sub>m"} are marked as internal by default, which prevents the
wenzelm@26870
  1005
  proof context from being polluted by ad-hoc variables.  The variable
wenzelm@26870
  1006
  names and type constraints given as arguments for @{command "guess"}
wenzelm@26870
  1007
  specify a prefix of obtained parameters explicitly in the text.
wenzelm@26870
  1008
wenzelm@26870
  1009
  It is important to note that the facts introduced by @{command
wenzelm@26870
  1010
  "obtain"} and @{command "guess"} may not be polymorphic: any
wenzelm@26870
  1011
  type-variables occurring here are fixed in the present context!
wenzelm@26870
  1012
*}
wenzelm@26870
  1013
wenzelm@26870
  1014
wenzelm@26870
  1015
section {* Calculational reasoning \label{sec:calculation} *}
wenzelm@26870
  1016
wenzelm@26870
  1017
text {*
wenzelm@26870
  1018
  \begin{matharray}{rcl}
wenzelm@28761
  1019
    @{command_def "also"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28761
  1020
    @{command_def "finally"} & : & @{text "proof(state) \<rightarrow> proof(chain)"} \\
wenzelm@28761
  1021
    @{command_def "moreover"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28761
  1022
    @{command_def "ultimately"} & : & @{text "proof(state) \<rightarrow> proof(chain)"} \\
wenzelm@28761
  1023
    @{command_def "print_trans_rules"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
wenzelm@28761
  1024
    @{attribute trans} & : & @{text attribute} \\
wenzelm@28761
  1025
    @{attribute sym} & : & @{text attribute} \\
wenzelm@28761
  1026
    @{attribute symmetric} & : & @{text attribute} \\
wenzelm@26870
  1027
  \end{matharray}
wenzelm@26870
  1028
wenzelm@26870
  1029
  Calculational proof is forward reasoning with implicit application
wenzelm@26870
  1030
  of transitivity rules (such those of @{text "="}, @{text "\<le>"},
wenzelm@26870
  1031
  @{text "<"}).  Isabelle/Isar maintains an auxiliary fact register
wenzelm@26870
  1032
  @{fact_ref calculation} for accumulating results obtained by
wenzelm@26870
  1033
  transitivity composed with the current result.  Command @{command
wenzelm@26870
  1034
  "also"} updates @{fact calculation} involving @{fact this}, while
wenzelm@26870
  1035
  @{command "finally"} exhibits the final @{fact calculation} by
wenzelm@26870
  1036
  forward chaining towards the next goal statement.  Both commands
wenzelm@26870
  1037
  require valid current facts, i.e.\ may occur only after commands
wenzelm@26870
  1038
  that produce theorems such as @{command "assume"}, @{command
wenzelm@26870
  1039
  "note"}, or some finished proof of @{command "have"}, @{command
wenzelm@26870
  1040
  "show"} etc.  The @{command "moreover"} and @{command "ultimately"}
wenzelm@26870
  1041
  commands are similar to @{command "also"} and @{command "finally"},
wenzelm@26870
  1042
  but only collect further results in @{fact calculation} without
wenzelm@26870
  1043
  applying any rules yet.
wenzelm@26870
  1044
wenzelm@26870
  1045
  Also note that the implicit term abbreviation ``@{text "\<dots>"}'' has
wenzelm@26870
  1046
  its canonical application with calculational proofs.  It refers to
wenzelm@26870
  1047
  the argument of the preceding statement. (The argument of a curried
wenzelm@26870
  1048
  infix expression happens to be its right-hand side.)
wenzelm@26870
  1049
wenzelm@26870
  1050
  Isabelle/Isar calculations are implicitly subject to block structure
wenzelm@26870
  1051
  in the sense that new threads of calculational reasoning are
wenzelm@26870
  1052
  commenced for any new block (as opened by a local goal, for
wenzelm@26870
  1053
  example).  This means that, apart from being able to nest
wenzelm@26870
  1054
  calculations, there is no separate \emph{begin-calculation} command
wenzelm@26870
  1055
  required.
wenzelm@26870
  1056
wenzelm@26870
  1057
  \medskip The Isar calculation proof commands may be defined as
wenzelm@26870
  1058
  follows:\footnote{We suppress internal bookkeeping such as proper
wenzelm@26870
  1059
  handling of block-structure.}
wenzelm@26870
  1060
wenzelm@26870
  1061
  \begin{matharray}{rcl}
wenzelm@26870
  1062
    @{command "also"}@{text "\<^sub>0"} & \equiv & @{command "note"}~@{text "calculation = this"} \\
wenzelm@30547
  1063
    @{command "also"}@{text "\<^sub>n+1"} & \equiv & @{command "note"}~@{text "calculation = trans [OF calculation this]"} \\[0.5ex]
wenzelm@26870
  1064
    @{command "finally"} & \equiv & @{command "also"}~@{command "from"}~@{text calculation} \\[0.5ex]
wenzelm@26870
  1065
    @{command "moreover"} & \equiv & @{command "note"}~@{text "calculation = calculation this"} \\
wenzelm@26870
  1066
    @{command "ultimately"} & \equiv & @{command "moreover"}~@{command "from"}~@{text calculation} \\
wenzelm@26870
  1067
  \end{matharray}
wenzelm@26870
  1068
wenzelm@26870
  1069
  \begin{rail}
wenzelm@26870
  1070
    ('also' | 'finally') ('(' thmrefs ')')?
wenzelm@26870
  1071
    ;
wenzelm@26870
  1072
    'trans' (() | 'add' | 'del')
wenzelm@26870
  1073
    ;
wenzelm@26870
  1074
  \end{rail}
wenzelm@26870
  1075
wenzelm@28760
  1076
  \begin{description}
wenzelm@26870
  1077
wenzelm@28760
  1078
  \item @{command "also"}~@{text "(a\<^sub>1 \<dots> a\<^sub>n)"} maintains the auxiliary
wenzelm@28760
  1079
  @{fact calculation} register as follows.  The first occurrence of
wenzelm@28760
  1080
  @{command "also"} in some calculational thread initializes @{fact
wenzelm@28760
  1081
  calculation} by @{fact this}. Any subsequent @{command "also"} on
wenzelm@28760
  1082
  the same level of block-structure updates @{fact calculation} by
wenzelm@28760
  1083
  some transitivity rule applied to @{fact calculation} and @{fact
wenzelm@28760
  1084
  this} (in that order).  Transitivity rules are picked from the
wenzelm@28760
  1085
  current context, unless alternative rules are given as explicit
wenzelm@28760
  1086
  arguments.
wenzelm@26870
  1087
wenzelm@28760
  1088
  \item @{command "finally"}~@{text "(a\<^sub>1 \<dots> a\<^sub>n)"} maintaining @{fact
wenzelm@28760
  1089
  calculation} in the same way as @{command "also"}, and concludes the
wenzelm@28760
  1090
  current calculational thread.  The final result is exhibited as fact
wenzelm@28760
  1091
  for forward chaining towards the next goal. Basically, @{command
wenzelm@28760
  1092
  "finally"} just abbreviates @{command "also"}~@{command
wenzelm@28760
  1093
  "from"}~@{fact calculation}.  Typical idioms for concluding
wenzelm@28760
  1094
  calculational proofs are ``@{command "finally"}~@{command
wenzelm@26870
  1095
  "show"}~@{text ?thesis}~@{command "."}'' and ``@{command
wenzelm@26870
  1096
  "finally"}~@{command "have"}~@{text \<phi>}~@{command "."}''.
wenzelm@26870
  1097
wenzelm@28760
  1098
  \item @{command "moreover"} and @{command "ultimately"} are
wenzelm@26870
  1099
  analogous to @{command "also"} and @{command "finally"}, but collect
wenzelm@26870
  1100
  results only, without applying rules.
wenzelm@26870
  1101
wenzelm@28760
  1102
  \item @{command "print_trans_rules"} prints the list of transitivity
wenzelm@28760
  1103
  rules (for calculational commands @{command "also"} and @{command
wenzelm@28760
  1104
  "finally"}) and symmetry rules (for the @{attribute symmetric}
wenzelm@28760
  1105
  operation and single step elimination patters) of the current
wenzelm@28760
  1106
  context.
wenzelm@26870
  1107
wenzelm@28760
  1108
  \item @{attribute trans} declares theorems as transitivity rules.
wenzelm@26870
  1109
wenzelm@28760
  1110
  \item @{attribute sym} declares symmetry rules, as well as
wenzelm@26894
  1111
  @{attribute "Pure.elim"}@{text "?"} rules.
wenzelm@26870
  1112
wenzelm@28760
  1113
  \item @{attribute symmetric} resolves a theorem with some rule
wenzelm@26870
  1114
  declared as @{attribute sym} in the current context.  For example,
wenzelm@26870
  1115
  ``@{command "assume"}~@{text "[symmetric]: x = y"}'' produces a
wenzelm@26870
  1116
  swapped fact derived from that assumption.
wenzelm@26870
  1117
wenzelm@26870
  1118
  In structured proof texts it is often more appropriate to use an
wenzelm@26870
  1119
  explicit single-step elimination proof, such as ``@{command
wenzelm@26870
  1120
  "assume"}~@{text "x = y"}~@{command "then"}~@{command "have"}~@{text
wenzelm@26870
  1121
  "y = x"}~@{command ".."}''.
wenzelm@26870
  1122
wenzelm@28760
  1123
  \end{description}
wenzelm@26870
  1124
*}
wenzelm@26870
  1125
wenzelm@28754
  1126
wenzelm@27040
  1127
section {* Proof by cases and induction \label{sec:cases-induct} *}
wenzelm@27040
  1128
wenzelm@27040
  1129
subsection {* Rule contexts *}
wenzelm@27040
  1130
wenzelm@27040
  1131
text {*
wenzelm@27040
  1132
  \begin{matharray}{rcl}
wenzelm@28761
  1133
    @{command_def "case"} & : & @{text "proof(state) \<rightarrow> proof(state)"} \\
wenzelm@28761
  1134
    @{command_def "print_cases"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
wenzelm@28761
  1135
    @{attribute_def case_names} & : & @{text attribute} \\
wenzelm@28761
  1136
    @{attribute_def case_conclusion} & : & @{text attribute} \\
wenzelm@28761
  1137
    @{attribute_def params} & : & @{text attribute} \\
wenzelm@28761
  1138
    @{attribute_def consumes} & : & @{text attribute} \\
wenzelm@27040
  1139
  \end{matharray}
wenzelm@27040
  1140
wenzelm@27040
  1141
  The puristic way to build up Isar proof contexts is by explicit
wenzelm@27040
  1142
  language elements like @{command "fix"}, @{command "assume"},
wenzelm@27040
  1143
  @{command "let"} (see \secref{sec:proof-context}).  This is adequate
wenzelm@27040
  1144
  for plain natural deduction, but easily becomes unwieldy in concrete
wenzelm@27040
  1145
  verification tasks, which typically involve big induction rules with
wenzelm@27040
  1146
  several cases.
wenzelm@27040
  1147
wenzelm@27040
  1148
  The @{command "case"} command provides a shorthand to refer to a
wenzelm@27040
  1149
  local context symbolically: certain proof methods provide an
wenzelm@27040
  1150
  environment of named ``cases'' of the form @{text "c: x\<^sub>1, \<dots>,
wenzelm@27040
  1151
  x\<^sub>m, \<phi>\<^sub>1, \<dots>, \<phi>\<^sub>n"}; the effect of ``@{command
wenzelm@27040
  1152
  "case"}~@{text c}'' is then equivalent to ``@{command "fix"}~@{text
wenzelm@27040
  1153
  "x\<^sub>1 \<dots> x\<^sub>m"}~@{command "assume"}~@{text "c: \<phi>\<^sub>1 \<dots>
wenzelm@27040
  1154
  \<phi>\<^sub>n"}''.  Term bindings may be covered as well, notably
wenzelm@27040
  1155
  @{variable ?case} for the main conclusion.
wenzelm@27040
  1156
wenzelm@27040
  1157
  By default, the ``terminology'' @{text "x\<^sub>1, \<dots>, x\<^sub>m"} of
wenzelm@27040
  1158
  a case value is marked as hidden, i.e.\ there is no way to refer to
wenzelm@27040
  1159
  such parameters in the subsequent proof text.  After all, original
wenzelm@27040
  1160
  rule parameters stem from somewhere outside of the current proof
wenzelm@27040
  1161
  text.  By using the explicit form ``@{command "case"}~@{text "(c
wenzelm@27040
  1162
  y\<^sub>1 \<dots> y\<^sub>m)"}'' instead, the proof author is able to
wenzelm@27040
  1163
  chose local names that fit nicely into the current context.
wenzelm@27040
  1164
wenzelm@27040
  1165
  \medskip It is important to note that proper use of @{command
wenzelm@27040
  1166
  "case"} does not provide means to peek at the current goal state,
wenzelm@27040
  1167
  which is not directly observable in Isar!  Nonetheless, goal
wenzelm@27040
  1168
  refinement commands do provide named cases @{text "goal\<^sub>i"}
wenzelm@27040
  1169
  for each subgoal @{text "i = 1, \<dots>, n"} of the resulting goal state.
wenzelm@27040
  1170
  Using this extra feature requires great care, because some bits of
wenzelm@27040
  1171
  the internal tactical machinery intrude the proof text.  In
wenzelm@27040
  1172
  particular, parameter names stemming from the left-over of automated
wenzelm@27040
  1173
  reasoning tools are usually quite unpredictable.
wenzelm@27040
  1174
wenzelm@27040
  1175
  Under normal circumstances, the text of cases emerge from standard
wenzelm@27040
  1176
  elimination or induction rules, which in turn are derived from
wenzelm@27040
  1177
  previous theory specifications in a canonical way (say from
wenzelm@27040
  1178
  @{command "inductive"} definitions).
wenzelm@27040
  1179
wenzelm@27040
  1180
  \medskip Proper cases are only available if both the proof method
wenzelm@27040
  1181
  and the rules involved support this.  By using appropriate
wenzelm@27040
  1182
  attributes, case names, conclusions, and parameters may be also
wenzelm@27040
  1183
  declared by hand.  Thus variant versions of rules that have been
wenzelm@27040
  1184
  derived manually become ready to use in advanced case analysis
wenzelm@27040
  1185
  later.
wenzelm@27040
  1186
wenzelm@27040
  1187
  \begin{rail}
wenzelm@27040
  1188
    'case' (caseref | '(' caseref ((name | underscore) +) ')')
wenzelm@27040
  1189
    ;
wenzelm@27040
  1190
    caseref: nameref attributes?
wenzelm@27040
  1191
    ;
wenzelm@27040
  1192
wenzelm@27040
  1193
    'case\_names' (name +)
wenzelm@27040
  1194
    ;
wenzelm@27040
  1195
    'case\_conclusion' name (name *)
wenzelm@27040
  1196
    ;
wenzelm@27040
  1197
    'params' ((name *) + 'and')
wenzelm@27040
  1198
    ;
wenzelm@27040
  1199
    'consumes' nat?
wenzelm@27040
  1200
    ;
wenzelm@27040
  1201
  \end{rail}
wenzelm@27040
  1202
wenzelm@28760
  1203
  \begin{description}
wenzelm@27040
  1204
  
wenzelm@28760
  1205
  \item @{command "case"}~@{text "(c x\<^sub>1 \<dots> x\<^sub>m)"} invokes a named local
wenzelm@28760
  1206
  context @{text "c: x\<^sub>1, \<dots>, x\<^sub>m, \<phi>\<^sub>1, \<dots>, \<phi>\<^sub>m"}, as provided by an
wenzelm@28760
  1207
  appropriate proof method (such as @{method_ref cases} and
wenzelm@28760
  1208
  @{method_ref induct}).  The command ``@{command "case"}~@{text "(c
wenzelm@28760
  1209
  x\<^sub>1 \<dots> x\<^sub>m)"}'' abbreviates ``@{command "fix"}~@{text "x\<^sub>1 \<dots>
wenzelm@28760
  1210
  x\<^sub>m"}~@{command "assume"}~@{text "c: \<phi>\<^sub>1 \<dots> \<phi>\<^sub>n"}''.
wenzelm@27040
  1211
wenzelm@28760
  1212
  \item @{command "print_cases"} prints all local contexts of the
wenzelm@27040
  1213
  current state, using Isar proof language notation.
wenzelm@27040
  1214
  
wenzelm@28760
  1215
  \item @{attribute case_names}~@{text "c\<^sub>1 \<dots> c\<^sub>k"} declares names for
wenzelm@28760
  1216
  the local contexts of premises of a theorem; @{text "c\<^sub>1, \<dots>, c\<^sub>k"}
wenzelm@28760
  1217
  refers to the \emph{suffix} of the list of premises.
wenzelm@27040
  1218
  
wenzelm@28760
  1219
  \item @{attribute case_conclusion}~@{text "c d\<^sub>1 \<dots> d\<^sub>k"} declares
wenzelm@28760
  1220
  names for the conclusions of a named premise @{text c}; here @{text
wenzelm@28760
  1221
  "d\<^sub>1, \<dots>, d\<^sub>k"} refers to the prefix of arguments of a logical formula
wenzelm@28760
  1222
  built by nesting a binary connective (e.g.\ @{text "\<or>"}).
wenzelm@27040
  1223
  
wenzelm@27040
  1224
  Note that proof methods such as @{method induct} and @{method
wenzelm@27040
  1225
  coinduct} already provide a default name for the conclusion as a
wenzelm@27040
  1226
  whole.  The need to name subformulas only arises with cases that
wenzelm@27040
  1227
  split into several sub-cases, as in common co-induction rules.
wenzelm@27040
  1228
wenzelm@28760
  1229
  \item @{attribute params}~@{text "p\<^sub>1 \<dots> p\<^sub>m \<AND> \<dots> q\<^sub>1 \<dots> q\<^sub>n"} renames
wenzelm@28760
  1230
  the innermost parameters of premises @{text "1, \<dots>, n"} of some
wenzelm@28760
  1231
  theorem.  An empty list of names may be given to skip positions,
wenzelm@28760
  1232
  leaving the present parameters unchanged.
wenzelm@27040
  1233
  
wenzelm@27040
  1234
  Note that the default usage of case rules does \emph{not} directly
wenzelm@27040
  1235
  expose parameters to the proof context.
wenzelm@27040
  1236
  
wenzelm@28760
  1237
  \item @{attribute consumes}~@{text n} declares the number of ``major
wenzelm@28760
  1238
  premises'' of a rule, i.e.\ the number of facts to be consumed when
wenzelm@28760
  1239
  it is applied by an appropriate proof method.  The default value of
wenzelm@28760
  1240
  @{attribute consumes} is @{text "n = 1"}, which is appropriate for
wenzelm@28760
  1241
  the usual kind of cases and induction rules for inductive sets (cf.\
wenzelm@28760
  1242
  \secref{sec:hol-inductive}).  Rules without any @{attribute
wenzelm@28760
  1243
  consumes} declaration given are treated as if @{attribute
wenzelm@28760
  1244
  consumes}~@{text 0} had been specified.
wenzelm@27040
  1245
  
wenzelm@27040
  1246
  Note that explicit @{attribute consumes} declarations are only
wenzelm@27040
  1247
  rarely needed; this is already taken care of automatically by the
wenzelm@27040
  1248
  higher-level @{attribute cases}, @{attribute induct}, and
wenzelm@27040
  1249
  @{attribute coinduct} declarations.
wenzelm@27040
  1250
wenzelm@28760
  1251
  \end{description}
wenzelm@27040
  1252
*}
wenzelm@27040
  1253
wenzelm@27040
  1254
wenzelm@27040
  1255
subsection {* Proof methods *}
wenzelm@27040
  1256
wenzelm@27040
  1257
text {*
wenzelm@27040
  1258
  \begin{matharray}{rcl}
wenzelm@28761
  1259
    @{method_def cases} & : & @{text method} \\
wenzelm@28761
  1260
    @{method_def induct} & : & @{text method} \\
wenzelm@28761
  1261
    @{method_def coinduct} & : & @{text method} \\
wenzelm@27040
  1262
  \end{matharray}
wenzelm@27040
  1263
wenzelm@27040
  1264
  The @{method cases}, @{method induct}, and @{method coinduct}
wenzelm@27040
  1265
  methods provide a uniform interface to common proof techniques over
wenzelm@27040
  1266
  datatypes, inductive predicates (or sets), recursive functions etc.
wenzelm@27040
  1267
  The corresponding rules may be specified and instantiated in a
wenzelm@27040
  1268
  casual manner.  Furthermore, these methods provide named local
wenzelm@27040
  1269
  contexts that may be invoked via the @{command "case"} proof command
wenzelm@27040
  1270
  within the subsequent proof text.  This accommodates compact proof
wenzelm@27040
  1271
  texts even when reasoning about large specifications.
wenzelm@27040
  1272
wenzelm@27040
  1273
  The @{method induct} method also provides some additional
wenzelm@27040
  1274
  infrastructure in order to be applicable to structure statements
wenzelm@27040
  1275
  (either using explicit meta-level connectives, or including facts
wenzelm@27040
  1276
  and parameters separately).  This avoids cumbersome encoding of
wenzelm@27040
  1277
  ``strengthened'' inductive statements within the object-logic.
wenzelm@27040
  1278
wenzelm@27040
  1279
  \begin{rail}
berghofe@37462
  1280
    'cases' '(no_simp)'? (insts * 'and') rule?
wenzelm@27040
  1281
    ;
berghofe@37462
  1282
    'induct' '(no_simp)'? (definsts * 'and') \\ arbitrary? taking? rule?
wenzelm@27040
  1283
    ;
wenzelm@27040
  1284
    'coinduct' insts taking rule?
wenzelm@27040
  1285
    ;
wenzelm@27040
  1286
wenzelm@27040
  1287
    rule: ('type' | 'pred' | 'set') ':' (nameref +) | 'rule' ':' (thmref +)
wenzelm@27040
  1288
    ;
berghofe@37462
  1289
    definst: name ('==' | equiv) term | '(' term ')' | inst
wenzelm@27040
  1290
    ;
wenzelm@27040
  1291
    definsts: ( definst *)
wenzelm@27040
  1292
    ;
wenzelm@27040
  1293
    arbitrary: 'arbitrary' ':' ((term *) 'and' +)
wenzelm@27040
  1294
    ;
wenzelm@27040
  1295
    taking: 'taking' ':' insts
wenzelm@27040
  1296
    ;
wenzelm@27040
  1297
  \end{rail}
wenzelm@27040
  1298
wenzelm@28760
  1299
  \begin{description}
wenzelm@27040
  1300
wenzelm@28760
  1301
  \item @{method cases}~@{text "insts R"} applies method @{method
wenzelm@27040
  1302
  rule} with an appropriate case distinction theorem, instantiated to
wenzelm@27040
  1303
  the subjects @{text insts}.  Symbolic case names are bound according
wenzelm@27040
  1304
  to the rule's local contexts.
wenzelm@27040
  1305
wenzelm@27040
  1306
  The rule is determined as follows, according to the facts and
wenzelm@27040
  1307
  arguments passed to the @{method cases} method:
wenzelm@27040
  1308
wenzelm@27040
  1309
  \medskip
wenzelm@27040
  1310
  \begin{tabular}{llll}
wenzelm@27040
  1311
    facts           &                 & arguments   & rule \\\hline
wenzelm@27040
  1312
                    & @{method cases} &             & classical case split \\
wenzelm@27040
  1313
                    & @{method cases} & @{text t}   & datatype exhaustion (type of @{text t}) \\
wenzelm@27040
  1314
    @{text "\<turnstile> A t"} & @{method cases} & @{text "\<dots>"} & inductive predicate/set elimination (of @{text A}) \\
wenzelm@27040
  1315
    @{text "\<dots>"}     & @{method cases} & @{text "\<dots> rule: R"} & explicit rule @{text R} \\
wenzelm@27040
  1316
  \end{tabular}
wenzelm@27040
  1317
  \medskip
wenzelm@27040
  1318
wenzelm@27040
  1319
  Several instantiations may be given, referring to the \emph{suffix}
wenzelm@27040
  1320
  of premises of the case rule; within each premise, the \emph{prefix}
wenzelm@27040
  1321
  of variables is instantiated.  In most situations, only a single
wenzelm@27040
  1322
  term needs to be specified; this refers to the first variable of the
wenzelm@37465
  1323
  last premise (it is usually the same for all cases).  The @{text
wenzelm@37465
  1324
  "(no_simp)"} option can be used to disable pre-simplification of
wenzelm@37465
  1325
  cases (see the description of @{method induct} below for details).
wenzelm@27040
  1326
wenzelm@28760
  1327
  \item @{method induct}~@{text "insts R"} is analogous to the
wenzelm@27040
  1328
  @{method cases} method, but refers to induction rules, which are
wenzelm@27040
  1329
  determined as follows:
wenzelm@27040
  1330
wenzelm@27040
  1331
  \medskip
wenzelm@27040
  1332
  \begin{tabular}{llll}
wenzelm@27040
  1333
    facts           &                  & arguments            & rule \\\hline
wenzelm@27040
  1334
                    & @{method induct} & @{text "P x"}        & datatype induction (type of @{text x}) \\
wenzelm@27040
  1335
    @{text "\<turnstile> A x"} & @{method induct} & @{text "\<dots>"}          & predicate/set induction (of @{text A}) \\
wenzelm@27040
  1336
    @{text "\<dots>"}     & @{method induct} & @{text "\<dots> rule: R"} & explicit rule @{text R} \\
wenzelm@27040
  1337
  \end{tabular}
wenzelm@27040
  1338
  \medskip
wenzelm@27040
  1339
  
wenzelm@27040
  1340
  Several instantiations may be given, each referring to some part of
wenzelm@27040
  1341
  a mutual inductive definition or datatype --- only related partial
wenzelm@27040
  1342
  induction rules may be used together, though.  Any of the lists of
wenzelm@27040
  1343
  terms @{text "P, x, \<dots>"} refers to the \emph{suffix} of variables
wenzelm@27040
  1344
  present in the induction rule.  This enables the writer to specify
wenzelm@27040
  1345
  only induction variables, or both predicates and variables, for
wenzelm@27040
  1346
  example.
wenzelm@37465
  1347
wenzelm@27040
  1348
  Instantiations may be definitional: equations @{text "x \<equiv> t"}
wenzelm@27040
  1349
  introduce local definitions, which are inserted into the claim and
wenzelm@27040
  1350
  discharged after applying the induction rule.  Equalities reappear
wenzelm@27040
  1351
  in the inductive cases, but have been transformed according to the
wenzelm@27040
  1352
  induction principle being involved here.  In order to achieve
wenzelm@27040
  1353
  practically useful induction hypotheses, some variables occurring in
wenzelm@37465
  1354
  @{text t} need to be fixed (see below).  Instantiations of the form
wenzelm@37465
  1355
  @{text t}, where @{text t} is not a variable, are taken as a
wenzelm@37465
  1356
  shorthand for \mbox{@{text "x \<equiv> t"}}, where @{text x} is a fresh
wenzelm@37465
  1357
  variable. If this is not intended, @{text t} has to be enclosed in
wenzelm@37465
  1358
  parentheses.  By default, the equalities generated by definitional
wenzelm@37465
  1359
  instantiations are pre-simplified using a specific set of rules,
wenzelm@37465
  1360
  usually consisting of distinctness and injectivity theorems for
wenzelm@37465
  1361
  datatypes. This pre-simplification may cause some of the parameters
wenzelm@37465
  1362
  of an inductive case to disappear, or may even completely delete
wenzelm@37465
  1363
  some of the inductive cases, if one of the equalities occurring in
wenzelm@37465
  1364
  their premises can be simplified to @{text False}.  The @{text
wenzelm@37465
  1365
  "(no_simp)"} option can be used to disable pre-simplification.
wenzelm@37465
  1366
  Additional rules to be used in pre-simplification can be declared
wenzelm@37465
  1367
  using the @{attribute_def induct_simp} attribute.
wenzelm@37465
  1368
wenzelm@27040
  1369
  The optional ``@{text "arbitrary: x\<^sub>1 \<dots> x\<^sub>m"}''
wenzelm@27040
  1370
  specification generalizes variables @{text "x\<^sub>1, \<dots>,
wenzelm@27040
  1371
  x\<^sub>m"} of the original goal before applying induction.  Thus
wenzelm@27040
  1372
  induction hypotheses may become sufficiently general to get the
wenzelm@27040
  1373
  proof through.  Together with definitional instantiations, one may
wenzelm@27040
  1374
  effectively perform induction over expressions of a certain
wenzelm@27040
  1375
  structure.
wenzelm@27040
  1376
  
wenzelm@27040
  1377
  The optional ``@{text "taking: t\<^sub>1 \<dots> t\<^sub>n"}''
wenzelm@27040
  1378
  specification provides additional instantiations of a prefix of
wenzelm@27040
  1379
  pending variables in the rule.  Such schematic induction rules
wenzelm@27040
  1380
  rarely occur in practice, though.
wenzelm@27040
  1381
wenzelm@28760
  1382
  \item @{method coinduct}~@{text "inst R"} is analogous to the
wenzelm@27040
  1383
  @{method induct} method, but refers to coinduction rules, which are
wenzelm@27040
  1384
  determined as follows:
wenzelm@27040
  1385
wenzelm@27040
  1386
  \medskip
wenzelm@27040
  1387
  \begin{tabular}{llll}
wenzelm@27040
  1388
    goal          &                    & arguments & rule \\\hline
wenzelm@27040
  1389
                  & @{method coinduct} & @{text x} & type coinduction (type of @{text x}) \\
wenzelm@27040
  1390
    @{text "A x"} & @{method coinduct} & @{text "\<dots>"} & predicate/set coinduction (of @{text A}) \\
wenzelm@27040
  1391
    @{text "\<dots>"}   & @{method coinduct} & @{text "\<dots> rule: R"} & explicit rule @{text R} \\
wenzelm@27040
  1392
  \end{tabular}
wenzelm@27040
  1393
  
wenzelm@27040
  1394
  Coinduction is the dual of induction.  Induction essentially
wenzelm@27040
  1395
  eliminates @{text "A x"} towards a generic result @{text "P x"},
wenzelm@27040
  1396
  while coinduction introduces @{text "A x"} starting with @{text "B
wenzelm@27040
  1397
  x"}, for a suitable ``bisimulation'' @{text B}.  The cases of a
wenzelm@27040
  1398
  coinduct rule are typically named after the predicates or sets being
wenzelm@27040
  1399
  covered, while the conclusions consist of several alternatives being
wenzelm@27040
  1400
  named after the individual destructor patterns.
wenzelm@27040
  1401
  
wenzelm@27040
  1402
  The given instantiation refers to the \emph{suffix} of variables
wenzelm@27040
  1403
  occurring in the rule's major premise, or conclusion if unavailable.
wenzelm@27040
  1404
  An additional ``@{text "taking: t\<^sub>1 \<dots> t\<^sub>n"}''
wenzelm@27040
  1405
  specification may be required in order to specify the bisimulation
wenzelm@27040
  1406
  to be used in the coinduction step.
wenzelm@27040
  1407
wenzelm@28760
  1408
  \end{description}
wenzelm@27040
  1409
wenzelm@27040
  1410
  Above methods produce named local contexts, as determined by the
wenzelm@27040
  1411
  instantiated rule as given in the text.  Beyond that, the @{method
wenzelm@27040
  1412
  induct} and @{method coinduct} methods guess further instantiations
wenzelm@27040
  1413
  from the goal specification itself.  Any persisting unresolved
wenzelm@27040
  1414
  schematic variables of the resulting rule will render the the
wenzelm@27040
  1415
  corresponding case invalid.  The term binding @{variable ?case} for
wenzelm@27040
  1416
  the conclusion will be provided with each case, provided that term
wenzelm@27040
  1417
  is fully specified.
wenzelm@27040
  1418
wenzelm@27040
  1419
  The @{command "print_cases"} command prints all named cases present
wenzelm@27040
  1420
  in the current proof state.
wenzelm@27040
  1421
wenzelm@27040
  1422
  \medskip Despite the additional infrastructure, both @{method cases}
wenzelm@27040
  1423
  and @{method coinduct} merely apply a certain rule, after
wenzelm@27040
  1424
  instantiation, while conforming due to the usual way of monotonic
wenzelm@27040
  1425
  natural deduction: the context of a structured statement @{text
wenzelm@27040
  1426
  "\<And>x\<^sub>1 \<dots> x\<^sub>m. \<phi>\<^sub>1 \<Longrightarrow> \<dots> \<phi>\<^sub>n \<Longrightarrow> \<dots>"}
wenzelm@27040
  1427
  reappears unchanged after the case split.
wenzelm@27040
  1428
wenzelm@27040
  1429
  The @{method induct} method is fundamentally different in this
wenzelm@27040
  1430
  respect: the meta-level structure is passed through the
wenzelm@27040
  1431
  ``recursive'' course involved in the induction.  Thus the original
wenzelm@27040
  1432
  statement is basically replaced by separate copies, corresponding to
wenzelm@27040
  1433
  the induction hypotheses and conclusion; the original goal context
wenzelm@27040
  1434
  is no longer available.  Thus local assumptions, fixed parameters
wenzelm@27040
  1435
  and definitions effectively participate in the inductive rephrasing
wenzelm@27040
  1436
  of the original statement.
wenzelm@27040
  1437
wenzelm@27040
  1438
  In induction proofs, local assumptions introduced by cases are split
wenzelm@27040
  1439
  into two different kinds: @{text hyps} stemming from the rule and
wenzelm@27040
  1440
  @{text prems} from the goal statement.  This is reflected in the
wenzelm@27040
  1441
  extracted cases accordingly, so invoking ``@{command "case"}~@{text
wenzelm@27040
  1442
  c}'' will provide separate facts @{text c.hyps} and @{text c.prems},
wenzelm@27040
  1443
  as well as fact @{text c} to hold the all-inclusive list.
wenzelm@27040
  1444
wenzelm@27040
  1445
  \medskip Facts presented to either method are consumed according to
wenzelm@27040
  1446
  the number of ``major premises'' of the rule involved, which is
wenzelm@27040
  1447
  usually 0 for plain cases and induction rules of datatypes etc.\ and
wenzelm@27040
  1448
  1 for rules of inductive predicates or sets and the like.  The
wenzelm@27040
  1449
  remaining facts are inserted into the goal verbatim before the
wenzelm@27040
  1450
  actual @{text cases}, @{text induct}, or @{text coinduct} rule is
wenzelm@27040
  1451
  applied.
wenzelm@27040
  1452
*}
wenzelm@27040
  1453
wenzelm@27040
  1454
wenzelm@27040
  1455
subsection {* Declaring rules *}
wenzelm@27040
  1456
wenzelm@27040
  1457
text {*
wenzelm@27040
  1458
  \begin{matharray}{rcl}
wenzelm@28761
  1459
    @{command_def "print_induct_rules"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\
wenzelm@28761
  1460
    @{attribute_def cases} & : & @{text attribute} \\
wenzelm@28761
  1461
    @{attribute_def induct} & : & @{text attribute} \\
wenzelm@28761
  1462
    @{attribute_def coinduct} & : & @{text attribute} \\
wenzelm@27040
  1463
  \end{matharray}
wenzelm@27040
  1464
wenzelm@27040
  1465
  \begin{rail}
wenzelm@27040
  1466
    'cases' spec
wenzelm@27040
  1467
    ;
wenzelm@27040
  1468
    'induct' spec
wenzelm@27040
  1469
    ;
wenzelm@27040
  1470
    'coinduct' spec
wenzelm@27040
  1471
    ;
wenzelm@27040
  1472
wenzelm@27141
  1473
    spec: (('type' | 'pred' | 'set') ':' nameref) | 'del'
wenzelm@27040
  1474
    ;
wenzelm@27040
  1475
  \end{rail}
wenzelm@27040
  1476
wenzelm@28760
  1477
  \begin{description}
wenzelm@27040
  1478
wenzelm@28760
  1479
  \item @{command "print_induct_rules"} prints cases and induct rules
wenzelm@28760
  1480
  for predicates (or sets) and types of the current context.
wenzelm@27040
  1481
  
wenzelm@28760
  1482
  \item @{attribute cases}, @{attribute induct}, and @{attribute
wenzelm@28760
  1483
  coinduct} (as attributes) declare rules for reasoning about
wenzelm@27141
  1484
  (co)inductive predicates (or sets) and types, using the
wenzelm@27141
  1485
  corresponding methods of the same name.  Certain definitional
wenzelm@27141
  1486
  packages of object-logics usually declare emerging cases and
wenzelm@27141
  1487
  induction rules as expected, so users rarely need to intervene.
wenzelm@27141
  1488
wenzelm@27141
  1489
  Rules may be deleted via the @{text "del"} specification, which
wenzelm@27141
  1490
  covers all of the @{text "type"}/@{text "pred"}/@{text "set"}
wenzelm@27141
  1491
  sub-categories simultaneously.  For example, @{attribute
wenzelm@27141
  1492
  cases}~@{text del} removes any @{attribute cases} rules declared for
wenzelm@27141
  1493
  some type, predicate, or set.
wenzelm@27040
  1494
  
wenzelm@27040
  1495
  Manual rule declarations usually refer to the @{attribute
wenzelm@27040
  1496
  case_names} and @{attribute params} attributes to adjust names of
wenzelm@27040
  1497
  cases and parameters of a rule; the @{attribute consumes}
wenzelm@27040
  1498
  declaration is taken care of automatically: @{attribute
wenzelm@27040
  1499
  consumes}~@{text 0} is specified for ``type'' rules and @{attribute
wenzelm@27040
  1500
  consumes}~@{text 1} for ``predicate'' / ``set'' rules.
wenzelm@27040
  1501
wenzelm@28760
  1502
  \end{description}
wenzelm@27040
  1503
*}
wenzelm@27040
  1504
wenzelm@26869
  1505
end