Zulip Chat Archive
Stream: new members
Topic: sorry in def doesn't warn
Alok Singh (Mar 05 2025 at 04:44):
this gives no warnings about the use of sorry. if i don't have sorry in the type signature, then the sorry in the body is at least warned about
theorem sorryInStmt {n: Nat} (f: Fin n → α) (i: Fin n)
: (ofFn f)[i]'sorry = f i
:= sorry
Sebastian Ullrich (Mar 05 2025 at 07:48):
Only because it fails before it even gets to the sorry. Could you please provide an #mwe?
Robin Arnez (Mar 05 2025 at 10:19):
If you mean
theorem sorryInStmt {n : Nat} (f : Fin n → α) (i : Fin n) : (List.ofFn f)[i]'sorry = f i := sorry
then it does warn for me.
Last updated: May 02 2025 at 03:31 UTC