We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 854e335 commit 8ec35d8Copy full SHA for 8ec35d8
tests/lean/run/6655.lean
@@ -52,6 +52,18 @@ example {α : Type} (c : α → α) (x : α) : c x = x := by
52
simp?
53
sorry
54
55
+/-!
56
+Example from comments of #6655. This used to suggest `simp only [Int.add_sub_cancel, p]`.
57
+(N.B. the goal at that point does not have `p` in it!)
58
+-/
59
+/-- info: Try this: simp only [Int.add_sub_cancel] -/
60
+#guard_msgs in
61
+example (a b : Int) : a + b - b = a := by
62
+ let p := 1
63
+ have h : p = 1 := by
64
+ simp only [p]
65
+ simp?
66
+
67
/-!
68
Example from https://github.com/leanprover/lean4/pull/7539 by JovanGerb.
69
This used to suggest `simp only [a, b] ` and `simp only [a, b]`
0 commit comments