Skip to content

Commit

Permalink
Keep TODOs in for future unproven string theorems
Browse files Browse the repository at this point in the history
Co-Authored-By: Bulhwi Cha <[email protected]>
  • Loading branch information
tjf801 and chabulhwi committed May 23, 2024
1 parent 2aabdc1 commit 8b65f75
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions Batteries/Data/String/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -990,6 +990,8 @@ theorem data_isPrefixOf_iff_isPrefixOf {s t : String} : s.1.isPrefixOf t.1 ↔ s
exact (isPrefixOf_cons.mp h).imp_right data_isPrefixOf_iff_isPrefixOf.mpr
termination_by s.length

-- TODO: substrEq
-- TODO: isPrefixOf
-- TODO: replace

@[nolint unusedHavesSuffices] -- false positive from unfolding String.takeWhileAux
Expand Down

0 comments on commit 8b65f75

Please sign in to comment.