diff -r e9ab4ad7bd15 -r 23307fd33906 src/Doc/Tutorial/Rules/Tacticals.thy --- a/src/Doc/Tutorial/Rules/Tacticals.thy Thu Jan 11 13:48:17 2018 +0100 +++ b/src/Doc/Tutorial/Rules/Tacticals.thy Fri Jan 12 14:08:53 2018 +0100 @@ -1,6 +1,6 @@ theory Tacticals imports Main begin -text{*REPEAT*} +text\REPEAT\ lemma "\P\Q; Q\R; R\S; P\ \ S" apply (drule mp, assumption) apply (drule mp, assumption) @@ -11,32 +11,32 @@ lemma "\P\Q; Q\R; R\S; P\ \ S" by (drule mp, assumption)+ -text{*ORELSE with REPEAT*} +text\ORELSE with REPEAT\ lemma "\Q\R; P\Q; x<5\P; Suc x < 5\ \ R" by (drule mp, (assumption|arith))+ -text{*exercise: what's going on here?*} +text\exercise: what's going on here?\ lemma "\P\Q\R; P\Q; P\ \ R" by (drule mp, (intro conjI)?, assumption+)+ -text{*defer and prefer*} +text\defer and prefer\ lemma "hard \ (P \ ~P) \ (Q\Q)" -apply (intro conjI) --{* @{subgoals[display,indent=0,margin=65]} *} -defer 1 --{* @{subgoals[display,indent=0,margin=65]} *} -apply blast+ --{* @{subgoals[display,indent=0,margin=65]} *} +apply (intro conjI) \\@{subgoals[display,indent=0,margin=65]}\ +defer 1 \\@{subgoals[display,indent=0,margin=65]}\ +apply blast+ \\@{subgoals[display,indent=0,margin=65]}\ oops lemma "ok1 \ ok2 \ doubtful" -apply (intro conjI) --{* @{subgoals[display,indent=0,margin=65]} *} -prefer 3 --{* @{subgoals[display,indent=0,margin=65]} *} +apply (intro conjI) \\@{subgoals[display,indent=0,margin=65]}\ +prefer 3 \\@{subgoals[display,indent=0,margin=65]}\ oops lemma "bigsubgoal1 \ bigsubgoal2 \ bigsubgoal3 \ bigsubgoal4 \ bigsubgoal5 \ bigsubgoal6" -apply (intro conjI) --{* @{subgoals[display,indent=0,margin=65]} *} -txt{* @{subgoals[display,indent=0,margin=65]} +apply (intro conjI) \\@{subgoals[display,indent=0,margin=65]}\ +txt\@{subgoals[display,indent=0,margin=65]} A total of 6 subgoals... -*} +\ oops