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.
24 lines
371 B
Plaintext
24 lines
371 B
Plaintext
2 years ago
|
import TestGame.Metadata
|
||
|
import Std.Tactic.RCases
|
||
|
import Mathlib.Tactic.Contrapose
|
||
|
|
||
|
Game "TestGame"
|
||
|
World "Contradiction"
|
||
|
Level 7
|
||
|
|
||
|
Title "Kontraposition"
|
||
|
|
||
|
Introduction
|
||
|
"
|
||
|
Im Gegensatz zum Widerspruch, wo
|
||
|
"
|
||
|
|
||
|
Statement
|
||
|
"Ein Widerspruch impliziert alles."
|
||
|
(A B : Prop) (h : ¬ B → ¬ A) (hA : A) : B := by
|
||
|
revert hA
|
||
|
contrapose
|
||
|
assumption
|
||
|
|
||
|
Tactics contradiction
|