lean icon indicating copy to clipboard operation
lean copied to clipboard

apply tactic produces incorrect proof

Open gebner opened this issue 4 years ago • 1 comments

def additive (α : Type*) := α

instance {α} [has_one α] : has_zero (additive α) := ⟨(1 : α)⟩

example : (0 : ℕ) = (0 : additive ℕ) :=
by apply eq.refl

gebner avatar Nov 01 '21 10:11 gebner

This is getting more and more interesting:

#eval tactic.is_def_eq `(0 : ℕ) `(0 : additive ℕ) -- succeeds!?!

gebner avatar Nov 01 '21 10:11 gebner