lean2/tests/lean/run/level_bug3.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

11 lines
199 B
Text

variables {a r : Type}
definition f a := Πr, (a -> r) -> r
lemma blah2 (sa : f a) (k : (a -> r)) :
sa r k = sa r k :=
sorry
lemma blah3 (sa : f a) (k : (a -> r)) :
sa r k = sa r k :=
rfl