diff -r 23a8c5ac35f8 -r 69916a850301 doc-src/TutorialI/Rules/Basic.thy --- a/doc-src/TutorialI/Rules/Basic.thy Sat Oct 17 01:05:59 2009 +0200 +++ b/doc-src/TutorialI/Rules/Basic.thy Sat Oct 17 14:43:18 2009 +0200 @@ -1,4 +1,3 @@ -(* ID: $Id$ *) theory Basic imports Main begin lemma conj_rule: "\ P; Q \ \ P \ (Q \ P)" @@ -149,9 +148,9 @@ lemma "\\(P\Q); \(R\Q)\ \ R" apply (erule_tac Q="R\Q" in contrapos_np) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply (intro impI) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} by (erule notE) text {* @@ -161,11 +160,11 @@ lemma "(P \ Q) \ R \ P \ Q \ R" apply (intro disjCI conjI) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply (elim conjE disjE) apply assumption - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} by (erule contrapos_np, rule conjI) text{* @@ -241,18 +240,18 @@ text{*rename_tac*} lemma "x < y \ \x y. P x (f y)" apply (intro allI) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply (rename_tac v w) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} oops lemma "\\x. P x \ P (h x); P a\ \ P(h (h a))" apply (frule spec) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply (drule mp, assumption) apply (drule spec) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} by (drule mp) lemma "\\x. P x \ P (f x); P a\ \ P(f (f a))" @@ -276,11 +275,11 @@ lemma "\\x. P x \ P (h x); P a\ \ P(h (h a))" apply (frule spec) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply (drule mp, assumption) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply (drule_tac x = "h a" in spec) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} by (drule mp) text {* @@ -290,15 +289,15 @@ lemma mult_dvd_mono: "\i dvd m; j dvd n\ \ i*j dvd (m*n :: nat)" apply (simp add: dvd_def) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply (erule exE) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply (erule exE) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply (rename_tac l) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply (rule_tac x="k*l" in exI) - --{* @{subgoals[display,indent=0,margin=65]} *} + --{* @{subgoals[display,indent=0,margin=65]} *} apply simp done