summaryrefslogtreecommitdiff
path: root/backends/lean/Base/Utils.lean
diff options
context:
space:
mode:
Diffstat (limited to 'backends/lean/Base/Utils.lean')
-rw-r--r--backends/lean/Base/Utils.lean6
1 files changed, 2 insertions, 4 deletions
diff --git a/backends/lean/Base/Utils.lean b/backends/lean/Base/Utils.lean
index b0032281..eacfe72b 100644
--- a/backends/lean/Base/Utils.lean
+++ b/backends/lean/Base/Utils.lean
@@ -1,6 +1,5 @@
import Lean
import Mathlib.Tactic.Core
-import Mathlib.Tactic.LeftRight
import Base.UtilsBase
/-
@@ -503,9 +502,8 @@ elab "split_disj " n:ident : tactic => do
example (x y : Int) (h0 : x ≤ y ∨ x ≥ y) : x ≤ y ∨ x ≥ y := by
split_disj h0
- . left; assumption
- . right; assumption
-
+ . apply Or.inl; assumption
+ . apply Or.inr; assumption
-- Tactic to split on an exists.
-- `h` must be an FVar