diff -r 37a92211a5d3 -r dbb95b825244 src/HOL/PreList.thy --- a/src/HOL/PreList.thy Fri Apr 16 04:06:52 2004 +0200 +++ b/src/HOL/PreList.thy Fri Apr 16 04:07:10 2004 +0200 @@ -6,13 +6,14 @@ header{*A Basis for Building the Theory of Lists*} -(*Is defined separately to serve as a basis for theory ToyList in the -documentation.*) - theory PreList = Wellfounded_Relations + Presburger + Recdef + Relation_Power + Parity: -(*belongs to theory Wellfounded_Recursion*) +text {* + Is defined separately to serve as a basis for theory ToyList in the + documentation. *} + lemmas wf_induct_rule = wf_induct [rule_format, case_names less, induct set: wf] + -- {* belongs to theory @{text Wellfounded_Recursion} *} end