a341643335
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
10 lines
282 B
Text
10 lines
282 B
Text
Set: pp::colors
|
||
Set: pp::unicode
|
||
Assumed: f
|
||
Assumed: g
|
||
∀ a b : Type, ∃ c : Type, (g a b) = (f c)
|
||
Bool
|
||
(λ a : Type,
|
||
(λ b : Type, ite Bool ((λ x : Type, ite Bool ((g a b) = (f x)) ⊥ ⊤) = (λ x : Type, ⊤)) ⊥ ⊤) =
|
||
(λ x : Type, ⊤)) =
|
||
(λ x : Type, ⊤)
|