lean2/tests/lean/run/361.lean

6 lines
109 B
Text

variables {P Q R : Prop}
theorem foo (H : P → Q → R) (x : P) : Q → R :=
begin
apply H,
exact x
end