equal
deleted
inserted
replaced
379 initially (via @{command_ref "then"}), and whether the final result |
379 initially (via @{command_ref "then"}), and whether the final result |
380 is meant to solve some pending goal. |
380 is meant to solve some pending goal. |
381 |
381 |
382 Goals may consist of multiple statements, resulting in a list of |
382 Goals may consist of multiple statements, resulting in a list of |
383 facts eventually. A pending multi-goal is internally represented as |
383 facts eventually. A pending multi-goal is internally represented as |
384 a meta-level conjunction (printed as @{text "&&"}), which is usually |
384 a meta-level conjunction (@{text "&&&"}), which is usually |
385 split into the corresponding number of sub-goals prior to an initial |
385 split into the corresponding number of sub-goals prior to an initial |
386 method application, via @{command_ref "proof"} |
386 method application, via @{command_ref "proof"} |
387 (\secref{sec:proof-steps}) or @{command_ref "apply"} |
387 (\secref{sec:proof-steps}) or @{command_ref "apply"} |
388 (\secref{sec:tactic-commands}). The @{method_ref induct} method |
388 (\secref{sec:tactic-commands}). The @{method_ref induct} method |
389 covered in \secref{sec:cases-induct} acts on multiple claims |
389 covered in \secref{sec:cases-induct} acts on multiple claims |