theory a1 imports Main begin section "Question 1: Types" text {* submit as part of a .txt or .pdf file *} section "Question 2: Lambda-Calculus" text {* submit as part of a .txt or .pdf file *} section "Question 3: Higher Order Unification" text {* submit as part of a .txt or .pdf file *} section "Question 4: Propositional Logic" lemma prop_a: "A \ A \ B" oops lemma prop_b: "A \ B \ A" oops lemma prop_c: "(P \ P) = P" oops lemma prop_d: "\\P \ P" oops lemma prop_e: "P \ \\P" oops lemma prop_f: "\\\P \ \P" oops lemma prop_g: "(A \ B \ C) = (A \ B \ C)" oops lemma prop_h: "(x = False) = (\ x)" oops lemma prop_i: "(P \ Q) = (\ (P \ \ Q))" oops lemma prop_j: "(P \ \ P) \ (\\ P \ P)" oops lemma prop_k: "(P \ (Q \ R)) \ ((P \ Q) \ (P \ R))" oops text {* Which of the above statements are provable only in a classical logic? *} end