Skip to content

Commit

Permalink
var name
Browse files Browse the repository at this point in the history
  • Loading branch information
joneugster committed Sep 5, 2024
1 parent 940ea61 commit 96e69cb
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions ImportGraph/Cli.lean
Original file line number Diff line number Diff line change
Expand Up @@ -154,8 +154,8 @@ def importGraphCLI (args : Cli.Parsed) : IO UInt32 := do
let graph₂ := match args.flag? "to" with
| none => graph.filter (fun n _ => n != to)
| some _ => graph
let gexFile := Graph.toGexf graph₂ p env
outFiles := outFiles.insert "gexf" gexFile
let gexfFile := Graph.toGexf graph₂ p env
outFiles := outFiles.insert "gexf" gexfFile
return outFiles

catch err =>
Expand Down

0 comments on commit 96e69cb

Please sign in to comment.