From 3898e69ad9f5318ca13765c0ed01be6f222fa335 Mon Sep 17 00:00:00 2001 From: luisacicolini Date: Tue, 1 Oct 2024 12:05:53 +0100 Subject: [PATCH] fix parentheses --- src/Init/Data/BitVec/Lemmas.lean | 2 +- 1 file changed, 1 insertion(+), 1 deletion(-) diff --git a/src/Init/Data/BitVec/Lemmas.lean b/src/Init/Data/BitVec/Lemmas.lean index 0168e52ebae6..44db8a636191 100644 --- a/src/Init/Data/BitVec/Lemmas.lean +++ b/src/Init/Data/BitVec/Lemmas.lean @@ -463,7 +463,7 @@ theorem toInt_pos_iff {w : Nat} {x : BitVec w} : 0 ≤ BitVec.toInt x ↔ 2 * x.toNat < 2 ^ w := by simp [toInt_eq_toNat_cond]; omega -theorem eq_zero_or_eq_one {a : BitVec 1} : a = 0#1 ∨ a = 1#1 := by +theorem eq_zero_or_eq_one (a : BitVec 1) : a = 0#1 ∨ a = 1#1 := by obtain ⟨a, ha⟩ := a simp only [Nat.reducePow] have acases : a = 0 ∨ a = 1 := by omega