lean2/tests/lean/run/app_builder_issue1.lean
Leonardo de Moura 19ebedd480 feat(library/type_context): improve type_context get_level_core, add virtual method for checking types whenever a metavariable is assigned
We add an example where app_builder fails without these new features.
That is, app_builder fails to solve the unification problem.
2016-01-03 17:58:27 -08:00

4 lines
127 B
Text

constant f {A : Type} (a : A) {B : Type} (b : B) : nat
example (a b c d : nat) : a = c → b = d → f a b = f c d :=
by simp