Skip to content

Commit a5cca0f

Browse files
mcdollurkud
andcommitted
feat: port Topology.UniformSpace.Cauchy (#2007)
Co-authored-by: Yury G. Kudryashov <urkud@urkud.name>
1 parent 7bfd7d1 commit a5cca0f

File tree

3 files changed

+773
-2
lines changed

3 files changed

+773
-2
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -977,6 +977,7 @@ import Mathlib.Topology.Separation
977977
import Mathlib.Topology.SubsetProperties
978978
import Mathlib.Topology.Support
979979
import Mathlib.Topology.UniformSpace.Basic
980+
import Mathlib.Topology.UniformSpace.Cauchy
980981
import Mathlib.Topology.UniformSpace.Separation
981982
import Mathlib.Util.AtomM
982983
import Mathlib.Util.Export

Mathlib/Logic/Equiv/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -20,6 +20,7 @@ import Mathlib.Logic.Function.Conjugate
2020
import Mathlib.Tactic.Convert
2121
import Mathlib.Tactic.Contrapose
2222
import Mathlib.Tactic.GeneralizeProofs
23+
import Mathlib.Tactic.Lift
2324

2425
/-!
2526
# Equivalence between types
@@ -1427,8 +1428,7 @@ theorem ofBijective_symm_apply_apply (f : α → β) (hf : Bijective f) (x : α)
14271428
(ofBijective f hf).symm_apply_apply x
14281429
#align equiv.of_bijective_symm_apply_apply Equiv.ofBijective_symm_apply_apply
14291430

1430-
-- Porting note: `lift` tactic is not implemented yet.
1431-
-- instance : CanLift (α → β) (α ≃ β) coeFn Bijective where prf f hf := ⟨ofBijective f hf, rfl⟩
1431+
instance : CanLift (α → β) (α ≃ β) (↑) Bijective where prf f hf := ⟨ofBijective f hf, rfl⟩
14321432

14331433
section
14341434

0 commit comments

Comments
 (0)