leanprover / theorem_proving_in_lean

Theorem proving in Lean
Apache License 2.0
47 stars 46 forks source link

Actually leave the type implicit since that's what the text says #54

Closed holtzermann17 closed 6 years ago

holtzermann17 commented 6 years ago

The text said that the type should be left implicit, but the notation preserved the type. This fixes it.

The proof goes through as expected!

example : ∃ x, x + 2 = 8 :=
begin
  let a := 3 * 2,
  existsi a,
  reflexivity
end