text cleanup
authorhaftmann
Tue, 19 Sep 2006 15:21:48 +0200
changeset 20591 7cbb224598b2
parent 20590 bf92900995f8
child 20592 527563e67194
text cleanup
src/HOL/PreList.thy
--- a/src/HOL/PreList.thy	Tue Sep 19 15:21:44 2006 +0200
+++ b/src/HOL/PreList.thy	Tue Sep 19 15:21:48 2006 +0200
@@ -4,14 +4,15 @@
     Copyright   2000 TU Muenchen
 *)
 
-header{*A Basis for Building the Theory of Lists*}
+header {* A Basis for Building the Theory of Lists *}
 
 theory PreList
 imports Wellfounded_Relations Presburger Relation_Power Binomial
 begin
 
 text {*
-  Is defined separately to serve as a basis for theory ToyList in the
-  documentation. *}
+  This is defined separately to serve as a basis for
+  theory ToyList in the documentation.
+*}
 
 end