lean2/tests/lean/run/level_bug2.lean
Leonardo de Moura 16b7bc3922 fix(kernel/default_converter): broken optimization
we must also check the universe levels when applying the optimization for
constraints of the form:

            f.{l_1 ... l_k} a_1 ... a_n  =?= f.{l_1' ... l_k'} b_1 ... b_n

The optimization tries to avoid unfolding f if we can establish that
a_i is definitionally equal to b_i for each i in [1, n]

closes #581
2015-05-06 18:32:41 -07:00

4 lines
149 B
Text

definition f (a : Type) := Π r : Type, (a → r) → r
definition blah2 {a : Type} {r : Type} (sa : f a) (k : a → r) : sa r k = sa r k :=
rfl