diff -r e4c5c7ffceea -r fee67c099d03 doc-src/IsarImplementation/Thy/Logic.thy --- a/doc-src/IsarImplementation/Thy/Logic.thy Tue May 03 21:40:14 2011 +0200 +++ b/doc-src/IsarImplementation/Thy/Logic.thy Tue May 03 21:44:05 2011 +0200 @@ -517,14 +517,14 @@ \infer[@{text "(assume)"}]{@{text "A \ A"}}{} \] \[ - \infer[@{text "(\\intro)"}]{@{text "\ \ \x. b[x]"}}{@{text "\ \ b[x]"} & @{text "x \ \"}} + \infer[@{text "(\\intro)"}]{@{text "\ \ \x. b[x]"}}{@{text "\ \ b[x]"} & @{text "x \ \"}} \qquad - \infer[@{text "(\\elim)"}]{@{text "\ \ b[a]"}}{@{text "\ \ \x. b[x]"}} + \infer[@{text "(\\elim)"}]{@{text "\ \ b[a]"}}{@{text "\ \ \x. b[x]"}} \] \[ - \infer[@{text "(\\intro)"}]{@{text "\ - A \ A \ B"}}{@{text "\ \ B"}} + \infer[@{text "(\\intro)"}]{@{text "\ - A \ A \ B"}}{@{text "\ \ B"}} \qquad - \infer[@{text "(\\elim)"}]{@{text "\\<^sub>1 \ \\<^sub>2 \ B"}}{@{text "\\<^sub>1 \ A \ B"} & @{text "\\<^sub>2 \ A"}} + \infer[@{text "(\\elim)"}]{@{text "\\<^sub>1 \ \\<^sub>2 \ B"}}{@{text "\\<^sub>1 \ A \ B"} & @{text "\\<^sub>2 \ A"}} \] \caption{Primitive inferences of Pure}\label{fig:prim-rules} \end{center} @@ -554,7 +554,7 @@ \cite{Berghofer-Nipkow:2000:TPHOL}). Observe that locally fixed parameters (as in @{text - "\\intro"}) need not be recorded in the hypotheses, because + "\\intro"}) need not be recorded in the hypotheses, because the simple syntactic types of Pure are always inhabitable. ``Assumptions'' @{text "x :: \"} for type-membership are only present as long as some @{text "x\<^isub>\"} occurs in the statement