Skip to content

Commit

Permalink
close goal in example
Browse files Browse the repository at this point in the history
  • Loading branch information
kmill authored and kim-em committed Nov 4, 2023
1 parent 3b88e16 commit 616f717
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions src/Init/Tactics.lean
Original file line number Diff line number Diff line change
Expand Up @@ -106,6 +106,7 @@ example : let n := 1; let k := 2; n + k = 3 := by
/- n✝ : Nat := 1
k✝ : Nat := 2
⊢ n✝ + k✝ = 3 -/
rfl
```
-/
syntax (name := intros) "intros" (ppSpace colGt (ident <|> hole))* : tactic
Expand Down

0 comments on commit 616f717

Please sign in to comment.