| author | paulson |
| Thu, 14 Sep 2000 11:34:13 +0200 | |
| changeset 9955 | 6ed42bcba707 |
| parent 9619 | 6125cc9efc18 |
| child 10212 | 33fe2d701ddd |
| 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 + |
| 9619 | 12 |
SVC_Oracle + While: |
| 8490 | 13 |
|
| 9066 | 14 |
theorems [cases type: bool] = case_split |
15 |
||
| 8490 | 16 |
end |