| author | wenzelm |
| Sat, 01 Apr 2000 20:21:39 +0200 | |
| changeset 8657 | b9475dad85ed |
| parent 8563 | 2746bc9a7ef2 |
| child 8756 | b03a0b219139 |
| permissions | -rw-r--r-- |
| 8563 | 1 |
(* Title: HOL/List.thy |
2 |
ID: $Id$ |
|
3 |
Author: Tobias Nipkow |
|
4 |
Copyright 2000 TU Muenchen |
|
5 |
||
6 |
A basis for building theory List on. Is defined separately to serve as a |
|
7 |
basis for theory ToyList in the documentation. |
|
8 |
*) |
|
| 8490 | 9 |
|
10 |
theory PreList = |
|
| 8563 | 11 |
Option + WF_Rel + NatBin + Recdef + Record + RelPow + Sexp + Calculation |
12 |
+ SVC_Oracle: |
|
| 8490 | 13 |
|
14 |
end |