Used locale interpretations everywhere. -> lemma had new name
--- a/src/HOL/MicroJava/Comp/CorrCompTp.thy Wed Apr 20 17:19:18 2005 +0200
+++ b/src/HOL/MicroJava/Comp/CorrCompTp.thy Wed Apr 20 17:19:42 2005 +0200
@@ -908,7 +908,7 @@
by (simp add: check_type_def states_lower)
lemma max_same_iter [simp]: "max (x::'a::linorder) (max x y) = max x y"
-by (simp del: max_assoc add: max_assoc [THEN sym])
+by (simp add: AC_max.assoc [THEN sym])
(* ******************************************************************* *)