doc-src/ZF/IFOL_examples.thy
changeset 48510 8f3069015441
parent 16417 9bc16273c2d4
equal deleted inserted replaced
48509:4854ced3e9d7 48510:8f3069015441
     1 header{*Examples of Intuitionistic Reasoning*}
     1 header{*Examples of Intuitionistic Reasoning*}
     2 
     2 
     3 theory IFOL_examples imports IFOL begin
     3 theory IFOL_examples imports "~~/src/FOL/IFOL" begin
     4 
     4 
     5 text{*Quantifier example from the book Logic and Computation*}
     5 text{*Quantifier example from the book Logic and Computation*}
     6 lemma "(EX y. ALL x. Q(x,y)) -->  (ALL x. EX y. Q(x,y))"
     6 lemma "(EX y. ALL x. Q(x,y)) -->  (ALL x. EX y. Q(x,y))"
     7   --{* @{subgoals[display,indent=0,margin=65]} *}
     7   --{* @{subgoals[display,indent=0,margin=65]} *}
     8 apply (rule impI)
     8 apply (rule impI)