``` {"cmd": "#eval 1 + 1"} {"cmd": "def foo : (fun ((x, y, z) : Nat × Nat × Nat) => x = x) = fun x => True := by sorry", "env": 0} {"tactic": "simp", "proofState": 0} ``` Expected: Goal closed Actual: `{"message": "Lean error:\nunknown constant 'foo.match_1'"}` This comes down to https://github.com/leanprover-community/repl/commit/66515025d9ccffa2be29718d31b816edd0675202 which eliminates both `foo` and `foo.match_1` from the env. I'm not sure why the `InfoTree` env has `foo` actually, but I've [made a question about this on Zulip](https://leanprover.zulipchat.com/#narrow/channel/239415-metaprogramming-.2F-tactics/topic/presence.20of.20decl.20in.20env.2Econstants.20of.20InfoTree.20of.20decl/near/492476303).