doc-src/IsarRef/Thy/Proof.thy
changeset 36366 5ab0f8859f9f
parent 36320 549be64e890f
child 37462 250f487b3034
equal deleted inserted replaced
36365:aaa9933039b3 36366:5ab0f8859f9f
    43   explained in \chref{ch:isar-framework}.
    43   explained in \chref{ch:isar-framework}.
    44 *}
    44 *}
    45 
    45 
    46 
    46 
    47 section {* Proof structure *}
    47 section {* Proof structure *}
       
    48 
       
    49 subsection {* Example proofs *}
       
    50 
       
    51 text {*
       
    52   \begin{matharray}{rcl}
       
    53     @{command_def "example_proof"} & : & @{text "local_theory \<rightarrow> proof(state)"} \\
       
    54   \end{matharray}
       
    55 
       
    56   \begin{description}
       
    57 
       
    58   \item @{command "example_proof"} opens an empty proof body.  This
       
    59   allows to experiment with Isar, without producing any persistent
       
    60   result.
       
    61 
       
    62   Structurally, this is like a vacous @{command "lemma"} statement
       
    63   followed by ``@{command "proof"}~@{text "-"}'', which means the
       
    64   example proof may be closed by a regular @{command "qed"}, or
       
    65   discontinued by @{command "oops"}.
       
    66 
       
    67   \end{description}
       
    68 *}
       
    69 
    48 
    70 
    49 subsection {* Blocks *}
    71 subsection {* Blocks *}
    50 
    72 
    51 text {*
    73 text {*
    52   \begin{matharray}{rcl}
    74   \begin{matharray}{rcl}