diff -r 05072ae0d435 -r 36a59e5d0039 src/HOL/Lattice/Lattice.thy --- a/src/HOL/Lattice/Lattice.thy Wed Sep 13 00:38:38 2006 +0200 +++ b/src/HOL/Lattice/Lattice.thy Wed Sep 13 12:05:50 2006 +0200 @@ -519,7 +519,7 @@ qed qed -instance fun :: (type, lattice) lattice +instance "fun" :: (type, lattice) lattice proof fix f g :: "'a \ 'b::lattice" show "\inf. is_inf f g inf" by rule (rule is_inf_fun) (* FIXME @{text "from \ show \ .."} does not work!? unification incompleteness!? *)