changeset 16417 | 9bc16273c2d4 |
parent 10844 | 0c0e7de7e9c5 |
child 42637 | 381fdcab0f36 |
--- a/doc-src/TutorialI/Rules/Blast.thy Fri Jun 17 11:35:35 2005 +0200 +++ b/doc-src/TutorialI/Rules/Blast.thy Fri Jun 17 16:12:49 2005 +0200 @@ -1,5 +1,5 @@ (* ID: $Id$ *) -theory Blast = Main: +theory Blast imports Main begin lemma "((\<exists>x. \<forall>y. p(x)=p(y)) = ((\<exists>x. q(x))=(\<forall>y. p(y)))) = ((\<exists>x. \<forall>y. q(x)=q(y)) = ((\<exists>x. p(x))=(\<forall>y. q(y))))"