diff -r e4c5c7ffceea -r fee67c099d03 doc-src/IsarRef/Thy/Framework.thy --- a/doc-src/IsarRef/Thy/Framework.thy Tue May 03 21:40:14 2011 +0200 +++ b/doc-src/IsarRef/Thy/Framework.thy Tue May 03 21:44:05 2011 +0200 @@ -424,7 +424,7 @@ \infer[(@{inference refinement})] {@{text "(\\<^vec>x. \<^vec>H \<^vec>x \ \<^vec>G' (\<^vec>a \<^vec>x))\ \ C\"}} {\begin{tabular}{rl} - @{text "sub\proof:"} & + @{text "sub\proof:"} & @{text "\<^vec>G \<^vec>a \ B \<^vec>a"} \\ @{text "goal:"} & @{text "(\\<^vec>x. \<^vec>H \<^vec>x \ B' \<^vec>x) \ C"} \\ @@ -436,7 +436,7 @@ \end{tabular}} \] - \noindent Here the @{text "sub\proof"} rule stems from the + \noindent Here the @{text "sub\proof"} rule stems from the main @{command fix}-@{command assume}-@{command show} outline of Isar (cf.\ \secref{sec:framework-subproof}): each assumption indicated in the text results in a marked premise @{text "G"} above. @@ -466,7 +466,7 @@ \medskip \begin{tabular}{rcl} - @{text "theory\stmt"} & = & @{command "theorem"}~@{text "statement proof |"}~~@{command "definition"}~@{text "\ | \"} \\[1ex] + @{text "theory\stmt"} & = & @{command "theorem"}~@{text "statement proof |"}~~@{command "definition"}~@{text "\ | \"} \\[1ex] @{text "proof"} & = & @{text "prfx\<^sup>*"}~@{command "proof"}~@{text "method\<^sup>? stmt\<^sup>*"}~@{command "qed"}~@{text "method\<^sup>?"} \\[1ex] @@ -582,7 +582,7 @@ \medskip \begin{tabular}{rcl} - @{command presume}~@{text A} & @{text "\"} & @{command assume}~@{text "\weak\discharge\ A"} \\ + @{command presume}~@{text A} & @{text "\"} & @{command assume}~@{text "\weak\discharge\ A"} \\ @{command def}~@{text "x \ a"} & @{text "\"} & @{command fix}~@{text x}~@{command assume}~@{text "\expansion\ x \ a"} \\ \end{tabular} \medskip @@ -591,14 +591,14 @@ \infer[(@{inference_def discharge})]{@{text "\\ - A \ #A \ B"}}{@{text "\\ \ B"}} \] \[ - \infer[(@{inference_def "weak\discharge"})]{@{text "\\ - A \ A \ B"}}{@{text "\\ \ B"}} + \infer[(@{inference_def "weak\discharge"})]{@{text "\\ - A \ A \ B"}}{@{text "\\ \ B"}} \] \[ \infer[(@{inference_def expansion})]{@{text "\\ - (x \ a) \ B a"}}{@{text "\\ \ B x"}} \] \medskip Note that @{inference discharge} and @{inference - "weak\discharge"} differ in the marker for @{prop A}, which is + "weak\discharge"} differ in the marker for @{prop A}, which is relevant when the result of a @{command fix}-@{command assume}-@{command show} outline is composed with a pending goal, cf.\ \secref{sec:framework-subproof}.