doc-src/IsarRef/Thy/Framework.thy
changeset 40476 515eab39b6c2
parent 36357 641a521bfc19
child 40964 482a8334ee9e
--- a/doc-src/IsarRef/Thy/Framework.thy	Wed Nov 10 20:43:22 2010 +0100
+++ b/doc-src/IsarRef/Thy/Framework.thy	Thu Nov 11 13:07:41 2010 +0100
@@ -649,25 +649,25 @@
 theorem True
 proof
 (*>*)
-  txt_raw {* \begin{minipage}[t]{0.4\textwidth} *}
+  txt_raw {* \begin{minipage}[t]{0.45\textwidth} *}
   {
     fix x
     have "B x" sorry %noproof
   }
   note `\<And>x. B x`
-  txt_raw {* \end{minipage}\quad\begin{minipage}[t]{0.4\textwidth} *}(*<*)next(*>*)
+  txt_raw {* \end{minipage}\quad\begin{minipage}[t]{0.45\textwidth} *}(*<*)next(*>*)
   {
     assume A
     have B sorry %noproof
   }
   note `A \<Longrightarrow> B`
-  txt_raw {* \end{minipage}\\[3ex]\begin{minipage}[t]{0.4\textwidth} *}(*<*)next(*>*)
+  txt_raw {* \end{minipage}\\[3ex]\begin{minipage}[t]{0.45\textwidth} *}(*<*)next(*>*)
   {
     def x \<equiv> a
     have "B x" sorry %noproof
   }
   note `B a`
-  txt_raw {* \end{minipage}\quad\begin{minipage}[t]{0.4\textwidth} *}(*<*)next(*>*)
+  txt_raw {* \end{minipage}\quad\begin{minipage}[t]{0.45\textwidth} *}(*<*)next(*>*)
   {
     obtain x where "A x" sorry %noproof
     have B sorry %noproof