1
(* Title: HOL/BCV/Types.thy
2
ID: $Id$
3
Author: Tobias Nipkow
4
Copyright 1999 TUM
5
6
Types for the register machine
7
*)
8
9
Types = Types0 +
10
11
instance typ :: order (le_typ_refl,le_typ_trans,le_typ_antisym,less_le_typ)
12
13
end