refactor: Move files and update toml
This commit is contained in:
parent
a957bb484c
commit
49ec0b6ea7
220 changed files with 832 additions and 832 deletions
|
@ -10,7 +10,7 @@ import Mathlib.Data.Nat.Notation
|
|||
|
||||
# TODO finder
|
||||
|
||||
This program finds all instances of `/<!> TODO: ...` (without the `<>`) in HepLean files.
|
||||
This program finds all instances of `/<!> TODO: ...` (without the `<>`) in PhysLean files.
|
||||
|
||||
## Note
|
||||
|
||||
|
@ -21,10 +21,10 @@ Parts of this file are adapted from `Mathlib.Tactic.Linter.TextBased`,
|
|||
open Lean System Meta
|
||||
|
||||
/-- Given a list of lines, outputs an error message and a line number. -/
|
||||
def HepLeanTODOItem : Type := Array String → Array (String × ℕ)
|
||||
def PhysLeanTODOItem : Type := Array String → Array (String × ℕ)
|
||||
|
||||
/-- Checks if a . -/
|
||||
def TODOFinder : HepLeanTODOItem := fun lines ↦ Id.run do
|
||||
def TODOFinder : PhysLeanTODOItem := fun lines ↦ Id.run do
|
||||
let enumLines := (lines.toList.enumFrom 1)
|
||||
let todos := enumLines.filterMap (fun (lno1, l1) ↦
|
||||
if l1.startsWith "/-! TODO:" then
|
||||
|
@ -45,7 +45,7 @@ def printTODO (todos : Array TODOContext) : IO Unit := do
|
|||
IO.println (s!"{e.path}:{e.lineNumber}: {e.statement}")
|
||||
|
||||
def filePathToGitPath (S : FilePath) (n : ℕ) : String :=
|
||||
"https://github.com/HEPLean/HepLean/blob/master/"++
|
||||
"https://github.com/HEPLean/PhysLean/blob/master/"++
|
||||
(S.toString.replace "." "/").replace "/lean" ".lean"
|
||||
++ "#L" ++ toString n
|
||||
|
||||
|
@ -67,7 +67,7 @@ def hepLeanLintFile (path : FilePath) : IO String := do
|
|||
def todoFileHeader : String := s!"
|
||||
# TODO List
|
||||
|
||||
This is an automatically generated list of TODOs appearing as `/-! TODO:...` in HepLean.
|
||||
This is an automatically generated list of TODOs appearing as `/-! TODO:...` in PhysLean.
|
||||
|
||||
Please feel free to contribute to the completion of these tasks.
|
||||
|
||||
|
@ -76,7 +76,7 @@ Please feel free to contribute to the completion of these tasks.
|
|||
|
||||
def main (args : List String) : IO UInt32 := do
|
||||
initSearchPath (← findSysroot)
|
||||
let mods : Name := `HepLean
|
||||
let mods : Name := `PhysLean
|
||||
let imp : Import := {module := mods}
|
||||
let mFile ← findOLean imp.module
|
||||
unless (← mFile.pathExists) do
|
||||
|
|
Loading…
Add table
Add a link
Reference in a new issue