Skip to content

Commit

Permalink
chore(Topology/Constructions): rename most type variables (#9863)
Browse files Browse the repository at this point in the history
Now we use letters X and Y for topological spaces, not Greek letters.

I didn't replace all letters; some lemmas need a large number of different letters. Volunteers for the last instances welcome.
  • Loading branch information
grunweg committed Jan 25, 2024
1 parent 2e59248 commit 9a290c2
Show file tree
Hide file tree
Showing 2 changed files with 377 additions and 377 deletions.
4 changes: 2 additions & 2 deletions Mathlib/CategoryTheory/Extensive.lean
Original file line number Diff line number Diff line change
Expand Up @@ -387,7 +387,7 @@ instance finitaryExtensive_TopCat : FinitaryExtensive TopCat.{u} := by
refine' ⟨⟨l, _⟩, ContinuousMap.ext fun a => (hl a).symm, TopCat.isTerminalPUnit.hom_ext _ _,
fun {l'} h₁ _ => ContinuousMap.ext fun x =>
hl' x (l' x) (ConcreteCategory.congr_hom h₁ x).symm⟩
apply (embedding_inl (α := X') (β := Y')).toInducing.continuous_iff.mpr
apply (embedding_inl (X := X') (Y := Y')).toInducing.continuous_iff.mpr
convert s.fst.2 using 1
exact (funext hl).symm
· refine' ⟨⟨hαY.symm⟩, ⟨PullbackCone.isLimitAux' _ _⟩⟩
Expand All @@ -404,7 +404,7 @@ instance finitaryExtensive_TopCat : FinitaryExtensive TopCat.{u} := by
refine' ⟨⟨l, _⟩, ContinuousMap.ext fun a => (hl a).symm, TopCat.isTerminalPUnit.hom_ext _ _,
fun {l'} h₁ _ =>
ContinuousMap.ext fun x => hl' x (l' x) (ConcreteCategory.congr_hom h₁ x).symm⟩
apply (embedding_inr (α := X') (β := Y')).toInducing.continuous_iff.mpr
apply (embedding_inr (X := X') (Y := Y')).toInducing.continuous_iff.mpr
convert s.fst.2 using 1
exact (funext hl).symm
· intro Z f
Expand Down
Loading

0 comments on commit 9a290c2

Please sign in to comment.