mathlib documentation

data.​list.​min_max

data.​list.​min_max

def list.​argmax₂ {α : Type u_1} {β : Type u_2} [decidable_linear_order β] :
(α → β)option αα → option α

Auxiliary definition to define argmax

Equations
def list.​argmax {α : Type u_1} {β : Type u_2} [decidable_linear_order β] :
(α → β)list αoption α

argmax f l returns some a, where a of l that maximises f a. If there are a b such that f a = f b, it returns whichever of a or b comes first in the list. argmax f [] = none`

Equations
def list.​argmin {α : Type u_1} {β : Type u_2} [decidable_linear_order β] :
(α → β)list αoption α

argmin f l returns some a, where a of l that minimises f a. If there are a b such that f a = f b, it returns whichever of a or b comes first in the list. argmin f [] = none`

Equations
@[simp]
theorem list.​argmax_two_self {α : Type u_1} {β : Type u_2} [decidable_linear_order β] (f : α → β) (a : α) :

@[simp]
theorem list.​argmax_nil {α : Type u_1} {β : Type u_2} [decidable_linear_order β] (f : α → β) :

@[simp]
theorem list.​argmin_nil {α : Type u_1} {β : Type u_2} [decidable_linear_order β] (f : α → β) :

@[simp]
theorem list.​argmax_singleton {α : Type u_1} {β : Type u_2} [decidable_linear_order β] {f : α → β} {a : α} :

@[simp]
theorem list.​argmin_singleton {α : Type u_1} {β : Type u_2} [decidable_linear_order β] {f : α → β} {a : α} :

@[simp]
theorem list.​foldl_argmax₂_eq_none {α : Type u_1} {β : Type u_2} [decidable_linear_order β] {f : α → β} {l : list α} {o : option α} :

theorem list.​argmax_mem {α : Type u_1} {β : Type u_2} [decidable_linear_order β] {f : α → β} {l : list α} {m : α} :
m list.argmax f lm l

theorem list.​argmin_mem {α : Type u_1} {β : Type u_2} [decidable_linear_order β] {f : α → β} {l : list α} {m : α} :
m list.argmin f lm l

@[simp]
theorem list.​argmax_eq_none {α : Type u_1} {β : Type u_2} [decidable_linear_order β] {f : α → β} {l : list α} :

@[simp]
theorem list.​argmin_eq_none {α : Type u_1} {β : Type u_2} [decidable_linear_order β] {f : α → β} {l : list α} :

theorem list.​le_argmax_of_mem {α : Type u_1} {β : Type u_2} [decidable_linear_order β] {f : α → β} {a m : α} {l : list α} :
a lm list.argmax f lf a f m

theorem list.​argmin_le_of_mem {α : Type u_1} {β : Type u_2} [decidable_linear_order β] {f : α → β} {a m : α} {l : list α} :
a lm list.argmin f lf m f a

theorem list.​argmax_concat {α : Type u_1} {β : Type u_2} [decidable_linear_order β] (f : α → β) (a : α) (l : list α) :
list.argmax f (l ++ [a]) = (list.argmax f l).cases_on (option.some a) (λ (c : α), ite (f a f c) (option.some c) (option.some a))

theorem list.​argmin_concat {α : Type u_1} {β : Type u_2} [decidable_linear_order β] (f : α → β) (a : α) (l : list α) :
list.argmin f (l ++ [a]) = (list.argmin f l).cases_on (option.some a) (λ (c : α), ite (f c f a) (option.some c) (option.some a))

theorem list.​argmax_cons {α : Type u_1} {β : Type u_2} [decidable_linear_order β] (f : α → β) (a : α) (l : list α) :
list.argmax f (a :: l) = (list.argmax f l).cases_on (option.some a) (λ (c : α), ite (f c f a) (option.some a) (option.some c))

theorem list.​argmin_cons {α : Type u_1} {β : Type u_2} [decidable_linear_order β] (f : α → β) (a : α) (l : list α) :
list.argmin f (a :: l) = (list.argmin f l).cases_on (option.some a) (λ (c : α), ite (f a f c) (option.some a) (option.some c))

theorem list.​index_of_argmax {α : Type u_1} {β : Type u_2} [decidable_linear_order β] [decidable_eq α] {f : α → β} {l : list α} {m : α} (a : m list.argmax f l) {a_1 : α} :
a_1 lf m f a_1list.index_of m l list.index_of a_1 l

