src/HOLCF/Lift2.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

Lift2 = Lift1 + 

default term

arities "lift" :: (term)po

rules

 inst_lift_po   "((op <<)::['a lift,'a lift]=>bool) = less_lift"

end