src/HOL/PreList.thy
changeset 16760 5c5f051aaaaa
parent 15298 a5bea99352d6
child 17042 da5cfaa258f7
equal deleted inserted replaced
16759:668e72b1c4d7 16760:5c5f051aaaaa
     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 Presburger Recdef Relation_Power Parity
    10 imports Wellfounded_Relations Presburger Relation_Power GCD
    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. *}