|
|
@ -741,28 +741,37 @@ open Topology
|
|
|
|
variable {G α : Type _} [Group G] [TopologicalSpace α] [T2Space α]
|
|
|
|
variable {G α : Type _} [Group G] [TopologicalSpace α] [T2Space α]
|
|
|
|
variable [MulAction G α] [ContinuousConstSMul G α] [FaithfulSMul G α] [LocallyMoving G α]
|
|
|
|
variable [MulAction G α] [ContinuousConstSMul G α] [FaithfulSMul G α] [LocallyMoving G α]
|
|
|
|
|
|
|
|
|
|
|
|
theorem proposition_3_4_2 {α : Type _} [TopologicalSpace α] [T2Space α] [LocallyCompactSpace α] (F : Ultrafilter α):
|
|
|
|
theorem exists_compact_closure_of_le_nhds {α : Type _} [TopologicalSpace α] [T2Space α] [LocallyCompactSpace α] (F : Filter α):
|
|
|
|
(∃ p : α, ClusterPt p F) ↔ ∃ S ∈ F, IsCompact (closure S) :=
|
|
|
|
(∃ p : α, F ≤ 𝓝 p) → ∃ S ∈ F, IsCompact (closure S) :=
|
|
|
|
by
|
|
|
|
by
|
|
|
|
constructor
|
|
|
|
intro ⟨p, p_le_nhds⟩
|
|
|
|
· intro ⟨p, p_clusterPt⟩
|
|
|
|
|
|
|
|
rw [Ultrafilter.clusterPt_iff] at p_clusterPt
|
|
|
|
|
|
|
|
have ⟨S, S_in_nhds, S_compact⟩ := (compact_basis_nhds p).ex_mem
|
|
|
|
have ⟨S, S_in_nhds, S_compact⟩ := (compact_basis_nhds p).ex_mem
|
|
|
|
use S
|
|
|
|
use S
|
|
|
|
constructor
|
|
|
|
constructor
|
|
|
|
exact p_clusterPt S_in_nhds
|
|
|
|
exact p_le_nhds S_in_nhds
|
|
|
|
rw [IsClosed.closure_eq S_compact.isClosed]
|
|
|
|
rw [IsClosed.closure_eq S_compact.isClosed]
|
|
|
|
exact S_compact
|
|
|
|
exact S_compact
|
|
|
|
· intro ⟨S, S_in_F, clS_compact⟩
|
|
|
|
|
|
|
|
|
|
|
|
theorem clusterPt_of_exists_compact_closure {α : Type _} [TopologicalSpace α] [T2Space α] [LocallyCompactSpace α] (F : Filter α) [Filter.NeBot F]:
|
|
|
|
|
|
|
|
(∃ S ∈ F, IsCompact (closure S)) → ∃ p : α, ClusterPt p F :=
|
|
|
|
|
|
|
|
by
|
|
|
|
|
|
|
|
intro ⟨S, S_in_F, clS_compact⟩
|
|
|
|
have F_le_principal_S : F ≤ Filter.principal (closure S) := by
|
|
|
|
have F_le_principal_S : F ≤ Filter.principal (closure S) := by
|
|
|
|
rw [Filter.le_principal_iff]
|
|
|
|
rw [Filter.le_principal_iff]
|
|
|
|
simp
|
|
|
|
|
|
|
|
apply Filter.sets_of_superset
|
|
|
|
apply Filter.sets_of_superset
|
|
|
|
exact S_in_F
|
|
|
|
exact S_in_F
|
|
|
|
exact subset_closure
|
|
|
|
exact subset_closure
|
|
|
|
let ⟨x, _, F_clusterPt⟩ := clS_compact F_le_principal_S
|
|
|
|
let ⟨x, _, F_clusterPt⟩ := clS_compact F_le_principal_S
|
|
|
|
use x
|
|
|
|
use x
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
theorem proposition_3_4_2 {α : Type _} [TopologicalSpace α] [T2Space α] [LocallyCompactSpace α] (F : Ultrafilter α):
|
|
|
|
|
|
|
|
(∃ p : α, ClusterPt p F) ↔ ∃ S ∈ F, IsCompact (closure S) :=
|
|
|
|
|
|
|
|
by
|
|
|
|
|
|
|
|
constructor
|
|
|
|
|
|
|
|
· simp only [Ultrafilter.clusterPt_iff, <-Ultrafilter.mem_coe]
|
|
|
|
|
|
|
|
exact exists_compact_closure_of_le_nhds (F : Filter α)
|
|
|
|
|
|
|
|
· exact clusterPt_of_exists_compact_closure (F : Filter α)
|
|
|
|
|
|
|
|
|
|
|
|
end HomeoGroup
|
|
|
|
end HomeoGroup
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
@ -830,21 +839,15 @@ by
|
|
|
|
· exact subset_trans clV_ss_W W_ss_U
|
|
|
|
· exact subset_trans clV_ss_W W_ss_U
|
|
|
|
· exact IsCompact.of_isClosed_subset W_compact isClosed_closure clV_ss_W
|
|
|
|
· exact IsCompact.of_isClosed_subset W_compact isClosed_closure clV_ss_W
|
|
|
|
|
|
|
|
|
|
|
|
/--
|
|
|
|
variable [LocallyDense G α] [LocallyCompactSpace α] [HasNoIsolatedPoints α]
|
|
|
|
# Proposition 3.5
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
This proposition gives an alternative definition for an ultrafilter to converge within a set `U`.
|
|
|
|
lemma proposition_3_5_1
|
|
|
|
This alternative definition should be reconstructible entirely from the algebraic structure of `G`.
|
|
|
|
{U : Set α} (U_in_basis : U ∈ RegularSupportBasis G α) (F: Filter α):
|
|
|
|
--/
|
|
|
|
(∃ p ∈ U, F ≤ nhds p)
|
|
|
|
theorem proposition_3_5 [LocallyDense G α] [LocallyCompactSpace α] [HasNoIsolatedPoints α]
|
|
|
|
→ ∃ V : RegularSupportBasis G α, V.val ⊆ U ∧ RSuppSubsets G V.val ⊆ RSuppOrbit F G•[U] :=
|
|
|
|
{U : Set α} (U_in_basis : U ∈ RegularSupportBasis G α) (F: Ultrafilter α):
|
|
|
|
|
|
|
|
(∃ p ∈ U, ClusterPt p F)
|
|
|
|
|
|
|
|
↔ ∃ V : RegularSupportBasis G α, V.val ⊆ U ∧ RSuppSubsets G V.val ⊆ RSuppOrbit F G•[U] :=
|
|
|
|
|
|
|
|
by
|
|
|
|
by
|
|
|
|
constructor
|
|
|
|
|
|
|
|
{
|
|
|
|
|
|
|
|
simp
|
|
|
|
simp
|
|
|
|
intro p p_in_U p_clusterPt
|
|
|
|
intro p p_in_U F_le_nhds_p
|
|
|
|
have U_regular : Regular U := RegularSupportBasis.regular U_in_basis
|
|
|
|
have U_regular : Regular U := RegularSupportBasis.regular U_in_basis
|
|
|
|
|
|
|
|
|
|
|
|
-- First, get a neighborhood of p that is a subset of the closure of the orbit of G_U
|
|
|
|
-- First, get a neighborhood of p that is a subset of the closure of the orbit of G_U
|
|
|
@ -931,8 +934,7 @@ by
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
|
|
|
|
|
|
|
-- We just need to show that h⁻¹ •'' W ∈ F, that is, h⁻¹ •'' W ∈ 𝓝 p
|
|
|
|
-- We just need to show that h⁻¹ •'' W ∈ F, that is, h⁻¹ •'' W ∈ 𝓝 p
|
|
|
|
rw [Ultrafilter.clusterPt_iff] at p_clusterPt
|
|
|
|
apply F_le_nhds_p
|
|
|
|
apply p_clusterPt
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
have basis := (RegularSupportBasis.isBasis G α).nhds_hasBasis (a := p)
|
|
|
|
have basis := (RegularSupportBasis.isBasis G α).nhds_hasBasis (a := p)
|
|
|
|
rw [basis.mem_iff]
|
|
|
|
rw [basis.mem_iff]
|
|
|
@ -953,8 +955,11 @@ by
|
|
|
|
· rw [mem_smulImage, inv_inv]
|
|
|
|
· rw [mem_smulImage, inv_inv]
|
|
|
|
exact hp_in_W
|
|
|
|
exact hp_in_W
|
|
|
|
· exact Eq.subset rfl
|
|
|
|
· exact Eq.subset rfl
|
|
|
|
}
|
|
|
|
|
|
|
|
{
|
|
|
|
theorem proposition_3_5_2
|
|
|
|
|
|
|
|
{U : Set α} (F: Filter α) [Filter.NeBot F]:
|
|
|
|
|
|
|
|
(∃ V : RegularSupportBasis G α, V.val ⊆ U ∧ RSuppSubsets G V.val ⊆ RSuppOrbit F G•[U]) → ∃ p ∈ U, ClusterPt p F :=
|
|
|
|
|
|
|
|
by
|
|
|
|
intro ⟨⟨V, V_in_basis⟩, ⟨V_ss_U, subsets_ss_orbit⟩⟩
|
|
|
|
intro ⟨⟨V, V_in_basis⟩, ⟨V_ss_U, subsets_ss_orbit⟩⟩
|
|
|
|
simp only at V_ss_U
|
|
|
|
simp only at V_ss_U
|
|
|
|
simp only at subsets_ss_orbit
|
|
|
|
simp only at subsets_ss_orbit
|
|
|
@ -982,7 +987,7 @@ by
|
|
|
|
apply smulImage_compact
|
|
|
|
apply smulImage_compact
|
|
|
|
assumption
|
|
|
|
assumption
|
|
|
|
|
|
|
|
|
|
|
|
have ⟨p, p_lim⟩ := (proposition_3_4_2 F).mpr ⟨g⁻¹ •'' V'.val, ⟨gV'_in_F, gV'_compact⟩⟩
|
|
|
|
have ⟨p, p_lim⟩ := clusterPt_of_exists_compact_closure _ ⟨g⁻¹ •'' V'.val, ⟨gV'_in_F, gV'_compact⟩⟩
|
|
|
|
use p
|
|
|
|
use p
|
|
|
|
constructor
|
|
|
|
constructor
|
|
|
|
swap
|
|
|
|
swap
|
|
|
@ -999,7 +1004,21 @@ by
|
|
|
|
apply V_ss_U
|
|
|
|
apply V_ss_U
|
|
|
|
apply clV'_ss_V
|
|
|
|
apply clV'_ss_V
|
|
|
|
exact p_lim
|
|
|
|
exact p_lim
|
|
|
|
}
|
|
|
|
|
|
|
|
|
|
|
|
/--
|
|
|
|
|
|
|
|
# Proposition 3.5
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
This proposition gives an alternative definition for an ultrafilter to converge within a set `U`.
|
|
|
|
|
|
|
|
This alternative definition should be reconstructible entirely from the algebraic structure of `G`.
|
|
|
|
|
|
|
|
--/
|
|
|
|
|
|
|
|
theorem proposition_3_5 {U : Set α} (U_in_basis : U ∈ RegularSupportBasis G α) (F: Ultrafilter α):
|
|
|
|
|
|
|
|
(∃ p ∈ U, ClusterPt p F)
|
|
|
|
|
|
|
|
↔ ∃ V : RegularSupportBasis G α, V.val ⊆ U ∧ RSuppSubsets G V.val ⊆ RSuppOrbit F G•[U] :=
|
|
|
|
|
|
|
|
by
|
|
|
|
|
|
|
|
constructor
|
|
|
|
|
|
|
|
· simp only [Ultrafilter.clusterPt_iff]
|
|
|
|
|
|
|
|
exact proposition_3_5_1 U_in_basis (F : Filter α)
|
|
|
|
|
|
|
|
· exact proposition_3_5_2 (F : Filter α)
|
|
|
|
|
|
|
|
|
|
|
|
end Ultrafilter
|
|
|
|
end Ultrafilter
|
|
|
|
|
|
|
|
|
|
|
@ -1026,15 +1045,16 @@ def IsRigidSubgroup.toSubgroup {S : Set G} (S_rigid : IsRigidSubgroup S) : Subgr
|
|
|
|
simp only [S_eq, SetLike.mem_coe]
|
|
|
|
simp only [S_eq, SetLike.mem_coe]
|
|
|
|
apply Subgroup.inv_mem
|
|
|
|
apply Subgroup.inv_mem
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
@[simp]
|
|
|
|
theorem IsRigidSubgroup.mem_subgroup {S : Set G} (S_rigid : IsRigidSubgroup S) (g : G):
|
|
|
|
theorem IsRigidSubgroup.mem_subgroup {S : Set G} (S_rigid : IsRigidSubgroup S) (g : G):
|
|
|
|
g ∈ S ↔ g ∈ S_rigid.toSubgroup := by rfl
|
|
|
|
g ∈ S_rigid.toSubgroup ↔ g ∈ S := by rfl
|
|
|
|
|
|
|
|
|
|
|
|
theorem IsRigidSubgroup.toSubgroup_neBot {S : Set G} (S_rigid : IsRigidSubgroup S) :
|
|
|
|
theorem IsRigidSubgroup.toSubgroup_neBot {S : Set G} (S_rigid : IsRigidSubgroup S) :
|
|
|
|
S_rigid.toSubgroup ≠ ⊥ :=
|
|
|
|
S_rigid.toSubgroup ≠ ⊥ :=
|
|
|
|
by
|
|
|
|
by
|
|
|
|
intro eq_bot
|
|
|
|
intro eq_bot
|
|
|
|
rw [Subgroup.eq_bot_iff_forall] at eq_bot
|
|
|
|
rw [Subgroup.eq_bot_iff_forall] at eq_bot
|
|
|
|
simp only [<-mem_subgroup] at eq_bot
|
|
|
|
simp only [mem_subgroup] at eq_bot
|
|
|
|
apply S_rigid.left
|
|
|
|
apply S_rigid.left
|
|
|
|
rw [Set.eq_singleton_iff_unique_mem]
|
|
|
|
rw [Set.eq_singleton_iff_unique_mem]
|
|
|
|
constructor
|
|
|
|
constructor
|
|
|
@ -1153,6 +1173,19 @@ theorem IsRigidSubgroup.toRegularSupportBasis_mono' {S T : Set G} (S_rigid : IsR
|
|
|
|
by
|
|
|
|
by
|
|
|
|
rw [<-IsRigidSubgroup.toRegularSupportBasis_mono]
|
|
|
|
rw [<-IsRigidSubgroup.toRegularSupportBasis_mono]
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
@[simp]
|
|
|
|
|
|
|
|
theorem IsRigidSubgroup.toRegularSupportBasis_rigidStabilizer {S : Set G} (S_rigid : IsRigidSubgroup S) :
|
|
|
|
|
|
|
|
G•[(S_rigid.toRegularSupportBasis α : Set α)] = S :=
|
|
|
|
|
|
|
|
by
|
|
|
|
|
|
|
|
sorry
|
|
|
|
|
|
|
|
-- TODO: prove that `G•[S_rigid.toRegularSupportBasis] = S`
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
@[simp]
|
|
|
|
|
|
|
|
theorem IsRigidSubgroup.toRegularSupportBasis_rigidStabilizer' {S : Set G} (S_rigid : IsRigidSubgroup S) (g : G):
|
|
|
|
|
|
|
|
g ∈ G•[(S_rigid.toRegularSupportBasis α : Set α)] ↔ g ∈ S :=
|
|
|
|
|
|
|
|
by
|
|
|
|
|
|
|
|
rw [<-SetLike.mem_coe, IsRigidSubgroup.toRegularSupportBasis_rigidStabilizer]
|
|
|
|
|
|
|
|
|
|
|
|
end toRegularSupportBasis
|
|
|
|
end toRegularSupportBasis
|
|
|
|
|
|
|
|
|
|
|
|
theorem IsRigidSubgroup.conj {U : Set G} (U_rigid : IsRigidSubgroup U) (g : G) : IsRigidSubgroup ((fun h => g * h * g⁻¹) '' U) := by
|
|
|
|
theorem IsRigidSubgroup.conj {U : Set G} (U_rigid : IsRigidSubgroup U) (g : G) : IsRigidSubgroup ((fun h => g * h * g⁻¹) '' U) := by
|
|
|
@ -1184,8 +1217,14 @@ def AlgebraicOrbit (F : Filter G) (U : Set G) : Set (Subgroup G) :=
|
|
|
|
{ (W_rigid.conj g).toSubgroup | (g ∈ U) (W ∈ F) (W_rigid : IsRigidSubgroup W) }
|
|
|
|
{ (W_rigid.conj g).toSubgroup | (g ∈ U) (W ∈ F) (W_rigid : IsRigidSubgroup W) }
|
|
|
|
|
|
|
|
|
|
|
|
structure RubinFilter (G : Type _) [Group G] where
|
|
|
|
structure RubinFilter (G : Type _) [Group G] where
|
|
|
|
filter : Filter G
|
|
|
|
-- Issue: It's *really hard* to generate ultrafilters on G that satisfy the other conditions of this rubinfilter
|
|
|
|
|
|
|
|
filter : Ultrafilter G
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
-- Note: the following condition cannot be met by ultrafilters in G,
|
|
|
|
|
|
|
|
-- and doesn't seem to be necessary
|
|
|
|
-- rigid_basis : ∀ S ∈ filter, ∃ T ⊆ S, IsRigidSubgroup T
|
|
|
|
-- rigid_basis : ∀ S ∈ filter, ∃ T ⊆ S, IsRigidSubgroup T
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
-- Equivalent formulation of convergence
|
|
|
|
converges : ∀ U ∈ filter,
|
|
|
|
converges : ∀ U ∈ filter,
|
|
|
|
IsRigidSubgroup U →
|
|
|
|
IsRigidSubgroup U →
|
|
|
|
∃ V : Set G, IsRigidSubgroup V ∧ V ⊆ U ∧ AlgebraicSubsets V ⊆ AlgebraicOrbit filter U
|
|
|
|
∃ V : Set G, IsRigidSubgroup V ∧ V ⊆ U ∧ AlgebraicSubsets V ⊆ AlgebraicOrbit filter U
|
|
|
@ -1193,21 +1232,23 @@ structure RubinFilter (G : Type _) [Group G] where
|
|
|
|
-- Only really used to prove that ∀ S : Rigid, T : Rigid, S T ∈ F, S ∩ T : Rigid
|
|
|
|
-- Only really used to prove that ∀ S : Rigid, T : Rigid, S T ∈ F, S ∩ T : Rigid
|
|
|
|
ne_bot : {1} ∉ filter
|
|
|
|
ne_bot : {1} ∉ filter
|
|
|
|
|
|
|
|
|
|
|
|
instance : Coe (RubinFilter G) (Filter G) where
|
|
|
|
instance : Coe (RubinFilter G) (Ultrafilter G) where
|
|
|
|
coe := RubinFilter.filter
|
|
|
|
coe := RubinFilter.filter
|
|
|
|
|
|
|
|
|
|
|
|
section Equivalence
|
|
|
|
section Equivalence
|
|
|
|
open Topology
|
|
|
|
open Topology
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
variable {G : Type _} [Group G]
|
|
|
|
variable (α : Type _)
|
|
|
|
variable (α : Type _)
|
|
|
|
variable [TopologicalSpace α] [MulAction G α] [ContinuousConstSMul G α]
|
|
|
|
variable [TopologicalSpace α] [T2Space α] [MulAction G α] [ContinuousConstSMul G α]
|
|
|
|
variable [FaithfulSMul G α] [T2Space α] [LocallyMoving G α]
|
|
|
|
variable [FaithfulSMul G α] [LocallyDense G α] [LocallyCompactSpace α] [HasNoIsolatedPoints α]
|
|
|
|
|
|
|
|
|
|
|
|
-- TODO: either see whether we actually need this step, or change these names to something memorable
|
|
|
|
-- TODO: either see whether we actually need this step, or change these names to something memorable
|
|
|
|
-- This is an attempt to convert a RubinFilter G back to an Ultrafilter α
|
|
|
|
-- This is an attempt to convert a RubinFilter G back to an Ultrafilter α
|
|
|
|
def RubinFilter.to_action_filter (F : RubinFilter G) : Filter α :=
|
|
|
|
def RubinFilter.to_action_filter (F : RubinFilter G) : Filter α :=
|
|
|
|
⨅ (S : { S : Set G // S ∈ F.filter ∧ IsRigidSubgroup S }), (Filter.principal (S.prop.right.toRegularSupportBasis α))
|
|
|
|
⨅ (S : { S : Set G // S ∈ F.filter ∧ IsRigidSubgroup S }), (Filter.principal (S.prop.right.toRegularSupportBasis α))
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
instance RubinFilter.to_action_filter_neBot {F : RubinFilter G} [Nonempty α] : Filter.NeBot (F.to_action_filter α) :=
|
|
|
|
instance RubinFilter.to_action_filter_neBot {F : RubinFilter G} [Nonempty α] : Filter.NeBot (F.to_action_filter α) :=
|
|
|
|
by
|
|
|
|
by
|
|
|
|
unfold to_action_filter
|
|
|
|
unfold to_action_filter
|
|
|
@ -1244,8 +1285,116 @@ instance RubinFilter.to_action_filter_neBot {F : RubinFilter G} [Nonempty α] :
|
|
|
|
exact Set.inter_subset_left S T
|
|
|
|
exact Set.inter_subset_left S T
|
|
|
|
exact Set.inter_subset_right S T
|
|
|
|
exact Set.inter_subset_right S T
|
|
|
|
|
|
|
|
|
|
|
|
-- lemma RubinFilter.mem_to_action_filter' (F : RubinFilter G) (U : Set α) :
|
|
|
|
-- theorem RubinFilter.to_action_filter_converges' (F : RubinFilter G) :
|
|
|
|
-- U ∈ F.to_action_filter α ↔ ∃ S : AlgebraicCentralizerBasis G, S.val ∈ F.filter,
|
|
|
|
-- ∀ U : Set α, U ∈ RegularSupportBasis G α → U ∈ F.to_action_filter →
|
|
|
|
|
|
|
|
-- ∃ V ⊆ F.to_action_filter, V ⊆ U ∧
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
theorem RubinFilter.to_action_filter_mem {F : RubinFilter G} {U : Set G} (U_rigid : IsRigidSubgroup U) :
|
|
|
|
|
|
|
|
U ∈ F.filter ↔ (U_rigid.toRegularSupportBasis α : Set α) ∈ F.to_action_filter α :=
|
|
|
|
|
|
|
|
by
|
|
|
|
|
|
|
|
sorry
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
theorem RubinFilter.to_action_filter_mem' {F : RubinFilter G} {U : Set α} (U_in_basis : U ∈ RegularSupportBasis G α) :
|
|
|
|
|
|
|
|
U ∈ F.to_action_filter α ↔ (G•[U] : Set G) ∈ F.filter :=
|
|
|
|
|
|
|
|
by
|
|
|
|
|
|
|
|
-- trickier to prove but should be possible
|
|
|
|
|
|
|
|
sorry
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
theorem RubinFilter.to_action_filter_clusterPt [Nonempty α] (F : RubinFilter G) :
|
|
|
|
|
|
|
|
∃ p : α, ClusterPt p (F.to_action_filter α) :=
|
|
|
|
|
|
|
|
by
|
|
|
|
|
|
|
|
have univ_in_basis : Set.univ ∈ RegularSupportBasis G α := by
|
|
|
|
|
|
|
|
rw [RegularSupportBasis.mem_iff]
|
|
|
|
|
|
|
|
simp
|
|
|
|
|
|
|
|
use {}
|
|
|
|
|
|
|
|
simp [RegularSupport.FiniteInter]
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
have univ_rigid : IsRigidSubgroup (G := G) Set.univ := by
|
|
|
|
|
|
|
|
constructor
|
|
|
|
|
|
|
|
simp [Set.eq_singleton_iff_unique_mem]
|
|
|
|
|
|
|
|
exact LocallyMoving.nontrivial_elem
|
|
|
|
|
|
|
|
use {}
|
|
|
|
|
|
|
|
simp
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
suffices ∃ p ∈ Set.univ, ClusterPt p (F.to_action_filter α) by
|
|
|
|
|
|
|
|
let ⟨p, _, clusterPt⟩ := this
|
|
|
|
|
|
|
|
use p
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
apply proposition_3_5_2 (G := G) (α := α)
|
|
|
|
|
|
|
|
simp
|
|
|
|
|
|
|
|
let ⟨S, S_rigid, _, S_subsets_ss_orbit⟩ := F.converges _ Filter.univ_mem univ_rigid
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
use S_rigid.toRegularSupportBasis α
|
|
|
|
|
|
|
|
constructor
|
|
|
|
|
|
|
|
simp
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
unfold RSuppSubsets RSuppOrbit
|
|
|
|
|
|
|
|
simp
|
|
|
|
|
|
|
|
intro T T_in_basis T_ss_S
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
let T' := G•[T]
|
|
|
|
|
|
|
|
have T_regular : Regular T := sorry -- easy
|
|
|
|
|
|
|
|
have T'_rigid : IsRigidSubgroup (T' : Set G) := sorry -- provable
|
|
|
|
|
|
|
|
have T'_ss_S : (T' : Set G) ⊆ S := sorry -- using one of our lovely theorems
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
have T'_in_subsets : T' ∈ AlgebraicSubsets S := by
|
|
|
|
|
|
|
|
unfold AlgebraicSubsets
|
|
|
|
|
|
|
|
simp
|
|
|
|
|
|
|
|
constructor
|
|
|
|
|
|
|
|
sorry -- prove that rigid subgroups are in the algebraic centralizer basis
|
|
|
|
|
|
|
|
exact T'_ss_S
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
let ⟨g, _, W, W_in_F, W_rigid, W_conj⟩ := S_subsets_ss_orbit T'_in_subsets
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
use g
|
|
|
|
|
|
|
|
constructor
|
|
|
|
|
|
|
|
sorry -- TODO: G•[univ] = top
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
let W' := W_rigid.toRegularSupportBasis α
|
|
|
|
|
|
|
|
have W'_regular : Regular (W' : Set α) := by
|
|
|
|
|
|
|
|
apply RegularSupportBasis.regular (G := G)
|
|
|
|
|
|
|
|
simp
|
|
|
|
|
|
|
|
use W'
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
constructor
|
|
|
|
|
|
|
|
rw [<-RubinFilter.to_action_filter_mem]
|
|
|
|
|
|
|
|
assumption
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
rw [<-rigidStabilizer_eq_iff (α := α) (G := G) ((smulImage_regular _ _).mp W'_regular) T_regular]
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
ext i
|
|
|
|
|
|
|
|
rw [rigidStabilizer_smulImage]
|
|
|
|
|
|
|
|
unfold_let at W_conj
|
|
|
|
|
|
|
|
rw [<-W_conj]
|
|
|
|
|
|
|
|
simp
|
|
|
|
|
|
|
|
constructor
|
|
|
|
|
|
|
|
· intro
|
|
|
|
|
|
|
|
use g⁻¹ * i * g
|
|
|
|
|
|
|
|
constructor
|
|
|
|
|
|
|
|
assumption
|
|
|
|
|
|
|
|
group
|
|
|
|
|
|
|
|
· intro ⟨j, j_in_W, gjg_eq_i⟩
|
|
|
|
|
|
|
|
rw [<-gjg_eq_i]
|
|
|
|
|
|
|
|
group
|
|
|
|
|
|
|
|
assumption
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
-- theorem RubinFilter.to_action_filter_le_nhds [Nonempty α] (F : RubinFilter G) :
|
|
|
|
|
|
|
|
-- ∃ p : α, (F.to_action_filter α) ≤ 𝓝 p :=
|
|
|
|
|
|
|
|
-- by
|
|
|
|
|
|
|
|
-- let ⟨p, p_clusterPt⟩ := to_action_filter_clusterPt α F
|
|
|
|
|
|
|
|
-- use p
|
|
|
|
|
|
|
|
-- intro S S_in_nhds
|
|
|
|
|
|
|
|
-- rw [(RegularSupportBasis.isBasis G α).mem_nhds_iff] at S_in_nhds
|
|
|
|
|
|
|
|
-- let ⟨T, T_in_basis, p_in_T, T_ss_S⟩ := S_in_nhds
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
-- suffices T ∈ F.to_action_filter α by
|
|
|
|
|
|
|
|
-- apply Filter.sets_of_superset (F.to_action_filter α) this T_ss_S
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
-- rw [RubinFilter.to_action_filter_mem' _ T_in_basis]
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
|
-- intro S p_in_S S_open
|
|
|
|
|
|
|
|
-- sorry
|
|
|
|
|
|
|
|
|
|
|
|
lemma RubinFilter.mem_to_action_filter (F : RubinFilter G) {U : Set G} (U_rigid : IsRigidSubgroup U) :
|
|
|
|
lemma RubinFilter.mem_to_action_filter (F : RubinFilter G) {U : Set G} (U_rigid : IsRigidSubgroup U) :
|
|
|
|
U ∈ F.filter ↔ (U_rigid.toRegularSupportBasis α : Set α) ∈ F.to_action_filter α :=
|
|
|
|
U ∈ F.filter ↔ (U_rigid.toRegularSupportBasis α : Set α) ∈ F.to_action_filter α :=
|
|
|
@ -1293,8 +1442,8 @@ by
|
|
|
|
|
|
|
|
|
|
|
|
have GS_ss_V : G•[S] ≤ V := by
|
|
|
|
have GS_ss_V : G•[S] ≤ V := by
|
|
|
|
rw [<-V_rigid.toRegularSupportBasis_eq (α := α)]
|
|
|
|
rw [<-V_rigid.toRegularSupportBasis_eq (α := α)]
|
|
|
|
simp
|
|
|
|
simp only [Set.le_eq_subset, SetLike.coe_subset_coe]
|
|
|
|
rw [<-rigidStabilizer_subset_iff G (α := α) S_regular (IsRigidSubgroup.toRegularSupportBasis_regular _ _)]
|
|
|
|
rw [<-rigidStabilizer_subset_iff G (α := α) S_regular (IsRigidSubgroup.toRegularSupportBasis_regular _ V_rigid)]
|
|
|
|
assumption
|
|
|
|
assumption
|
|
|
|
|
|
|
|
|
|
|
|
-- TODO: show that G•[S] ∈ AlgebraicSubsets V
|
|
|
|
-- TODO: show that G•[S] ∈ AlgebraicSubsets V
|
|
|
@ -1314,8 +1463,7 @@ by
|
|
|
|
use g
|
|
|
|
use g
|
|
|
|
constructor
|
|
|
|
constructor
|
|
|
|
{
|
|
|
|
{
|
|
|
|
rw [<-SetLike.mem_coe]
|
|
|
|
|
|
|
|
rw [U_rigid.toRegularSupportBasis_eq (α := α)]
|
|
|
|
|
|
|
|
assumption
|
|
|
|
assumption
|
|
|
|
}
|
|
|
|
}
|
|
|
|
|
|
|
|
|
|
|
@ -1334,7 +1482,7 @@ by
|
|
|
|
exact S_regular
|
|
|
|
exact S_regular
|
|
|
|
|
|
|
|
|
|
|
|
ext i
|
|
|
|
ext i
|
|
|
|
rw [rigidStabilizer_smulImage, <-Wconj_eq_GS, <-IsRigidSubgroup.mem_subgroup, <-SetLike.mem_coe, IsRigidSubgroup.toRegularSupportBasis_eq]
|
|
|
|
rw [rigidStabilizer_smulImage, <-Wconj_eq_GS]
|
|
|
|
simp
|
|
|
|
simp
|
|
|
|
constructor
|
|
|
|
constructor
|
|
|
|
· intro gig_in_W
|
|
|
|
· intro gig_in_W
|
|
|
@ -1350,8 +1498,8 @@ by
|
|
|
|
|
|
|
|
|
|
|
|
instance RubinFilterSetoid (G : Type _) [Group G] : Setoid (RubinFilter G) where
|
|
|
|
instance RubinFilterSetoid (G : Type _) [Group G] : Setoid (RubinFilter G) where
|
|
|
|
r F F' := ∀ (U : Set G), IsRigidSubgroup U →
|
|
|
|
r F F' := ∀ (U : Set G), IsRigidSubgroup U →
|
|
|
|
((∃ V : Set G, V ≤ U ∧ AlgebraicSubsets V ⊆ AlgebraicOrbit F U)
|
|
|
|
((∃ V : Set G, V ≤ U ∧ AlgebraicSubsets V ⊆ AlgebraicOrbit F.filter U)
|
|
|
|
↔ (∃ V' : Set G, V' ≤ U ∧ AlgebraicSubsets V' ⊆ AlgebraicOrbit F' U))
|
|
|
|
↔ (∃ V' : Set G, V' ≤ U ∧ AlgebraicSubsets V' ⊆ AlgebraicOrbit F'.filter U))
|
|
|
|
iseqv := by
|
|
|
|
iseqv := by
|
|
|
|
constructor
|
|
|
|
constructor
|
|
|
|
· intros
|
|
|
|
· intros
|
|
|
@ -1390,8 +1538,10 @@ variable [Group G]
|
|
|
|
variable [TopologicalSpace α] [Nonempty α] [T2Space α] [HasNoIsolatedPoints α] [LocallyCompactSpace α]
|
|
|
|
variable [TopologicalSpace α] [Nonempty α] [T2Space α] [HasNoIsolatedPoints α] [LocallyCompactSpace α]
|
|
|
|
variable [MulAction G α] [ContinuousConstSMul G α] [FaithfulSMul G α] [LocallyMoving G α] [LocallyDense G α]
|
|
|
|
variable [MulAction G α] [ContinuousConstSMul G α] [FaithfulSMul G α] [LocallyMoving G α] [LocallyDense G α]
|
|
|
|
|
|
|
|
|
|
|
|
def RubinFilter.fromElement (x : α) : RubinFilter G where
|
|
|
|
instance RubinFilter.fromElement_neBot (x : α) : Filter.NeBot (⨅ (S ∈ 𝓝 x), Filter.principal (G•[S] : Set G)) := by sorry
|
|
|
|
filter := ⨅ (S ∈ 𝓝 x), Filter.principal G•[S]
|
|
|
|
|
|
|
|
|
|
|
|
noncomputable def RubinFilter.fromElement (x : α) : RubinFilter G where
|
|
|
|
|
|
|
|
filter := @Ultrafilter.of _ (⨅ (S ∈ 𝓝 x), Filter.principal (G•[S] : Set G)) (RubinFilter.fromElement_neBot G α x)
|
|
|
|
converges := by
|
|
|
|
converges := by
|
|
|
|
sorry
|
|
|
|
sorry
|
|
|
|
ne_bot := by
|
|
|
|
ne_bot := by
|
|
|
|