Skip to content

Commit

Permalink
fix
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Jan 14, 2025
1 parent a9c19df commit b1378c9
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions REPL/Lean/InfoTree.lean
Original file line number Diff line number Diff line change
Expand Up @@ -63,8 +63,8 @@ def kind : Info → String
| .ofCustomInfo _ => "CustomInfo"
| .ofFVarAliasInfo _ => "FVarAliasInfo"
| .ofFieldRedeclInfo _ => "FieldRedeclInfo"
| .ofOmissionInfo _ => "OmissionInfo"
| .ofChoiceInfo _ => "ChoiceInfo"
| .ofDelabTermInfo _ => "DelabTermInfo"

/-- The `Syntax` for a `Lean.Elab.Info`, if there is one. -/
def stx? : Info → Option Syntax
Expand All @@ -80,8 +80,8 @@ def stx? : Info → Option Syntax
| .ofCustomInfo info => info.stx
| .ofFVarAliasInfo _ => none
| .ofFieldRedeclInfo info => info.stx
| .ofOmissionInfo info => info.stx
| .ofChoiceInfo info => info.stx
| .ofDelabTermInfo info => info.stx

/-- Is the `Syntax` for this `Lean.Elab.Info` original, or synthetic? -/
def isOriginal (i : Info) : Bool :=
Expand Down

0 comments on commit b1378c9

Please sign in to comment.