Commit cbe69a6 1 parent 4afcacf commit cbe69a6 Copy full SHA for cbe69a6
File tree 2 files changed +3
-3
lines changed
2 files changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -3,7 +3,6 @@ Copyright (c) 2015 Microsoft Corporation. All rights reserved.
3
3
Released under Apache 2.0 license as described in the file LICENSE.
4
4
Authors: Leonardo de Moura
5
5
-/
6
- import Batteries.Logic
7
6
import Mathlib.Mathport.Rename
8
7
9
8
/-!
@@ -51,7 +50,7 @@ def EqvGen.Setoid : Setoid α :=
51
50
#align eqv_gen.setoid EqvGen.Setoid
52
51
53
52
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
55
54
(Quot.lift (Quotient.mk (EqvGen.Setoid r)) (fun x y h ↦ Quot.sound (EqvGen.rel x y h))) H)
56
55
#align quot.exact Quot.exact
57
56
Original file line number Diff line number Diff line change @@ -3,7 +3,8 @@ Copyright (c) 2022 Arthur Paulino. All rights reserved.
3
3
Released under Apache 2.0 license as described in the file LICENSE.
4
4
Authors: Arthur Paulino, Gabriel Ebner, Kyle Miller
5
5
-/
6
- import Batteries.Logic
6
+ import Lean.Meta.Tactic.Util
7
+ import Lean.Elab.Tactic.Basic
7
8
8
9
/-!
9
10
# The `use` tactic
You can’t perform that action at this time.
0 commit comments