| author | paulson | 
| Wed, 14 Feb 2001 13:01:02 +0100 | |
| changeset 11117 | 55358999077d | 
| parent 10519 | ade64af4c57c | 
| child 11483 | f4d10044a2cd | 
| permissions | -rw-r--r-- | 
(* Title: HOL/Main.thy ID: $Id$ Author: Tobias Nipkow Copyright 2000 TU Muenchen Theory Main includes everything. Note that theory PreList already includes most HOL theories. *) theory Main = Map + String: (*belongs to theory List*) declare lists_mono [mono] declare map_cong [recdef_cong] lemmas rev_induct [case_names Nil snoc] = rev_induct and rev_cases [case_names Nil snoc] = rev_exhaust end