Skip to content

Commit

Permalink
Update RupAddResult.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser authored and kim-em committed Nov 19, 2024
1 parent a5e74f4 commit 5372af3
Showing 1 changed file with 1 addition and 1 deletion.
Original file line number Diff line number Diff line change
Expand Up @@ -815,7 +815,7 @@ theorem confirmRupHint_preserves_invariant_helper {n : Nat} (f : DefaultFormula
have k'_in_bounds : k' < acc.2.1.length := by
simp only [List.length_cons, Nat.succ_eq_add_one] at k'_succ_in_bounds
exact Nat.lt_of_succ_lt_succ k'_succ_in_bounds
exact h2 (acc.2.1.get ⟨k', k'_in_bounds⟩) <| List.get_mem acc.snd.fst k' k'_in_bounds
exact h2 (acc.2.1.get ⟨k', k'_in_bounds⟩) <| List.get_mem acc.snd.fst ⟨k', k'_in_bounds
· next l_ne_i =>
apply Or.inl
constructor
Expand Down

0 comments on commit 5372af3

Please sign in to comment.