doc-src/TutorialI/Rules/Basic.thy
changeset 12408 2884148a9fe9
parent 12390 2fa13b499975
child 13550 5a176b8dda84
--- a/doc-src/TutorialI/Rules/Basic.thy	Thu Dec 06 13:00:25 2001 +0100
+++ b/doc-src/TutorialI/Rules/Basic.thy	Thu Dec 06 13:01:07 2001 +0100
@@ -160,7 +160,7 @@
 *};
 
 lemma "(P \<or> Q) \<and> R \<Longrightarrow> P \<or> Q \<and> R"
-apply (intro conjI disjCI)
+apply (intro disjCI conjI)
 	--{* @{subgoals[display,indent=0,margin=65]} *}
 
 apply (elim conjE disjE)
@@ -362,9 +362,9 @@
 
 lemma "(\<exists>x. P x) \<or> (\<exists>x. Q x) \<Longrightarrow> \<exists>x. P x \<or> Q x"
 apply (elim exE disjE)
- apply (intro exI disjCI)
+ apply (intro exI disjI1)
  apply assumption
-apply (intro exI disjI2) (*or else we get disjCI*)
+apply (intro exI disjI2)
 apply assumption
 done