Documentation

Mathlib.Data.Fintype.Prod

fintype instance for the product of two fintypes. #

theorem Set.toFinset_prod {α : Type u_1} {β : Type u_2} (s : Set α) (t : Set β) [inst : Fintype s] [inst : Fintype t] [inst : Fintype ↑(s ×ˢ t)] :
theorem Set.toFinset_off_diag {α : Type u_1} {s : Set α} [inst : DecidableEq α] [inst : Fintype s] [inst : Fintype ↑(Set.offDiag s)] :
instance instFintypeProd (α : Type u_1) (β : Type u_2) [inst : Fintype α] [inst : Fintype β] :
Fintype (α × β)
Equations
@[simp]
theorem Finset.univ_product_univ {α : Type u_1} {β : Type u_2} [inst : Fintype α] [inst : Fintype β] :
Finset.univ ×ᶠ Finset.univ = Finset.univ
@[simp]
theorem Fintype.card_prod (α : Type u_1) (β : Type u_2) [inst : Fintype α] [inst : Fintype β] :
@[simp]
theorem infinite_prod {α : Type u_2} {β : Type u_1} :
instance Pi.infinite_of_left {ι : Sort u_1} {π : ιType u_2} [inst : ∀ (i : ι), Nontrivial (π i)] [inst : Infinite ι] :
Infinite ((i : ι) → π i)
Equations
theorem Pi.infinite_of_exists_right {ι : Type u_1} {π : ιType u_2} (i : ι) [inst : Infinite (π i)] [inst : ∀ (i : ι), Nonempty (π i)] :
Infinite ((i : ι) → π i)

If at least one π i is infinite and the rest nonempty, the pi type of all π is infinite.

instance Pi.infinite_of_right {ι : Type u_1} {π : ιType u_2} [inst : ∀ (i : ι), Infinite (π i)] [inst : Nonempty ι] :
Infinite ((i : ι) → π i)

See Pi.infinite_of_exists_right for the case that only one π i is infinite.

Equations
instance Function.infinite_of_left {ι : Sort u_1} {π : Type u_2} [inst : Nontrivial π] [inst : Infinite ι] :
Infinite (ιπ)

Non-dependent version of Pi.infinite_of_left.

Equations