Skip to content

Commit

Permalink
chore: test for issue #4064
Browse files Browse the repository at this point in the history
closes #4064
  • Loading branch information
leodemoura committed May 7, 2024
1 parent dfde4ee commit 0304061
Showing 1 changed file with 11 additions and 0 deletions.
11 changes: 11 additions & 0 deletions tests/lean/run/4064.lean
Original file line number Diff line number Diff line change
@@ -0,0 +1,11 @@
import Lean

def test : Lean.CoreM (List Lean.Name) := do
let .thmInfo tval ← Lean.getConstInfo `And.left | unreachable!
return tval.all

/--
info: [`And.left]
-/
#guard_msgs in
#eval test

0 comments on commit 0304061

Please sign in to comment.