diff -r 77e3ffb5aeb3 -r 4cfe65cfd369 src/Doc/Isar_Ref/First_Order_Logic.thy --- a/src/Doc/Isar_Ref/First_Order_Logic.thy Sun Feb 07 19:33:42 2016 +0100 +++ b/src/Doc/Isar_Ref/First_Order_Logic.thy Sun Feb 07 19:43:40 2016 +0100 @@ -418,47 +418,47 @@ have "A \ B" proof assume A - show B sorry %noproof + show B \ qed text_raw \\end{minipage}\qquad\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) - have "A \ B" and A sorry %noproof + have "A \ B" and A \ then have B .. text_raw \\end{minipage}\\[3ex]\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) - have A sorry %noproof + have A \ then have "A \ B" .. - have B sorry %noproof + have B \ then have "A \ B" .. text_raw \\end{minipage}\qquad\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) - have "A \ B" sorry %noproof + have "A \ B" \ then have C proof assume A - then show C sorry %noproof + then show C \ next assume B - then show C sorry %noproof + then show C \ qed text_raw \\end{minipage}\\[3ex]\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) - have A and B sorry %noproof + have A and B \ then have "A \ B" .. text_raw \\end{minipage}\qquad\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) - have "A \ B" sorry %noproof + have "A \ B" \ then obtain A and B .. text_raw \\end{minipage}\\[3ex]\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) - have "\" sorry %noproof + have "\" \ then have A .. text_raw \\end{minipage}\qquad\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) @@ -470,12 +470,12 @@ have "\ A" proof assume A - then show "\" sorry %noproof + then show "\" \ qed text_raw \\end{minipage}\qquad\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) - have "\ A" and A sorry %noproof + have "\ A" and A \ then have B .. text_raw \\end{minipage}\\[3ex]\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) @@ -483,24 +483,24 @@ have "\x. B x" proof fix x - show "B x" sorry %noproof + show "B x" \ qed text_raw \\end{minipage}\qquad\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) - have "\x. B x" sorry %noproof + have "\x. B x" \ then have "B a" .. text_raw \\end{minipage}\\[3ex]\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) have "\x. B x" proof - show "B a" sorry %noproof + show "B a" \ qed text_raw \\end{minipage}\qquad\begin{minipage}[t]{0.4\textwidth}\(*<*)next(*>*) - have "\x. B x" sorry %noproof + have "\x. B x" \ then obtain a where "B a" .. text_raw \\end{minipage}\