changeset 15131 | c69542757a4d |
parent 14577 | dbb95b825244 |
child 15140 | 322485b816ac |
--- a/src/HOL/PreList.thy Mon Aug 16 14:21:54 2004 +0200 +++ b/src/HOL/PreList.thy Mon Aug 16 14:22:27 2004 +0200 @@ -6,8 +6,9 @@ header{*A Basis for Building the Theory of Lists*} -theory PreList = - Wellfounded_Relations + Presburger + Recdef + Relation_Power + Parity: +theory PreList +import Wellfounded_Relations Presburger Recdef Relation_Power Parity +begin text {* Is defined separately to serve as a basis for theory ToyList in the