@@ -52,16 +52,20 @@ theorem getElem_ofFnLEAux (f : Fin n → Bool) (i) (h : i < n) (h' : i < m) :
5252@[simp] theorem getElem_ofFnLE (f : Fin n → Bool) (i) (h : i < n) : (ofFnLE f)[i] = f ⟨i, h⟩ :=
5353 getElem_ofFnLEAux ..
5454
55- theorem getLsb'_ofFnLE (f : Fin n → Bool) (i) : (ofFnLE f).getLsb' i = f i := by simp
55+ theorem getLsb_ofFnLE (f : Fin n → Bool) (i) : (ofFnLE f).getLsb i = f i := by simp
56+
57+ @[deprecated (since := "2025-06-17")] alias getLsb'_ofFnLE := getLsb_ofFnLE
5658
5759theorem getLsbD_ofFnLE (f : Fin n → Bool) (i) :
5860 (ofFnLE f).getLsbD i = if h : i < n then f ⟨i, h⟩ else false := by
5961 split
6062 · next h => rw [getLsbD_eq_getElem h, getElem_ofFnLE]
6163 · next h => rw [getLsbD_of_ge _ _ (Nat.ge_of_not_lt h)]
6264
63- @[simp] theorem getMsb'_ofFnLE (f : Fin n → Bool) (i) : (ofFnLE f).getMsb' i = f i.rev := by
64- simp [getMsb'_eq_getLsb', Fin.rev]; congr 2 ; omega
65+ @[simp] theorem getMsb_ofFnLE (f : Fin n → Bool) (i) : (ofFnLE f).getMsb i = f i.rev := by
66+ simp [getMsb_eq_getLsb, Fin.rev]; congr 2 ; omega
67+
68+ @[deprecated (since := "2025-06-17")] alias getMsb'_ofFnLE := getMsb_ofFnLE
6569
6670theorem getMsbD_ofFnLE (f : Fin n → Bool) (i) :
6771 (ofFnLE f).getMsbD i = if h : i < n then f (Fin.rev ⟨i, h⟩) else false := by
@@ -88,16 +92,20 @@ theorem msb_ofFnLE (f : Fin n → Bool) :
8892@[simp] theorem getElem_ofFnBE (f : Fin n → Bool) (i) (h : i < n) :
8993 (ofFnBE f)[i] = f (Fin.rev ⟨i, h⟩) := by simp [ofFnBE]
9094
91- theorem getLsb'_ofFnBE (f : Fin n → Bool) (i) : (ofFnBE f).getLsb' i = f i.rev := by
95+ theorem getLsb_ofFnBE (f : Fin n → Bool) (i) : (ofFnBE f).getLsb i = f i.rev := by
9296 simp
9397
98+ @[deprecated (since := "2025-06-17")] alias getLsb'_ofFnBE := getLsb_ofFnBE
99+
94100theorem getLsbD_ofFnBE (f : Fin n → Bool) (i) :
95101 (ofFnBE f).getLsbD i = if h : i < n then f (Fin.rev ⟨i, h⟩) else false := by
96102 simp [ofFnBE, getLsbD_ofFnLE]
97103
98- @[simp] theorem getMsb'_ofFnBE (f : Fin n → Bool) (i) : (ofFnBE f).getMsb' i = f i := by
104+ @[simp] theorem getMsb_ofFnBE (f : Fin n → Bool) (i) : (ofFnBE f).getMsb i = f i := by
99105 simp [ofFnBE]
100106
107+ @[deprecated (since := "2025-06-17")] alias getMsb'_ofFnBE := getMsb_ofFnBE
108+
101109theorem getMsbD_ofFnBE (f : Fin n → Bool) (i) :
102110 (ofFnBE f).getMsbD i = if h : i < n then f ⟨i, h⟩ else false := by
103111 simp [ofFnBE, getMsbD_ofFnLE]
0 commit comments