theory a1 imports Main begin section "Question 1: Lambda-Calculus" text {* submit as part of a .txt or .pdf file *} section "Question 2: Higher Order Unification" text {* submit as part of a .txt or .pdf file *} section "Question 3: Propositional Logic" lemma prop_a: "A \ B \ B" oops lemma prop_b: "(P \ P) = P" oops lemma prop_c: "\\P \ P" oops lemma prop_d: "(A \ B \ C) = (A \ B \ C)" oops lemma prop_e: "(\ x) = (x = False)" oops lemma prop_f: "(a \ b) = (\ (a \ \ b))" oops text {* Which of the above statements are provable only in a classical logic? *} section "Question 4: Higher Order Logic" lemma hol_a: "(\x. \y. R x y) \ (\y. \x. R x y)" oops lemma hol_b: "(\x. P x \ Q x) \ ((\x. P x) \ (\x. Q x))" oops lemma hol_c: "False = (\P. P)" oops lemma hol_d: "\R::bool \ bool \ bool. ((\x. \y. R x y) \ \(\y. \x. R x y))" oops lemma hol_e: "(\x. \ (R x) \ RM x) \ (\x. \ RM x \ R x)" oops lemma hol_f: "\(\x. \ (R x) \ R (M x)); (\x. R x)\ \ (\x. R x \ R (M (M x)))" oops text {* Formalise and prove the following statement using only the proof methods and rules as earlier in this question. If every poor person has a rich mother, then there is a rich person with a rich grandmother. *} lemma rich_grandmothers: "formalise_the_statement_here" oops end