Theory Cube_Dissection
theory Cube_Dissection
imports Complex_Main "HOL-Library.Disjoint_Sets" "HOL-Library.Infinite_Set"
begin
text "Proof that a cube can't be dissected into a finite number of subcubes of different size
This formalization is heavily inspired by the Lean proof of the same fact, \<^cite>‹leanproof›.
One goal of this project, is that by restricting to cubes of dimension 3 the logic will
be easier to follow"
section "Basic definitions"
subsection "point and cube definitions"
record point = px:: real py::real pz::real
record cube = point:: point width::real