theorem list.​index_of_argmin {α : Type u_1} {β : Type u_2} [decidable_linear_order β] [decidable_eq α] {f : α → β} {l : list α} {m : α} (a : m list.argmin f l) {a_1 : α} :
a_1 lf a_1 f mlist.index_of m l list.index_of a_1 l

theorem list.​mem_argmax_iff {α : Type u_1} {β : Type u_2} [decidable_linear_order β] [decidable_eq α] {f : α → β} {m : α} {l : list α} :
m list.argmax f l m l (∀ (a : α), a lf a f m) ∀ (a : α), a lf m f alist.index_of m l list.index_of a l

theorem list.​argmax_eq_some_iff {α : Type u_1} {β : Type u_2} [decidable_linear_order β] [decidable_eq α] {f : α → β} {m : α} {l : list α} :
list.argmax f l = option.some m m l (∀ (a : α), a lf a f m) ∀ (a : α), a lf m f alist.index_of m l list.index_of a l

theorem list.​mem_argmin_iff {α : Type u_1} {β : Type u_2} [decidable_linear_order β] [decidable_eq α] {f : α → β} {m : α} {l : list α} :
m list.argmin f l m l (∀ (a : α), a lf m f a) ∀ (a : α), a lf a f mlist.index_of m l list.index_of a l

theorem list.​argmin_eq_some_iff {α : Type u_1} {β : Type u_2} [decidable_linear_order β] [decidable_eq α] {f : α → β} {m : α} {l : list α} :
list.argmin f l = option.some m m l (∀ (a : α), a lf m f a) ∀ (a : α), a lf a f mlist.index_of m l list.index_of a l

def list.​maximum {α : Type u_1} [decidable_linear_order α] :
list αwith_bot α

maximum l returns an with_bot α, the largest element of l for nonempty lists, and for []

Equations
def list.​minimum {α : Type u_1} [decidable_linear_order α] :
list αwith_top α

minimum l returns an with_top α, the smallest element of l for nonempty lists, and for []

Equations
@[simp]

@[simp]

@[simp]
theorem list.​maximum_singleton {α : Type u_1} [decidable_linear_order α] (a : α) :

@[simp]
theorem list.​minimum_singleton {α : Type u_1} [decidable_linear_order α] (a : α) :

theorem list.​maximum_mem {α : Type u_1} [decidable_linear_order α] {l : list α} {m : α} :
l.maximum = mm l

theorem list.​minimum_mem {α : Type u_1} [decidable_linear_order α] {l : list α} {m : α} :
l.minimum = mm l

@[simp]
theorem list.​maximum_eq_none {α : Type u_1} [decidable_linear_order α] {l : list α} :

@[simp]
theorem list.​minimum_eq_none {α : Type u_1} [decidable_linear_order α] {l : list α} :

theorem list.​le_maximum_of_mem {α : Type u_1} [decidable_linear_order α] {a m : α} {l : list α} :
a ll.maximum = ma m

theorem list.​minimum_le_of_mem {α : Type u_1} [decidable_linear_order α] {a m : α} {l : list α} :
a ll.minimum = mm a

theorem list.​le_maximum_of_mem' {α : Type u_1} [decidable_linear_order α] {a : α} {l : list α} :
a la l.maximum

theorem list.​le_minimum_of_mem' {α : Type u_1} [decidable_linear_order α] {a : α} {l : list α} :
a ll.minimum a

theorem list.​maximum_concat {α : Type u_1} [decidable_linear_order α] (a : α) (l : list α) :
(l ++ [a]).maximum = max l.maximum a

theorem list.​minimum_concat {α : Type u_1} [decidable_linear_order α] (a : α) (l : list α) :
(l ++ [a]).minimum = min l.minimum a

theorem list.​maximum_cons {α : Type u_1} [decidable_linear_order α] (a : α) (l : list α) :

theorem list.​minimum_cons {α : Type u_1} [decidable_linear_order α] (a : α) (l : list α) :

theorem list.​maximum_eq_coe_iff {α : Type u_1} [decidable_linear_order α] {m : α} {l : list α} :
l.maximum = m m l ∀ (a : α), a la m

theorem list.​minimum_eq_coe_iff {α : Type u_1} [decidable_linear_order α] {m : α} {l : list α} :
l.minimum = m m l ∀ (a : α), a lm a