blob: 1533960150c468e2fb52a451480299efb8f046f7 (
plain)
1
2
3
4
5
6
7
8
9
10
|
Generalizable Variables A.
Class Test A := { test : A }.
Lemma mylemma : forall `{Test A}, test = test.
Admitted. (* works fine *)
Definition mylemma' := forall `{Test A}, test = test.
About mylemma'.
|