| author | wenzelm | 
| Wed, 11 Oct 2006 22:55:14 +0200 | |
| changeset 20977 | dbf1eca9b34e | 
| parent 20591 | 7cbb224598b2 | 
| child 21256 | 47195501ecf7 | 
| permissions | -rw-r--r-- | 
| 10519 | 1 | (* Title: HOL/PreList.thy | 
| 8563 | 2 | ID: $Id$ | 
| 10733 | 3 | Author: Tobias Nipkow and Markus Wenzel | 
| 8563 | 4 | Copyright 2000 TU Muenchen | 
| 5 | *) | |
| 8490 | 6 | |
| 20591 | 7 | header {* A Basis for Building the Theory of Lists *}
 | 
| 12020 | 8 | |
| 15131 | 9 | theory PreList | 
| 17508 | 10 | imports Wellfounded_Relations Presburger Relation_Power Binomial | 
| 15131 | 11 | begin | 
| 12397 | 12 | |
| 14577 | 13 | text {*
 | 
| 20591 | 14 | This is defined separately to serve as a basis for | 
| 15 | theory ToyList in the documentation. | |
| 16 | *} | |
| 14577 | 17 | |
| 8490 | 18 | end |