Skip to content

Commit

Permalink
chore: expand comment
Browse files Browse the repository at this point in the history
  • Loading branch information
tobiasgrosser committed Jan 2, 2025
1 parent a127c9d commit 3c0d9bf
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion src/Lean/Elab/Tactic/BVDecide/Frontend/Normalize.lean
Original file line number Diff line number Diff line change
Expand Up @@ -222,7 +222,8 @@ def rewriteRulesPass (maxSteps : Nat) : Pass where
return newGoal

/--
Responsible for applying short-circuit optimizations for `*`.
Responsible for applying short-circuit optimizations for `*`, e.g.,
translating `x1 * y == x2 * y` to `!(!x1 == x2 && !x1 * y == x2 * y)`.
-/
def shortCircuitPass (maxSteps : Nat) : Pass where
name := `shortCircuitPass
Expand Down

0 comments on commit 3c0d9bf

Please sign in to comment.