src/HOL/MicroJava/J/JBasis.thy
author nipkow
Wed, 06 Sep 2000 08:04:41 +0200
changeset 9870 2374ba026fc6
parent 8116 759f712f8f06
child 10042 7164dc0d24d8
permissions -rw-r--r--
less_induct -> nat_less_induct

(*  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 \\<Rightarrow> bool"
 "unique  \\<equiv> nodups \\<circ> map fst"

end