src/HOLCF/Lift1.thy
author sandnerr
Mon, 09 Dec 1996 19:16:20 +0100
changeset 2356 125260ef480c
child 2357 dd2e5e655fd2
permissions -rw-r--r--
Theories Lift1, Lift2 and Lift3 inserted below HOLCF.thy

Lift1 = Tr2 + 

default term

datatype 'a lift  = Undef | Def('a)

arities "lift" :: (term)term

consts less_lift    :: "['a lift, 'a lift] => bool"
       UU_lift      :: "'a lift"

defs 
 
 less_lift_def  "less_lift x y == (x=y | x=Undef)"


end