diff -r 5ab0f8859f9f -r 641a521bfc19 doc-src/IsarRef/Thy/Framework.thy --- a/doc-src/IsarRef/Thy/Framework.thy Mon Apr 26 21:45:08 2010 +0200 +++ b/doc-src/IsarRef/Thy/Framework.thy Mon Apr 26 21:50:28 2010 +0200 @@ -79,8 +79,7 @@ text_raw {*\medskip\begin{minipage}{0.6\textwidth}*} (*<*) -lemma True -proof +example_proof (*>*) assume "x \ A" and "x \ B" then have "x \ A \ B" .. @@ -107,8 +106,7 @@ *} (*<*) -lemma True -proof +example_proof (*>*) assume "x \ A" and "x \ B" then have "x \ A \ B" by (rule IntI) @@ -130,8 +128,7 @@ text_raw {*\medskip\begin{minipage}{0.6\textwidth}*} (*<*) -lemma True -proof +example_proof (*>*) have "x \ \\" proof @@ -178,8 +175,7 @@ text_raw {*\medskip\begin{minipage}{0.6\textwidth}*} (*<*) -lemma True -proof +example_proof (*>*) assume "x \ \\" then have C @@ -212,8 +208,7 @@ *} (*<*) -lemma True -proof +example_proof (*>*) assume "x \ \\" then obtain A where "x \ A" and "A \ \" .. @@ -817,8 +812,7 @@ *} text_raw {* \begingroup\footnotesize *} -(*<*)lemma True -proof +(*<*)example_proof (*>*) txt_raw {* \begin{minipage}[t]{0.18\textwidth} *} have "A \ B" @@ -877,8 +871,7 @@ text_raw {*\begin{minipage}{0.5\textwidth}*} (*<*) -lemma True -proof +example_proof (*>*) have "\x y. A x \ B y \ C x y" proof - @@ -987,8 +980,7 @@ *} (*<*) -lemma True -proof +example_proof (*>*) have "a = b" sorry also have "\ = c" sorry