src/Doc/Isar_Ref/Proof.thy
changeset 61166 5976fe402824
parent 61164 2a03ae772c60
child 61337 4645502c3c64
equal deleted inserted replaced
61165:8020249565fb 61166:5976fe402824
   830   \chref{ch:gen-tools} and \partref{part:hol}).
   830   \chref{ch:gen-tools} and \partref{part:hol}).
   831 
   831 
   832   \begin{matharray}{rcl}
   832   \begin{matharray}{rcl}
   833     @{command_def "print_rules"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\[0.5ex]
   833     @{command_def "print_rules"}@{text "\<^sup>*"} & : & @{text "context \<rightarrow>"} \\[0.5ex]
   834     @{method_def "-"} & : & @{text method} \\
   834     @{method_def "-"} & : & @{text method} \\
   835     @{method_def "goals"} & : & @{text method} \\
   835     @{method_def "goal_cases"} & : & @{text method} \\
   836     @{method_def "fact"} & : & @{text method} \\
   836     @{method_def "fact"} & : & @{text method} \\
   837     @{method_def "assumption"} & : & @{text method} \\
   837     @{method_def "assumption"} & : & @{text method} \\
   838     @{method_def "this"} & : & @{text method} \\
   838     @{method_def "this"} & : & @{text method} \\
   839     @{method_def (Pure) "rule"} & : & @{text method} \\
   839     @{method_def (Pure) "rule"} & : & @{text method} \\
   840     @{attribute_def (Pure) "intro"} & : & @{text attribute} \\
   840     @{attribute_def (Pure) "intro"} & : & @{text attribute} \\
   845     @{attribute_def "of"} & : & @{text attribute} \\
   845     @{attribute_def "of"} & : & @{text attribute} \\
   846     @{attribute_def "where"} & : & @{text attribute} \\
   846     @{attribute_def "where"} & : & @{text attribute} \\
   847   \end{matharray}
   847   \end{matharray}
   848 
   848 
   849   @{rail \<open>
   849   @{rail \<open>
   850     @@{method goals} (@{syntax name}*)
   850     @@{method goal_cases} (@{syntax name}*)
   851     ;
   851     ;
   852     @@{method fact} @{syntax thmrefs}?
   852     @@{method fact} @{syntax thmrefs}?
   853     ;
   853     ;
   854     @@{method (Pure) rule} @{syntax thmrefs}?
   854     @@{method (Pure) rule} @{syntax thmrefs}?
   855     ;
   855     ;
   884   Note that command @{command_ref "proof"} without any method actually
   884   Note that command @{command_ref "proof"} without any method actually
   885   performs a single reduction step using the @{method_ref (Pure) rule}
   885   performs a single reduction step using the @{method_ref (Pure) rule}
   886   method; thus a plain \emph{do-nothing} proof step would be ``@{command
   886   method; thus a plain \emph{do-nothing} proof step would be ``@{command
   887   "proof"}~@{text "-"}'' rather than @{command "proof"} alone.
   887   "proof"}~@{text "-"}'' rather than @{command "proof"} alone.
   888 
   888 
   889   \item @{method "goals"}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} turns the current subgoals
   889   \item @{method "goal_cases"}~@{text "a\<^sub>1 \<dots> a\<^sub>n"} turns the current subgoals
   890   into cases within the context (see also \secref{sec:cases-induct}). The
   890   into cases within the context (see also \secref{sec:cases-induct}). The
   891   specified case names are used if present; otherwise cases are numbered
   891   specified case names are used if present; otherwise cases are numbered
   892   starting from 1.
   892   starting from 1.
   893 
   893 
   894   Invoking cases in the subsequent proof body via the @{command_ref case}
   894   Invoking cases in the subsequent proof body via the @{command_ref case}