e218b92a9d
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
9 lines
263 B
Text
9 lines
263 B
Text
Set: pp::colors
|
||
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, ⊤)
|