src/HOL/MicroJava/Comp/TypeInf.thy
changeset 17778 93d7e524417a
parent 16417 9bc16273c2d4
child 35416 d8d7d1b785af
equal deleted inserted replaced
17777:05f5532a8289 17778:93d7e524417a
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author:     Martin Strecker
     3     Author:     Martin Strecker
     4 *)
     4 *)
     5 
     5 
     6 (* Exact position in theory hierarchy still to be determined *)
     6 (* Exact position in theory hierarchy still to be determined *)
     7 theory TypeInf imports  WellType begin
     7 theory TypeInf
       
     8 imports "../J/WellType"
       
     9 begin
     8 
    10 
     9 
    11 
    10 
    12 
    11 (**********************************************************************)
    13 (**********************************************************************)
    12 ;
    14 ;