src/FOL/ex/int.thy
author wenzelm
Thu, 24 Jan 2002 22:42:14 +0100
changeset 12847 afa356dbcb15
parent 9205 f171fa6a0989
child 16417 9bc16273c2d4
permissions -rw-r--r--
fixed subgoal_tac; fails on non-existent subgoal;

(*  Title:      FOL/ex/int.thy
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1991  University of Cambridge

Intuitionistic First-Order Logic.
*)

theory int = IFOL:

end