THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Proof that a cube (in dimension n ≥ 3) cannot be cubed: There does not exist a partition of a cube into finitely many smaller cubes (at least two) of different sizes.
We follow the proof described here: http://www.alaricstephen.com/main-featured/2017/9/28/cubing-a-cube-proof
Given three intervals I, J, K
such that J ⊂ I
,
neither endpoint of J
coincides with an endpoint of I
, ¬ (K ⊆ J)
and
K
does not lie completely to the left nor completely to the right of J
.
Then I ∩ K \ J
is nonempty.
A (hyper)-cube (in standard orientation) is a vector b
consisting of the bottom-left point
of the cube, a width w
and a proof that w > 0
. We use functions from fin n
to denote vectors.
Instances for theorems_100.82.cube
- theorems_100.82.cube.has_sizeof_inst
- pairwise_disjoint : pairwise (disjoint on theorems_100.«82».cube.to_set ∘ cs)
- Union_eq : (⋃ (i : ι), (cs i).to_set) = theorems_100.«82».cube.unit_cube.to_set
- injective : function.injective (theorems_100.«82».cube.w ∘ cs)
- three_le : 3 ≤ n
A finite family of (at least 2) cubes partitioning the unit cube with different sizes
The width of any cube in the partition cannot be 1.
The top of a cube (which is the bottom of the cube shifted up by its width) must be covered by bottoms of (other) cubes in the family.
A valley is a square on which cubes in the family of cubes are placed, so that the cubes
completely cover the valley and none of those cubes is partially outside the square.
We also require that no cube on it has the same size as the valley (so that there are at least
two cubes on the valley).
This is the main concept in the formalization.
We prove that the smallest cube on a valley has another valley on the top of it, which
gives an infinite sequence of cubes in the partition, which contradicts the finiteness.
A valley is characterized by a cube c
(which is not a cube in the family cs) by considering
the bottom face of c
.
The bottom of the unit cube is a valley
Every cube in the valley must be smaller than it
There are at least two cubes in a valley
We let mi
be the (index for the) smallest cube in the valley c
Equations
- theorems_100.«82».mi h v = classical.some _
The top of mi
cannot be 1, since there is a larger cube in the valley
If mi
lies on the boundary of the valley in dimension j, then this lemma expresses that all
other cubes on the same boundary extend further from the boundary.
More precisely, there is a j-th coordinate x : ℝ
in the valley, but not in mi
,
such that every cube that shares a (particular) j-th coordinate with mi
also contains j-th
coordinate x
mi
cannot lie on the boundary of the valley. Otherwise, the cube adjacent to it in the j
-th
direction will intersect one of the neighbouring cubes on the same boundary as mi
.
The same result that mi
cannot lie on the boundary of the valley written as inequalities.
The top of mi
gives rise to a new valley, since the neighbouring cubes extend further upward
than mi
.
We get a sequence of cubes whose size is decreasing
Equations
- theorems_100.«82».sequence_of_cubes h (k + 1) = let v : theorems_100.«82».valley cs (cs (theorems_100.«82».sequence_of_cubes h k).val).shift_up := _ in ⟨theorems_100.«82».mi h v _inst_1, _⟩
- theorems_100.«82».sequence_of_cubes h 0 = let v : theorems_100.«82».valley cs theorems_100.«82».cube.unit_cube := _ in ⟨theorems_100.«82».mi h v _inst_1, _⟩
The infinite sequence of cubes contradicts the finiteness of the family.
Dissection of Cubes: A cube cannot be cubed.