src/HOLCF/Lift3.thy
changeset 10834 a7897aebbffc
parent 3034 9c44acc3c6fa
equal deleted inserted replaced
10833:c0844a30ea4e 10834:a7897aebbffc
    27  flift2_def
    27  flift2_def
    28   "flift2 f == (LAM x. (case x of 
    28   "flift2 f == (LAM x. (case x of 
    29                    Undef => UU
    29                    Undef => UU
    30                  | Def y => Def (f y)))"
    30                  | Def y => Def (f y)))"
    31  liftpair_def
    31  liftpair_def
    32   "liftpair x  == (case (cfst`x) of 
    32   "liftpair x  == (case (cfst$x) of 
    33                   Undef  => UU
    33                   Undef  => UU
    34                 | Def x1 => (case (csnd`x) of 
    34                 | Def x1 => (case (csnd$x) of 
    35                                Undef => UU
    35                                Undef => UU
    36                              | Def x2 => Def (x1,x2)))"
    36                              | Def x2 => Def (x1,x2)))"
    37 
    37 
    38 end
    38 end
    39 
    39