Skip to content

Commit

Permalink
implies
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Aug 30, 2024
1 parent 6dc33a1 commit 3c90f51
Show file tree
Hide file tree
Showing 2 changed files with 4 additions and 4 deletions.
2 changes: 1 addition & 1 deletion ImportGraph/Cli.lean
Original file line number Diff line number Diff line change
Expand Up @@ -77,7 +77,7 @@ def importGraphCLI (args : Cli.Parsed) : IO UInt32 := do
let toModule := ImportGraph.getModule to
let includeLean := args.hasFlag "include-lean"
let includeStd := args.hasFlag "include-std" || includeLean
let includeDeps := args.hasFlag "include-deps" || includeStd
let includeDeps := args.hasFlag "include-deps" || args.hasFlag "mark-module" || includeStd
let filter (n : Name) : Bool :=
toModule.isPrefixOf n ||
bif isPrefixOf `Std n then includeStd else
Expand Down
6 changes: 3 additions & 3 deletions Main.lean
Original file line number Diff line number Diff line change
Expand Up @@ -21,9 +21,9 @@ def graph : Cmd := `[Cli|
"from" : ModuleName; "Only show the downstream dependencies of the specified module."
"exclude-meta"; "Exclude any files starting with `Mathlib.[Tactic|Lean|Util|Mathport]`."
"include-deps"; "Include used files from other libraries (not including Lean itself and `std`)"
"mark-module"; "visually highlight the current module. Only sensible in combination with `--include-deps`"
"include-std"; "Include used files from the Lean standard library (implies 'include-deps')"
"include-lean"; "Include used files from Lean itself (implies 'include-deps' and 'include-std')"
"mark-module"; "Visually highlight the current module. (implies `--include-deps`)"
"include-std"; "Include used files from the Lean standard library (implies `--include-deps`)"
"include-lean"; "Include used files from Lean itself (implies `--include-deps` and `--include-std`)"

ARGS:
...outputs : String; "Filename(s) for the output. \
Expand Down

0 comments on commit 3c90f51

Please sign in to comment.