src/HOL/Main.thy
changeset 10261 bb2f1e859177
parent 9876 a069795f1060
child 10386 581a5a143994
equal deleted inserted replaced
10260:6c31c8bb78e8 10261:bb2f1e859177
     2 (*theory Main includes everything; note that theory
     2 (*theory Main includes everything; note that theory
     3   PreList already includes most HOL theories*)
     3   PreList already includes most HOL theories*)
     4 
     4 
     5 theory Main = Map + String:
     5 theory Main = Map + String:
     6 
     6 
     7 (*actually belongs to theory List*)
     7 (*belongs to theory List*)
     8 lemmas [mono] = lists_mono
     8 declare lists_mono [mono]
     9 lemmas [recdef_cong] = map_cong
     9 declare map_cong [recdef_cong]
    10 
    10 
    11 end
    11 end