doc-src/TutorialI/Rules/Force.thy
changeset 10341 6eb91805a012
parent 10295 8eb12693cead
child 11407 138919f1a135
equal deleted inserted replaced
10340:0a380ac80e7d 10341:6eb91805a012
       
     1 (* ID:         $Id$ *)
     1 theory Force = Main:
     2 theory Force = Main:
     2 
     3 
     3 
     4 
     4 
     5 
     5 lemma "(\<forall>x. P x) \<and> (\<exists>x. Q x) \<longrightarrow> (\<forall>x. P x \<and> Q x)"
     6 lemma "(\<forall>x. P x) \<and> (\<exists>x. Q x) \<longrightarrow> (\<forall>x. P x \<and> Q x)"