Skip to content

Commit

Permalink
to pass nix test, adding Newline file back in
Browse files Browse the repository at this point in the history
  • Loading branch information
kmill committed May 7, 2024
1 parent 147cac0 commit d283ac3
Showing 1 changed file with 10 additions and 0 deletions.
10 changes: 10 additions & 0 deletions src/lake/Lake/Util/Newline.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1,10 @@
/-
Copyright (c) 2023 Mario Carneiro. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Mario Carneiro
-/

namespace Lake

/-- This is the same as `String.replace text "\r\n" "\n"`, but more efficient. -/
@[inline, deprecated] partial def crlf2lf (text : String) : String := text.crlfToLf

0 comments on commit d283ac3

Please sign in to comment.