src/FOL/ex/int.thy
author ballarin
Tue, 02 Aug 2005 16:52:21 +0200
changeset 17000 552df70f52c2
parent 16417 9bc16273c2d4
permissions -rw-r--r--
First version of interpretation in locales. Not yet fully functional.

(*  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 imports IFOL begin

end