src/HOL/List.thy
changeset 58916 229765cc3414
parent 58889 5b7a9633cfa8
child 58956 a816aa3ff391
equal deleted inserted replaced
58915:7d673ab6a8d9 58916:229765cc3414
     3 *)
     3 *)
     4 
     4 
     5 section {* The datatype of finite lists *}
     5 section {* The datatype of finite lists *}
     6 
     6 
     7 theory List
     7 theory List
     8 imports Sledgehammer Code_Numeral Lifting_Set Lifting_Option Lifting_Product
     8 imports Sledgehammer Code_Numeral Lifting_Set
     9 begin
     9 begin
    10 
    10 
    11 datatype (set: 'a) list =
    11 datatype (set: 'a) list =
    12     Nil  ("[]")
    12     Nil  ("[]")
    13   | Cons (hd: 'a) (tl: "'a list")  (infixr "#" 65)
    13   | Cons (hd: 'a) (tl: "'a list")  (infixr "#" 65)