| author | nipkow | 
| Fri, 24 Nov 2000 16:49:27 +0100 | |
| changeset 10519 | ade64af4c57c | 
| parent 10386 | 581a5a143994 | 
| child 11483 | f4d10044a2cd | 
| permissions | -rw-r--r-- | 
| 10519 | 1 | (* Title: HOL/Main.thy | 
| 2 | ID: $Id$ | |
| 3 | Author: Tobias Nipkow | |
| 4 | Copyright 2000 TU Muenchen | |
| 9619 | 5 | |
| 10519 | 6 | Theory Main includes everything. | 
| 7 | Note that theory PreList already includes most HOL theories. | |
| 8 | *) | |
| 9619 | 9 | |
| 9650 
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
 wenzelm parents: 
9619diff
changeset | 10 | theory Main = Map + String: | 
| 
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
 wenzelm parents: 
9619diff
changeset | 11 | |
| 10261 | 12 | (*belongs to theory List*) | 
| 13 | declare lists_mono [mono] | |
| 14 | declare map_cong [recdef_cong] | |
| 10386 | 15 | lemmas rev_induct [case_names Nil snoc] = rev_induct | 
| 16 | and rev_cases [case_names Nil snoc] = rev_exhaust | |
| 9768 | 17 | |
| 9650 
6f0b89f2a1f9
Main now new-style theory; added Main.ML for compatibility;
 wenzelm parents: 
9619diff
changeset | 18 | end |