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