src/ZF/OrdQuant.thy
changeset 13174 85d3c0981a16
parent 13172 03a5afa7b888
child 13175 81082cfa5618
--- a/src/ZF/OrdQuant.thy	Wed May 22 18:55:47 2002 +0200
+++ b/src/ZF/OrdQuant.thy	Wed May 22 19:34:01 2002 +0200
@@ -60,10 +60,6 @@
 
 (** Now some very basic ZF theorems **)
 
-(*FIXME: move to ZF.thy or even to FOL.thy??*)
-lemma [simp]: "((P-->Q) <-> (P-->R)) <-> (P --> (Q<->R))"
-by blast
-
 (*FIXME: move to Rel.thy*)
 lemma trans_imp_trans_on: "trans(r) ==> trans[A](r)"
 by (unfold trans_def trans_on_def, blast)