src/CTT/bool.thy
changeset 13894 8018173a7979
parent 13893 19849d258890
child 13895 b6105462ccd3
--- a/src/CTT/bool.thy	Sat Apr 05 16:00:00 2003 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,19 +0,0 @@
-(*  Title: 	CTT/bool
-    ID:         $Id$
-    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
-    Copyright   1991  University of Cambridge
-
-The two-element type (booleans and conditionals)
-*)
-
-Bool = CTT +
-
-consts Bool		:: "t"
-       true,false	:: "i"
-       cond		:: "[i,i,i]=>i"
-rules
-  Bool_def	"Bool == T+T"
-  true_def	"true == inl(tt)"
-  false_def	"false == inr(tt)"
-  cond_def	"cond(a,b,c) == when(a, %u.b, %u.c)"
-end