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 |
|
|
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 =
|
12919
|
11 |
Wellfounded_Relations + NatSimprocs + Recdef + Relation_Power:
|
12020
|
12 |
|
|
13 |
(*belongs to theory Divides*)
|
12304
|
14 |
declare dvdI [intro?] dvdE [elim?] dvd_trans [trans]
|
8490
|
15 |
|
12397
|
16 |
(*belongs to theory Nat*)
|
|
17 |
lemmas less_induct = nat_less_induct [rule_format, case_names less]
|
|
18 |
|
10261
|
19 |
(*belongs to theory Wellfounded_Recursion*)
|
12397
|
20 |
lemmas wf_induct_rule = wf_induct [rule_format, case_names less, induct set: wf]
|
9066
|
21 |
|
8490
|
22 |
end
|