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 5cb41d9 commit 2816e77Copy full SHA for 2816e77
src/Init/Data/Option/Lemmas.lean
@@ -1028,7 +1028,7 @@ variable [BEq α]
1028
· intro h
1029
infer_instance
1030
1031
-@[simp, grind =] theorem beq_none {o : Option α} : (o == none) = o.isNone := by cases o <;> simp
+@[simp] theorem beq_none {o : Option α} : (o == none) = o.isNone := by cases o <;> simp
1032
1033
@[simp, grind =]
1034
theorem filter_beq_self [ReflBEq α] {p : α → Bool} {o : Option α} : (o.filter p == o) = o.all p := by
0 commit comments