Skip to content

Commit 9a290c2

Browse files
committed
chore(Topology/Constructions): rename most type variables (#9863)
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.
1 parent 2e59248 commit 9a290c2

File tree

2 files changed

+377
-377
lines changed

2 files changed

+377
-377
lines changed

Mathlib/CategoryTheory/Extensive.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -387,7 +387,7 @@ instance finitaryExtensive_TopCat : FinitaryExtensive TopCat.{u} := by
387387
refine' ⟨⟨l, _⟩, ContinuousMap.ext fun a => (hl a).symm, TopCat.isTerminalPUnit.hom_ext _ _,
388388
fun {l'} h₁ _ => ContinuousMap.ext fun x =>
389389
hl' x (l' x) (ConcreteCategory.congr_hom h₁ x).symm⟩
390-
apply (embedding_inl (α := X') (β := Y')).toInducing.continuous_iff.mpr
390+
apply (embedding_inl (X := X') (Y := Y')).toInducing.continuous_iff.mpr
391391
convert s.fst.2 using 1
392392
exact (funext hl).symm
393393
· refine' ⟨⟨hαY.symm⟩, ⟨PullbackCone.isLimitAux' _ _⟩⟩
@@ -404,7 +404,7 @@ instance finitaryExtensive_TopCat : FinitaryExtensive TopCat.{u} := by
404404
refine' ⟨⟨l, _⟩, ContinuousMap.ext fun a => (hl a).symm, TopCat.isTerminalPUnit.hom_ext _ _,
405405
fun {l'} h₁ _ =>
406406
ContinuousMap.ext fun x => hl' x (l' x) (ConcreteCategory.congr_hom h₁ x).symm⟩
407-
apply (embedding_inr (α := X') (β := Y')).toInducing.continuous_iff.mpr
407+
apply (embedding_inr (X := X') (Y := Y')).toInducing.continuous_iff.mpr
408408
convert s.fst.2 using 1
409409
exact (funext hl).symm
410410
· intro Z f

0 commit comments

Comments
 (0)