File tree Expand file tree Collapse file tree 5 files changed +2
-13
lines changed
Expand file tree Collapse file tree 5 files changed +2
-13
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 @@ -283,9 +283,6 @@ instance [GetElem? cont Nat elem dom] [h : LawfulGetElem cont Nat elem dom] :
283283macro_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-
289286end Fin
290287
291288namespace List
Original file line number Diff line number Diff line change @@ -1933,9 +1933,7 @@ syntax "get_elem_tactic_trivial" : tactic
19331933
19341934macro_rules | `(tactic| get_elem_tactic_extensible) => `(tactic| omega)
19351935macro_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]`
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`"
Original file line number Diff line number Diff line change @@ -6,7 +6,7 @@ import Std.Data.HashMap
66
77set_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
1111open Std
1212
You can’t perform that action at this time.
0 commit comments