Skip to content

Commit

Permalink
Test imported declaration
Browse files Browse the repository at this point in the history
  • Loading branch information
TwoFX committed Feb 3, 2025
1 parent 3a4f10d commit 23e0105
Showing 1 changed file with 9 additions and 3 deletions.
12 changes: 9 additions & 3 deletions tests/lean/run/recommendedSpelling.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2,11 +2,10 @@ import Lean

/-!
Test the `recommended_spelling` command.
TODO: once we use this command in Init, we can test that recommended spellings from imported
modules are reported correctly.
-/

recommended_spelling "bland" for "🥤" in [And]

/--
Conjuction
Expand Down Expand Up @@ -56,6 +55,13 @@ info: some
#guard_msgs in
#eval findDocString? `«term_☋_»

/--
info: some
"`And a b`, or `a ∧ b`, is the conjunction of propositions. It can be\nconstructed and destructed like a pair: if `ha : a` and `hb : b` then\n`⟨ha, hb⟩ : a ∧ b`, and if `h : a ∧ b` then `h.left : a` and `h.right : b`.\n\n\nConventions for notations in identifiers:\n\n * The recommended spelling of `∧` in identifiers is `and`.\n\n * The recommended spelling of `/\\` in identifiers is `and` (prefer `∧` over `/\\`).\n\n * The recommended spelling of `🥤` in identifiers is `bland`."
-/
#guard_msgs in
#eval findDocString? `And

/-- info: 1 -/
#guard_msgs in
#eval do
Expand Down

0 comments on commit 23e0105

Please sign in to comment.