diff -r 634cd44bb1d3 -r c49a8ebd30cc src/Doc/Implementation/Proof.thy --- a/src/Doc/Implementation/Proof.thy Thu Nov 05 00:02:30 2015 +0100 +++ b/src/Doc/Implementation/Proof.thy Thu Nov 05 00:17:13 2015 +0100 @@ -58,14 +58,14 @@ notepad begin { - fix x -- \all potential occurrences of some \x::\\ are fixed\ + fix x \ \all potential occurrences of some \x::\\ are fixed\ { - have "x::'a \ x" -- \implicit type assignment by concrete occurrence\ + have "x::'a \ x" \ \implicit type assignment by concrete occurrence\ by (rule reflexive) } - thm this -- \result still with fixed type \'a\\ + thm this \ \result still with fixed type \'a\\ } - thm this -- \fully general result for arbitrary \?x::?'a\\ + thm this \ \fully general result for arbitrary \?x::?'a\\ end text \The Isabelle/Isar proof context manages the details of term