author | paulson |
Tue, 11 May 2004 10:47:15 +0200 | |
changeset 14732 | 967db86e853c |
parent 14577 | dbb95b825244 |
child 15131 | c69542757a4d |
permissions | -rw-r--r-- |
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 |
|
14430
5cb24165a2e1
new material from Avigad, and simplified treatment of division by 0
paulson
parents:
14125
diff
changeset
|
9 |
theory PreList = |
5cb24165a2e1
new material from Avigad, and simplified treatment of division by 0
paulson
parents:
14125
diff
changeset
|
10 |
Wellfounded_Relations + Presburger + Recdef + Relation_Power + Parity: |
12397 | 11 |
|
14577 | 12 |
text {* |
13 |
Is defined separately to serve as a basis for theory ToyList in the |
|
14 |
documentation. *} |
|
15 |
||
12397 | 16 |
lemmas wf_induct_rule = wf_induct [rule_format, case_names less, induct set: wf] |
14577 | 17 |
-- {* belongs to theory @{text Wellfounded_Recursion} *} |
9066 | 18 |
|
8490 | 19 |
end |