diff -r 788e902f3c59 -r b8d89db3e238 doc-src/IsarImplementation/Thy/Logic.thy --- a/doc-src/IsarImplementation/Thy/Logic.thy Sun Oct 17 20:00:23 2010 +0100 +++ b/doc-src/IsarImplementation/Thy/Logic.thy Sun Oct 17 20:25:36 2010 +0100 @@ -286,7 +286,7 @@ polymorphic constants that the user-level type-checker would reject due to violation of type class restrictions. - \medskip An \emph{atomic} term is either a variable or constant. + \medskip An \emph{atomic term} is either a variable or constant. The logical category \emph{term} is defined inductively over atomic terms, with abstraction and application as follows: @{text "t = b | x\<^isub>\ | ?x\<^isub>\ | c\<^isub>\ | \\<^isub>\. t | t\<^isub>1 t\<^isub>2"}. Parsing and printing takes care of @@ -929,9 +929,9 @@ \end{tabular} \medskip - \noindent Thus we essentially impose nesting levels on propositions - formed from @{text "\"} and @{text "\"}. At each level there is a - prefix of parameters and compound premises, concluding an atomic + Thus we essentially impose nesting levels on propositions formed + from @{text "\"} and @{text "\"}. At each level there is a prefix + of parameters and compound premises, concluding an atomic proposition. Typical examples are @{text "\"}-introduction @{text "(A \ B) \ A \ B"} or mathematical induction @{text "P 0 \ (\n. P n \ P (Suc n)) \ P n"}. Even deeper nesting occurs in well-founded