File tree Expand file tree Collapse file tree 1 file changed +4
-3
lines changed
src/Std/Tactic/BVDecide/Bitblast/BVExpr/Circuit/Lemmas/Operations Expand file tree Collapse file tree 1 file changed +4
-3
lines changed Original file line number Diff line number Diff line change @@ -10,7 +10,9 @@ import Std.Tactic.BVDecide.Bitblast.BVExpr.Circuit.Lemmas.Const
1010
1111/-!
1212This module contains the verification of the bitblaster for `BitVec.clz` from
13- `Impl.Operations.Clz`.
13+ `Impl.Operations.Clz`. We prove that the accumulator of the `go` function
14+ at step`n` represents the portion of the `ite` nodes in the AIG constructed for
15+ bits `0` until `n`.
1416-/
1517
1618namespace Std.Tactic.BVDecide
@@ -46,8 +48,7 @@ theorem go_denote_eq {w : Nat} (aig : AIG α)
4648 split at hgo
4749 · case isTrue h =>
4850 simp at hgo
49- rw [← hgo]
50- rw [go_denote_eq]
51+ rw [← hgo, go_denote_eq]
5152 · intro idx hidx
5253 rw [AIG.LawfulVecOperator.denote_mem_prefix (f := RefVec.ite)]
5354 · simp [hx]
You can’t perform that action at this time.
0 commit comments