src/HOL/PreList.thy
changeset 15298 a5bea99352d6
parent 15231 96d5b6e2b6e4
child 16760 5c5f051aaaaa
equal deleted inserted replaced
15297:0aff5d912422 15298:a5bea99352d6
     5 *)
     5 *)
     6 
     6 
     7 header{*A Basis for Building the Theory of Lists*}
     7 header{*A Basis for Building the Theory of Lists*}
     8 
     8 
     9 theory PreList
     9 theory PreList
    10 imports Wellfounded_Relations Barith Recdef Relation_Power Parity
    10 imports Wellfounded_Relations Presburger Recdef Relation_Power Parity
    11 begin
    11 begin
    12 
    12 
    13 text {*
    13 text {*
    14   Is defined separately to serve as a basis for theory ToyList in the
    14   Is defined separately to serve as a basis for theory ToyList in the
    15   documentation. *}
    15   documentation. *}