Skip to content
This repository was archived by the owner on Aug 29, 2024. It is now read-only.

Commit

Permalink
perf: add another dsimp into If.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
hargoniX committed Jun 25, 2024
1 parent be4fb62 commit f4033ce
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions LeanSAT/AIG/If.lean
Original file line number Diff line number Diff line change
Expand Up @@ -63,6 +63,7 @@ theorem denote_mkIfCached {aig : AIG α} {input : TernaryInput aig} :
if ⟦aig, input.discr, assign⟧ then ⟦aig, input.lhs, assign⟧ else ⟦aig, input.rhs, assign⟧ := by
rw [if_as_bool]
unfold mkIfCached
dsimp
simp only [TernaryInput.cast, Ref_cast', id_eq, Int.reduceNeg, denote_mkOrCached,
denote_projected_entry, denote_mkAndCached, denote_mkNotCached]
congr 2
Expand Down

0 comments on commit f4033ce

Please sign in to comment.