You cannot select more than 25 topics Topics must start with a letter or number, can include dashes ('-') and can be up to 35 characters long.
lean4game/server/adam/Adam/Levels/Implication/L03_Apply.lean

36 lines
915 B
Plaintext

import Adam.Metadata
2 years ago
import Mathlib
2 years ago
Game "Adam"
World "Implication"
Level 3
2 years ago
Title "Apply"
2 years ago
Introduction
"
2 years ago
Sein Kollege zieht eine Linie unter deinen Beweis, schreibt ein durchgestrichenes ~`revert`~
hin und gibt dir das Blatt wieder.
"
2 years ago
2 years ago
Statement (A B : Prop) (hA : A) (h : A → B) : B := by
2 years ago
Hint "**Robo**: Da hat er natürlich recht, normalerweise ist es viel schöner mit
2 years ago
`apply {h}` die Implikation anzuwenden."
2 years ago
apply h
2 years ago
Hint "**Du**: Und jetzt genügt es also `A` zu zeigen."
2 years ago
assumption
2 years ago
Conclusion "**Robo** Übrigens mit `apply LEMMA` kannst auch jedes Lemma anwenden, dessen
Aussage mit dem Goal übereinstimmt.
Die beiden Fragenden schauen das Blatt an und murmeln zustimmend."
2 years ago
NewTactic apply
DisabledTactic revert tauto
2 years ago
-- Katex notes
-- `\\( \\)` or `$ $` for inline
-- and `$$ $$` block.
-- align block:
2 years ago
-- $$\\begin{aligned} 2x - 4 &= 6 \\\\ 2x &= 10 \\\\ x &= 5 \\end{aligned}$$