lean2/tests/lean/584c.lean

30 lines
471 B
Text
Raw Permalink Normal View History

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