File tree Expand file tree Collapse file tree 1 file changed +3
-3
lines changed
Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Original file line number Diff line number Diff 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
184183builtin_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}"
You can’t perform that action at this time.
0 commit comments