Many other files modified as follows:
s|Sign.cterm|cterm|g
s|Sign.ctyp|ctyp|g
s|Sign.rep_cterm|rep_cterm|g
s|Sign.rep_ctyp|rep_ctyp|g
s|Sign.pprint_cterm|pprint_cterm|g
s|Sign.pprint_ctyp|pprint_ctyp|g
s|Sign.string_of_cterm|string_of_cterm|g
s|Sign.string_of_ctyp|string_of_ctyp|g
s|Sign.term_of|term_of|g
s|Sign.typ_of|typ_of|g
s|Sign.read_cterm|read_cterm|g
s|Sign.read_insts|read_insts|g
s|Sign.cfun|cterm_fun|g
(*  Title: 	CCL/hered.thy
    ID:         $Id$
    Author: 	Martin Coen
    Copyright   1993  University of Cambridge
Hereditary Termination - cf. Martin Lo\"f
Note that this is based on an untyped equality and so lam x.b(x) is only 
hereditarily terminating if ALL x.b(x) is.  Not so useful for functions!
*)
Hered = Type +
consts
      (*** Predicates ***)
  HTTgen     ::       "i set => i set"
  HTT        ::       "i set"
rules
  (*** Definitions of Hereditary Termination ***)
  HTTgen_def 
  "HTTgen(R) == {t. t=true | t=false | (EX a b.t=<a,b>      & a : R & b : R) | \
\                                      (EX f.  t=lam x.f(x) & (ALL x.f(x) : R))}"
  HTT_def       "HTT == gfp(HTTgen)"
end