Skip to content

Commit 681d9aa

Browse files
committed
chore: add public modifiers in Lean.Elab.Tactic.Ext
1 parent 663df8f commit 681d9aa

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

src/Lean/Elab/Tactic/Ext.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -178,8 +178,7 @@ def realizeExtIffTheorem (extName : Name) : Elab.Command.CommandElabM Name := do
178178
### Attribute
179179
-/
180180

181-
abbrev extExtension := Meta.Ext.extExtension
182-
abbrev getExtTheorems := Meta.Ext.getExtTheorems
181+
open Ext
183182

184183
builtin_initialize registerBuiltinAttribute {
185184
name := `ext
@@ -220,7 +219,8 @@ builtin_initialize registerBuiltinAttribute {
220219
-/
221220

222221
/-- Apply a single extensionality theorem to `goal`. -/
223-
def applyExtTheoremAt (goal : MVarId) : MetaM (List MVarId) := goal.withContext do
222+
-- Tis is public for now as it is used internally in `aesop`.
223+
public def applyExtTheoremAt (goal : MVarId) : MetaM (List MVarId) := goal.withContext do
224224
let tgt ← goal.getType'
225225
unless tgt.isAppOfArity ``Eq 3 do
226226
throwError "This extensionality tactic only applies to equalities, not{indentExpr tgt}"

0 commit comments

Comments
 (0)