header {* Automated Reasoning, Exercise Sheet 2 *} theory ex2 imports Main begin text {* Prove the following lemmas in Isabelle *} lemma one: "(P \ (Q \ R)) \ ((P \ Q) \ (P \ R))" oops lemma two: "\\P \ P" oops lemma three: "(P \ Q \ R) \ ((P \ Q) \ (P \ R))" oops lemma four: "(\P \ Q) \ (\Q \ P)" oops lemma five: "P \ \P" oops text {* To fully understand the proofs you have constructed, try drawing out the proof trees that correspond to the proof steps accepted by Isabelle. *} end