src/ZF/Coind/Types.thy
changeset 16417 9bc16273c2d4
parent 13339 0f89104dd377
child 35762 af3ff2ba4c54
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     2     ID:         $Id$
     2     ID:         $Id$
     3     Author:     Jacob Frost, Cambridge University Computer Laboratory
     3     Author:     Jacob Frost, Cambridge University Computer Laboratory
     4     Copyright   1995  University of Cambridge
     4     Copyright   1995  University of Cambridge
     5 *)
     5 *)
     6 
     6 
     7 theory Types = Language:
     7 theory Types imports Language begin
     8 
     8 
     9 consts
     9 consts
    10   Ty :: i               (* Datatype of types *)
    10   Ty :: i               (* Datatype of types *)
    11   TyConst :: i          (* Abstract type of type constants *)
    11   TyConst :: i          (* Abstract type of type constants *)
    12 
    12