diff -r 493d9c4d7ed5 -r c296c75f4cf4 src/HOL/Algebra/Lattice.thy --- a/src/HOL/Algebra/Lattice.thy Wed Dec 28 15:08:12 2011 +0100 +++ b/src/HOL/Algebra/Lattice.thy Wed Dec 28 20:03:13 2011 +0100 @@ -1285,22 +1285,18 @@ by default auto next fix B - assume B: "B \ carrier ?L" - show "EX s. least ?L s (Upper ?L B)" - proof - from B show "least ?L (\ B) (Upper ?L B)" - by (fastforce intro!: least_UpperI simp: Upper_def) - qed + assume "B \ carrier ?L" + then have "least ?L (\ B) (Upper ?L B)" + by (fastforce intro!: least_UpperI simp: Upper_def) + then show "EX s. least ?L s (Upper ?L B)" .. next fix B - assume B: "B \ carrier ?L" - show "EX i. greatest ?L i (Lower ?L B)" - proof - from B show "greatest ?L (\ B \ A) (Lower ?L B)" - txt {* @{term "\ B"} is not the infimum of @{term B}: - @{term "\ {} = UNIV"} which is in general bigger than @{term "A"}! *} - by (fastforce intro!: greatest_LowerI simp: Lower_def) - qed + assume "B \ carrier ?L" + then have "greatest ?L (\ B \ A) (Lower ?L B)" + txt {* @{term "\ B"} is not the infimum of @{term B}: + @{term "\ {} = UNIV"} which is in general bigger than @{term "A"}! *} + by (fastforce intro!: greatest_LowerI simp: Lower_def) + then show "EX i. greatest ?L i (Lower ?L B)" .. qed text {* An other example, that of the lattice of subgroups of a group,