Skip to content

Commit e87858f

Browse files
committed
chore: fix typos
1 parent 5db666d commit e87858f

File tree

1 file changed

+2
-2
lines changed

1 file changed

+2
-2
lines changed

src/Lean/Meta/Tactic/Grind/Order/Proof.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -51,7 +51,7 @@ def mkTransCore (p₁ : ProofInfo) (p₂ : ProofInfo) (v : NodeId) : OrderM Proo
5151
return { w := p₁.w, k.strict := s₁ || s₂, proof := h }
5252

5353
/--
54-
Assume `pi₁` is `{ w := u, k := k₁, proof := p₁ }` and `pi₂` is `{ w := w, k := k₂, proof := p₂ }`
54+
Assume `p₁` is `{ w := u, k := k₁, proof := p₁ }` and `p₂` is `{ w := w, k := k₂, proof := p₂ }`
5555
`p₁` is the proof for edge `u -(k₁)→ w` and `p₂` the proof for edge `w -(k₂)-> v`.
5656
Then, this function returns a proof for edge `u -(k₁+k₂) -> v`.
5757
@@ -72,7 +72,7 @@ def mkTransOffset (p₁ : ProofInfo) (p₂ : ProofInfo) (v : NodeId) : OrderM Pr
7272
return { w := p₁.w, k.k := k, k.strict := s₁ || s₂, proof := h }
7373

7474
/--
75-
Assume `pi₁` is `{ w := u, k := k₁, proof := p₁ }` and `pi₂` is `{ w := w, k := k₂, proof := p₂ }`
75+
Assume `p₁` is `{ w := u, k := k₁, proof := p₁ }` and `p₂` is `{ w := w, k := k₂, proof := p₂ }`
7676
`p₁` is the proof for edge `u -(k₁)→ w` and `p₂` the proof for edge `w -(k₂)-> v`.
7777
Then, this function returns a proof for edge `u -(k₁+k₂) -> v`.
7878

0 commit comments

Comments
 (0)