diff -r 9c50eb3bff50 -r ddb3ac3fef45 src/Doc/Implementation/Logic.thy --- a/src/Doc/Implementation/Logic.thy Wed Nov 04 18:14:28 2015 +0100 +++ b/src/Doc/Implementation/Logic.thy Wed Nov 04 18:32:47 2015 +0100 @@ -19,11 +19,11 @@ Derivations are relative to a logical theory, which declares type constructors, constants, and axioms. Theory declarations support schematic polymorphism, which is strictly speaking outside the - logic.\footnote{This is the deeper logical reason, why the theory + logic.\<^footnote>\This is the deeper logical reason, why the theory context \\\ is separate from the proof context \\\ of the core calculus: type constructors, term constants, and facts (proof constants) may involve arbitrary type schemes, but the type - of a locally fixed term parameter is also fixed!} + of a locally fixed term parameter is also fixed!\ \ @@ -531,9 +531,9 @@ the simple syntactic types of Pure are always inhabitable. ``Assumptions'' \x :: \\ for type-membership are only present as long as some \x\<^sub>\\ occurs in the statement - body.\footnote{This is the key difference to ``\\HOL\'' in + body.\<^footnote>\This is the key difference to ``\\HOL\'' in the PTS framework @{cite "Barendregt-Geuvers:2001"}, where hypotheses - \x : A\ are treated uniformly for propositions and types.} + \x : A\ are treated uniformly for propositions and types.\ \<^medskip> The axiomatization of a theory is implicitly closed by