Skip to content

Commit cbe69a6

Browse files
committed
chore: removing unnecessary imports of Batteries.Logic (#14522)
1 parent 4afcacf commit cbe69a6

File tree

2 files changed

+3
-3
lines changed

2 files changed

+3
-3
lines changed

Mathlib/Init/Data/Quot.lean

+1-2
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,6 @@ Copyright (c) 2015 Microsoft Corporation. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Leonardo de Moura
55
-/
6-
import Batteries.Logic
76
import Mathlib.Mathport.Rename
87

98
/-!
@@ -51,7 +50,7 @@ def EqvGen.Setoid : Setoid α :=
5150
#align eqv_gen.setoid EqvGen.Setoid
5251

5352
theorem Quot.exact {a b : α} (H : Quot.mk r a = Quot.mk r b) : EqvGen r a b :=
54-
@Quotient.exact _ (EqvGen.Setoid r) a b (congr_arg
53+
@Quotient.exact _ (EqvGen.Setoid r) a b (congrArg
5554
(Quot.lift (Quotient.mk (EqvGen.Setoid r)) (fun x y h ↦ Quot.sound (EqvGen.rel x y h))) H)
5655
#align quot.exact Quot.exact
5756

Mathlib/Tactic/Use.lean

+2-1
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,8 @@ Copyright (c) 2022 Arthur Paulino. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Arthur Paulino, Gabriel Ebner, Kyle Miller
55
-/
6-
import Batteries.Logic
6+
import Lean.Meta.Tactic.Util
7+
import Lean.Elab.Tactic.Basic
78

89
/-!
910
# The `use` tactic

0 commit comments

Comments
 (0)