theory Test imports Main begin lemma fixes x :: int shows "x > 0 \ x * x > 0" by simp lemma "\ x. drinks x \ (\ y. drinks y)" by blast lemma "(\ x. P x) = (\ x. P x)" by auto end