You signed in with another tab or window. Reload to refresh your session.You signed out in another tab or window. Reload to refresh your session.You switched accounts on another tab or window. Reload to refresh your session.Dismiss alert
This bug extremely rarely arises when working with metaprogramming.
The following is the only case it's encountered.
Though mathlib is involved, I don't think it can ever fix a function from standard library, so I put the issue here.
Steps to Reproduce
import Mathlib
example := bylet S := Finset.range 10000let P := ∏ a ∈ S, a
have t : P = (∏ a ∈ S, a) := by rfl
have : (?a : Finset ℕ) = ?b := by
exact t
example := bylet S := Finset.range 10000let P := ∏ a ∈ S, a
have t : P = (∏ a ∈ S, a) := by rfl
have : @Eq (Finset ℕ) ?a ?b := by
exact t
Expected behavior: No error.
Actual behavior: Error maximum recursion depth has been reached throws on the exacts.
Versions
4.9.0
4.11.0-rc2
latest version test now going on
The text was updated successfully, but these errors were encountered:
Description
This bug extremely rarely arises when working with metaprogramming.
The following is the only case it's encountered.
Though mathlib is involved, I don't think it can ever fix a function from standard library, so I put the issue here.
Steps to Reproduce
Expected behavior: No error.
Actual behavior: Error
maximum recursion depth has been reached
throws on theexact
s.Versions
The text was updated successfully, but these errors were encountered: