2013-09-02 19:29:21 +00:00
|
|
|
|
Set: pp::colors
|
2013-09-03 17:44:51 +00:00
|
|
|
|
Set: pp::unicode
|
2013-09-01 02:15:48 +00:00
|
|
|
|
Assumed: N
|
|
|
|
|
Assumed: h
|
|
|
|
|
Proved: CongrH
|
2013-09-02 19:29:21 +00:00
|
|
|
|
Set: lean::pp::implicit
|
2013-12-19 21:12:39 +00:00
|
|
|
|
Variable h : N → N → N
|
2013-12-22 01:02:16 +00:00
|
|
|
|
Theorem CongrH {a1 a2 b1 b2 : N} (H1 : @eq N a1 b1) (H2 : @eq N a2 b2) : @eq N (h a1 a2) (h b1 b2) :=
|
|
|
|
|
@Congr N (λ x : N, N) (h a1) (h b1) a2 b2 (@Congr N (λ x : N, N → N) h h a1 b1 (@Refl (N → N → N) h) H1) H2
|
2013-09-02 19:29:21 +00:00
|
|
|
|
Set: lean::pp::implicit
|
2013-12-19 21:12:39 +00:00
|
|
|
|
Variable h : N → N → N
|
2013-12-19 20:46:14 +00:00
|
|
|
|
Theorem CongrH {a1 a2 b1 b2 : N} (H1 : a1 = b1) (H2 : a2 = b2) : h a1 a2 = h b1 b2 := Congr (Congr (Refl h) H1) H2
|
2013-09-01 02:15:48 +00:00
|
|
|
|
Proved: Example1
|
2013-09-02 19:29:21 +00:00
|
|
|
|
Set: lean::pp::implicit
|
2013-12-22 01:02:16 +00:00
|
|
|
|
Theorem Example1 (a b c d : N) (H : @eq N a b ∧ @eq N b c ∨ @eq N a d ∧ @eq N d c) : @eq N (h a b) (h c b) :=
|
|
|
|
|
@DisjCases
|
|
|
|
|
(@eq N a b ∧ @eq N b c)
|
|
|
|
|
(@eq N a d ∧ @eq N d c)
|
2013-12-19 20:46:14 +00:00
|
|
|
|
(h a b == h c b)
|
2013-09-01 02:15:48 +00:00
|
|
|
|
H
|
2013-12-22 01:02:16 +00:00
|
|
|
|
(λ H1 : @eq N a b ∧ @eq N b c,
|
|
|
|
|
@CongrH a
|
|
|
|
|
b
|
|
|
|
|
c
|
|
|
|
|
b
|
|
|
|
|
(@Trans N a b c (@Conjunct1 (@eq N a b) (@eq N b c) H1) (@Conjunct2 (@eq N a b) (@eq N b c) H1))
|
|
|
|
|
(@Refl N b))
|
|
|
|
|
(λ H1 : @eq N a d ∧ @eq N d c,
|
|
|
|
|
@CongrH a
|
|
|
|
|
b
|
|
|
|
|
c
|
|
|
|
|
b
|
|
|
|
|
(@Trans N a d c (@Conjunct1 (@eq N a d) (@eq N d c) H1) (@Conjunct2 (@eq N a d) (@eq N d c) H1))
|
|
|
|
|
(@Refl N b))
|
2013-09-01 02:15:48 +00:00
|
|
|
|
Proved: Example2
|
2013-09-02 19:29:21 +00:00
|
|
|
|
Set: lean::pp::implicit
|
2013-12-22 01:02:16 +00:00
|
|
|
|
Theorem Example2 (a b c d : N) (H : @eq N a b ∧ @eq N b c ∨ @eq N a d ∧ @eq N d c) : @eq N (h a b) (h c b) :=
|
|
|
|
|
@DisjCases
|
|
|
|
|
(@eq N a b ∧ @eq N b c)
|
|
|
|
|
(@eq N a d ∧ @eq N d c)
|
|
|
|
|
(@eq N (h a b) (h c b))
|
2013-09-01 02:15:48 +00:00
|
|
|
|
H
|
2013-12-22 01:02:16 +00:00
|
|
|
|
(λ H1 : @eq N a b ∧ @eq N b c,
|
|
|
|
|
@CongrH a
|
|
|
|
|
b
|
|
|
|
|
c
|
|
|
|
|
b
|
|
|
|
|
(@Trans N a b c (@Conjunct1 (a == b) (@eq N b c) H1) (@Conjunct2 (@eq N a b) (b == c) H1))
|
|
|
|
|
(@Refl N b))
|
|
|
|
|
(λ H1 : @eq N a d ∧ @eq N d c,
|
|
|
|
|
@CongrH a
|
|
|
|
|
b
|
|
|
|
|
c
|
|
|
|
|
b
|
|
|
|
|
(@Trans N a d c (@Conjunct1 (a == d) (@eq N d c) H1) (@Conjunct2 (@eq N a d) (d == c) H1))
|
|
|
|
|
(@Refl N b))
|
2013-09-01 02:15:48 +00:00
|
|
|
|
Proved: Example3
|
2013-09-02 19:29:21 +00:00
|
|
|
|
Set: lean::pp::implicit
|
2013-12-19 20:46:14 +00:00
|
|
|
|
Theorem Example3 (a b c d e : N) (H : a = b ∧ b = e ∧ b = c ∨ a = d ∧ d = c) : h a b = h c b :=
|
2013-09-01 02:15:48 +00:00
|
|
|
|
DisjCases
|
|
|
|
|
H
|
2013-09-01 17:34:57 +00:00
|
|
|
|
(λ H1 : a = b ∧ b = e ∧ b = c, CongrH (Trans (Conjunct1 H1) (Conjunct2 (Conjunct2 H1))) (Refl b))
|
|
|
|
|
(λ H1 : a = d ∧ d = c, CongrH (Trans (Conjunct1 H1) (Conjunct2 H1)) (Refl b))
|
2013-09-01 02:15:48 +00:00
|
|
|
|
Proved: Example4
|
2013-09-02 19:29:21 +00:00
|
|
|
|
Set: lean::pp::implicit
|
2013-12-19 20:46:14 +00:00
|
|
|
|
Theorem Example4 (a b c d e : N) (H : a = b ∧ b = e ∧ b = c ∨ a = d ∧ d = c) : h a c = h c a :=
|
2013-09-01 02:15:48 +00:00
|
|
|
|
DisjCases
|
|
|
|
|
H
|
2013-09-01 17:34:57 +00:00
|
|
|
|
(λ H1 : a = b ∧ b = e ∧ b = c,
|
|
|
|
|
let AeqC := Trans (Conjunct1 H1) (Conjunct2 (Conjunct2 H1)) in CongrH AeqC (Symm AeqC))
|
|
|
|
|
(λ H1 : a = d ∧ d = c, let AeqC := Trans (Conjunct1 H1) (Conjunct2 H1) in CongrH AeqC (Symm AeqC))
|