2016-01-14 06:10:15 +00:00
|
|
|
open subtype
|
2016-01-14 06:13:04 +00:00
|
|
|
set_option blast.strategy "cc"
|
2016-01-14 06:10:15 +00:00
|
|
|
|
2016-01-14 05:44:32 +00:00
|
|
|
example (f g : Π {A : Type₁}, A → A → A) (h : nat → nat) (a b : nat) :
|
|
|
|
h = f a → h b = f a b :=
|
|
|
|
by blast
|
|
|
|
|
2016-01-17 03:53:36 +00:00
|
|
|
example (f g : Π {A : Type₁}, A → A → A) (h : nat → nat) (a b : nat) :
|
|
|
|
h = f a → h b = f a b :=
|
|
|
|
by blast
|
|
|
|
|
2016-01-14 06:10:15 +00:00
|
|
|
example (f g : Π {A : Type₁} (a b : A), {x : A | x ≠ b}) (h : Π (b : nat), {x : nat | x ≠ b}) (a b₁ b₂ : nat) :
|
|
|
|
h = f a → b₁ = b₂ → h b₁ == f a b₂ :=
|
2016-01-14 05:44:32 +00:00
|
|
|
by blast
|