src/HOL/Main.thy
author wenzelm
Fri, 03 Nov 2000 21:27:06 +0100
changeset 10379 93630e0c5ae9
parent 10261 bb2f1e859177
child 10386 581a5a143994
permissions -rw-r--r--
improved handling of "that": insert into goal, only declare as Pure "intro"; eliminated functor;


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

end