File tree Expand file tree Collapse file tree 4 files changed +1
-12
lines changed
Expand file tree Collapse file tree 4 files changed +1
-12
lines changed Original file line number Diff line number Diff line change @@ -86,6 +86,3 @@ theorem Membership.get_elem_helper {i n : Nat} {r : Std.Range} (h₁ : i ∈ r)
8686
8787macro_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)
Original file line number Diff line number Diff line change @@ -285,9 +285,6 @@ instance [GetElem? cont Nat elem dom] [h : LawfulGetElem cont Nat elem dom] :
285285macro_rules
286286 | `(tactic| get_elem_tactic_extensible) => `(tactic| (with_reducible apply Fin.val_lt_of_le); get_elem_tactic_extensible; done)
287287
288- macro_rules
289- | `(tactic| get_elem_tactic_trivial) => `(tactic| (with_reducible apply Fin.val_lt_of_le); get_elem_tactic_trivial; done)
290-
291288end Fin
292289
293290namespace List
Original file line number Diff line number Diff line change @@ -1896,9 +1896,7 @@ syntax "get_elem_tactic_trivial" : tactic
18961896
18971897macro_rules | `(tactic| get_elem_tactic_extensible) => `(tactic| omega)
18981898macro_rules | `(tactic| get_elem_tactic_extensible) => `(tactic| simp +arith; done)
1899-
1900- macro_rules | `(tactic| get_elem_tactic_trivial) => `(tactic| omega)
1901- macro_rules | `(tactic| get_elem_tactic_trivial) => `(tactic| simp +arith; done)
1899+ macro_rules | `(tactic| get_elem_tactic_extensible) => `(tactic| trivial)
19021900
19031901/--
19041902`get_elem_tactic` is the tactic automatically called by the notation `arr[i]`
Original file line number Diff line number Diff line change @@ -51,6 +51,3 @@ import Lean.Elab.Tactic.TreeTacAttr
5151import Lean.Elab.Tactic.ExposeNames
5252import Lean.Elab.Tactic.SimpArith
5353import 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`"
You can’t perform that action at this time.
0 commit comments