src/FOL/ex/Classical.thy
changeset 42789 3a84b6947932
parent 36319 8feb2c4bef1a
child 51717 9e7d1c139569
equal deleted inserted replaced
42788:9984232a0c68 42789:3a84b6947932
   434     (\<exists>v. C(v) &                                                        
   434     (\<exists>v. C(v) &                                                        
   435           (\<forall>y. ((C(y) & Q(w,y,y)) & OO(w,g) --> ~P(v,y)) &            
   435           (\<forall>y. ((C(y) & Q(w,y,y)) & OO(w,g) --> ~P(v,y)) &            
   436                   ((C(y) & Q(w,y,y)) & OO(w,b) --> P(v,y) & OO(v,b)))))  
   436                   ((C(y) & Q(w,y,y)) & OO(w,b) --> P(v,y) & OO(v,b)))))  
   437    -->                   
   437    -->                   
   438    ~ (\<exists>x. A(x) & (\<forall>y. C(y) --> (\<forall>z. D(x,y,z))))"
   438    ~ (\<exists>x. A(x) & (\<forall>y. C(y) --> (\<forall>z. D(x,y,z))))"
   439 by (tactic{*Blast.depth_tac @{claset} 12 1*})
   439 by (blast 12)
   440    --{*Needed because the search for depths below 12 is very slow*}
   440    --{*Needed because the search for depths below 12 is very slow*}
   441 
   441 
   442 
   442 
   443 text{*Halting problem II: credited to M. Bruschi by Li Dafa in JAR 18(1), p.105*}
   443 text{*Halting problem II: credited to M. Bruschi by Li Dafa in JAR 18(1), p.105*}
   444 lemma "((\<exists>x. A(x) & (\<forall>y. C(y) --> (\<forall>z. D(x,y,z)))) -->        
   444 lemma "((\<exists>x. A(x) & (\<forall>y. C(y) --> (\<forall>z. D(x,y,z)))) -->