Skip to content

Commit

Permalink
fix: cond reflection bug in bv_decide (#6517)
Browse files Browse the repository at this point in the history
This PR fixes a slight bug that was created in the reflection of `bif`
in `bv_decide`.

Tagged as changelog-no as the code in question isn't in an RC yet.
  • Loading branch information
hargoniX authored Jan 3, 2025
1 parent 7b496bf commit 58d178e
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Std/Tactic/BVDecide/Reflect.lean
Original file line number Diff line number Diff line change
Expand Up @@ -156,7 +156,7 @@ theorem or_congr (lhs rhs lhs' rhs' : Bool) (h1 : lhs' = lhs) (h2 : rhs' = rhs)

theorem cond_congr (discr lhs rhs discr' lhs' rhs' : Bool) (h1 : discr' = discr) (h2 : lhs' = lhs)
(h3 : rhs' = rhs) :
(bif discr' = true then lhs' else rhs') = (bif discr = true then lhs else rhs) := by
(bif discr' then lhs' else rhs') = (bif discr then lhs else rhs) := by
simp[*]

theorem false_of_eq_true_of_eq_false (h₁ : x = true) (h₂ : x = false) : False := by
Expand Down

0 comments on commit 58d178e

Please sign in to comment.