lean2/tests/lean/exact_partial.lean

5 lines
91 B
Text

example (a b : Prop) : a → b → a ∧ b :=
begin
intros,
exact (and.intro _ _),
end