lean2/tests/lean/run/indbug2.lean

9 lines
196 B
Text
Raw Normal View History

set_option pp.implicit true
set_option pp.universes true
context
parameter {A : Type}
definition foo : A → A → Type := (λ x y, Type)
inductive bar {a b : A} (f : foo a b) :=
bar2 : bar f
end