theory a1 imports Main begin text \ Question 1 \ text \ Insert your answer here, or in a separate .pdf or .txt file \ text \ Question 2 \ text \ Insert your answer here, or in a separate .pdf or .txt file \ text \ Question 3 \ lemma prop_a: "B \ A \ B \ C" sorry lemma prop_b: "(A \ B) \ (B \ C) \ (C \ D) \ A \ D" sorry lemma prop_c: "((A \ B) \ C) = (A \ C \ C \ B)" sorry lemma prop_d: "(\P) = (\\\P)" sorry lemma prop_e: "(A\B) = (\ (\B \ A))" sorry lemma prop_f: "((A\C)\(C\A)\(A\D))\D" sorry text \ Question 4 \ lemma hol_a: "(\x. P x) \ (\x. Q x) \ (\x. Q x \ P x)" sorry lemma hol_b: "(\x. P x \ Q x) \ (\x. P x) \ (\x. Q x)" sorry lemma hol_c: "(\x. P x \ Q x) \ ((\x. Q x) \ W) \ ((\x. P x)\ Z) \ W \ Z" sorry lemma hol_d: "(\x. R x x) \\(\ x y. R y x \ \ R x y)" sorry end