19ebedd480
We add an example where app_builder fails without these new features. That is, app_builder fails to solve the unification problem.
4 lines
127 B
Text
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
|