refactor: some docs

This commit is contained in:
jstoobysmith 2025-02-14 08:50:24 +00:00
parent 1b8360fda8
commit e1303cbcf8
14 changed files with 46 additions and 46 deletions

View file

@ -3,7 +3,7 @@ Copyright (c) 2024 Joseph Tooby-Smith. All rights reserved.
Released under Apache 2.0 license.
Authors: Joseph Tooby-Smith
-/
import HepLean.Meta.Basic
import PhysLean.Meta.Basic
import ImportGraph.Imports
/-!
@ -11,7 +11,7 @@ import ImportGraph.Imports
-/
open Lean System Meta HepLean
open Lean System Meta PhysLean
def Imports.RedundentImports (imp : Import) : MetaM UInt32 := do
@ -25,5 +25,5 @@ def Imports.RedundentImports (imp : Import) : MetaM UInt32 := do
unsafe def main (_ : List String) : IO UInt32 := do
initSearchPath (← findSysroot)
let imports ← allImports
let _ ← CoreM.withImportModules #[`HepLean] (imports.mapM Imports.RedundentImports).run'
let _ ← CoreM.withImportModules #[`PhysLean] (imports.mapM Imports.RedundentImports).run'
return 0