Skip to content

Commit

Permalink
chore: format to avoid multiple goals (#10979)
Browse files Browse the repository at this point in the history
  • Loading branch information
adomani committed Feb 26, 2024
1 parent fb56e88 commit 7eae15a
Showing 1 changed file with 3 additions and 3 deletions.
Expand Up @@ -206,9 +206,9 @@ theorem compExactValue_correctness_of_stream_eq_some :
nextContinuants, nextNumerator, nextDenominator]
have hfr : (IntFractPair.of (1 / ifp_n.fr)).fr = f := rfl
rw [one_div, if_neg _, ← one_div, hfr]
field_simp [hA, hB]
ac_rfl
rwa [inv_eq_one_div, hfr]
· field_simp [hA, hB]
ac_rfl
· rwa [inv_eq_one_div, hfr]
#align generalized_continued_fraction.comp_exact_value_correctness_of_stream_eq_some GeneralizedContinuedFraction.compExactValue_correctness_of_stream_eq_some

open GeneralizedContinuedFraction (of_terminatedAt_n_iff_succ_nth_intFractPair_stream_eq_none)
Expand Down

0 comments on commit 7eae15a

Please sign in to comment.