lean2/tests/lean/binder_overload.lean.expected.out

8 lines
331 B
Text
Raw Normal View History

{x : ∈ S| x > 0} : set
{x : ∈ s| x > 0} : finset
@set.sep.{1} nat (λ (x : nat), nat.gt x (nat.of_num 0)) S : set.{1} nat
@finset.sep.{1} nat (λ (a b : nat), nat.has_decidable_eq a b) (λ (x : nat), nat.gt x (nat.of_num 0))
(λ (a : nat), nat.decidable_ge a (nat.succ (nat.of_num 0)))
s :
finset.{1} nat