PhysLean/scripts/check_file_imports.lean

111 lines
3.8 KiB
Text
Raw Normal View History

/-
Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
Released under Apache 2.0 license.
Authors: Joseph Tooby-Smith
-/
2024-06-26 08:54:54 -04:00
import Batteries.Lean.HashSet
import Lean
/-!
# Check file imports
This file checks that the imports in `HepLean.lean` are sorted and complete.
It can be run from the terminal using
`lake exe check_file_imports`.
## Note on adaptation
The functions
`addModulesIn`, `expectedHepLeanImports`, and `checkMissingImports`
are adapted from `batteries.scripts.check_imports.lean` authored by Joe Hendrix.
-/
open Lean System Meta
/-- Recursively finds files in directory. -/
partial def addModulesIn (recurse : Bool) (prev : Array Name) (root : Name := .anonymous)
(path : FilePath) : IO (Array Name) := do
let mut r := prev
for entry in ← path.readDir do
if ← entry.path.isDir then
if recurse then
r ← addModulesIn recurse r (root.mkStr entry.fileName) entry.path
else
let .some mod := FilePath.fileStem entry.fileName
| continue
r := r.push (root.mkStr mod)
pure r
/-- Compute imports expected by `HepLean.lean` by looking at file structure. -/
def expectedHepLeanImports : IO (Array Name) := do
let mut needed := #[]
for top in ← FilePath.readDir "HepLean" do
let nm := `HepLean
let rootname := FilePath.withExtension top.fileName ""
let root := nm.mkStr rootname.toString
if ← top.path.isDir then
needed ← addModulesIn (recurse := true) needed (root := root) top.path
else
needed :=
needed.push root
pure needed
def listDif : (a: List String) → (b : List String) → (List String × List String)
| [], [] => ([], [])
| a :: as, [] => (a :: as, [])
| [], b :: bs => ([], b :: bs)
| a :: as, b :: bs =>
if a = b then listDif as bs
else (a :: (listDif as bs).1, b :: (listDif as bs).2)
/-- Checks whether an array `imports` is sorted after `Init` is removed. -/
def arrayImportSorted (imports : Array Import) : IO Bool := do
let X := (imports.map (fun x => x.module.toString)).filter (fun x => x != "Init")
let mut warned := false
if ! X = X.qsort (· < ·) then
IO.print s!"Import file is not sorted. \n"
let ldif := listDif X.toList (X.qsort (· < ·)).toList
let lzip := List.zip ldif.1 ldif.2
let lstring := String.intercalate "\n" (lzip.map (fun x => s!"{x.1} > {x.2}"))
println! lstring
warned := true
pure warned
/-- Checks every file in `reqImports` is imported into `modData`
return true if this is NOT the case. -/
def checkMissingImports (modData : ModuleData) (reqImports : Array Name) :
IO Bool := do
2024-10-03 13:58:48 +00:00
let names : Std.HashSet Name := Std.HashSet.ofArray (modData.imports.map (·.module))
let mut warned := false
2024-07-30 07:51:07 -04:00
let nameArray := reqImports.filterMap (
fun req => if !names.contains req then
some req
else
none)
if nameArray.size ≠ 0 then
let nameArraySort := nameArray.qsort (·.toString < ·.toString)
IO.print s!"Files are not imported add the following to the `HepLean` file: \n"
for name in nameArraySort do
IO.print s!"import {name}\n"
warned := true
pure warned
def main (_ : List String) : IO UInt32 := do
initSearchPath (← findSysroot)
2024-08-30 10:11:55 -04:00
let mods : Name := `HepLean
2024-06-27 08:43:57 -04:00
let imp : Import := {module := mods}
let mFile ← findOLean imp.module
unless (← mFile.pathExists) do
throw <| IO.userError s!"object file '{mFile}' of module {imp.module} does not exist"
let (hepLeanMod, _) ← readModuleData mFile
let eHepLeanImports ← expectedHepLeanImports
let sortedWarned ← arrayImportSorted hepLeanMod.imports
let warned ← checkMissingImports hepLeanMod eHepLeanImports
if (warned sortedWarned) then
throw <| IO.userError s!"The HepLean module is not sorted, or has missing imports."
IO.println s!"Import check complete."
pure 0