src/HOL/MicroJava/J/Decl.ML
author wenzelm
Sat, 20 Jan 2001 00:34:46 +0100
changeset 10946 c03f7dcee8b2
parent 10925 5ffe7ed8899a
permissions -rw-r--r--
instance int :: ordered_ring moved to Ring_and_Field_Example, because it changes the way that int expressions get simplified, violating the strict library principle (cf. README.html);

(*  Title:      HOL/MicroJava/J/Decl.ML
    ID:         $Id$
    Author:     David von Oheimb
    Copyright   1999 Technische Universitaet Muenchen
*)

Goalw [is_class_def, class_def] "finite {C. is_class G C}";
by (fold_goals_tac [dom_def]);
by (rtac finite_dom_map_of 1);
qed "finite_is_class";