Skip to content

Commit

Permalink
test: macro scopes in Conv.congr (#1955)
Browse files Browse the repository at this point in the history
  • Loading branch information
digama0 authored Dec 14, 2022
1 parent d5fb32a commit 52d00e8
Showing 1 changed file with 3 additions and 0 deletions.
3 changes: 3 additions & 0 deletions tests/lean/conv1.lean
Original file line number Diff line number Diff line change
Expand Up @@ -242,3 +242,6 @@ example : ((x + y) + z : Nat) = x + (y + z) := by conv => pattern (occs := 5) _
example : ((x + y) + z : Nat) = x + (y + z) := by conv => pattern (occs := 2 5) _ + _
example : ((x + y) + z : Nat) = x + (y + z) := by conv => pattern (occs := 1 5) _ + _
example : ((x + y) + z : Nat) = x + (y + z) := by conv => pattern (occs := 1 2 5) _ + _

macro "bla" : term => `(?a)
example : 1 = 1 := by conv => apply bla; congr

0 comments on commit 52d00e8

Please sign in to comment.