src/HOLCF/Holcfb.thy
author paulson
Thu, 18 Jan 1996 10:38:29 +0100
changeset 1444 23ceb1dc9755
parent 1274 ea0668a1c0ba
child 1479 21eb5e156d91
permissions -rw-r--r--
trivial updates

(*  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"
defs

theleast_def    "theleast P == (@z.(P z & (!n.P n --> z<=n)))"

(* start 8bit 1 *)
(* end 8bit 1 *)

end