diff -r 89d19aa73081 -r aa894a49f77d src/HOL/Library/Convex.thy --- a/src/HOL/Library/Convex.thy Sun Apr 17 22:38:50 2016 +0200 +++ b/src/HOL/Library/Convex.thy Mon Apr 18 14:30:32 2016 +0100 @@ -65,13 +65,13 @@ lemma convex_UNIV[intro,simp]: "convex UNIV" unfolding convex_def by auto -lemma convex_Inter: "(\s\f. convex s) \ convex(\f)" +lemma convex_Inter: "(\s. s\f \ convex s) \ convex(\f)" unfolding convex_def by auto lemma convex_Int: "convex s \ convex t \ convex (s \ t)" unfolding convex_def by auto -lemma convex_INT: "\i\A. convex (B i) \ convex (\i\A. B i)" +lemma convex_INT: "(\i. i \ A \ convex (B i)) \ convex (\i\A. B i)" unfolding convex_def by auto lemma convex_Times: "convex s \ convex t \ convex (s \ t)"