diff -r 4b03e3586f7f -r 31781b2de73d src/HOL/Lattice/Lattice.thy --- a/src/HOL/Lattice/Lattice.thy Thu Jun 14 22:59:42 2007 +0200 +++ b/src/HOL/Lattice/Lattice.thy Thu Jun 14 23:04:36 2007 +0200 @@ -232,7 +232,7 @@ show "x \ x" .. show "x \ x \ y" .. fix z assume "z \ x" and "z \ x \ y" - show "z \ x" by assumption + show "z \ x" by fact qed theorem join_meet_absorb: "x \ (x \ y) = x"