author | paulson |
Fri, 12 May 2000 15:05:02 +0200 | |
changeset 8862 | 78643f8449c6 |
parent 8840 | 18b76c137c41 |
child 9066 | b1e874e38dab |
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 = |
|
8862 | 11 |
Option + WF_Rel + NatSimprocs + Recdef + Record + RelPow + Calculation + |
12 |
SVC_Oracle: |
|
8490 | 13 |
|
14 |
end |