diff -r aaa9933039b3 -r 5ab0f8859f9f doc-src/IsarRef/Thy/Proof.thy --- a/doc-src/IsarRef/Thy/Proof.thy Mon Apr 26 21:36:44 2010 +0200 +++ b/doc-src/IsarRef/Thy/Proof.thy Mon Apr 26 21:45:08 2010 +0200 @@ -46,6 +46,28 @@ section {* Proof structure *} +subsection {* Example proofs *} + +text {* + \begin{matharray}{rcl} + @{command_def "example_proof"} & : & @{text "local_theory \ proof(state)"} \\ + \end{matharray} + + \begin{description} + + \item @{command "example_proof"} opens an empty proof body. This + allows to experiment with Isar, without producing any persistent + result. + + Structurally, this is like a vacous @{command "lemma"} statement + followed by ``@{command "proof"}~@{text "-"}'', which means the + example proof may be closed by a regular @{command "qed"}, or + discontinued by @{command "oops"}. + + \end{description} +*} + + subsection {* Blocks *} text {*