src/ZF/ex/LList.thy
changeset 11354 9b80fe19407f
parent 11316 b4e71bd751e4
child 12867 5c900a821a7c
equal deleted inserted replaced
11353:7f6eff7bc97a 11354:9b80fe19407f
    12 STILL NEEDS:
    12 STILL NEEDS:
    13 co_recursion for defining lconst, flip, etc.
    13 co_recursion for defining lconst, flip, etc.
    14 a typing rule for it, based on some notion of "productivity..."
    14 a typing rule for it, based on some notion of "productivity..."
    15 *)
    15 *)
    16 
    16 
    17 LList = Datatype +
    17 LList = Main +
    18 
    18 
    19 consts
    19 consts
    20   llist  :: i=>i
    20   llist  :: i=>i
    21 
    21 
    22 codatatype
    22 codatatype