Skip to content

Commit

Permalink
make robust against a failure in a nightly
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Feb 11, 2024
1 parent d95fb9c commit 9618fa9
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion ImportGraph/Cli.lean
Original file line number Diff line number Diff line change
Expand Up @@ -38,7 +38,7 @@ def importGraphCLI (args : Cli.Parsed) : IO UInt32 := do
searchPathRef.set compile_time_search_path%
let dotFile ← try unsafe withImportModules #[{module := to}] {} (trustLevel := 1024) fun env => do
let mut graph := env.importGraph
if let .some f := from? then
if let Option.some f := from? then
graph := graph.downstreamOf (NameSet.empty.insert f)
if ¬(args.hasFlag "include-deps") then
let p := ImportGraph.getModule to
Expand Down

0 comments on commit 9618fa9

Please sign in to comment.