Zulip Chat Archive

Stream: Is there code for X?

Topic: zipWith


Scott Morrison (Sep 13 2023 at 11:11):

What is the closest we have to:

set_option autoImplicit true

@[simp] theorem zipWith_data {A : Array α} {B : Array β} {f : α  β  γ} :
    (Array.zipWith A B f).data = List.zipWith f A.data B.data := by
  sorry

Anything characterising Array.zipWith would be helpful!

Martin Dvořák (Sep 13 2023 at 11:18):

docs#Array.zipWith
There doesn't seem to be much.

Eric Rodriguez (Sep 13 2023 at 11:25):

@loogle Array.zipWith, List.zipWith

loogle (Sep 13 2023 at 11:25):

:shrug: nothing found

Eric Rodriguez (Sep 13 2023 at 11:25):

@loogle Array.zipWith

loogle (Sep 13 2023 at 11:25):

:shrug: nothing found

Scott Morrison (Sep 13 2023 at 11:26):

Yeah... :-) Sorry, I'd already got that far privately, should have specified.

Eric Rodriguez (Sep 13 2023 at 11:26):

Amazing news...

Damiano Testa (Sep 13 2023 at 11:29):

Whenever I see these attempts, I am always reminded of the old time and "let me Google that for you"!. With loogle, I would really welcome a "let me Loogle that for you!"


Last updated: Dec 20 2023 at 11:08 UTC