src/HOL/MicroJava/J/JBasis.thy
author oheimb
Wed, 06 Dec 2000 19:09:34 +0100
changeset 10612 779af7c58743
parent 10042 7164dc0d24d8
child 11026 a50365d21144
permissions -rw-r--r--
improved superclass entry for classes and definition status of is_class, class corrected recursive definitions of "method" and "fields" Beware: some proofs are incomplete (sorry, oops), preliminary comments with DvO:

(*  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