Format area axioms for easier linking.

finite-set-exercises
Joshua Potter 2023-05-06 12:01:37 -06:00
parent b632097ce2
commit 74f52f02b8
1 changed files with 28 additions and 59 deletions

View File

@ -28,91 +28,80 @@ introduced by Apostol. He denotes this function as `a`.
-/ -/
axiom area : ∀ ⦃x⦄, x ∈ 𝓜 axiom area : ∀ ⦃x⦄, x ∈ 𝓜
/-- /-! ## Nonnegative Property
The nonnegative property.
For each set `S` in `𝓜`, we have `a(S) ≥ 0`. For each set `S` in `𝓜`, we have `a(S) ≥ 0`.
-/ -/
axiom area_ge_zero {S : Set ℝ²} (h : S ∈ 𝓜): area h ≥ 0 axiom area_ge_zero {S : Set ℝ²} (h : S ∈ 𝓜): area h ≥ 0
/-- /-! ## Additive Property
The additive property (i).
If `S` and `T` are in `𝓜`, then `S T` in `𝓜`. If `S` and `T` are in `𝓜`, then `S T` in `𝓜`, `S ∩ T` in `𝓜`, and
`a(S T) = a(S) + a(T) - a(S ∩ T)`.
-/ -/
axiom measureable_imp_union_measurable {S T : Set ℝ²} (hS : S ∈ 𝓜) (hT : T ∈ 𝓜) axiom measureable_imp_union_measurable {S T : Set ℝ²} (hS : S ∈ 𝓜) (hT : T ∈ 𝓜)
: S T ∈ 𝓜 : S T ∈ 𝓜
/--
The additive property (ii).
If `S` and `T` are in `𝓜`, then `S ∩ T` in `𝓜`.
-/
axiom measurable_imp_inter_measurable {S T : Set ℝ²} (hS : S ∈ 𝓜) (hT : T ∈ 𝓜) axiom measurable_imp_inter_measurable {S T : Set ℝ²} (hS : S ∈ 𝓜) (hT : T ∈ 𝓜)
: S ∩ T ∈ 𝓜 : S ∩ T ∈ 𝓜
/--
The additive property (iii).
If `S` and `T` are in `𝓜`, then `a(S T) = a(S) + a(T) - a(S ∩ T)`.
-/
axiom union_area_eq_area_add_area_sub_inter_area axiom union_area_eq_area_add_area_sub_inter_area
{S T : Set ℝ²} (hS : S ∈ 𝓜) (hT : T ∈ 𝓜) {S T : Set ℝ²} (hS : S ∈ 𝓜) (hT : T ∈ 𝓜)
: area (measureable_imp_union_measurable hS hT) = : area (measureable_imp_union_measurable hS hT) =
area hS + area hT - area (measurable_imp_inter_measurable hS hT) area hS + area hT - area (measurable_imp_inter_measurable hS hT)
/-- /-! ## Difference Property
The difference property (i).
If `S` and `T` are in `𝓜` with `S ⊆ T`, then `T - S` is in `𝓜`. If `S` and `T` are in `𝓜` with `S ⊆ T`, then `T - S` is in `𝓜` and
`a(T - S) = a(T) - a(S)`.
-/ -/
axiom measureable_imp_diff_measurable axiom measureable_imp_diff_measurable
{S T : Set ℝ²} (hS : S ∈ 𝓜) (hT : T ∈ 𝓜) (h : S ⊆ T) {S T : Set ℝ²} (hS : S ∈ 𝓜) (hT : T ∈ 𝓜) (h : S ⊆ T)
: T \ S ∈ 𝓜 : T \ S ∈ 𝓜
/--
The difference property (ii).
If `S` and `T` are in `𝓜` with `S ⊆ T`, then `a(T - S) = a(T) - a(S)`.
-/
axiom diff_area_eq_area_sub_area axiom diff_area_eq_area_sub_area
{S T : Set ℝ²} (hS : S ∈ 𝓜) (hT : T ∈ 𝓜) (h : S ⊆ T) {S T : Set ℝ²} (hS : S ∈ 𝓜) (hT : T ∈ 𝓜) (h : S ⊆ T)
: area (measureable_imp_diff_measurable hS hT h) = area hT - area hS : area (measureable_imp_diff_measurable hS hT h) = area hT - area hS
/-- /-! ## Invariance Under Congruence
Invariance under congruence (i).
If a set `S` is in `𝓜` and if `T` is congruent to `S`, then `T` is also in `𝓜`.. If a set `S` is in `𝓜` and if a set `T` is congruent to `S`, then `T` is also in
`𝓜` and `a(S) = a(T)`.
-/ -/
axiom measurable_congruent_imp_measurable axiom measurable_congruent_imp_measurable
{S T : Set ℝ²} (hS : S ∈ 𝓜) (h : congruent S T) {S T : Set ℝ²} (hS : S ∈ 𝓜) (h : congruent S T)
: T ∈ 𝓜 : T ∈ 𝓜
/--
Invariance under congruence (ii).
If a set `S` is in `𝓜` and if `T` is congruent to `S`, then `a(S) = a(T)`.
-/
axiom congruent_imp_area_eq_area axiom congruent_imp_area_eq_area
{S T : Set ℝ²} (hS : S ∈ 𝓜) (h : congruent S T) {S T : Set ℝ²} (hS : S ∈ 𝓜) (h : congruent S T)
: area hS = area (measurable_congruent_imp_measurable hS h) : area hS = area (measurable_congruent_imp_measurable hS h)
/--
Choice of scale (i).
Every rectangle `R` is in `𝓜`. /-! ## Choice of Scale
(i) Every rectangle `R` is in `𝓜`.
(ii) If the edges of rectangle `R` have lengths `h` and `k`, then `a(R) = hk`.
-/ -/
axiom rectangle_measurable (R : Rectangle) axiom rectangle_measurable (R : Rectangle)
: R.set_def ∈ 𝓜 : R.set_def ∈ 𝓜
/--
Choice of scale (ii).
If the edges of rectangle `R` have lengths `h` and `k`, then `a(R) = hk`.
-/
axiom rectangle_area_eq_mul_edge_lengths (R : Rectangle) axiom rectangle_area_eq_mul_edge_lengths (R : Rectangle)
: area (rectangle_measurable R) = R.width * R.height : area (rectangle_measurable R) = R.width * R.height
/-! ## Exhaustion property
Let `Q` be a set that can be enclosed between two step regions `S` and `T`, so
that (1.1) `S ⊆ Q ⊆ T`. If there is one and only one number `k` which satisfies
the inequalities `a(S) ≤ k ≤ a(T)` for all step regions `S` and `T` satisfying
(1.1), then `Q` is measurable and `a(Q) = k`.
-/
/-- /--
Every step region is measurable. This follows from the choice of scale axiom, Every step region is measurable. This follows from the choice of scale axiom,
and the fact all step regions are equivalent to the union of a collection of and the fact all step regions are equivalent to the union of a collection of
@ -121,36 +110,16 @@ rectangles.
theorem step_function_measurable (S : Function.Step) : S.set_def ∈ 𝓜 := by theorem step_function_measurable (S : Function.Step) : S.set_def ∈ 𝓜 := by
sorry sorry
/--
Exhaustion property.
Let `Q` be a set that can be enclosed between two step regions `S` and `T`, so
that (1.1) `S ⊆ Q ⊆ T`. If there is one and only one number `k` which satisfies
the inequalities `a(S) ≤ k ≤ a(T)` for all step regions `S` and `T` satisfying
(1.1), then `Q` is measurable and `a(Q) = k`.
-/
def forall_subset_between_step_imp_le_between_area (k : ) (Q : Set ℝ²) := def forall_subset_between_step_imp_le_between_area (k : ) (Q : Set ℝ²) :=
∀ S T : Function.Step, ∀ S T : Function.Step,
(hS : S.set_def ⊆ Q) → (hS : S.set_def ⊆ Q) →
(hT : Q ⊆ T.set_def) → (hT : Q ⊆ T.set_def) →
area (step_function_measurable S) ≤ k ∧ k ≤ area (step_function_measurable T) area (step_function_measurable S) ≤ k ∧ k ≤ area (step_function_measurable T)
/--
Exhaustion property (i).
If there exists some `k` satisfying the description in the above `def`, then `Q`
is measurable.
-/
axiom exhaustion_exists_unique_imp_measurable (Q : Set ℝ²) axiom exhaustion_exists_unique_imp_measurable (Q : Set ℝ²)
: (∃! k : , forall_subset_between_step_imp_le_between_area k Q) : (∃! k : , forall_subset_between_step_imp_le_between_area k Q)
→ Q ∈ 𝓜 → Q ∈ 𝓜
/--
Exhaustion property (ii).
If there exists some `k` satisfying the description in the above `def`, then `Q`
satisfies `a(Q) = k`.
-/
axiom exhaustion_exists_unique_imp_area_eq (Q : Set ℝ²) axiom exhaustion_exists_unique_imp_area_eq (Q : Set ℝ²)
: ∃ k : , : ∃ k : ,
(h : forall_subset_between_step_imp_le_between_area k Q ∧ (h : forall_subset_between_step_imp_le_between_area k Q ∧