src/HOLCF/holcfb.thy
changeset 13897 f62f9a75f685
parent 13896 717bd79b976f
child 13898 9410d2eb9563
--- a/src/HOLCF/holcfb.thy	Sat Apr 05 17:03:38 2003 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,25 +0,0 @@
-(*  Title: 	HOLCF/holcfb.thy
-    ID:         $Id$
-    Author: 	Franz Regensburger
-    Copyright   1993  Technische Universitaet Muenchen
-
-Basic definitions for the embedding of LCF into HOL.
-
-*)
-
-Holcfb = Nat + 
-
-consts
-
-theleast     :: "(nat=>bool)=>nat"
-
-rules
-
-theleast_def    "theleast(P) == (@z.(P(z) & (!n.P(n)-->z<=n)))"
-
-end
-
-
-
-
-