src/HOL/Library/Coinductive_List.thy
changeset 27368 9f90ac19e32b
parent 25595 6c48275f9c76
child 27487 c8a6ce181805
equal deleted inserted replaced
27367:a75d71c73362 27368:9f90ac19e32b
     4 *)
     4 *)
     5 
     5 
     6 header {* Potentially infinite lists as greatest fixed-point *}
     6 header {* Potentially infinite lists as greatest fixed-point *}
     7 
     7 
     8 theory Coinductive_List
     8 theory Coinductive_List
     9 imports List
     9 imports Plain List
    10 begin
    10 begin
    11 
    11 
    12 subsection {* List constructors over the datatype universe *}
    12 subsection {* List constructors over the datatype universe *}
    13 
    13 
    14 definition "NIL = Datatype.In0 (Datatype.Numb 0)"
    14 definition "NIL = Datatype.In0 (Datatype.Numb 0)"