src/HOL/Main.thy
author berghofe
Mon, 29 Jan 2001 13:28:15 +0100
changeset 10989 87f8a7644f91
parent 10519 ade64af4c57c
child 11483 f4d10044a2cd
permissions -rw-r--r--
New function complete_split_rule for complete splitting of partially splitted rules (as generated by inductive definition package).

(*  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