natural-number-game

Solututions to the Natural Number Game

NameSizeMode
..
proposition.lean 1293B -rw-r--r--
01
02
03
04
05
06
07
08
09
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
example (P Q : Prop) (p : P) (h : P → Q) : Q :=
begin
  apply h,
  exact p,
end

lemma imp_self (P : Prop) : P → P :=
begin
  intro p,
  exact p,
end

lemma maze (P Q R S T U: Prop)
           (p : P)
           (h : P → Q)
           (i : Q → R)
           (j : Q → T)
           (k : S → T)
           (l : T → U) : U :=
begin
  apply l,
  apply j,
  apply h,
  exact p,
end

example (P Q : Prop) : P → (Q → P) :=
begin
  intros p q,
  exact p,
end

example (P Q R : Prop) : (P → (Q → R)) → ((P → Q) → (P → R)) :=
begin
  intros h1 h2 p,
  apply h1,
  exact p,
  apply h2,
  exact p,
end

lemma imp_trans (P Q R : Prop) : (P → Q) → ((Q → R) → (P → R)) :=
begin
  intros hpq hqr p,
  apply hqr,
  apply hpq,
  exact p,
end

lemma contrapositive (P Q : Prop) : (P → Q) → (¬ Q → ¬ P) :=
begin
  repeat {rw not_iff_imp_false},
  intros hpq not_q p,
  apply not_q,
  apply hpq,
  exact p,
end

example (A B C D E F G H I J K L : Prop)
        ( f1 : A → B) ( f2 : B → E) ( f3 : E → D) 
        ( f4 : D → A) ( f5 : E → F) ( f6 : F → C) 
        ( f7 : B → C) ( f8 : F → G) ( f9 : G → J)
        (f10 : I → J) (f11 : J → I) (f12 : I → H) 
        (f13 : E → H) (f14 : H → K) (f15 : I → L) : A → L :=
begin
  cc,
end