theory s2 imports Main begin (* Question 1 *) lemma a: "(\ x. \ y. R x y) = (\ y. \ x. R x y)" oops lemma b: "((\ x. P x) \ (\ x. Q x)) = (\ x. P x \ Q x)" oops lemma c: "(\ P. P = True \ P = False) \ (\ P. (\ P \ P) \ P)" oops lemma d: "(\ P. P = True \ P = False) \ (\ P. (\\ P) = P)" oops lemma e: "((\P. \x. (R x \ P x) \ P (SOME x. P x)) \ (\ x y. Q x y \ R y)) \ ((\x. \y. Q x y) \ (\f. \x. Q x (f x)))" oops (* Question 2 -- drinker formula *) (* part (a) *) lemma df: "\ x. D x \ (\ x. D x)" oops (* part (b) *) (* Question 3 *) (* Question 4 *) end