src/HOL/PreList.thy
changeset 14125 bf8edef6c1f1
parent 13878 90ca3815e4b2
child 14430 5cb24165a2e1
--- a/src/HOL/PreList.thy	Tue Jul 22 11:05:02 2003 +0200
+++ b/src/HOL/PreList.thy	Thu Jul 24 16:35:51 2003 +0200
@@ -2,19 +2,14 @@
     ID:         $Id$
     Author:     Tobias Nipkow and Markus Wenzel
     Copyright   2000 TU Muenchen
-
-A basis for building theory List on. Is defined separately to serve as a
-basis for theory ToyList in the documentation.
 *)
 
-theory PreList =
-  Wellfounded_Relations + Presburger + Recdef + Relation_Power:
+header{*A Basis for Building the Theory of Lists*}
 
-(*belongs to theory Divides*)
-declare dvdI [intro?]  dvdE [elim?]  dvd_trans [trans]
+(*Is defined separately to serve as a basis for theory ToyList in the
+documentation.*)
 
-(*belongs to theory Nat*)
-lemmas less_induct = nat_less_induct [rule_format, case_names less]
+theory PreList = Wellfounded_Relations + Presburger + Recdef + Relation_Power:
 
 (*belongs to theory Wellfounded_Recursion*)
 lemmas wf_induct_rule = wf_induct [rule_format, case_names less, induct set: wf]