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 |
|
14125
|
7 |
header{*A Basis for Building the Theory of Lists*}
|
12020
|
8 |
|
15131
|
9 |
theory PreList
|
15298
|
10 |
imports Wellfounded_Relations Presburger Recdef Relation_Power Parity
|
15131
|
11 |
begin
|
12397
|
12 |
|
14577
|
13 |
text {*
|
|
14 |
Is defined separately to serve as a basis for theory ToyList in the
|
|
15 |
documentation. *}
|
|
16 |
|
12397
|
17 |
lemmas wf_induct_rule = wf_induct [rule_format, case_names less, induct set: wf]
|
14577
|
18 |
-- {* belongs to theory @{text Wellfounded_Recursion} *}
|
9066
|
19 |
|
8490
|
20 |
end
|