diff -r ee42cba50933 -r e0825405d398 src/Doc/Isar_Ref/First_Order_Logic.thy --- a/src/Doc/Isar_Ref/First_Order_Logic.thy Mon Oct 12 21:42:14 2015 +0200 +++ b/src/Doc/Isar_Ref/First_Order_Logic.thy Mon Oct 12 22:03:24 2015 +0200 @@ -231,7 +231,8 @@ ``@{text "\ A \ B \ A \ B"}'' coincides with the original axiomatization of @{thm disjE}. - \medskip We continue propositional logic by introducing absurdity + \<^medskip> + We continue propositional logic by introducing absurdity with its characteristic elimination. Plain truth may then be defined as a proposition that is trivially true. \ @@ -248,8 +249,8 @@ unfolding true_def .. text \ - \medskip Now negation represents an implication towards - absurdity: + \<^medskip> + Now negation represents an implication towards absurdity: \ definition @@ -374,7 +375,7 @@ can now be summarized as follows, using the native Isar statement format of \secref{sec:framework-stmt}. - \medskip + \<^medskip> \begin{tabular}{l} @{text "impI: \ A \ B \ A \ B"} \\ @{text "impD: \ A \ B \ A \ B"} \\[1ex] @@ -398,7 +399,7 @@ @{text "exI: \ B a \ \x. B x"} \\ @{text "exE: \ \x. B x \ a \ B a"} \end{tabular} - \medskip + \<^medskip> This essentially provides a declarative reading of Pure rules as Isar reasoning patterns: the rule statements tells how a @@ -511,7 +512,8 @@ (*>*) text \ - \bigskip Of course, these proofs are merely examples. As + \<^bigskip> + Of course, these proofs are merely examples. As sketched in \secref{sec:framework-subproof}, there is a fair amount of flexibility in expressing Pure deductions in Isar. Here the user is asked to express himself adequately, aiming at proof texts of