theory week03A_exercise imports Main begin text \ exercise on slide #5: - derive the classical contradiction rule (\P =\ False) =\ P in Isabelle - define nor and nand in Isabelle - show nor x x = nand x x - derive safe intro and elim rules for them - use these in anautomated proof of nor x x = nand x x\ thm ccontr lemma "(\P \ False) \ P" (* TODO *) oops text \nor and nand\ definition nor (* TODO *) lemma norI: (* TODO *) lemma norE: (* TODO *) lemma "nor P P \ \P" (* TODO *) oops definition nand (* TODO *) lemma nandI: (* TODO *) lemma nandE: (* TODO *) (* show nor x x = nand x x *) end