src/ZF/ex/LList.thy
changeset 1155 928a16e02f9f
parent 810 91c68f74f458
child 1401 0c439768f45c
equal deleted inserted replaced
1154:bc295e3dc078 1155:928a16e02f9f
    47   lconst_def  "lconst(a) == lfp(univ(a), %l. LCons(a,l))"
    47   lconst_def  "lconst(a) == lfp(univ(a), %l. LCons(a,l))"
    48 
    48 
    49 rules
    49 rules
    50   flip_LNil   "flip(LNil) = LNil"
    50   flip_LNil   "flip(LNil) = LNil"
    51 
    51 
    52   flip_LCons  "[| x:bool; l: llist(bool) |] ==> \
    52   flip_LCons  "[| x:bool; l: llist(bool) |] ==> 
    53 \              flip(LCons(x,l)) = LCons(not(x), flip(l))"
    53               flip(LCons(x,l)) = LCons(not(x), flip(l))"
    54 
    54 
    55 end
    55 end
    56 
    56