File tree Expand file tree Collapse file tree 3 files changed +773
-2
lines changed Expand file tree Collapse file tree 3 files changed +773
-2
lines changed Original file line number Diff line number Diff line change @@ -977,6 +977,7 @@ import Mathlib.Topology.Separation
977
977
import Mathlib.Topology.SubsetProperties
978
978
import Mathlib.Topology.Support
979
979
import Mathlib.Topology.UniformSpace.Basic
980
+ import Mathlib.Topology.UniformSpace.Cauchy
980
981
import Mathlib.Topology.UniformSpace.Separation
981
982
import Mathlib.Util.AtomM
982
983
import Mathlib.Util.Export
Original file line number Diff line number Diff line change @@ -20,6 +20,7 @@ import Mathlib.Logic.Function.Conjugate
20
20
import Mathlib.Tactic.Convert
21
21
import Mathlib.Tactic.Contrapose
22
22
import Mathlib.Tactic.GeneralizeProofs
23
+ import Mathlib.Tactic.Lift
23
24
24
25
/-!
25
26
# Equivalence between types
@@ -1427,8 +1428,7 @@ theorem ofBijective_symm_apply_apply (f : α → β) (hf : Bijective f) (x : α)
1427
1428
(ofBijective f hf).symm_apply_apply x
1428
1429
#align equiv.of_bijective_symm_apply_apply Equiv.ofBijective_symm_apply_apply
1429
1430
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⟩
1432
1432
1433
1433
section
1434
1434
You can’t perform that action at this time.
0 commit comments