src/HOL/HOL.thy
changeset 80948 572970d15ab0
parent 80934 8e72f55295fd
child 81092 c92efbf32bfe
--- a/src/HOL/HOL.thy	Tue Sep 24 21:41:01 2024 +0200
+++ b/src/HOL/HOL.thy	Thu Sep 26 14:44:37 2024 +0100
@@ -633,6 +633,11 @@
   shows R
   using assms by (elim impCE)
 
+text \<open>The analogous introduction rule for conjunction, above, is even constructive\<close>
+lemma context_disjE:
+  assumes major: "P \<or> Q" and minor: "P \<Longrightarrow> R" "\<not>P \<Longrightarrow> Q \<Longrightarrow> R"
+  shows R
+  by (iprover intro: disjE [OF major] disjE [OF excluded_middle] assms)
 
 text \<open>Classical \<open>\<longleftrightarrow>\<close> elimination.\<close>
 lemma iffCE: