src/HOLCF/Void.thy
author regensbu
Thu, 29 Jun 1995 16:28:40 +0200
changeset 1168 74be52691d62
parent 243 c22b85994e17
child 1479 21eb5e156d91
permissions -rw-r--r--
The curried version of HOLCF is now just called HOLCF. The old uncurried version is no longer supported

(*  Title: 	HOLCF/void.thy
    ID:         $Id$
    Author: 	Franz Regensburger
    Copyright   1993  Technische Universitaet Muenchen

Definition of type void with partial order. Void is the prototype for
all types in class 'po'

Type void  is defined as a set Void over type bool.
*)

Void = Holcfb +

types void 0

arities void :: term

consts
  Void		:: "bool set"
  UU_void_Rep	:: "bool"	
  Rep_Void	:: "void => bool"
  Abs_Void	:: "bool => void"
  UU_void	:: "void"
  less_void	:: "[void,void] => bool"	

defs

  (* The unique element in Void is False:bool *)

  UU_void_Rep_def	"UU_void_Rep == False"
  Void_def		"Void == {x. x = UU_void_Rep}"

   (*defining the abstract constants*)

  UU_void_def	"UU_void == Abs_Void(UU_void_Rep)"  
  less_void_def "less_void x y == (Rep_Void x = Rep_Void y)"  

rules

  (*faking a type definition... *)
  (* void is isomorphic to Void *)

  Rep_Void		"Rep_Void(x):Void"		
  Rep_Void_inverse	"Abs_Void(Rep_Void(x)) = x"	
  Abs_Void_inverse	"y:Void ==> Rep_Void(Abs_Void(y)) = y"

end