# HG changeset patch # User wenzelm # Date 1007562996 -3600 # Node ID 2fa13b49997597aed3064b5efab5aff0a54e6192 # Parent 23bd419144ebcbae4d25488a62c2c73affb292ba adapted intr/elim uses; diff -r 23bd419144eb -r 2fa13b499975 doc-src/TutorialI/Rules/Basic.thy --- a/doc-src/TutorialI/Rules/Basic.thy Wed Dec 05 14:32:10 2001 +0100 +++ b/doc-src/TutorialI/Rules/Basic.thy Wed Dec 05 15:36:36 2001 +0100 @@ -150,7 +150,7 @@ lemma "\\(P\Q); \(R\Q)\ \ R" apply (erule_tac Q="R\Q" in contrapos_np) --{* @{subgoals[display,indent=0,margin=65]} *} -apply intro +apply (intro impI) --{* @{subgoals[display,indent=0,margin=65]} *} by (erule notE) @@ -160,7 +160,7 @@ *}; lemma "(P \ Q) \ R \ P \ Q \ R" -apply intro +apply (intro conjI disjCI) --{* @{subgoals[display,indent=0,margin=65]} *} apply (elim conjE disjE) @@ -211,7 +211,7 @@ text{*rename_tac*} lemma "x < y \ \x y. P x (f y)" -apply intro +apply (intro allI) --{* @{subgoals[display,indent=0,margin=65]} *} apply (rename_tac v w) --{* @{subgoals[display,indent=0,margin=65]} *} @@ -361,21 +361,22 @@ lemma "(\x. P x) \ (\x. Q x) \ \x. P x \ Q x" -apply elim - apply intro +apply (elim exE disjE) + apply (intro exI disjCI) apply assumption apply (intro exI disjI2) (*or else we get disjCI*) apply assumption done lemma "(P\Q) \ (Q\P)" -apply intro -apply elim +apply (intro disjCI impI) +apply (elim notE) +apply (intro impI) apply assumption done lemma "(P\Q)\(P\R) \ P \ (Q\R)" -apply intro +apply (intro disjCI conjI) apply (elim conjE disjE) apply blast apply blast diff -r 23bd419144eb -r 2fa13b499975 doc-src/TutorialI/Rules/Forward.thy --- a/doc-src/TutorialI/Rules/Forward.thy Wed Dec 05 14:32:10 2001 +0100 +++ b/doc-src/TutorialI/Rules/Forward.thy Wed Dec 05 15:36:36 2001 +0100 @@ -117,7 +117,7 @@ *} lemma "2 \ u \ u*m \ Suc(u*n)" -apply intro +apply (intro notI) txt{* before using arg_cong @{subgoals[display,indent=0,margin=65]} diff -r 23bd419144eb -r 2fa13b499975 doc-src/TutorialI/Rules/Tacticals.thy --- a/doc-src/TutorialI/Rules/Tacticals.thy Wed Dec 05 14:32:10 2001 +0100 +++ b/doc-src/TutorialI/Rules/Tacticals.thy Wed Dec 05 15:36:36 2001 +0100 @@ -17,23 +17,23 @@ text{*exercise: what's going on here?*} lemma "\P\Q\R; P\Q; P\ \ R" -by (drule mp, intro?, assumption+)+ +by (drule mp, (intro conjI)?, assumption+)+ text{*defer and prefer*} lemma "hard \ (P \ ~P) \ (Q\Q)" -apply intro --{* @{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 --{* @{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 --{* @{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... *} @@ -44,7 +44,7 @@ (*needed??*) lemma "(P\Q) \ (R\S) \ PP" -apply elim +apply (elim conjE disjE) oops lemma "((P\Q) \ R) \ (Q \ (P\S)) \ PP"