diff -r ad91cf279f06 -r e4dc78f4e51e doc-src/TutorialI/IsarOverview/Isar/Logic.thy --- a/doc-src/TutorialI/IsarOverview/Isar/Logic.thy Mon Jul 08 15:01:58 2002 +0200 +++ b/doc-src/TutorialI/IsarOverview/Isar/Logic.thy Mon Jul 08 15:03:04 2002 +0200 @@ -699,10 +699,10 @@ thus "(x,z) \ r*" . next fix x' x y - assume step: "(x',x) \ r" and + assume 1: "(x',x) \ r" and IH: "(y,z) \ r* \ (x,z) \ r*" and B: "(y,z) \ r*" - from step IH[OF B] show "(x',z) \ r*" by(rule rtc.step) + from 1 IH[OF B] show "(x',z) \ r*" by(rule rtc.step) qed qed