Skip to content

Commit a539cf8

Browse files
committed
fix test output
1 parent 27616c8 commit a539cf8

File tree

1 file changed

+0
-5
lines changed

1 file changed

+0
-5
lines changed

BatteriesTest/print_prefix.lean

Lines changed: 0 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -129,16 +129,11 @@ def testMatchProof : (n : Nat) → Fin n → Unit
129129

130130
/--
131131
info: testMatchProof (n : Nat) : Fin n → Unit
132-
testMatchProof._cstage1 (n : Nat) : Fin n → Unit
133-
testMatchProof._cstage2 : _obj → _obj → _obj
134132
testMatchProof._sunfold (n : Nat) : Fin n → Unit
135133
testMatchProof._unsafe_rec (n : Nat) : Fin n → Unit
136134
testMatchProof.match_1.{u_1} (motive : (x : Nat) → Fin x → Sort u_1) (x✝ : Nat) (x✝¹ : Fin x✝)
137135
(h_1 : (n : Nat) → (isLt : 0 < n) → motive n ⟨0, isLt⟩)
138136
(h_2 : (as i : Nat) → (h : i.succ < as.succ) → motive as.succ ⟨i.succ, h⟩) : motive x✝ x✝¹
139-
testMatchProof.match_1._cstage1.{u_1} (motive : (x : Nat) → Fin x → Sort u_1) (x✝ : Nat) (x✝¹ : Fin x✝)
140-
(h_1 : (n : Nat) → (isLt : 0 < n) → motive n ⟨0, isLt⟩)
141-
(h_2 : (as i : Nat) → (h : i.succ < as.succ) → motive as.succ ⟨i.succ, h⟩) : motive x✝ x✝¹
142137
testMatchProof.proof_1 (as i : Nat) (h : i.succ < as.succ) : i.succ ≤ as
143138
testMatchProof.proof_2 (as i : Nat) (h : i.succ < as.succ) : i.succ ≤ as
144139
-/

0 commit comments

Comments
 (0)