I can prove the following lemma:
lemma lem1: assumes "(a::real) ≤ b / c" and "c > 0" shows "a * c ≤ b"
using assms
using pos_le_divide_eq[of "c" "a" "b"] by auto
however, if I use bound variables, the proof does not work.
lemma lem2: assumes "∀a b c. (a::real) ≤ b / c" and "∀c. c > 0" shows "∀a b c. a * c ≤ b"
using assms
using pos_le_divide_eq[of "c" "a" "b"]
Inserting the ∀ quantifier into the pos_le_divide_eq changes the data type so that is not possible. How can I solve lem2?