diff -r a645a0e6d790 -r 48fdff264eb2 src/HOL/Algebra/Lattice.thy --- a/src/HOL/Algebra/Lattice.thy Fri Jun 26 00:14:10 2015 +0200 +++ b/src/HOL/Algebra/Lattice.thy Fri Jun 26 10:20:33 2015 +0200 @@ -589,7 +589,7 @@ lemma (in weak_upper_semilattice) finite_sup_insertI: assumes P: "!!l. least L l (Upper L (insert x A)) ==> P l" and xA: "finite A" "x \ carrier L" "A \ carrier L" - shows "P (\ (insert x A))" + shows "P (\(insert x A))" proof (cases "A = {}") case True with P and xA show ?thesis by (simp add: finite_sup_least) @@ -828,7 +828,7 @@ lemma (in weak_lower_semilattice) finite_inf_insertI: assumes P: "!!i. greatest L i (Lower L (insert x A)) ==> P i" and xA: "finite A" "x \ carrier L" "A \ carrier L" - shows "P (\ (insert x A))" + shows "P (\(insert x A))" proof (cases "A = {}") case True with P and xA show ?thesis by (simp add: finite_inf_greatest) @@ -856,7 +856,7 @@ lemma (in weak_lower_semilattice) inf_of_two_greatest: "[| x \ carrier L; y \ carrier L |] ==> - greatest L (\ {x, y}) (Lower L {x, y})" + greatest L (\{x, y}) (Lower L {x, y})" proof (unfold inf_def) assume L: "x \ carrier L" "y \ carrier L" with inf_of_two_exists obtain s where "greatest L s (Lower L {x, y})" by fast @@ -904,8 +904,8 @@ proof - (* FIXME: improved simp, see weak_join_assoc above *) have "(x \ y) \ z = z \ (x \ y)" by (simp only: meet_comm) - also from L have "... .= \ {z, x, y}" by (simp add: weak_meet_assoc_lemma) - also from L have "... = \ {x, y, z}" by (simp add: insert_commute) + also from L have "... .= \{z, x, y}" by (simp add: weak_meet_assoc_lemma) + also from L have "... = \{x, y, z}" by (simp add: insert_commute) also from L have "... .= x \ (y \ z)" by (simp add: weak_meet_assoc_lemma [symmetric]) finally show ?thesis by (simp add: L) qed @@ -1286,15 +1286,15 @@ next fix B assume "B \ carrier ?L" - then have "least ?L (\ B) (Upper ?L B)" + 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 \ 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"}! *} + 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