Skip to content

Commit

Permalink
feat(topology/algebra/mul_action): add_torsor.connected_space (#16471)
Browse files Browse the repository at this point in the history
Add the lemma that an `add_torsor` for a connected space is itself a connected space, given `has_continuous_vadd`.
  • Loading branch information
jsm28 committed Sep 21, 2022
1 parent ae9b867 commit a6d28ae
Showing 1 changed file with 20 additions and 0 deletions.
20 changes: 20 additions & 0 deletions src/topology/algebra/mul_action.lean
Expand Up @@ -3,6 +3,7 @@ Copyright (c) 2021 Yury Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov
-/
import algebra.add_torsor
import topology.algebra.constructions
import group_theory.group_action.prod
import group_theory.group_action.basic
Expand Down Expand Up @@ -169,3 +170,22 @@ has_continuous_smul_Inf $ set.forall_range_iff.mpr h
by { rw inf_eq_infi, refine has_continuous_smul_infi (λ b, _), cases b; assumption }

end lattice_ops

section add_torsor

variables (G : Type*) (P : Type*) [add_group G] [add_torsor G P] [topological_space G]
variables [preconnected_space G] [topological_space P] [has_continuous_vadd G P]
include G

/-- An `add_torsor` for a connected space is a connected space. This is not an instance because
it loops for a group as a torsor over itself. -/
protected lemma add_torsor.connected_space : connected_space P :=
{ is_preconnected_univ :=
begin
convert is_preconnected_univ.image ((equiv.vadd_const (classical.arbitrary P)) : G → P)
(continuous_id.vadd continuous_const).continuous_on,
rw [set.image_univ, equiv.range_eq_univ]
end,
to_nonempty := infer_instance }

end add_torsor

0 comments on commit a6d28ae

Please sign in to comment.