Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 040ebea

Browse files
fix(analysis/normed_space/normed_group_quotient): put lemmas inside namespace (#7653)
1 parent c1e9f94 commit 040ebea

File tree

1 file changed

+6
-2
lines changed

1 file changed

+6
-2
lines changed

src/analysis/normed_space/normed_group_quotient.lean

Lines changed: 6 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -416,6 +416,10 @@ begin
416416
simp only [(quotient_norm_eq_zero_iff S x).mpr hker, normed_mk.apply, zero_mul],
417417
end
418418

419+
end add_subgroup
420+
421+
namespace normed_group_hom
422+
419423
/-- `is_quotient f`, for `f : M ⟶ N` means that `N` is isomorphic to the quotient of `M`
420424
by the kernel of `f`. -/
421425
structure is_quotient (f : normed_group_hom M N) : Prop :=
@@ -451,7 +455,7 @@ lemma lift_unique {N : Type*} [semi_normed_group N] (S : add_subgroup M)
451455
begin
452456
intro h,
453457
ext,
454-
rcases surjective_normed_mk _ x with ⟨x,rfl⟩,
458+
rcases add_subgroup.surjective_normed_mk _ x with ⟨x,rfl⟩,
455459
change (g.comp (S.normed_mk) x) = _,
456460
simpa only [h]
457461
end
@@ -488,4 +492,4 @@ begin
488492
{ exact ⟨0, f.ker.zero_mem, by simp⟩ }
489493
end
490494

491-
end add_subgroup
495+
end normed_group_hom

0 commit comments

Comments
 (0)