Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Aug 10, 2024
1 parent 1279860 commit a13dba6
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Batteries/Data/ByteArray.lean
Original file line number Diff line number Diff line change
Expand Up @@ -132,7 +132,7 @@ private def ofFnAux (f : Fin n → UInt8) : ByteArray := go 0 (mkEmpty n) where
termination_by n - i

@[csimp] private theorem ofFn_eq_ofFnAux : @ofFn = @ofFnAux := by
funext n f; ext; simp [ofFnAux, Array.ofFn, ofFnAux_data, mkEmpty]
funext n f; ext1; simp [ofFnAux, Array.ofFn, ofFnAux_data, mkEmpty]
where
ofFnAux_data {n} (f : Fin n → UInt8) (i) {acc} :
(ofFnAux.go f i acc).data = Array.ofFn.go f i acc.data := by
Expand Down

0 comments on commit a13dba6

Please sign in to comment.