Eliminated the prediates flat,chfin
Changed theorems with flat(x::'a) to (x::'a::flat)
Since flat<chfin theorems adm_flat,adm_flatdom are eliminated.
Use adm_chain_finite and adm_chfindom instead!
Examples do not use flat_flat any more
(* Title: HOLCF/Discrete.thy
ID: $Id$
Author: Tobias Nipkow
Copyright 1997 TUM
Discrete CPOs
*)
Discrete = Discrete1 +
instance discr :: (term)cpo (discr_cpo)
constdefs
undiscr :: ('a::term)discr => 'a
"undiscr x == (case x of Discr y => y)"
end