Skip to content

Commit

Permalink
Update src/Std/Sat/AIG/Basic.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Markus Himmel <markus@lean-fro.org>
  • Loading branch information
hargoniX and TwoFX authored Aug 8, 2024
1 parent 949ed3f commit ca1e212
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/Std/Sat/AIG/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -284,8 +284,8 @@ structure Entrypoint (α : Type) [DecidableEq α] [Hashable α] where
/--
Transform an `Entrypoint` into a graphviz string. Useful for debugging purposes.
-/
def toGraphviz {α : Type} [DecidableEq α] [ToString α] [Hashable α] (entry : Entrypoint α)
: String :=
def toGraphviz {α : Type} [DecidableEq α] [ToString α] [Hashable α] (entry : Entrypoint α) :
String :=
let ⟨⟨decls, _, hinv⟩, ⟨idx, h⟩⟩ := entry
let (dag, s) := go "" decls hinv idx h |>.run .empty
let nodes := s.fold (fun x y ↦ x ++ toGraphvizString decls y) ""
Expand Down

0 comments on commit ca1e212

Please sign in to comment.