improved superclass entry for classes and definition status of is_class, class
corrected recursive definitions of "method" and "fields"
cleanup of many proofs, removed superfluous tactics and theorems
(* Title: HOL/MicroJava/J/JBasis.thy
ID: $Id$
Author: David von Oheimb
Copyright 1999 TU Muenchen
Some auxiliary definitions.
*)
JBasis = Main +
constdefs
unique :: "('a \\<times> 'b) list => bool"
"unique == nodups \\<circ> map fst"
end