src/FOL/ex/Intuitionistic.thy
changeset 31974 e81979a703a4
parent 16417 9bc16273c2d4
child 51798 ad3a241def73
equal deleted inserted replaced
31973:a89f758dba5b 31974:e81979a703a4
     1 (*  Title:      FOL/ex/Intuitionistic
     1 (*  Title:      FOL/ex/Intuitionistic.thy
     2     ID:         $Id$
       
     3     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     2     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     4     Copyright   1991  University of Cambridge
     3     Copyright   1991  University of Cambridge
     5 *)
     4 *)
     6 
     5 
     7 header{*Intuitionistic First-Order Logic*}
     6 header {* Intuitionistic First-Order Logic *}
     8 
     7 
     9 theory Intuitionistic imports IFOL begin
     8 theory Intuitionistic
       
     9 imports IFOL
       
    10 begin
    10 
    11 
    11 (*
    12 (*
    12 Single-step ML commands:
    13 Single-step ML commands:
    13 by (IntPr.step_tac 1)
    14 by (IntPr.step_tac 1)
    14 by (biresolve_tac safe_brls 1);
    15 by (biresolve_tac safe_brls 1);
   420 lemma "ALL x. P(x,f(x)) <-> (EX y. (ALL z. P(z,y) --> P(z,f(x))) & P(x,y))"
   421 lemma "ALL x. P(x,f(x)) <-> (EX y. (ALL z. P(z,y) --> P(z,f(x))) & P(x,y))"
   421 by (tactic{*IntPr.fast_tac 1*})
   422 by (tactic{*IntPr.fast_tac 1*})
   422 
   423 
   423 end
   424 end
   424 
   425 
   425