removed obsolete cla_dist_concl;
authorwenzelm
Sat, 31 Dec 2005 21:49:39 +0100
changeset 18531 ce7b80b7c84e
parent 18530 d995aecddc15
child 18532 0347c1bba406
removed obsolete cla_dist_concl;
src/FOL/FOL.thy
src/HOL/HOL.thy
--- a/src/FOL/FOL.thy	Sat Dec 31 21:49:38 2005 +0100
+++ b/src/FOL/FOL.thy	Sat Dec 31 21:49:39 2005 +0100
@@ -24,15 +24,6 @@
 use "FOL_lemmas1.ML"
 theorems case_split = case_split_thm [case_names True False, cases type: o]
 
-lemma cla_dist_concl:
-  assumes x: "~Z_Z ==> PROP X_X"
-    and z: "PROP Y_Y ==> Z_Z"
-    and y: "PROP X_X ==> PROP Y_Y"
-  shows Z_Z
-  apply (rule classical)
-  apply (erule x [THEN y, THEN z])
-  done
-
 use "cladata.ML"
 setup Cla.setup
 setup cla_setup
--- a/src/HOL/HOL.thy	Sat Dec 31 21:49:38 2005 +0100
+++ b/src/HOL/HOL.thy	Sat Dec 31 21:49:39 2005 +0100
@@ -909,15 +909,6 @@
 
 subsubsection {* Classical Reasoner setup *}
 
-lemma cla_dist_concl:
-  assumes x: "~Z_Z ==> PROP X_X"
-    and z: "PROP Y_Y ==> Z_Z"
-    and y: "PROP X_X ==> PROP Y_Y"
-  shows Z_Z
-  apply (rule classical)
-  apply (erule x [THEN y, THEN z])
-  done
-
 use "cladata.ML"
 setup hypsubst_setup