lean2/tests/lean/584b.lean

28 lines
376 B
Text
Raw Normal View History

2015-05-07 21:24:30 +00:00
section
variable (A : Type)
section
variables (a b : A)
variable (H : a = b)
definition tst₁ := a
check @tst₁
variable {A}
definition tst₂ := a
check @tst₂ -- A is implicit
lemma symm₂ : b = a := eq.symm H
check @symm₂
end
variable (a : A)
definition tst₃ := a
check @tst₃ -- A is explicit again
end