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: f
|
|
|
|
|
Assumed: g
|
2013-09-01 17:34:57 +00:00
|
|
|
|
∀ a b : Type, ∃ c : Type, (g a b) = (f c)
|
2013-09-09 05:54:22 +00:00
|
|
|
|
∀ a b : Type, ∃ c : Type, (g a b) = (f c) : Bool
|
2013-09-01 17:34:57 +00:00
|
|
|
|
(λ a : Type,
|
2013-10-29 23:20:02 +00:00
|
|
|
|
(λ b : Type, if ((λ x : Type, if ((g a b) == (f x)) ⊥ ⊤) == (λ x : Type, ⊤)) ⊥ ⊤) ==
|
|
|
|
|
(λ x : Type, ⊤)) ==
|
2013-09-01 17:34:57 +00:00
|
|
|
|
(λ x : Type, ⊤)
|