src/LCF/LCF.thy
changeset 41310 65631ca437c9
parent 36452 d37c6eed8117
child 47025 b2b8ae61d6ad
equal deleted inserted replaced
41309:2e9bf718a7a1 41310:65631ca437c9
    16 classes cpo < "term"
    16 classes cpo < "term"
    17 default_sort cpo
    17 default_sort cpo
    18 
    18 
    19 typedecl tr
    19 typedecl tr
    20 typedecl void
    20 typedecl void
    21 typedecl ('a,'b) "*"    (infixl "*" 6)
    21 typedecl ('a,'b) prod  (infixl "*" 6)
    22 typedecl ('a,'b) "+"    (infixl "+" 5)
    22 typedecl ('a,'b) sum  (infixl "+" 5)
    23 
    23 
    24 arities
    24 arities
    25   "fun" :: (cpo, cpo) cpo
    25   "fun" :: (cpo, cpo) cpo
    26   "*" :: (cpo, cpo) cpo
    26   prod :: (cpo, cpo) cpo
    27   "+" :: (cpo, cpo) cpo
    27   sum :: (cpo, cpo) cpo
    28   tr :: cpo
    28   tr :: cpo
    29   void :: cpo
    29   void :: cpo
    30 
    30 
    31 consts
    31 consts
    32  UU     :: "'a"
    32  UU     :: "'a"