doc-src/TutorialI/Rules/Blast.thy
changeset 16417 9bc16273c2d4
parent 10844 0c0e7de7e9c5
child 42637 381fdcab0f36
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     1 (* ID:         $Id$ *)
     1 (* ID:         $Id$ *)
     2 theory Blast = Main:
     2 theory Blast imports Main begin
     3 
     3 
     4 lemma "((\<exists>x. \<forall>y. p(x)=p(y)) = ((\<exists>x. q(x))=(\<forall>y. p(y))))   =    
     4 lemma "((\<exists>x. \<forall>y. p(x)=p(y)) = ((\<exists>x. q(x))=(\<forall>y. p(y))))   =    
     5        ((\<exists>x. \<forall>y. q(x)=q(y)) = ((\<exists>x. p(x))=(\<forall>y. q(y))))"
     5        ((\<exists>x. \<forall>y. q(x)=q(y)) = ((\<exists>x. p(x))=(\<forall>y. q(y))))"
     6 by blast
     6 by blast
     7 
     7