Files
NNG/Game/Levels/OldProposition/Level_7.lean
2024-03-11 19:10:20 +01:00

27 lines
642 B
Lean4

import Game.Metadata
import Game.MyNat.Addition
World "Proposition"
Level 7
Title "(P → Q) → ((Q → R) → (P → R))"
open MyNat
Introduction ""
/-- From $P \implies Q$ and $Q \implies R$ we can deduce $P \implies R$. -/
Statement
(P Q R : Prop) : (P Q) ((Q R) (P R)) := by
Hint (hidden := true)"If you start with `intro hpq` and then `intro hqr`
the dust will clear a bit."
intro hpq
Hint (hidden := true) "Now try `intro hqr`."
intro hqr
Hint "So this level is really about showing transitivity of $\\implies$,
if you like that sort of language."
intro p
apply hqr
apply hpq
exact p