Skip to content

Commit 4741f3c

Browse files
committed
chore: cleanup after renaming get_elem_tactic_trivial
1 parent e4ec332 commit 4741f3c

File tree

5 files changed

+2
-13
lines changed

5 files changed

+2
-13
lines changed

src/Init/Data/Range/Basic.lean

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -86,6 +86,3 @@ theorem Membership.get_elem_helper {i n : Nat} {r : Std.Range} (h₁ : i ∈ r)
8686

8787
macro_rules
8888
| `(tactic| get_elem_tactic_extensible) => `(tactic| apply Membership.get_elem_helper; assumption; rfl)
89-
90-
macro_rules
91-
| `(tactic| get_elem_tactic_trivial) => `(tactic| apply Membership.get_elem_helper; assumption; rfl)

src/Init/GetElem.lean

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -283,9 +283,6 @@ instance [GetElem? cont Nat elem dom] [h : LawfulGetElem cont Nat elem dom] :
283283
macro_rules
284284
| `(tactic| get_elem_tactic_extensible) => `(tactic| (with_reducible apply Fin.val_lt_of_le); get_elem_tactic_extensible; done)
285285

286-
macro_rules
287-
| `(tactic| get_elem_tactic_trivial) => `(tactic| (with_reducible apply Fin.val_lt_of_le); get_elem_tactic_trivial; done)
288-
289286
end Fin
290287

291288
namespace List

src/Init/Tactics.lean

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1933,9 +1933,7 @@ syntax "get_elem_tactic_trivial" : tactic
19331933

19341934
macro_rules | `(tactic| get_elem_tactic_extensible) => `(tactic| omega)
19351935
macro_rules | `(tactic| get_elem_tactic_extensible) => `(tactic| simp +arith; done)
1936-
1937-
macro_rules | `(tactic| get_elem_tactic_trivial) => `(tactic| omega)
1938-
macro_rules | `(tactic| get_elem_tactic_trivial) => `(tactic| simp +arith; done)
1936+
macro_rules | `(tactic| get_elem_tactic_extensible) => `(tactic| trivial)
19391937

19401938
/--
19411939
`get_elem_tactic` is the tactic automatically called by the notation `arr[i]`

src/Lean/Elab/Tactic.lean

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -51,6 +51,3 @@ import Lean.Elab.Tactic.TreeTacAttr
5151
import Lean.Elab.Tactic.ExposeNames
5252
import Lean.Elab.Tactic.SimpArith
5353
import Lean.Elab.Tactic.Lets
54-
55-
elab "get_elem_tactic_trivial" : tactic => do
56-
throwError "`get_elem_tactic_trivial` has been renamed to `get_elem_tactic_extensible`"

tests/lean/run/grind_indexmap.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ import Std.Data.HashMap
66

77
set_option grind.warning false
88

9-
macro_rules | `(tactic| get_elem_tactic_trivial) => `(tactic| grind)
9+
macro_rules | `(tactic| get_elem_tactic_extensible) => `(tactic| grind)
1010

1111
open Std
1212

0 commit comments

Comments
 (0)