Zulip Chat Archive

Stream: mathlib4

Topic: port progress


Scott Morrison (Nov 13 2022 at 07:06):

I'm about to test a bot that may post regularly to this thread. Expect some noise as I convince cron to work.

port-progress bot (Nov 13 2022 at 07:08):

Total files in mathlib: 2725
Longest import chain in mathlib: 145
Ported files in mathlib: 30 (1.1% of total)
Ported lines in mathlib: 9160 (1.0% of total)
Longest unported chain in mathlib: 135

port-progress bot (Nov 13 2022 at 07:12):

Total files in mathlib: 2725
Longest import chain in mathlib: 145
Ported files in mathlib: 30 (1.1% of total)
Ported lines in mathlib: 9160 (1.0% of total)
Longest unported chain in mathlib: 135

port-progress bot (Nov 13 2022 at 07:17):

Total files in mathlib: 2725
Longest import chain in mathlib: 145
Ported files in mathlib: 30 (1.1% of total)
Ported lines in mathlib: 9160 (1.0% of total)
Longest unported chain in mathlib: 135

Scott Morrison (Nov 13 2022 at 07:19):

Thanks cron, once a day will do nicely from now on!

Scott Morrison (Nov 13 2022 at 07:21):

If anyone would like to see the longest unported chain, please run leanproject port-progress inside mathlib. I'm happy to take suggestions on a useful way for the bot to post this.

Eric Wieser (Nov 13 2022 at 11:13):

nit: maybe have the bot format as

Total files in mathlib 2725
Longest import chain in mathlib 145
Ported files in mathlib 30 (1.1% of total)
Ported lines in mathlib 9160 (1.0% of total)
Longest unported chain in mathlib 135

Scott Morrison (Nov 13 2022 at 11:48):

The bot just runs leanproject port-progress | head -n 5 | zulip-send ..., and there's not really room for formatting in there. :-)

Kyle Miller (Nov 13 2022 at 12:01):

@Scott Morrison This should do it:

leanproject port-progress | head -n 5 | awk 'BEGIN{ FS=":"; print "| | |\n|--|--|"} {print "| " $1 ": | " $2 " |"}' | zulip-send ...

port-progress bot (Nov 13 2022 at 12:06):

Total files in mathlib: 2726
Longest import chain in mathlib: 145
Ported files in mathlib: 30 (1.1% of total)
Ported lines in mathlib: 9160 (1.0% of total)
Longest unported chain in mathlib: 135

Eric Wieser (Nov 13 2022 at 13:42):

I would have suggested a --markdown flag to port-progress, but I guess that works too...

Jireh Loreaux (Nov 13 2022 at 15:39):

I do love awk

port-progress bot (Nov 13 2022 at 18:02):

Total files in mathlib: 2732
Longest import chain in mathlib: 142
Ported files in mathlib: 30 (1.1% of total)
Ported lines in mathlib: 9046 (1.0% of total)
Longest unported chain in mathlib: 132

Mario Carneiro (Nov 13 2022 at 18:11):

could the "ported files" and "ported lines" lines be changed to something like 30 / 2732 = 1.1%? That way you can also see the number of total lines in mathlib and trendline that as well instead of trying to reconstruct it from the 1.1%

Scott Morrison (Nov 13 2022 at 22:28):

file#analysis/normed_space/star/gelfand_duality is our new "champion", ending the longest unported import chain.

port-progress bot (Nov 13 2022 at 22:31):

Ported files: 30/2732 (1.1% of total)
Ported lines: 9046/914410 (1.0% of total)
Longest unported import chain: 132/142 (7.0% progress)

Scott Morrison (Nov 13 2022 at 22:33):

@Patrick Massot, this is in https://github.com/leanprover-community/mathlib-tools/pull/139. I can probably have my bot run off the branch for a while, to avoid cutting too many releases.

Patrick Massot (Nov 13 2022 at 22:37):

I'm not sure about this new display. On my phone I can see the information in the text version because it wraps line whereas the table version requires painful scrolling

Patrick Massot (Nov 13 2022 at 22:37):

This isn't a strong opinion however.

Patrick Massot (Nov 13 2022 at 22:39):

Releasing mathlibtools isn't super time consuming but doing it several times a week is maybe a bit excessive. If you and your bot are the only user of some new feature then we can probably wait to batch features a bit.

Yaël Dillies (Nov 13 2022 at 22:39):

If we're separating progress into a third column, we might as well remove the brackets (and maybe the "of total"/"of progress")

Patrick Massot (Nov 13 2022 at 22:39):

That being said, I'm also very happy if I can help the port by doing grunt releasing work on pypi

Mario Carneiro (Nov 13 2022 at 22:39):

well, one of the divisions is calculated differently from the others so it might be a bit confusing

Gabriel Ebner (Nov 13 2022 at 22:40):

We could also cut down the descriptions a bit "longest unported import chain" -> "longest chain" would make it almost fit I think.

Yaël Dillies (Nov 13 2022 at 22:41):

Mario Carneiro said:

well, one of the divisions is calculated differently from the others so it might be a bit confusing

Longgest unported chain: 10/142 sounds like a better phrasing to me anyway

Mario Carneiro (Nov 13 2022 at 22:41):

but 10 isn't a measure of anything there

Mario Carneiro (Nov 13 2022 at 22:41):

these are not related chains

Mario Carneiro (Nov 13 2022 at 22:42):

the longest chain in mathlib has length 142, and the longest chain of unported files has length 132

Yaël Dillies (Nov 13 2022 at 22:43):

Then why are we even printing progress on this if it doesn't mean anything?

Mario Carneiro (Nov 13 2022 at 22:43):

it's comparing the heights of the two posets which is a meaningful measure

Mario Carneiro (Nov 13 2022 at 22:43):

but the difference of heights isn't itself the height of something

Yaël Dillies (Nov 13 2022 at 22:44):

A better stat would be the number of unported files below the longest chain, but I think we're bikeshedding here

Scott Morrison (Nov 13 2022 at 22:44):

Yes. :-)

Mario Carneiro (Nov 13 2022 at 22:44):

isn't that going to be almost everything?

Yaël Dillies (Nov 13 2022 at 22:45):

I don't see how that's any less meaning ful than longest path! (as opposed to longest unported path)

Mario Carneiro (Nov 13 2022 at 22:46):

if we assume infinite bandwidth, after 132 rounds of PR merging all of mathlib will be ported

Yaël Dillies (Nov 13 2022 at 22:46):

Yeah, so 142 is meaningless :wink:

Yaël Dillies (Nov 13 2022 at 22:46):

and the progress is too

Mario Carneiro (Nov 13 2022 at 22:46):

142 is how many rounds there would be starting from scratch

Scott Morrison (Nov 13 2022 at 22:47):

Further, 142 will change over time!

Scott Morrison (Nov 13 2022 at 22:47):

If people continue doing refactoring work on mathlib3 to remove spurious imports, that number will decrease.

Scott Morrison (Nov 13 2022 at 22:47):

In fact, it has already dropped some.

Mario Carneiro (Nov 13 2022 at 22:47):

yeah, it's important to have both numbers because they chase each other

Mario Carneiro (Nov 13 2022 at 22:47):

the number of files went up though

Scott Morrison (Nov 13 2022 at 22:47):

And this is exactly why I've included the 142. :-)

Yaël Dillies (Nov 13 2022 at 22:48):

Uh, I thought you were arguing for removing it :sweat_smile:

Jireh Loreaux (Nov 14 2022 at 01:14):

Scott Morrison said:

file#analysis/normed_space/star/gelfand_duality is our new "champion", ending the longest unported import chain.

I guess it's my turn to wear the scarlet "A" :sweat_smile: ? I'll have a look at the chain to see if anything stands out.

Jireh Loreaux (Nov 14 2022 at 01:15):

And unfortunately it's about to be superseded because of #17164 ... :embarrassed:

port-progress bot (Nov 14 2022 at 18:02):

Total files in mathlib: 2743
Longest import chain in mathlib: 134
Ported files in mathlib: 34 (1.2% of total)
Ported lines in mathlib: 10584 (1.2% of total)
Longest unported chain in mathlib: 124

Johan Commelin (Nov 14 2022 at 18:16):

Where's our pretty tables?

Scott Morrison (Nov 14 2022 at 20:39):

Oops. I have two open PRs against mathlib-tools. I guess I had run pip3 install . against the other one, and my bot ran using that.

port-progress bot (Nov 14 2022 at 21:57):

Ported files: 35/2744 (1.3% of total)
Ported lines: 10767/913983 (1.2% of total)
Longest unported import chain: 124/134 (7.5% progress)

Jireh Loreaux (Nov 14 2022 at 22:26):

Finally had a chance to look at this long chain. topology.noetherian_space was a bit surprising to me, but I'm not really familiar at all with that part of the library. Ultimately though, this chain requires Liouville's theorem and the Cauchy integral formula, so it's bound to be rather long (I'm not sure exactly how long).The pieces after that are expected I think. It seems that there is a lot of roaming around in topology and measure theory maybe some of which can be short-circuited, but I'm not at all sure about that.

Heather Macbeth (Nov 14 2022 at 22:36):

Perhaps we could prove that the exponential function is convex without appealing to its derivative. Then

analysis.convex.specific_functions

would probably not need to import the chain

'analysis.normed_space.operator_norm', 'analysis.normed_space.multilinear', 'analysis.normed_space.bounded_linear_maps', 'analysis.calculus.fderiv', 'analysis.calculus.deriv', 'analysis.calculus.local_extr', 'analysis.calculus.mean_value', 'analysis.calculus.cont_diff', 'analysis.calculus.inverse', 'analysis.special_functions.exp_deriv', 'analysis.special_functions.complex.log_deriv', 'analysis.special_functions.pow_deriv', 'analysis.convex.specific_functions'

Mario Carneiro (Nov 14 2022 at 22:37):

what is the full chain?

Heather Macbeth (Nov 14 2022 at 22:38):

['logic.equiv.defs', 'order.synonym', 'order.compare', 'order.monotone', 'order.lattice', 'order.bounded_order', 'algebra.order.monoid.defs', 'algebra.order.sub.defs', 'algebra.order.group.defs', 'algebra.order.ring.defs', 'algebra.order.ring.canonical', 'data.nat.order.basic', 'data.nat.order.lemmas', 'algebra.group_power.ring', 'algebra.group_power.order', 'data.nat.pow', 'algebra.group_power.lemmas', 'algebra.group_power.default', 'data.list.big_operators', 'data.list.count', 'data.list.lattice', 'data.list.nodup', 'data.list.dedup', 'data.list.perm', 'data.multiset.basic', 'algebra.big_operators.multiset', 'data.multiset.bind', 'data.multiset.powerset', 'data.multiset.nodup', 'data.multiset.dedup', 'data.multiset.finset_ops', 'data.finset.basic', 'data.finset.card', 'data.finset.option', 'data.finset.lattice', 'data.finset.powerset', 'data.fintype.basic', 'data.finset.sort', 'data.set.finite', 'order.conditionally_complete_lattice', 'order.copy', 'order.filter.basic', 'order.filter.prod', 'order.filter.bases', 'order.filter.at_top_bot', 'order.filter.cofinite', 'order.filter.ultrafilter', 'topology.basic', 'topology.tactic', 'topology.order', 'topology.maps', 'topology.constructions', 'topology.continuous_on', 'topology.bases', 'topology.subset_properties', 'topology.connected', 'topology.separation', 'topology.dense_embedding', 'topology.homeomorph', 'topology.continuous_function.basic', 'topology.sets.opens', 'topology.sets.closeds', 'topology.noetherian_space', 'topology.quasi_separated', 'topology.sets.compacts', 'topology.algebra.group', 'topology.algebra.ring', 'topology.algebra.field', 'topology.algebra.order.basic', 'topology.algebra.order.intermediate_value', 'topology.algebra.order.compact', 'topology.metric_space.basic', 'topology.metric_space.lipschitz', 'topology.metric_space.antilipschitz', 'topology.metric_space.isometry', 'analysis.normed.group.basic', 'analysis.normed.group.infinite_sum', 'analysis.normed.field.basic', 'analysis.normed_space.basic', 'analysis.normed.order.basic', 'analysis.locally_convex.basic', 'analysis.locally_convex.balanced_core_hull', 'analysis.locally_convex.bounded', 'topology.algebra.uniform_convergence', 'topology.algebra.module.strong_topology', 'analysis.normed_space.operator_norm', 'analysis.normed_space.multilinear', 'analysis.normed_space.bounded_linear_maps', 'analysis.calculus.fderiv', 'analysis.calculus.deriv', 'analysis.calculus.local_extr', 'analysis.calculus.mean_value', 'analysis.calculus.cont_diff', 'analysis.calculus.inverse', 'analysis.special_functions.exp_deriv', 'analysis.special_functions.complex.log_deriv', 'analysis.special_functions.pow_deriv', 'analysis.convex.specific_functions', 'analysis.mean_inequalities', 'measure_theory.integral.mean_inequalities', 'measure_theory.function.simple_func_dense', 'measure_theory.function.strongly_measurable.basic', 'measure_theory.function.ae_eq_fun', 'measure_theory.function.lp_space', 'measure_theory.function.lp_order', 'measure_theory.function.l1_space', 'measure_theory.function.simple_func_dense_lp', 'measure_theory.integral.set_to_l1', 'measure_theory.integral.bochner', 'measure_theory.integral.set_integral', 'measure_theory.constructions.prod', 'measure_theory.group.measure', 'measure_theory.constructions.pi', 'measure_theory.measure.lebesgue', 'measure_theory.measure.haar_lebesgue', 'measure_theory.integral.interval_integral', 'analysis.special_functions.integrals', 'analysis.special_functions.non_integrable', 'measure_theory.integral.circle_integral', 'analysis.complex.cauchy_integral', 'analysis.complex.liouville', 'analysis.complex.polynomial', 'analysis.normed_space.spectrum', 'analysis.normed_space.star.spectrum', 'analysis.normed_space.star.gelfand_duality']

Scott Morrison (Nov 14 2022 at 22:48):

If we merge #17507 (just sayin') then leanproject import-graph will automatically annotate these long import chains according to modules with are not really used.

port-progress bot (Nov 14 2022 at 22:50):

mathlib port progress (data.rat.order)
Ported files: 29/126 (23.0% of total)
Ported lines: 10397/39435 (26.4% of total)
Longest unported chain: 16/26 (38.5% progress)

Mario Carneiro (Nov 14 2022 at 22:50):

do we have something which can make displays like the one I made before, with * in front of unused modules?

Mario Carneiro (Nov 14 2022 at 22:51):

sweet, from 1% to 23%

Scott Morrison (Nov 14 2022 at 22:51):

At present only graphical. Nothing text mode.

Scott Morrison (Nov 14 2022 at 22:51):

Ah -- notice the new header

Mario Carneiro (Nov 14 2022 at 22:51):

what does it mean?

Scott Morrison (Nov 14 2022 at 22:51):

This is progress up to data.rat.order.

Scott Morrison (Nov 14 2022 at 22:52):

I thought having some intermediate milestones might be encouraging / useful.

Scott Morrison (Nov 14 2022 at 22:53):

I can easily modify (after #17507) leanproject port-progress so that it prints the longest chain, annotated with *s. It is already printing the longest chain, and elsewhere in leanproject is code to compute the *s.

Mario Carneiro (Nov 14 2022 at 22:54):

How about putting the longest unported chain, with the *, in a <details> after the table?

Mario Carneiro (Nov 14 2022 at 22:55):

I guess that won't be a one-liner though

Scott Morrison (Nov 14 2022 at 22:55):

Sure. I can alternatively add a hyperlink.

Kevin Buzzard (Nov 14 2022 at 22:55):

It's not entirely clear to me that making the longest chain shorter is actually worthwhile progress. Just because it represents some sort of inf for the porting process doesn't imply that if we make it shorter it will actually make porting happen more quickly

Mario Carneiro (Nov 14 2022 at 22:55):

do you have something to link to?

Scott Morrison (Nov 14 2022 at 22:55):

I'm about to add a hyperlink to the rendered import-graph.

Mario Carneiro (Nov 14 2022 at 22:56):

making the chain shorter is refactoring work which makes it easier to reach particular targets

Scott Morrison (Nov 14 2022 at 22:56):

This will include the * information (as grey shading).

Scott Morrison (Nov 14 2022 at 22:56):

I think reporting the longest chain is quite useful: it gives people constructive work to be doing on the mathlib3 side. :-)

Mario Carneiro (Nov 14 2022 at 22:56):

I'm not sure that watching the chain over time is that useful though

Scott Morrison (Nov 14 2022 at 22:57):

I agree. But I want to make sure it is easy for people to look at the chain.

Mario Carneiro (Nov 14 2022 at 22:57):

once you have done some work to optimize a chain, it's usually better to go find a different chain elsewhere in the hierarchy

Mario Carneiro (Nov 14 2022 at 22:57):

but the longest chain is at least easy to pinpoint

Kevin Buzzard (Nov 14 2022 at 22:58):

I understand that, but if we have ten things to do and we decide to rearrange stuff to make the first thing quicker to do but the total longer to do, are we really gaining anything? We still have to port all the files, regardless of how much extra work you want to put in rearranging them. I understand it's important to get linarith working quickly but I don't understand why it's important to make the borel cantelli lemma rely on fewer imports

Mario Carneiro (Nov 14 2022 at 22:58):

I think it is important for the future that we get mathlib's dependency creep under control

Scott Morrison (Nov 14 2022 at 22:58):

leanproject import-graph --from tactic.basic --to interesting_target --show-unused will show you a picture of whatever chain you like.

Scott Morrison (Nov 14 2022 at 22:59):

I've stated adding assert_not_exists statements in my refactoring PRs, exactly to constrain import creep. But it is hard to do this well.

Mario Carneiro (Nov 14 2022 at 23:00):

The mathlib4 dependency hierarchy is going to look significantly different from mathlib once everything shakes out

Scott Morrison (Nov 14 2022 at 23:00):

Kevin, there is also a parallelisation argument. If we're optimistic about the number of people porting / number of simultaneous PRs we can cope with, broader shallower trees are better.

Mario Carneiro (Nov 14 2022 at 23:00):

because std is taking a bunch of the low level files and tactics need to be more stratified in order to optimize precompiledModules behavior

Scott Morrison (Nov 14 2022 at 23:00):

I suspect the borel cantelli lemmas is also limiting our CI times.

Mario Carneiro (Nov 14 2022 at 23:02):

note that it's not the borel cantelli lemma in particular we care about, but rather every file downstream of the refactored import edges

Mario Carneiro (Nov 14 2022 at 23:03):

the borel cantelli lemma is just a single target we can easily point to which holds up a big chain of imports

Mario Carneiro (Nov 14 2022 at 23:03):

the fact that it's a long chain means it's more likely to have unnecessary linearization in it

Kevin Buzzard (Nov 14 2022 at 23:03):

I'm just saying that it's not immediately obvious to me that shortening the depth definitely means shortening the length of the port and it might lengthen it. On the other hand if you can see other reasons for doing it then go ahead!

port-progress bot (Nov 14 2022 at 23:17):

mathlib port progress data.rat.order
Ported files: 29/126 (23.0% of total)
Ported lines: 10397/39435 (26.4% of total)
Longest unported chain: 16/26 (38.5% progress)

Jireh Loreaux (Nov 14 2022 at 23:21):

Kevin, I agree that it's probably not worth paying attention to the longest chain in a month or so, but I think focused effort up front to clean up the hierarchy could be useful.

Junyan Xu (Nov 14 2022 at 23:29):

Notice that I contributed to the chain (specifically the link analysis.complex.liouville -> polynomial) by golfing the fundamental theorem of algebra using Liouville (#17343). I wonder what the import graph looks like before and after the PR. However it's near the end of the chain, and the next file analysis.normed_space.spectrum does need algebraic closedness of C, so it needs the algebraic hierarchy up to docs#is_alg_closed, but maybe it doesn't need that much complex analysis.

Heather Macbeth (Nov 14 2022 at 23:52):

I played with the tool, speculatively deleting various imports (without compiling, or checking that my proposed file-reorganization or more-elementary-reproofs actually worked). I conjecture that one could get the Gelfand duality chain from 124 down to 114, something like

['logic.equiv.defs', 'order.synonym', 'order.compare', 'order.monotone', 'order.lattice', 'order.bounded_order', 'algebra.order.monoid.defs', 'algebra.order.sub.defs', 'algebra.order.group.defs', 'algebra.order.ring.defs', 'algebra.order.ring.canonical', 'data.nat.order.basic', 'data.nat.order.lemmas', 'algebra.group_power.ring', 'algebra.group_power.order', 'data.nat.pow', 'algebra.group_power.lemmas', 'algebra.group_power.default', 'data.list.big_operators', 'data.list.count', 'data.list.lattice', 'data.list.nodup', 'data.list.dedup', 'data.list.perm', 'data.multiset.basic', 'algebra.big_operators.multiset', 'data.multiset.bind', 'data.multiset.powerset', 'data.multiset.nodup', 'data.multiset.dedup', 'data.multiset.finset_ops', 'data.finset.basic', 'data.finset.card', 'data.finset.option', 'data.finset.lattice', 'data.finset.powerset', 'data.fintype.basic', 'data.finset.sort', 'data.set.finite', 'order.conditionally_complete_lattice', 'order.copy', 'order.filter.basic', 'order.filter.prod', 'order.filter.bases', 'order.filter.lift', 'order.filter.small_sets', 'topology.basic', 'topology.tactic', 'topology.order', 'topology.maps', 'topology.constructions', 'topology.continuous_on', 'topology.bases', 'topology.subset_properties', 'topology.connected', 'topology.separation', 'topology.dense_embedding', 'topology.homeomorph', 'topology.continuous_function.basic', 'topology.sets.opens', 'topology.sets.closeds', 'topology.noetherian_space', 'topology.quasi_separated', 'topology.sets.compacts', 'topology.algebra.group', 'topology.algebra.ring', 'topology.algebra.field', 'topology.algebra.order.basic', 'topology.algebra.order.intermediate_value', 'topology.algebra.order.compact', 'topology.metric_space.basic', 'topology.metric_space.lipschitz', 'topology.metric_space.antilipschitz', 'topology.metric_space.isometry', 'analysis.normed.group.basic', 'analysis.normed.group.infinite_sum', 'analysis.normed.field.basic', 'analysis.normed_space.basic', 'analysis.asymptotics.asymptotics', 'analysis.asymptotics.theta', 'analysis.special_functions.exp', 'analysis.special_functions.trigonometric.basic', 'analysis.special_functions.trigonometric.angle', 'analysis.special_functions.complex.arg', 'analysis.special_functions.complex.log', 'analysis.special_functions.pow', 'analysis.convex.specific_functions', 'analysis.mean_inequalities', 'measure_theory.integral.mean_inequalities', 'measure_theory.function.simple_func_dense', 'measure_theory.function.strongly_measurable.basic', 'measure_theory.function.ae_eq_fun', 'measure_theory.function.lp_space', 'measure_theory.function.lp_order', 'measure_theory.function.l1_space', 'measure_theory.function.simple_func_dense_lp', 'measure_theory.integral.set_to_l1', 'measure_theory.integral.bochner', 'measure_theory.integral.set_integral', 'measure_theory.constructions.prod', 'measure_theory.group.measure', 'measure_theory.constructions.pi', 'measure_theory.measure.lebesgue', 'measure_theory.measure.haar_lebesgue', 'measure_theory.integral.interval_integral', 'analysis.special_functions.integrals', 'analysis.special_functions.non_integrable', 'measure_theory.integral.circle_integral', 'analysis.complex.cauchy_integral', 'analysis.complex.liouville', 'analysis.complex.polynomial', 'analysis.normed_space.spectrum', 'analysis.normed_space.star.spectrum', 'analysis.normed_space.star.gelfand_duality']

Past this it is difficult. Observations:

  • measure theory unifies the integral (considered in L^1 spaces) with L^p spaces, and so needs a full theory of raising to the power of p, even though the construction "raise to the power of 1" is much more elementary than the construction "raise to the power of p"
  • the construction of raising to the power of p is itself not done directly using data.complex.exponential (which is a low-level file), but also requires the construction of trig functions, because the junk value chosen for a negative power is exp (y log x) cos (πy). And trig functions require a lot of topology (one chooses pi by the intermediate value theorem).

Scott Morrison (Nov 15 2022 at 00:02):

The first difficulty seems like a reasonable choice. The second one is a bit unfortunate. :-)

port-progress bot (Nov 15 2022 at 00:13):

mathlib port progress
Ported files: 35/2747 (1.3% of total)
Ported lines: 10767/914414 (1.2% of total)
Longest unported chain: 125/135 (7.4% progress)

Jireh Loreaux (Nov 15 2022 at 00:59):

FYI: analysis.normed_space.spectrum needs a bunch of complex analysis, including a direct application of Liouville's theorem, so the FTA golf into a separate file is no big deal.

port-progress bot (Nov 15 2022 at 04:04):

mathlib port progress data.rat.order
Ported files: 29/126 (23.0% of total)
Ported lines: 10397/39435 (26.4% of total)
Longest unported chain: 16/26 (38.5% progress)

port-progress bot (Nov 15 2022 at 04:08):

mathlib port progress algebra.order.field.defs
Ported files: 26/75 (34.7% of total)
Ported lines: 9637/26110 (36.9% of total)
Longest unported chain: 10/20 (50.0% progress)

port-progress bot (Nov 15 2022 at 04:54):

mathlib port progress all
Ported files: 35/2749 (1.3% of total)
Ported lines: 10767/913469 (1.2% of total)
Longest unported chain: 125/135 (7.4% progress)

Junyan Xu (Nov 15 2022 at 05:06):

port-progress bot said:

mathlib port progress algebra.order.field.defs

The first row shouldn't be restricted to the first column, I think.

Scott Morrison (Nov 15 2022 at 05:08):

I think vanilla markdown doesn't support that.

Junyan Xu (Nov 15 2022 at 05:09):

Then maybe don't include the first row in the table.

Scott Morrison (Nov 15 2022 at 05:09):

meh

port-progress bot (Nov 15 2022 at 05:10):

mathlib port progress topology.metric_space.basic
Ported files: 31/527 (5.9% of total)
Ported lines: 10457/211423 (4.9% of total)
Longest unported chain: 71/81 (12.3% progress)

Scott Morrison (Nov 15 2022 at 05:10):

I could just drop the words mathlib port progress. But I'm finding it hard to care about the whitespace. :-)

Junyan Xu (Nov 15 2022 at 05:11):

Or you could put the file name in the second column

Scott Morrison (Nov 15 2022 at 05:18):

Okay, I did that.

Scott Morrison (Nov 15 2022 at 05:20):

The graphs linked in the progress reports indicate files which "aren't really used" in a faint gray. Can people distinguish these?

Scott Morrison (Nov 15 2022 at 05:20):

The graph for topology.metric_space.basic is covered with gray. If anyone wants to have a go at cleaning up imports there ...

Moritz Doll (Nov 15 2022 at 09:55):

fyi: I am splitting of some parts of topology.algebra.order.basic

Moritz Doll (Nov 15 2022 at 09:56):

that is a monstrum of 3000 lines and should be split anyways

Yaël Dillies (Nov 15 2022 at 10:06):

Oh actually I have thoughts about this one specifically

Moritz Doll (Nov 15 2022 at 10:07):

I am only moving out the linear ordered field, this seems to be very sensible - there were quite a few files that never used the field parts

Yaël Dillies (Nov 15 2022 at 10:07):

The first half has no algebra in it, so it shouldn't be in topology.algebra.order, but rather topology.order

Moritz Doll (Nov 15 2022 at 10:08):

I think then our refactors are disjoint enough to not cause problems

Moritz Doll (Nov 15 2022 at 10:09):

#17549

Yaël Dillies (Nov 15 2022 at 10:10):

Okay, I will do the split I want myself :thumbs_up:

Sebastien Gouezel (Nov 15 2022 at 13:37):

#17549 looks good to me. @Yaël Dillies , is that compatible with your plans?

Yaël Dillies (Nov 15 2022 at 13:43):

This looks very fine

Riccardo Brasca (Nov 15 2022 at 16:38):

Do we have something like a list of who is working on which file somewhere? I would like to start working on the port, avoiding duplicating the efforts...

David Renshaw (Nov 15 2022 at 16:38):

https://github.com/leanprover-community/mathlib/wiki/mathlib4-port-status

Jireh Loreaux (Nov 15 2022 at 16:39):

I think this is on the wiki, but you can get it with the port-status script too.

David Renshaw (Nov 15 2022 at 16:39):

and for tactics https://github.com/leanprover-community/mathlib4/issues/430

Riccardo Brasca (Nov 15 2022 at 16:39):

Thanks!

Adam Topaz (Nov 15 2022 at 16:41):

Do we also have a script which shows which files are ready to be ported (because their imports have already been ported)?

Adam Topaz (Nov 15 2022 at 16:41):

There was some discussion of such a thing at some point, but I haven't been following this thread closely enough to remember whether it actually happened. And I would also like to start working on porting (once I can find some time)

Jireh Loreaux (Nov 15 2022 at 16:43):

That is part of the port-status output

Jireh Loreaux (Nov 15 2022 at 16:44):

leanproject import-graph also has some port-related features now (like node highlighting)

Riccardo Brasca (Nov 15 2022 at 16:47):

So suppose I want to work on algebra.pempty_instances (chosen at random). Is it OK to open a WIP PR to inform everybody that I am working on it?

Heather Macbeth (Nov 15 2022 at 16:48):

@Riccardo Brasca You should edit the wiki:
https://github.com/leanprover-community/mathlib/wiki/mathlib4-port-status

Heather Macbeth (Nov 15 2022 at 16:49):

(from No to No: wip riccardo)

Riccardo Brasca (Nov 15 2022 at 16:50):

I think open the WIP PR can in any case be useful. A beginner in Lean4 (like me) will probably be quite slow, but maybe the file I am on is needed for something more important, and with the PR people can work on it.

Heather Macbeth (Nov 15 2022 at 16:51):

(The advantage of editing the wiki is that then your WIP riccardo message will be displayed when other people who are looking for a task run the port-status script. So it serves a different function from opening the PR.)

Riccardo Brasca (Nov 15 2022 at 16:52):

Sure, I totally agree editing the wiki is useful. I just don't want to block someone else because I am slow.

Adam Topaz (Nov 15 2022 at 16:52):

Jireh Loreaux said:

That is part of the port-status output

Should this info be displayed in the wiki?

Heather Macbeth (Nov 15 2022 at 16:55):

Probably a good idea, but which wiki do you mean?

Adam Topaz (Nov 15 2022 at 16:56):

The port status wiki

Adam Topaz (Nov 15 2022 at 16:56):

https://github.com/leanprover-community/mathlib/wiki/mathlib4-port-status

Adam Topaz (Nov 15 2022 at 16:57):

Well, I suppose if this list changes very frequently, then maybe it shouldn't be displayed there.

Jireh Loreaux (Nov 15 2022 at 16:57):

I think not, because it is regenerated each time.

Jireh Loreaux (Nov 15 2022 at 16:57):

(deleted)

Adam Topaz (Nov 15 2022 at 16:57):

yeah I noticed it (and edited my message)

Yakov Pechersky (Nov 15 2022 at 16:58):

@Adam Topaz, the pdf that is generated also highlights nodes in a green "port complete", blue "PR exists", and neonish blue "all direct parents have port complete"

Adam Topaz (Nov 15 2022 at 16:59):

What PDF are you referring to? The script didn't generate any PDF for me.

Yakov Pechersky (Nov 15 2022 at 16:59):

ah: leanproject import-graph --to algebra.order.ring.defs --exclude-tactics algebra.order.ring.pdf --port-status --reduce

Yakov Pechersky (Nov 15 2022 at 16:59):

the crucial flag there is --port-status

Yakov Pechersky (Nov 15 2022 at 17:00):

That, or a similar command, is what is used to make those links up top like https://tqft.net/mathlib4/2022-11-15/algebra.order.field.defs.pdf

Heather Macbeth (Nov 15 2022 at 17:01):

I misunderstood what Adam was asking. I thought he was suggesting adding a sentence like "You can see the current list of port-able files (which is autogenerated by the information on this wiki page) by running the script scripts/port-status.py in mathlib" to the page
https://github.com/leanprover-community/mathlib/wiki/mathlib4-port-status
Maybe this wouldn't hurt?

Adam Topaz (Nov 15 2022 at 17:01):

Thanks!

Jireh Loreaux (Nov 15 2022 at 17:04):

Of course, that script is reading the wiki page, so before you add anything you should either read the script to see what it's doing or else ask someone who knows to make sure that where you add it doesn't break the script. :smiley:

Heather Macbeth (Nov 15 2022 at 17:05):

Indeed, I was hoping someone more confident would take on that task for me :)

Arien Malec (Nov 15 2022 at 17:05):

So the workflow is to generate the graph, look for a cyan node, assess portability, then what?

Generate a PR, mark that on the wiki page? Is the overall flow documented anywhere?

Jireh Loreaux (Nov 15 2022 at 17:07):

If you want to get started porting, see here: https://github.com/leanprover-community/mathlib4/wiki

Yakov Pechersky (Nov 15 2022 at 17:07):

You won't hurt the wiki! So I've added that sentence and a reference to a leanproject invocation too

Jireh Loreaux (Nov 15 2022 at 17:07):

@Arien Malec to see which files you might want to port, you want to run the port-status script inside mathlib.

Riccardo Brasca (Nov 15 2022 at 17:07):

The video is very helpful

Heather Macbeth (Nov 15 2022 at 17:09):

By the way, Yakov, did you ever implement this?

Yakov Pechersky said:

Anyway, to make ready defer to PR, one just has to add two lines here: https://github.com/leanprover-community/mathlib-tools/blob/67f1bda7637d17a9f765ecade305d3f9ffc93e7c/mathlibtools/lib.py#L1047-L1050
Specifically:

if not target_node.get("status"):
  continue

I think it would be helpful (it's another thing that I'm not confident enough to touch myself).

Yakov Pechersky (Nov 15 2022 at 17:10):

My start porting flow is -- generate the graph. Either pick a cyan node, or a white node that has parents that are blue. Update my mathlib3port clone via a git pull. Copy the file I care about in mathlib4 like cp ../mathlib3port/Mathbin/Logic/Equiv/Basic.lean Mathlib/Logic/Equiv/, possible having to do a mkdir. Add the file to Mathlib.lean, go to the file, rename Mathbin to Mathlib, git checkout -b pechersky/port-logic-equiv-basic; git add ...; git commit; git push ..., make a PR, change the wiki.

Adam Topaz (Nov 15 2022 at 17:12):

Can we add a TLDR section to https://github.com/leanprover-community/mathlib4/wiki (or elsewhere) with approximately what Yakov said?

Yakov Pechersky (Nov 15 2022 at 17:12):

@Heather Macbeth I haven't yet. I'd like to refactor the coloring a little so that it's easier to express our logic, which is why I have https://github.com/leanprover-community/mathlib-tools/pull/137. That refactor will allow us to tag ready nodes with "ready", and more cleanly have the logic of what ready overrides or not

Mario Carneiro (Nov 15 2022 at 17:13):

Also don't forget to record the mathlib SHA in that workflow @Yakov Pechersky

Yakov Pechersky (Nov 15 2022 at 17:13):

In particular, I hope this refactored logic is clearer: https://github.com/leanprover-community/mathlib-tools/pull/137/files#diff-51e32bc74d90e9d3fbf16a3cee752c906ce94722236bf3cc539fbba76b286ec1R37-R44

Yakov Pechersky (Nov 15 2022 at 17:14):

Yes, of course. I was describing just how to start on the port!

Jireh Loreaux (Nov 15 2022 at 17:14):

@Mario Carneiro which mathlib SHA should we take? Presumably the one used by math3port? But how do I find which mathlib3 SHA corresponds to the current mathlib3port I have?

Mario Carneiro (Nov 15 2022 at 17:15):

No, I mean when you git pull mathlib3port and pick a starting point, it is important to record what version you based your port on, that's the only part we can't automate

Mario Carneiro (Nov 15 2022 at 17:15):

It should be in the commit message for mathlib3port

Jireh Loreaux (Nov 15 2022 at 17:16):

All I see in the log is bump to nightly-2022-11-14

Heather Macbeth (Nov 15 2022 at 17:16):

One suggested addition to that workflow: I've been making my first commit just the raw mathport output. The idea is that this would give a better diff for reviewers to look at. See e.g. mathlib4#585. Can the people who are doing port reviews comment on whether this is indeed useful?

Mario Carneiro (Nov 15 2022 at 17:16):

well, it is the mathport nightly name, but that is good enough

Mario Carneiro (Nov 15 2022 at 17:16):

we still need to improve the workflow here but some information is better than none

Jireh Loreaux (Nov 15 2022 at 17:16):

But don't we want the actual mathlib3 SHA so that we can verify it later?

Mario Carneiro (Nov 15 2022 at 17:17):

we do

Mario Carneiro (Nov 15 2022 at 17:17):

I believe the mathlib SHA is stored in a file on that mathport nightly releasee

Riccardo Brasca (Nov 15 2022 at 17:18):

Adam Topaz said:

Can we add a TLDR section to https://github.com/leanprover-community/mathlib4/wiki (or elsewhere) with approximately what Yakov said?

Yes please, this conversation is already becoming too technical to follow :sweat_smile:

Mario Carneiro (Nov 15 2022 at 17:20):

hey @Gabriel Ebner , don't suppose I can get you to improve the mathlib3port CI to put the file with the mathlib SHA in either the commit message or in the root of the mathlib3port repo?

Mario Carneiro (Nov 15 2022 at 17:21):

having to download a 200MB .tar.gz just to find this info feels really unnecesssary

Gabriel Ebner (Nov 15 2022 at 17:24):

Which 200M tar.gz is the info in?

Gabriel Ebner (Nov 15 2022 at 17:30):

(I just noticed that we create a rev file but then only tar the .tlean and .ast.json files...)

Mario Carneiro (Nov 15 2022 at 17:39):

I thought it was in the produced mathlib3-synport but maybe I'm misremembering your earlier comments about the rev file

Gabriel Ebner (Nov 15 2022 at 17:51):

I thought so too... but apparently it was excluded from the tarball all this time.

Mario Carneiro (Nov 15 2022 at 17:55):

is the rev in the CI log?

Jon Eugster (Nov 15 2022 at 17:56):

@Yakov Pechersky Heather Macbeth said:

By the way, Yakov, did you ever implement this?

Scott implemented this in mathlib-tools#133, so it's fixed in the newest version of mathlib-tools.

Gabriel Ebner (Nov 15 2022 at 17:56):

Yes, it's in the CI log. And soon it's also going to be in the tarballs as intended.

Mario Carneiro (Nov 15 2022 at 17:57):

the release notes are also a good place to put it

port-progress bot (Nov 15 2022 at 18:04):

mathlib port progress topology.metric_space.basic
Ported files: 31/528 (5.9% of total)
Ported lines: 10457/211869 (4.9% of total)
Longest unported chain: 71/81 (12.3% progress)

Jireh Loreaux (Nov 15 2022 at 21:11):

@Mario Carneiro or @Gabriel Ebner : could you post the SHAs from the last few nightly releases somewhere, or tell me where I can find them?

Gabriel Ebner (Nov 15 2022 at 21:12):

https://github.com/leanprover-community/mathport/actions/runs/3459238046/jobs/5774422152 should have the revision for the 11/14 nightly.

Gabriel Ebner (Nov 15 2022 at 21:13):

If you wait a couple of hours, we should also hopefully have an upstream-rev file in mathlib3port.

Jireh Loreaux (Nov 15 2022 at 21:15):

Thanks. In case anyone else needs it the SHA for the 11/14 nightly is: aab56fd783b265168f660d6b46709961153c4c20

port-progress bot (Nov 15 2022 at 23:42):

mathlib port progress algebra.order.field.defs
Ported files: 26/75 (34.7% of total)
Ported lines: 9637/26113 (36.9% of total)
Longest unported chain: 10/20 (50.0% progress)

port-progress bot (Nov 15 2022 at 23:46):

mathlib port progress data.rat.order
Ported files: 29/128 (22.7% of total)
Ported lines: 10397/40185 (25.9% of total)
Longest unported chain: 16/26 (38.5% progress)

port-progress bot (Nov 15 2022 at 23:50):

mathlib port progress category_theory.limits.yoneda
Ported files: 23/97 (23.7% of total)
Ported lines: 8711/36359 (24.0% of total)
Longest unported chain: 28/37 (24.3% progress)

port-progress bot (Nov 15 2022 at 23:53):

mathlib port progress data.fintype.basic
Ported files: 28/229 (12.2% of total)
Ported lines: 10323/84925 (12.2% of total)
Longest unported chain: 36/46 (21.7% progress)

port-progress bot (Nov 15 2022 at 23:57):

mathlib port progress topology.metric_space.basic
Ported files: 31/528 (5.9% of total)
Ported lines: 10457/211934 (4.9% of total)
Longest unported chain: 71/81 (12.3% progress)

Moritz Doll (Nov 16 2022 at 00:06):

if a gray file is imported in the target file that means that this import is completely unnecessary (modulo transitive imports), right?

Mario Carneiro (Nov 16 2022 at 00:07):

Mathlib usually doesn't have completely unnecessary imports. Rather, what happens is that A -> B -> C because B has theorems B1 and B2 and C needs B2 and B1 needs A but C doesn't use A

Mario Carneiro (Nov 16 2022 at 00:09):

this is fixed by splitting B into two files B1, B2, so that you get A -> B1 and B2 -> C and hence C no longer transitively imports A

Moritz Doll (Nov 16 2022 at 00:10):

hmm, but if I remove topology.uniform_space.complete_separated from the imports in topology.metric_space.basic it compiles just fine

Scott Morrison (Nov 16 2022 at 00:10):

Yes, that happens too. :-)

Scott Morrison (Nov 16 2022 at 00:11):

You may find this makes someone unhappy downstream, in which case you simply add the import back in there.

Mario Carneiro (Nov 16 2022 at 00:11):

Oh, I thought we had a linter for that but maybe not

Moritz Doll (Nov 16 2022 at 00:11):

I would have guessed we had a linter for that

Mario Carneiro (Nov 16 2022 at 00:11):

It wouldn't be too hard to modify this module_refs program to calculate all unnecessary direct import edges

Scott Morrison (Nov 16 2022 at 00:13):

In particular if you just run scripts/modules_used.lean X, and diff that with the imports of X, it should be telling you direct imports that can be removed.

Mario Carneiro (Nov 16 2022 at 00:13):

how about making a CI job for that? :)

Scott Morrison (Nov 16 2022 at 00:13):

That's probably somewhat expensive to run across all of mathlib.

Scott Morrison (Nov 16 2022 at 00:13):

I'm not sure we want it in every CI run. But we could decide that later.

Mario Carneiro (Nov 16 2022 at 00:14):

Sorry, I meant a one-off job

Mario Carneiro (Nov 16 2022 at 00:14):

I think you can speed it up a bit by collecting all results simultaneously

Mario Carneiro (Nov 16 2022 at 00:15):

plus, you don't need to follow recursive references: since there are no intermediate files in a direct import, some declaration in B must directly reference some declaration in A for the A -> B import to be necessary

Mario Carneiro (Nov 16 2022 at 00:20):

Is the set of direct imports of a module available to lean 3 code? Does leanproject get this info by reading import lines?

Scott Morrison (Nov 16 2022 at 00:25):

There is lean --deps on the command line.

Scott Morrison (Nov 16 2022 at 00:25):

and leanproject calls that

Scott Morrison (Nov 16 2022 at 00:26):

afaik it's not otherwise available

Scott Morrison (Nov 16 2022 at 00:26):

I think if we don't care about efficiency it's just a few lines in bash to achieve this with existing code.

Scott Morrison (Nov 16 2022 at 00:26):

I'm happy to do that, but if you're doing it without following recursive references I won't duplicate!

Mario Carneiro (Nov 16 2022 at 00:46):

lean --deps gives me transitive dependencies in my tests

port-progress bot (Nov 16 2022 at 00:47):

mathlib port progress all
Ported files: 35/2753 (1.3% of total)
Ported lines: 10767/914005 (1.2% of total)
Longest unported chain: 125/135 (7.4% progress)

Mario Carneiro (Nov 16 2022 at 00:48):

Here's a program that does the hard part of the work:

import system.io

meta def decls_used_in : declaration  name_set  name_set
| d ns :=
  let process (v : expr) : name_set :=
    v.fold ns $ λ e _ ns, if e.is_constant then ns.insert e.const_name else ns in
  match d with
  | (declaration.defn _ _ _ v _ _) := process v
  | (declaration.thm _ _ _ v)      := process v.get
  | _ := ns
  end

meta def main : io unit := do
  env  io.run_tactic tactic.get_env,
  let map := env.fold (native.rb_map.mk string name_set) (λ d map,
    match env.decl_olean d.to_name with
    | some tgt := map.insert tgt (decls_used_in d ((map.find tgt).get_or_else mk_name_set))
    | none := map
    end),
  map.mfold () $ λ mod ns _, do
    io.print_ln sformat!"module: {mod}",
    let mods := ns.fold (native.mk_rb_set) (λ n mods, match env.decl_olean n with
    | some tgt := mods.insert tgt
    | none := mods
    end),
    mods.mfold () $ λ mod _, do
      io.print_ln sformat!"needs: {mod}"

Scott Morrison (Nov 16 2022 at 00:50):

Ok, I should have known you were going to do it. :-)

Mario Carneiro (Nov 16 2022 at 00:50):

This will report the module name followed by every module that it directly references (which is hopefully a superset of the direct imports and a subset of the transitive imports). By taking the set difference of "direct imports - reported imports" we get some useful data

Scott Morrison (Nov 16 2022 at 00:51):

Okay, I will hook that up.

Scott Morrison (Nov 16 2022 at 01:38):

Okay, here's the preliminary output: https://gist.github.com/semorrison/e136333cce63c8ffcc080a8997f2a6da

Scott Morrison (Nov 16 2022 at 01:38):

This is not super-duper useful, because often one needs to replace the unneeded import by some of its transitive dependencies, rather than just deleting an unneeded import.

Mario Carneiro (Nov 16 2022 at 01:39):

I was just about to say, you can also derive what transitive imports you need to reintroduce from this data

Scott Morrison (Nov 16 2022 at 01:39):

Yes.

Scott Morrison (Nov 16 2022 at 01:39):

But it's not quite as trivial as the first step I did. :-)

Mario Carneiro (Nov 16 2022 at 01:40):

do you have the unfiltered output of the lean program?

Mario Carneiro (Nov 16 2022 at 01:40):

If I had both the import graph and the direct-use graph I could throw them in mathematica or something to do the graph munging

Scott Morrison (Nov 16 2022 at 01:42):

reqs.gz

Scott Morrison (Nov 16 2022 at 01:43):

I'm already processing it / comparing with existing imports in mathematica.

Scott Morrison (Nov 16 2022 at 01:43):

So I can continue doing that. (But if you want to do it too, please let me know so I stop. :-)

Mario Carneiro (Nov 16 2022 at 01:43):

Eh, I'll let you do it if you have the data

Mario Carneiro (Nov 16 2022 at 01:46):

this will be a great PR, it is a low hanging fruit that will pay huge dividends across the library

Scott Morrison (Nov 16 2022 at 01:54):

Okay, it's looking good. A few spot checks seem to be working out.

Scott Morrison (Nov 16 2022 at 01:55):

Should I try to minimize diffs? i.e. preserving order of existing imports where possible?

Scott Morrison (Nov 16 2022 at 01:56):

or is it okay if for any file where I need to touch the import block I completely replace it with alphabetised imports?

Mario Carneiro (Nov 16 2022 at 01:57):

alphabetizing sounds fine to me

Scott Morrison (Nov 16 2022 at 01:58):

This is going to touch 1497 / 2854 files in mathlib, if all goes well. :-)

Mario Carneiro (Nov 16 2022 at 01:58):

You have to be careful with tactic imports though, I assume you are already handling that

Scott Morrison (Nov 16 2022 at 01:59):

Yes. I'm ignoring them in the processing. So the replacement process will fish them out, and tack them onto the new import list.

Scott Morrison (Nov 16 2022 at 01:59):

So far I've only done about 5 spot checks, so things will presumably still go horribly wrong.

Mario Carneiro (Nov 16 2022 at 01:59):

I mean that tactics are falsely marked as unused

Mario Carneiro (Nov 16 2022 at 01:59):

which could affect your graph calculation

Scott Morrison (Nov 16 2022 at 01:59):

Yes -- so I'll just preserve all the current import tactic.* lines.

Mario Carneiro (Nov 16 2022 at 02:00):

how are the new imports being calculated?

Scott Morrison (Nov 16 2022 at 02:00):

needed \ transitive imports of needed

Mario Carneiro (Nov 16 2022 at 02:01):

I would add direct imports which are needed to that list

Mario Carneiro (Nov 16 2022 at 02:02):

that way you aren't unnecessarily eliminating transitive dependencies

Mario Carneiro (Nov 16 2022 at 02:03):

not sure if that helps with the diff

Mario Carneiro (Nov 16 2022 at 02:05):

Actually if you take the list of direct imports, subtract unneeded ones, then append "needed \ transitive imports of needed", it will avoid the superfluous reordering as well

Scott Morrison (Nov 16 2022 at 02:15):

Okay, so the new procedure for new imports is:

  • take the existing imports, keeping only those that are tactic.*, meta.*, or are needed
  • then add everything in (needed \ transitive imports of needed)
  • finally, remove duplicates without reordering

Scott Morrison (Nov 16 2022 at 02:15):

I think that matches the discussion so far. It will touch 1340 files.

Scott Morrison (Nov 16 2022 at 02:20):

gah, mathematica is munging unicode. :-)

Arien Malec (Nov 16 2022 at 02:21):

I don't have permission for mathlib but I started work on the very small data.char, PR #609

Gabriel Ebner (Nov 16 2022 at 02:27):

could you post the SHAs from the last few nightly releases somewhere, or tell me where I can find them?

They are now available in the upstream-rev file in mathlib3port, the commit message, and the README: https://github.com/leanprover-community/mathlib3port

Scott Morrison (Nov 16 2022 at 02:42):

Ah, so this procedure is missing some tactics imports. I think I need to also add (all transitively imported tactics which are not implied by other imports).

Jireh Loreaux (Nov 16 2022 at 02:46):

@Arien Malec do you mind if I just push to your branch? I had just done this file and I can fix the errors.

Arien Malec (Nov 16 2022 at 02:46):

awesome

Mario Carneiro (Nov 16 2022 at 02:58):

Yes, that was what I was afraid of. Basically, pretend that all tactic.* files are in the needed list for every module

Mario Carneiro (Nov 16 2022 at 03:00):

I think you can combine that with the transitive reduction part, just add all transitively imported tactic.* files to "needed" for the purpose of the rest of the computation

Scott Morrison (Nov 16 2022 at 03:08):

Yes, this part seems okay now.

Scott Morrison (Nov 16 2022 at 03:09):

I've discovered a problem with the original data, actually.

Scott Morrison (Nov 16 2022 at 03:09):

We need to follow the @[ancestor] tag, as well as just inspecting declarations for references.

Scott Morrison (Nov 16 2022 at 03:09):

I'm hoping I can just patch this up by hand.

Scott Morrison (Nov 16 2022 at 03:18):

Hmm, there are quite a few problems caused by the @[ancestor] issue. Continuing by hand for now, but ...

Scott Morrison (Nov 16 2022 at 03:23):

There are also a certain number of imports which are only need for notation.

Mario Carneiro (Nov 16 2022 at 04:25):

what's the @[ancestor] issue?

Mario Carneiro (Nov 16 2022 at 04:26):

I would have expected that if A extends B as a class, there will be some reference to B in the declared parent instance

Scott Morrison (Nov 16 2022 at 04:28):

With old_structure_cmd unfortunately that's not the case. :-(

Scott Morrison (Nov 16 2022 at 15:12):

Okay, #17568 touches 595 files in mathlib, but I think does it.

Riccardo Brasca (Nov 16 2022 at 15:22):

Should we just don't merge anything else for a couple of hours and merge this immediately?

Anne Baanen (Nov 16 2022 at 15:29):

I went through all the non-import changes (using git diff c34a1aa4263bdf585dd705508c11d3b75836049e | grep '^[+-]' | grep -v '^[-+]import') and have just a few comments. If it builds, let's merge!

port-progress bot (Nov 16 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 26/75 (34.7% of total)
Ported lines: 9642/26118 (36.9% of total)
Longest unported chain: 10/20 (50.0% progress)

port-progress bot (Nov 16 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 29/128 (22.7% of total)
Ported lines: 10410/40198 (25.9% of total)
Longest unported chain: 16/26 (38.5% progress)

port-progress bot (Nov 16 2022 at 18:11):

mathlib port progress category_theory.limits.yoneda
Ported files: 23/97 (23.7% of total)
Ported lines: 8719/36367 (24.0% of total)
Longest unported chain: 28/37 (24.3% progress)

port-progress bot (Nov 16 2022 at 18:15):

mathlib port progress data.fintype.basic
Ported files: 28/229 (12.2% of total)
Ported lines: 10336/85027 (12.2% of total)
Longest unported chain: 36/46 (21.7% progress)

port-progress bot (Nov 16 2022 at 18:19):

mathlib port progress topology.metric_space.basic
Ported files: 31/513 (6.0% of total)
Ported lines: 10474/206781 (5.1% of total)
Longest unported chain: 69/79 (12.7% progress)

port-progress bot (Nov 16 2022 at 19:01):

mathlib port progress all
Ported files: 35/2755 (1.3% of total)
Ported lines: 10784/913656 (1.2% of total)
Longest unported chain: 123/133 (7.5% progress)

Riccardo Brasca (Nov 17 2022 at 16:13):

port-status.py lists algebra.order.hom.basic as ready to port, but I don't think it is, since it imports tactic.positivity.

Heather Macbeth (Nov 17 2022 at 16:14):

rss-bot said:

feat: positivity tactic (mathlib4#578)

  • [x] depends on #574

Implements the positivity tactic core, plus several of the positivity extensions. Most of the remaining extensions are blocked on theory files.

Co-authored-by: Scott Morrison <scott.morrison@gmail.com>

Authored-by: digama0 (commit)

Riccardo Brasca (Nov 17 2022 at 16:15):

ops, I need to update my master branch

Jireh Loreaux (Nov 17 2022 at 17:27):

How do I #lint in mathlib 4?

Riccardo Brasca (Nov 17 2022 at 17:35):

#lint works for me.

Alex J. Best (Nov 17 2022 at 17:36):

you need Std.Tactic.Lintimported I guess

Riccardo Brasca (Nov 17 2022 at 17:36):

The wiki says to add

import Std.Tactic.Lint.Frontend
import Std.Tactic.Lint.Misc

Jireh Loreaux (Nov 17 2022 at 17:37):

Ah, I was missing Frontend. Thanks.

port-progress bot (Nov 17 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 26/73 (35.6% of total)
Ported lines: 9670/25739 (37.6% of total)
Longest unported chain: 9/19 (52.6% progress)

Heather Macbeth (Nov 17 2022 at 18:06):

Has the port-progress bot stopped generating and hosting the PDF import graph? (It was still doing this yesterday.). That was a useful feature.

port-progress bot (Nov 17 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 30/126 (23.8% of total)
Ported lines: 10625/39668 (26.8% of total)
Longest unported chain: 15/25 (40.0% progress)

port-progress bot (Nov 17 2022 at 18:12):

mathlib port progress category_theory.limits.yoneda
Ported files: 22/95 (23.2% of total)
Ported lines: 7871/35513 (22.2% of total)
Longest unported chain: 27/36 (25.0% progress)

port-progress bot (Nov 17 2022 at 18:16):

mathlib port progress data.fintype.basic
Ported files: 29/221 (13.1% of total)
Ported lines: 11013/84854 (13.0% of total)
Longest unported chain: 33/43 (23.3% progress)

port-progress bot (Nov 17 2022 at 18:19):

mathlib port progress topology.metric_space.basic
Ported files: 33/500 (6.6% of total)
Ported lines: 11339/206207 (5.5% of total)
Longest unported chain: 66/76 (13.2% progress)

port-progress bot (Nov 17 2022 at 19:00):

mathlib port progress all
Ported files: 38/2755 (1.4% of total)
Ported lines: 11672/913532 (1.3% of total)
Longest unported chain: 116/126 (7.9% progress)

Scott Morrison (Nov 17 2022 at 22:46):

Oh... when I changed the table format I didn't update the regex that was inserting the links.

Scott Morrison (Nov 17 2022 at 22:46):

(insert obligatory link to SO...)

port-progress bot (Nov 18 2022 at 00:49):

mathlib port progress algebra.order.field.defs
Ported files: 26/73 (35.6% of total)
Ported lines: 9670/25739 (37.6% of total)
Longest unported chain: 9/19 (52.6% progress)

port-progress bot (Nov 18 2022 at 00:53):

mathlib port progress data.rat.order
Ported files: 30/126 (23.8% of total)
Ported lines: 10625/39668 (26.8% of total)
Longest unported chain: 15/25 (40.0% progress)

port-progress bot (Nov 18 2022 at 00:57):

mathlib port progress category_theory.limits.yoneda
Ported files: 22/95 (23.2% of total)
Ported lines: 7871/35513 (22.2% of total)
Longest unported chain: 27/36 (25.0% progress)

port-progress bot (Nov 18 2022 at 01:00):

mathlib port progress data.fintype.basic
Ported files: 30/221 (13.6% of total)
Ported lines: 11084/84854 (13.1% of total)
Longest unported chain: 33/43 (23.3% progress)

port-progress bot (Nov 18 2022 at 01:05):

mathlib port progress topology.metric_space.basic
Ported files: 36/500 (7.2% of total)
Ported lines: 12113/206285 (5.9% of total)
Longest unported chain: 66/76 (13.2% progress)

port-progress bot (Nov 18 2022 at 01:45):

mathlib port progress all
Ported files: 41/2756 (1.5% of total)
Ported lines: 12450/913326 (1.4% of total)
Longest unported chain: 116/126 (7.9% progress)

Heather Macbeth (Nov 18 2022 at 10:50):

Feature request: Could we add mathlib4 curves to the graphs at
https://leanprover-community.github.io/mathlib_stats.html
of number of files and number of lines over time? That is, display mathlib3 and mathlib4 on the same graph.

port-progress bot (Nov 18 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 33/73 (45.2% of total)
Ported lines: 13400/25823 (51.9% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 18 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 37/126 (29.4% of total)
Ported lines: 14359/39756 (36.1% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 18 2022 at 18:11):

mathlib port progress category_theory.limits.yoneda
Ported files: 27/90 (30.0% of total)
Ported lines: 10548/30300 (34.8% of total)
Longest unported chain: 26/36 (27.8% progress)

port-progress bot (Nov 18 2022 at 18:15):

mathlib port progress data.fintype.basic
Ported files: 37/185 (20.0% of total)
Ported lines: 14818/73234 (20.2% of total)
Longest unported chain: 26/39 (33.3% progress)

port-progress bot (Nov 18 2022 at 18:18):

mathlib port progress topology.metric_space.basic
Ported files: 43/510 (8.4% of total)
Ported lines: 15859/205604 (7.7% of total)
Longest unported chain: 63/76 (17.1% progress)

port-progress bot (Nov 18 2022 at 19:00):

mathlib port progress all
Ported files: 49/2769 (1.8% of total)
Ported lines: 16389/912462 (1.8% of total)
Longest unported chain: 113/126 (10.3% progress)

Scott Morrison (Nov 18 2022 at 21:33):

Huh, why is order.lattice not showing up in bright blue in these graphs? It looks like it should be ready to port.

Yakov Pechersky (Nov 18 2022 at 21:34):

It probably has some dependency which is getting hidden in the output

Ruben Van de Velde (Nov 18 2022 at 21:39):

Maybe the tool realized it needed tactic ports? Either that or the typo on the wiki page that I've fixed (I forgot the "no" before "wip")

Scott Morrison (Nov 18 2022 at 21:41):

Ah, typo would explain it.

port-progress bot (Nov 19 2022 at 18:05):

mathlib port progress algebra.order.field.defs
Ported files: 33/73 (45.2% of total)
Ported lines: 13403/25826 (51.9% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 19 2022 at 18:10):

mathlib port progress data.rat.order
Ported files: 37/126 (29.4% of total)
Ported lines: 14362/39759 (36.1% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 19 2022 at 18:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 27/90 (30.0% of total)
Ported lines: 10551/30303 (34.8% of total)
Longest unported chain: 26/36 (27.8% progress)

port-progress bot (Nov 19 2022 at 18:18):

mathlib port progress data.fintype.basic
Ported files: 37/185 (20.0% of total)
Ported lines: 14821/73237 (20.2% of total)
Longest unported chain: 26/39 (33.3% progress)

port-progress bot (Nov 19 2022 at 18:23):

mathlib port progress topology.metric_space.basic
Ported files: 43/510 (8.4% of total)
Ported lines: 15862/205622 (7.7% of total)
Longest unported chain: 63/76 (17.1% progress)

port-progress bot (Nov 19 2022 at 19:25):

mathlib port progress all
Ported files: 49/2770 (1.8% of total)
Ported lines: 16396/912497 (1.8% of total)
Longest unported chain: 113/126 (10.3% progress)

port-progress bot (Nov 20 2022 at 01:12):

mathlib port progress algebra.order.field.defs
Ported files: 35/73 (47.9% of total)
Ported lines: 13647/30688 (44.5% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 20 2022 at 01:15):

mathlib port progress data.rat.order
Ported files: 39/126 (31.0% of total)
Ported lines: 14606/49374 (29.6% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 20 2022 at 01:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 27/90 (30.0% of total)
Ported lines: 10551/30303 (34.8% of total)
Longest unported chain: 26/36 (27.8% progress)

port-progress bot (Nov 20 2022 at 01:22):

mathlib port progress data.fintype.basic
Ported files: 39/186 (21.0% of total)
Ported lines: 15065/83481 (18.0% of total)
Longest unported chain: 26/39 (33.3% progress)

port-progress bot (Nov 20 2022 at 01:26):

mathlib port progress topology.metric_space.basic
Ported files: 45/511 (8.8% of total)
Ported lines: 16106/223920 (7.2% of total)
Longest unported chain: 63/76 (17.1% progress)

port-progress bot (Nov 20 2022 at 02:06):

mathlib port progress all
Ported files: 51/2771 (1.8% of total)
Ported lines: 16640/955250 (1.7% of total)
Longest unported chain: 113/126 (10.3% progress)

Scott Morrison (Nov 20 2022 at 02:32):

If anyone is looking for things to do on the mathlib3 side, clicking on the "longest unported chain" links above, and identifying if there are file splits / lemma rearrangements that can remove the need (or delay the import) of files marked with -, could be helpful.

Scott Morrison (Nov 20 2022 at 02:32):

The longest chain overall is still to analysis.normed_space.star.gelfand_duality, but it has impressively few files marked - now.

port-progress bot (Nov 20 2022 at 18:03):

mathlib port progress algebra.order.field.defs
Ported files: 37/73 (50.7% of total)
Ported lines: 15070/30688 (49.1% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 20 2022 at 18:07):

mathlib port progress data.rat.order
Ported files: 42/126 (33.3% of total)
Ported lines: 16109/49379 (32.6% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 20 2022 at 18:10):

mathlib port progress category_theory.limits.yoneda
Ported files: 28/90 (31.1% of total)
Ported lines: 10680/30303 (35.2% of total)
Longest unported chain: 25/36 (30.6% progress)

port-progress bot (Nov 20 2022 at 18:14):

mathlib port progress data.fintype.basic
Ported files: 42/186 (22.6% of total)
Ported lines: 16568/83486 (19.8% of total)
Longest unported chain: 26/39 (33.3% progress)

port-progress bot (Nov 20 2022 at 18:17):

mathlib port progress topology.metric_space.basic
Ported files: 50/511 (9.8% of total)
Ported lines: 17759/223933 (7.9% of total)
Longest unported chain: 63/76 (17.1% progress)

port-progress bot (Nov 20 2022 at 18:58):

mathlib port progress all
Ported files: 60/2771 (2.2% of total)
Ported lines: 18819/955260 (2.0% of total)
Longest unported chain: 113/126 (10.3% progress)

port-progress bot (Nov 20 2022 at 23:57):

mathlib port progress (algebra.order.field.defs)
Ported files: 36/73 (49.3% of total)
Ported lines: 18630/33252 (56.0% of total)
Longest unported chain: 11/19 (42.1% progress)

port-progress bot (Nov 21 2022 at 00:00):

mathlib port progress (data.rat.order)
Ported files: 83/126 (65.9% of total)
Ported lines: 36152/51951 (69.6% of total)
Longest unported chain: 11/25 (56.0% progress)

port-progress bot (Nov 21 2022 at 00:03):

mathlib port progress (category_theory.limits.yoneda)
Ported files: 62/90 (68.9% of total)
Ported lines: 22152/32832 (67.5% of total)
Longest unported chain: 9/36 (75.0% progress)

port-progress bot (Nov 21 2022 at 00:07):

mathlib port progress (data.fintype.basic)
Ported files: 143/186 (76.9% of total)
Ported lines: 69870/86128 (81.1% of total)
Longest unported chain: 11/39 (71.8% progress)

port-progress bot (Nov 21 2022 at 00:10):

mathlib port progress (topology.metric_space.basic)
Ported files: 460/511 (90.0% of total)
Ported lines: 209186/226635 (92.3% of total)
Longest unported chain: 11/76 (85.5% progress)

Scott Morrison (Nov 21 2022 at 00:12):

Sorry, recent updates seem to have completely borked the port-progress-bot, and I'm about to get on a plane.

Scott Morrison (Nov 21 2022 at 00:23):

It seems that it has everything backwards.:-)

Riccardo Brasca (Nov 21 2022 at 09:58):

I think something nasty happened with algebra.order.absolute_value. The port status script marks it as ready to port, since it's only import, algebra.order.hom.basic is ported (this is correct). The problem is that algebra.order.hom.basic imports tactic.positivity (both in mathlib3 and mathlib4). But now the two diverge, in mathlib3 the imports are

import tactic.norm_num
import algebra.order.field.power

while in mathlib4 are

import Mathlib.Tactic.Positivity.Basic
import Mathlib.Tactic.NormNum.Basic
import Mathlib.Init.Data.Int.Order

(this is the whole Mathlib/Tactic/Positivity file). The point is that algebra/hom/group.lean is transitively imported in algebra.order.absolute_value (and really needed, already in the first declaration), while this file is not ported.

What should we do? It's not easy to fix the import in Mathlib/Tactic/Positivity, since the real ones do not exist.

Mario Carneiro (Nov 21 2022 at 10:20):

the simple fix would be to add import algebra.hom.group to algebra.order.absolute_value

Mario Carneiro (Nov 21 2022 at 10:21):

alternatively, the port-status program could look at transitive imports when deciding that a file is ready to port. I guess there is a reason it is not already doing so, e.g. this includes a bunch of unnecessary stuff

Riccardo Brasca (Nov 21 2022 at 10:21):

In this concrete case I think it is enough to add a note in the port-status page

Riccardo Brasca (Nov 21 2022 at 10:21):

I don't if we can do something more sistematic

Mario Carneiro (Nov 21 2022 at 10:21):

I mean, pulling in and accidentally relying on transitive imports is an issue that comes up all the time

Mario Carneiro (Nov 21 2022 at 10:22):

I don't think the solution should be to add imports to Mathlib.Tactic.Positivity, the original imports were too much anyway

Ruben Van de Velde (Nov 21 2022 at 10:23):

Hrm, this was fixed in leanproject import-graph --exclude-tactics already, that shows that algebra.order.absolute_value depends on an absolute spaghetti of unported files

Ruben Van de Velde (Nov 21 2022 at 10:24):

Mario Carneiro (Nov 21 2022 at 10:25):

An in between alternative would be to "inline" the imports of tactic files when determining the "direct" imports of a file

Ruben Van de Velde (Nov 21 2022 at 10:25):

(positivity pulls in norm_num which needs data.rat.cast which needs... a lot)

Riccardo Brasca (Nov 21 2022 at 10:25):

Ruben Van de Velde said:

Hrm, this was fixed in leanproject import-graph --exclude-tactics already, that shows that algebra.order.absolute_value depends on an absolute spaghetti of unported files

Maybe the script needs to be updated? It is still shown, at least for me.

Ruben Van de Velde (Nov 21 2022 at 10:26):

https://github.com/leanprover-community/mathlib-tools/commit/76edd6f66c23e9f4cbd0b7d9d0484d928d839b4e

Ruben Van de Velde (Nov 21 2022 at 10:26):

I think we previously discussed a divergence between port_status.py and leanproject

Eric Wieser (Nov 21 2022 at 10:52):

Yes we did, here

Eric Wieser (Nov 21 2022 at 10:52):

Ruben Van de Velde said:

https://github.com/leanprover-community/mathlib-tools/commit/76edd6f66c23e9f4cbd0b7d9d0484d928d839b4e

This commit has not been released, so almost no one is using this code

Eric Wieser (Nov 21 2022 at 10:52):

Which is an argument in favor of moving all this stuff out of mathlibtools

Riccardo Brasca (Nov 21 2022 at 10:59):

I missed that discussion. I don't have an opinion, but we should surely have only one tool.

Patrick Massot (Nov 21 2022 at 11:04):

Again, if the only problem is I don't have time to review mathlibtools PR then anyone should feel free to merge PRs that don't touch the core functionalities (around the olean cache). If you need me to release a new version to pypi then simply tell me.

port-progress bot (Nov 21 2022 at 18:04):

mathlib port progress (algebra.order.field.defs)
Ported files: 41/79 (51.9% of total)
Ported lines: 20121/34881 (57.7% of total)
Longest unported chain: 11/19 (42.1% progress)

port-progress bot (Nov 21 2022 at 18:08):

mathlib port progress (data.rat.order)
Ported files: 85/128 (66.4% of total)
Ported lines: 36754/52553 (69.9% of total)
Longest unported chain: 11/25 (56.0% progress)

port-progress bot (Nov 21 2022 at 18:11):

mathlib port progress (category_theory.limits.yoneda)
Ported files: 62/90 (68.9% of total)
Ported lines: 22152/32832 (67.5% of total)
Longest unported chain: 9/36 (75.0% progress)

port-progress bot (Nov 21 2022 at 18:14):

mathlib port progress (data.fintype.basic)
Ported files: 143/186 (76.9% of total)
Ported lines: 69874/86132 (81.1% of total)
Longest unported chain: 11/39 (71.8% progress)

port-progress bot (Nov 21 2022 at 18:18):

mathlib port progress (topology.metric_space.basic)
Ported files: 460/511 (90.0% of total)
Ported lines: 209275/226724 (92.3% of total)
Longest unported chain: 11/76 (85.5% progress)

port-progress bot (Nov 21 2022 at 18:22):

mathlib port progress (all)
Ported files: 2709/2770 (97.8% of total)
Ported lines: 939750/958259 (98.1% of total)
Longest unported chain: 11/126 (91.3% progress)

Jireh Loreaux (Nov 21 2022 at 18:26):

Wow! We ported a few thousand files really quickly? And people said this would take a while. :upside_down:

Kevin Buzzard (Nov 21 2022 at 18:32):

yeah I pulled an all-nighter on Sunday, I was pretty annoyed that I had to go to sleep when there were just 61 files to go. OK not really.

Scott Morrison (Nov 22 2022 at 00:06):

Ah, I was hoping to get off the plane and someone would have diagnosed this. :-)

Scott Morrison (Nov 22 2022 at 00:07):

These reports are created using leanproject --port-progress, if someone wants to have a look.

Jireh Loreaux (Nov 22 2022 at 00:18):

Sorry, been busy with other things.

Yakov Pechersky (Nov 22 2022 at 00:31):

    def delete_ported(self) -> 'ImportGraph':
        """Delete all nodes marked as ported during port_status"""
        H = self.subgraph({node for node, attrs in self.nodes(data=True)
                          if attrs.get("status") and attrs.get("status").ported})
        H.base_path = self.base_path
        return H

I think this is missing a not!

Yakov Pechersky (Nov 22 2022 at 00:32):

https://github.com/leanprover-community/mathlib-tools/pull/151

Scott Morrison (Nov 22 2022 at 00:44):

Looks good running locally. I've asked the bot to run again.

port-progress bot (Nov 22 2022 at 00:47):

mathlib port progress algebra.order.field.defs
Ported files: 38/79 (48.1% of total)
Ported lines: 14776/34898 (42.3% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 22 2022 at 00:51):

mathlib port progress data.rat.order
Ported files: 43/128 (33.6% of total)
Ported lines: 15819/52574 (30.1% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 22 2022 at 00:54):

mathlib port progress category_theory.limits.yoneda
Ported files: 28/90 (31.1% of total)
Ported lines: 10684/32837 (32.5% of total)
Longest unported chain: 25/36 (30.6% progress)

Moritz Doll (Nov 22 2022 at 00:55):

the links to the pdf seem to be broken

port-progress bot (Nov 22 2022 at 00:58):

mathlib port progress data.fintype.basic
Ported files: 43/186 (23.1% of total)
Ported lines: 16278/86159 (18.9% of total)
Longest unported chain: 26/39 (33.3% progress)

port-progress bot (Nov 22 2022 at 01:01):

mathlib port progress topology.metric_space.basic
Ported files: 51/511 (10.0% of total)
Ported lines: 17473/226793 (7.7% of total)
Longest unported chain: 63/76 (17.1% progress)

port-progress bot (Nov 22 2022 at 01:05):

mathlib port progress all
Ported files: 61/2770 (2.2% of total)
Ported lines: 18545/958364 (1.9% of total)
Longest unported chain: 113/126 (10.3% progress)

Scott Morrison (Nov 22 2022 at 05:17):

The pdf links are curently broken because leanproject import-graph X.pdf fails with

Node names and attributes should not contain ":" unless they are quoted with "".
For example the string 'attribute:data1' should be written as '"attribute:data1"'.

I suspect this came from https://github.com/leanprover-community/mathlib-tools/pull/149, but won't have a chance to look until tomorrow.

Yakov Pechersky (Nov 22 2022 at 12:17):

It still works locally for me, strange.

Yakov Pechersky (Nov 22 2022 at 15:52):

(base)   mathlib git:(master) leanproject import-graph --to algebra.order.ring.defs --exclude-tactics algebra.order.ring.pdf --port-status --mathlib4 ~/math/mathlib4 --reduce
(base)   mathlib git:(master) wslview algebra.order.ring.pdf

image.png

Yakov Pechersky (Nov 22 2022 at 15:52):

And the links are clickable

port-progress bot (Nov 22 2022 at 18:23):

mathlib port progress algebra.order.field.defs
Ported files: 39/79 (49.4% of total)
Ported lines: 14865/34898 (42.6% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 22 2022 at 18:26):

mathlib port progress data.rat.order
Ported files: 44/128 (34.4% of total)
Ported lines: 15908/52580 (30.3% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 22 2022 at 18:29):

mathlib port progress data.nat.choose.basic
Ported files: 40/125 (32.0% of total)
Ported lines: 15032/52149 (28.8% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 22 2022 at 18:33):

mathlib port progress category_theory.limits.yoneda
Ported files: 28/90 (31.1% of total)
Ported lines: 10684/32837 (32.5% of total)
Longest unported chain: 25/36 (30.6% progress)

port-progress bot (Nov 22 2022 at 18:37):

mathlib port progress data.fintype.basic
Ported files: 44/188 (23.4% of total)
Ported lines: 16367/86326 (19.0% of total)
Longest unported chain: 26/39 (33.3% progress)

Scott Morrison (Nov 22 2022 at 18:37):

@Yakov Pechersky, mathlib-tools#137 unintentionally clobbered the --show-unused flag.

Scott Morrison (Nov 22 2022 at 18:38):

Previously, in the presence of --show-unused it was finding the unused imports, and setting their fillcolor to grey. Then the --port-status flag was overwriting the colors, but it wasn't actually overwriting anything that was still white.

Scott Morrison (Nov 22 2022 at 18:38):

Now --port-status simply overwrites the fill colors that --show-unused had produced.

Scott Morrison (Nov 22 2022 at 18:38):

Would you be able to fix that?

port-progress bot (Nov 22 2022 at 18:40):

mathlib port progress topology.metric_space.basic
Ported files: 52/511 (10.2% of total)
Ported lines: 17562/226885 (7.7% of total)
Longest unported chain: 63/76 (17.1% progress)

Scott Morrison (Nov 22 2022 at 18:44):

Yakov Pechersky said:

It still works locally for me, strange.

I couldn't get it to work, but after https://github.com/leanprover-community/mathlib-tools/pull/152 it's fine.

Scott Morrison (Nov 22 2022 at 18:45):

Could you check that that works at your end?

port-progress bot (Nov 22 2022 at 19:19):

mathlib port progress all
Ported files: 62/2773 (2.2% of total)
Ported lines: 18634/959275 (1.9% of total)
Longest unported chain: 113/126 (10.3% progress)

Yakov Pechersky (Nov 23 2022 at 03:14):

https://github.com/leanprover-community/mathlib-tools/pull/153

Yakov Pechersky (Nov 23 2022 at 03:14):

That fixes the --show-unused clobber

Yakov Pechersky (Nov 23 2022 at 03:14):

And yes, links work locally for me

Scott Morrison (Nov 23 2022 at 03:16):

Great, thanks! Running port-progress-bot using mathlib-tools#153 now.

port-progress bot (Nov 23 2022 at 03:20):

mathlib port progress algebra.order.field.defs
Ported files: 39/79 (49.4% of total)
Ported lines: 14865/34898 (42.6% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 23 2022 at 03:23):

mathlib port progress data.rat.order
Ported files: 45/128 (35.2% of total)
Ported lines: 16008/52580 (30.4% of total)
Longest unported chain: 12/25 (52.0% progress)

Scott Morrison (Nov 23 2022 at 03:26):

@Yakov Pechersky, hmm, those last two were running with your PR, but it still seems the gray is being clobbered.

Yakov Pechersky (Nov 23 2022 at 03:26):

image.png

Yakov Pechersky (Nov 23 2022 at 03:26):

I see gray for 2 nodes there, green for one, white for the last

Scott Morrison (Nov 23 2022 at 03:30):

Oh! My browser had a cached version.

Scott Morrison (Nov 23 2022 at 03:30):

Ah, but we need a slightly more complicated logic, I think.

Yakov Pechersky (Nov 23 2022 at 03:30):

cache invalidation and off by one errors, the three hard things about programming

Scott Morrison (Nov 23 2022 at 03:30):

Green/Dark blue/Light blue should all clobber gray.

Scott Morrison (Nov 23 2022 at 03:31):

It's just white that shouldn't clobber gray.

Yakov Pechersky (Nov 23 2022 at 03:31):

:+1: will make happen

Scott Morrison (Nov 23 2022 at 03:33):

I think maybe similarly with --mathlib4: there's no point showing the red outline for files that have already been ported.

Yakov Pechersky (Nov 23 2022 at 04:15):

OK, try it now

Riccardo Brasca (Nov 23 2022 at 12:06):

Is it correct that we now have a bot that add the "frozen file" header in mathlib automatically? I am thinking of #17686

Scott Morrison (Nov 23 2022 at 13:16):

It is not quite automatic. It makes the PR, but someone needs to double check it and hit merge. The last commit it made was incorrect, so perhaps it is still a WIP. :-)

port-progress bot (Nov 23 2022 at 13:22):

mathlib port progress algebra.order.field.defs
Ported files: 39/79 (49.4% of total)
Ported lines: 14865/34898 (42.6% of total)
Longest unported chain: 7/19 (63.2% progress)

Eric Rodriguez (Nov 23 2022 at 13:26):

#17630 I'd appreciate a review on this, which should make the task of checking which files are still in sync far easier.

port-progress bot (Nov 23 2022 at 13:26):

mathlib port progress data.rat.order
Ported files: 45/128 (35.2% of total)
Ported lines: 16008/52580 (30.4% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 23 2022 at 13:29):

mathlib port progress data.nat.choose.basic
Ported files: 41/125 (32.8% of total)
Ported lines: 15132/52149 (29.0% of total)
Longest unported chain: 12/25 (52.0% progress)

Johan Commelin (Nov 23 2022 at 13:31):

Eric Rodriguez said:

#17630 I'd appreciate a review on this, which should make the task of checking which files are still in sync far easier.

I just tested it, and it looks good. But the 1 < len(argv) is a bit hacky.

Johan Commelin (Nov 23 2022 at 13:31):

I think you could even just enable this by default.

Scott Morrison (Nov 23 2022 at 13:32):

:racecar:, just wrote the same thing on the PR.

port-progress bot (Nov 23 2022 at 13:33):

mathlib port progress category_theory.limits.yoneda
Ported files: 28/90 (31.1% of total)
Ported lines: 10684/32837 (32.5% of total)
Longest unported chain: 25/36 (30.6% progress)

port-progress bot (Nov 23 2022 at 13:36):

mathlib port progress data.fintype.basic
Ported files: 45/188 (23.9% of total)
Ported lines: 16467/86326 (19.1% of total)
Longest unported chain: 26/39 (33.3% progress)

port-progress bot (Nov 23 2022 at 13:40):

mathlib port progress topology.metric_space.basic
Ported files: 54/511 (10.6% of total)
Ported lines: 17899/226885 (7.9% of total)
Longest unported chain: 63/76 (17.1% progress)

port-progress bot (Nov 23 2022 at 14:24):

mathlib port progress all
Ported files: 69/2773 (2.5% of total)
Ported lines: 19679/959511 (2.1% of total)
Longest unported chain: 113/126 (10.3% progress)

port-progress bot (Nov 23 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 39/79 (49.4% of total)
Ported lines: 14865/34898 (42.6% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 23 2022 at 18:07):

mathlib port progress data.rat.order
Ported files: 45/128 (35.2% of total)
Ported lines: 16008/52580 (30.4% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 23 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 41/125 (32.8% of total)
Ported lines: 15132/52149 (29.0% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 23 2022 at 18:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 28/90 (31.1% of total)
Ported lines: 10684/32837 (32.5% of total)
Longest unported chain: 25/36 (30.6% progress)

port-progress bot (Nov 23 2022 at 18:18):

mathlib port progress data.fintype.basic
Ported files: 46/188 (24.5% of total)
Ported lines: 16633/86326 (19.3% of total)
Longest unported chain: 26/39 (33.3% progress)

port-progress bot (Nov 23 2022 at 18:22):

mathlib port progress topology.metric_space.basic
Ported files: 55/511 (10.8% of total)
Ported lines: 18065/226885 (8.0% of total)
Longest unported chain: 63/76 (17.1% progress)

port-progress bot (Nov 23 2022 at 19:06):

mathlib port progress all
Ported files: 69/2773 (2.5% of total)
Ported lines: 19679/959511 (2.1% of total)
Longest unported chain: 113/126 (10.3% progress)

Scott Morrison (Nov 23 2022 at 20:42):

logic.embedding.basic and data.finite.defs are newly available for porting.

Kevin Buzzard (Nov 23 2022 at 20:54):

I'll do logic.embedding.basic

Eric Wieser (Nov 23 2022 at 20:59):

The problem with #17686 is not that the bot was broken, but that the yaml file was wrong!

Eric Wieser (Nov 23 2022 at 21:00):

I'll update the bot today or tomorrow to make it more obvious when that happens

Arien Malec (Nov 23 2022 at 21:05):

data.finite.defs looks doable for me.

Kevin Buzzard (Nov 23 2022 at 21:10):

Wait -- logic.embedding.basic seems to need tactic.lift which doesn't seem to be ported? There's some instance of can_lift early on. Do I just skip it?

Scott Morrison (Nov 23 2022 at 21:50):

Yes, we've been skipping instances for lift.

Eric Wieser (Nov 23 2022 at 22:29):

Are open PRs supposed to be marked "Yes" in the port status page?

Eric Wieser (Nov 23 2022 at 22:30):

I just noticed that https://github.com/leanprover-community/mathlib/pull/17686 (which is on the queue) adds a "ported" comment to a file that actually isn't ported yet, but rather just has a PR open

Ruben Van de Velde (Nov 23 2022 at 22:32):

Open PRs should be "no wip"

Eric Wieser (Nov 23 2022 at 22:33):

Looking more closely, this is the gray area where it's on the mathlib4 queue

Yakov Pechersky (Nov 23 2022 at 23:22):

It should have a PR number but not have Yes

Yakov Pechersky (Nov 23 2022 at 23:23):

Right now the syntax is stringly typed, if we switch to the other format (check the wiki for the new page) I think it'll be clearer

Scott Morrison (Nov 24 2022 at 01:48):

I have been using bors merge and then switching to Yes before waiting for it to actually hit master. Hopefully this hasn't caused to many problems. I can be more conservative if so.

Riccardo Brasca (Nov 24 2022 at 08:15):

bors failed on #17686, should we try again? Maybe merging master

Ruben Van de Velde (Nov 24 2022 at 08:50):

I'd just retry

Floris van Doorn (Nov 24 2022 at 08:53):

we should fix the timeout/slowdown in linear_algebra/matrix/sesquilinear_form.lean:322:0

Riccardo Brasca (Nov 24 2022 at 09:13):

I am having a look

Eric Wieser (Nov 24 2022 at 09:16):

@Scott Morrison: no, no problems caused; just surprised to see the bot mention an open PR

Eric Wieser (Nov 24 2022 at 09:18):

It would be great if someone could review #17693, since otherwise the old version of the bot will run at 0 UTC tonight and clobber the output that's currently in #17686.

Riccardo Brasca (Nov 24 2022 at 09:45):

#17705 for the timeout. I think squeezing the simp is enough.

port-progress bot (Nov 24 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 43/79 (54.4% of total)
Ported lines: 17756/34927 (50.8% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 24 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 50/128 (39.1% of total)
Ported lines: 19376/52607 (36.8% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 24 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 46/125 (36.8% of total)
Ported lines: 18500/52181 (35.5% of total)
Longest unported chain: 12/25 (52.0% progress)

port-progress bot (Nov 24 2022 at 18:15):

mathlib port progress category_theory.limits.yoneda
Ported files: 31/90 (34.4% of total)
Ported lines: 12267/32866 (37.3% of total)
Longest unported chain: 25/36 (30.6% progress)

port-progress bot (Nov 24 2022 at 18:18):

mathlib port progress data.fintype.basic
Ported files: 52/188 (27.7% of total)
Ported lines: 20072/86176 (23.3% of total)
Longest unported chain: 26/39 (33.3% progress)

port-progress bot (Nov 24 2022 at 18:22):

mathlib port progress topology.metric_space.basic
Ported files: 61/512 (11.9% of total)
Ported lines: 21504/226950 (9.5% of total)
Longest unported chain: 63/76 (17.1% progress)

port-progress bot (Nov 24 2022 at 19:03):

mathlib port progress all
Ported files: 76/2774 (2.7% of total)
Ported lines: 23221/959618 (2.4% of total)
Longest unported chain: 113/126 (10.3% progress)

Riccardo Brasca (Nov 25 2022 at 10:10):

Is it doable to have a script that update the hash in #port-status if the diff is only

+> THIS FILE IS SYNCHRONIZED WITH MATHLIB4.
+> https://github.com/leanprover-community/mathlib4/pull/*
+> Any changes to this file require a corresponding PR to mathlib4.
+

Currently port_status.py gives several results like that, and we are sure that in these cases updating the hash cannot hurt.

port-progress bot (Nov 25 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 45/79 (57.0% of total)
Ported lines: 19315/35065 (55.1% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 25 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 54/128 (42.2% of total)
Ported lines: 21411/52772 (40.6% of total)
Longest unported chain: 11/25 (56.0% progress)

Eric Wieser (Nov 25 2022 at 18:11):

I don't think we should even both updating #port-status, we should just report the file as unchanged

port-progress bot (Nov 25 2022 at 18:12):

mathlib port progress data.nat.choose.basic
Ported files: 50/125 (40.0% of total)
Ported lines: 20535/52346 (39.2% of total)
Longest unported chain: 11/25 (56.0% progress)

port-progress bot (Nov 25 2022 at 18:15):

mathlib port progress category_theory.limits.yoneda
Ported files: 32/90 (35.6% of total)
Ported lines: 13364/32890 (40.6% of total)
Longest unported chain: 25/36 (30.6% progress)

Ruben Van de Velde (Nov 25 2022 at 18:18):

Looks like algebra.order.sub.defs and order.min_max are up for grabs now

port-progress bot (Nov 25 2022 at 18:19):

mathlib port progress data.fintype.basic
Ported files: 56/184 (30.4% of total)
Ported lines: 22115/85605 (25.8% of total)
Longest unported chain: 24/38 (36.8% progress)

port-progress bot (Nov 25 2022 at 18:22):

mathlib port progress topology.metric_space.basic
Ported files: 65/516 (12.6% of total)
Ported lines: 23555/227232 (10.4% of total)
Longest unported chain: 59/73 (19.2% progress)

port-progress bot (Nov 25 2022 at 19:01):

mathlib port progress all
Ported files: 80/2778 (2.9% of total)
Ported lines: 25296/960957 (2.6% of total)
Longest unported chain: 109/123 (11.4% progress)

Kevin Buzzard (Nov 26 2022 at 15:32):

Can somebody show me an example of exactly what to type to generate one of these pdfs? I've read the manual but I must be understanding what path to file looks like or something, and I couldn't see an example in the manual

Kevin Buzzard (Nov 26 2022 at 15:34):

I'm in Ubuntu and happy to install anything

Ruben Van de Velde (Nov 26 2022 at 16:20):

Not at my laptop right now, so I can't promise it's exact, but something like leanproject import-graph --to data.nat.basic --no-tactics someNameForOutputFile.pdf

Jireh Loreaux (Nov 26 2022 at 16:24):

It's --exclude-tactics and you want --port-status too.

Scott Morrison (Nov 26 2022 at 16:40):

The port-progress-bot is running:

leanproject import-graph --to $target --exclude-tactics --reduce --port-status --show-unused --mathlib4 $tmp_dir/mathlib4 $graph_dir/$today/$target.pdf

Scott Morrison (Nov 26 2022 at 16:40):

--reduce is very helpful for making readable graphs. It removes all the transitively redundant edges.

Scott Morrison (Nov 26 2022 at 16:41):

--show-unused shades files which are not directly required by the --to file in grey. They indicate places where some refactoring might be useful!

Scott Morrison (Nov 26 2022 at 16:41):

--mathlib4 <dir> outlines in red any unported files that nevertheless exist as adhoc ports in the mathlib4 repo.

Scott Morrison (Nov 26 2022 at 16:42):

--port-status is the flag that highlights things in

  • green: already ported
  • light blue: ready to port
  • darker blue: PR open, please review

Kevin Buzzard (Nov 26 2022 at 17:06):

buzzard@buster:~/lean-projects/mathlib$ leanproject import-graph --to src/topology/uniform_space/compare_reals.lean --exclude-tactics --reduce --port-status --show-unused --mathlib4 ~/tmp/mathlib4 compare_reals.pdf
Usage: leanproject import-graph [OPTIONS] [OUTPUT]
Try "leanproject import-graph -h" for help.

Error: no such option: --show-unused
buzzard@buster:~/lean-projects/mathlib$ leanproject --version
leanproject, version 1.3.0
buzzard@buster:~/lean-projects/mathlib$

Help me I am stupid. I cannot get this thing to work

Kevin Buzzard (Nov 26 2022 at 17:07):

buzzard@buster:~/lean-projects/mathlib$ leanproject import-graph --to topology.uniform_space.compare_reals --exclude-tactics --reduce --port-status --show-unused --mathlib4 ~/tmp/mathlib4 compare_reals.pdf
Usage: leanproject import-graph [OPTIONS] [OUTPUT]
Try "leanproject import-graph -h" for help.

Error: no such option: --show-unused
buzzard@buster:~/lean-projects/mathlib$

Kevin Buzzard (Nov 26 2022 at 17:25):

leanproject import-graph --to data.nat.basic --exclude-tactics --port-status datanatbasic.pdf

This works for me :-) But I get no colours.

Scott Morrison (Nov 26 2022 at 17:30):

I find you have to run it inside the src/ directory.

Scott Morrison (Nov 26 2022 at 17:30):

You may need to update mathlib-tools, possibly even by checking out master and running pip3 install . or equivalent.

Arien Malec (Nov 26 2022 at 17:32):

pip3 install git+https://github.com/leanprover-community/mathlib-tools I think.

port-progress bot (Nov 26 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 46/79 (58.2% of total)
Ported lines: 19522/35065 (55.7% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 26 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 58/128 (45.3% of total)
Ported lines: 22366/52776 (42.4% of total)
Longest unported chain: 11/25 (56.0% progress)

port-progress bot (Nov 26 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 54/125 (43.2% of total)
Ported lines: 21490/52350 (41.1% of total)
Longest unported chain: 11/25 (56.0% progress)

port-progress bot (Nov 26 2022 at 18:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 33/90 (36.7% of total)
Ported lines: 13571/32890 (41.3% of total)
Longest unported chain: 25/36 (30.6% progress)

port-progress bot (Nov 26 2022 at 18:18):

mathlib port progress data.fintype.basic
Ported files: 60/184 (32.6% of total)
Ported lines: 23070/85609 (26.9% of total)
Longest unported chain: 24/38 (36.8% progress)

port-progress bot (Nov 26 2022 at 18:22):

mathlib port progress topology.metric_space.basic
Ported files: 69/508 (13.6% of total)
Ported lines: 24510/225082 (10.9% of total)
Longest unported chain: 57/71 (19.7% progress)

Kevin Buzzard (Nov 26 2022 at 18:27):

leanproject import-graph --to data.set.basic --exclude-tactics --reduce --port-status --show-unused data_set_basic.pdf
is still giving me no colours :-(

Jireh Loreaux (Nov 26 2022 at 18:50):

Kevin, did you uninstall mathlibtools and then reinstall from source?

port-progress bot (Nov 26 2022 at 19:02):

mathlib port progress all
Ported files: 84/2779 (3.0% of total)
Ported lines: 26251/961117 (2.7% of total)
Longest unported chain: 108/122 (11.5% progress)

Kevin Buzzard (Nov 26 2022 at 20:06):

buzzard@buster:~/lean-projects/mathlib/src$ which mathlibtools
buzzard@buster:~/lean-projects/mathlib/src$ pip3 install git+https://github.com/leanprover-community/mathlib-tools
Collecting git+https://github.com/leanprover-community/mathlib-tools
  Cloning https://github.com/leanprover-community/mathlib-tools to /tmp/pip-req-build-73wrnf7t
  Running command git clone -q https://github.com/leanprover-community/mathlib-tools /tmp/pip-req-build-73wrnf7t
Requirement already satisfied: Click in /usr/lib/python3/dist-packages (from mathlibtools==1.3.0) (7.0)
Requirement already satisfied: PyGithub in /home/buzzard/.local/lib/python3.8/site-packages (from mathlibtools==1.3.0) (1.55)
Requirement already satisfied: PyYAML>=3.13 in /usr/lib/python3/dist-packages (from mathlibtools==1.3.0) (5.3.1)
Requirement already satisfied: atomicwrites in /home/buzzard/.local/lib/python3.8/site-packages (from mathlibtools==1.3.0) (1.4.1)
Requirement already satisfied: certifi in /usr/lib/python3/dist-packages (from mathlibtools==1.3.0) (2019.11.28)
Requirement already satisfied: gitpython>=2.1.11 in /home/buzzard/.local/lib/python3.8/site-packages (from mathlibtools==1.3.0) (3.1.27)
Requirement already satisfied: networkx in /home/buzzard/.local/lib/python3.8/site-packages (from mathlibtools==1.3.0) (2.8.5)
Requirement already satisfied: pydot in /home/buzzard/.local/lib/python3.8/site-packages (from mathlibtools==1.3.0) (1.4.2)
Requirement already satisfied: requests in /usr/lib/python3/dist-packages (from mathlibtools==1.3.0) (2.22.0)
Requirement already satisfied: toml>=0.10.0 in /home/buzzard/.local/lib/python3.8/site-packages (from mathlibtools==1.3.0) (0.10.2)
Requirement already satisfied: tqdm in /home/buzzard/.local/lib/python3.8/site-packages (from mathlibtools==1.3.0) (4.64.0)
Requirement already satisfied: pynacl>=1.4.0 in /home/buzzard/.local/lib/python3.8/site-packages (from PyGithub->mathlibtools==1.3.0) (1.5.0)
Requirement already satisfied: deprecated in /home/buzzard/.local/lib/python3.8/site-packages (from PyGithub->mathlibtools==1.3.0) (1.2.13)
Requirement already satisfied: pyjwt>=2.0 in /home/buzzard/.local/lib/python3.8/site-packages (from PyGithub->mathlibtools==1.3.0) (2.4.0)
Requirement already satisfied: gitdb<5,>=4.0.1 in /home/buzzard/.local/lib/python3.8/site-packages (from gitpython>=2.1.11->mathlibtools==1.3.0) (4.0.9)
Requirement already satisfied: pyparsing>=2.1.4 in /home/buzzard/.local/lib/python3.8/site-packages (from pydot->mathlibtools==1.3.0) (2.4.7)
Requirement already satisfied: cffi>=1.4.1 in /home/buzzard/.local/lib/python3.8/site-packages (from pynacl>=1.4.0->PyGithub->mathlibtools==1.3.0) (1.15.1)
Requirement already satisfied: wrapt<2,>=1.10 in /home/buzzard/.local/lib/python3.8/site-packages (from deprecated->PyGithub->mathlibtools==1.3.0) (1.14.1)
Requirement already satisfied: smmap<6,>=3.0.1 in /home/buzzard/.local/lib/python3.8/site-packages (from gitdb<5,>=4.0.1->gitpython>=2.1.11->mathlibtools==1.3.0) (5.0.0)
Requirement already satisfied: pycparser in /home/buzzard/.local/lib/python3.8/site-packages (from cffi>=1.4.1->pynacl>=1.4.0->PyGithub->mathlibtools==1.3.0) (2.21)
Building wheels for collected packages: mathlibtools
  Building wheel for mathlibtools (setup.py) ... done
  Created wheel for mathlibtools: filename=mathlibtools-1.3.0-py3-none-any.whl size=32333 sha256=03155bc7342ea6eed34dff78752f72e6b4e525bcfe323098d2ffe4f4ec390c07
  Stored in directory: /tmp/pip-ephem-wheel-cache-x770e9pg/wheels/f6/e0/22/e72429590e4b7ea5a0aa076e96f5d0673c84c830db7a5e86e2
Successfully built mathlibtools
Installing collected packages: mathlibtools
Successfully installed mathlibtools-1.3.0
buzzard@buster:~/lean-projects/mathlib/src$ leanproject import-graph --to data.set.basic --exclude-tactics --reduce --port-status --show-unused data_set_basic2.pdf
evince data_set_basic2.pdf
buzzard@buster:~/lean-projects/mathlib/src$ evince data_set_basic2.pdf

gives me no colours :anguish:

Scott Morrison (Nov 26 2022 at 22:00):

try scripts/mk_all.sh?

Yakov Pechersky (Nov 26 2022 at 23:04):

Kevin, if you run the command to save a dot file instead of a pdf, what does that file look like?

Mario Carneiro (Nov 26 2022 at 23:08):

I always end up with pixelated PDFs with the usual command

Yakov Pechersky (Nov 26 2022 at 23:55):

My hypothesis is that this Mario's and Kevin's issue is due to the graphviz library that's on their system, that is implicitly used by leanproject

port-progress bot (Nov 27 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 46/79 (58.2% of total)
Ported lines: 19522/35065 (55.7% of total)
Longest unported chain: 7/19 (63.2% progress)

port-progress bot (Nov 27 2022 at 18:07):

mathlib port progress data.rat.order
Ported files: 59/128 (46.1% of total)
Ported lines: 22461/52776 (42.6% of total)
Longest unported chain: 11/25 (56.0% progress)

port-progress bot (Nov 27 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 55/125 (44.0% of total)
Ported lines: 21585/52350 (41.2% of total)
Longest unported chain: 11/25 (56.0% progress)

port-progress bot (Nov 27 2022 at 18:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 33/90 (36.7% of total)
Ported lines: 13571/32890 (41.3% of total)
Longest unported chain: 25/36 (30.6% progress)

port-progress bot (Nov 27 2022 at 18:18):

mathlib port progress data.fintype.basic
Ported files: 61/184 (33.2% of total)
Ported lines: 23165/85609 (27.1% of total)
Longest unported chain: 24/38 (36.8% progress)

port-progress bot (Nov 27 2022 at 18:22):

mathlib port progress topology.metric_space.basic
Ported files: 70/508 (13.8% of total)
Ported lines: 24605/225082 (10.9% of total)
Longest unported chain: 57/71 (19.7% progress)

port-progress bot (Nov 27 2022 at 18:59):

mathlib port progress all
Ported files: 85/2779 (3.1% of total)
Ported lines: 26346/961126 (2.7% of total)
Longest unported chain: 108/122 (11.5% progress)

David Michael Roberts (Nov 27 2022 at 22:14):

What does the 108/122 mean under longest unported chain (in "all").

Jireh Loreaux (Nov 27 2022 at 22:18):

There are 108 files in the chain left to port (so we have ported 14 of them).

Jireh Loreaux (Nov 27 2022 at 22:18):

It's kind of backwards from the rest of the port progress information.

Scott Morrison (Nov 27 2022 at 22:26):

Technically it is not really a fraction. It means that the longest import chain in mathlib3 is 122 files long, and then once you remove all the ported files the longest chain is 108 files long. That chain need not be a subset of the original chain!

Jireh Loreaux (Nov 27 2022 at 22:38):

Hmmm. when I click the longest imported chain, some files have - next to them. Is that supposed to mean that no declaration from that file was used in a later file? If that's the case, then I think there's a bug; maybe it's not picking up on instances which are used? In particular, analysis.complex.polynomial includes the fact is_alg_closed ℂ which gets used in analysis.normed_space.spectrumin the declaration map_polynomial_aeval which uses map_polynomial_aeval_of_nonempty which has an argument of is_alg_closed.

Jireh Loreaux (Nov 27 2022 at 22:38):

If you remove that import then that declaration complains.

Jireh Loreaux (Nov 27 2022 at 22:40):

Or is the point that this declaration map_polynomial_aeval doesn't get used in gelfand_duality.lean and hence the import analysis.complex.polynomial wasn't necessary for declarations in that file?

Scott Morrison (Nov 27 2022 at 22:43):

Yes, it's only about what is used in the very last file in the chain.

Scott Morrison (Nov 27 2022 at 22:43):

So if you see

- A
  B
  C

then it may well be that B needs A. However C only uses parts of B that do not need A!

Jireh Loreaux (Nov 27 2022 at 22:44):

Right, and that's not always something we want to change.

Scott Morrison (Nov 27 2022 at 22:44):

There is a known bug, however, which is that this analysis does not follow the @[ancestor] tag, so when using old_structure_cmd it will miss dependencies on parent classes.

Scott Morrison (Nov 27 2022 at 22:44):

That's right: a - is not a certain sign that anything is wrong.

Scott Morrison (Nov 27 2022 at 22:44):

but a long chain of them is suspicious.

Scott Morrison (Nov 27 2022 at 23:13):

A few new porting targets available:

algebra.group_with_zero.semiconj
algebra.ring.commute
algebra.regular.basic

I've been trying to stay on top of #queue4, but I suspect there are a bunch of mislabelled PRs out there too. If anyone notices PRs that are ready for review but not marked as such, please remind the authors about labelling! :-)

Kevin Buzzard (Nov 27 2022 at 23:51):

Ooh I never knew about #queue4 ! So we're finally into algebra?

Scott Morrison (Nov 28 2022 at 02:00):

Just mentioning this here so more people see it, and take heart: on mathlib4#757, Jireh's PR description is "porting notes: another perfect shot by mathport!"

Scott Morrison (Nov 28 2022 at 02:22):

We're blazing along today.

algebra.group_with_zero.commute

is now available.

Heather Macbeth (Nov 28 2022 at 02:26):

I see mathlib4#728 order.min_max has been merged, but the wiki still shows

order.min_max: 'No mathlib4##728 71ca477041bcd6d7c745fe555dc49735c12944b7'

Is this intentional or should I update?

Scott Morrison (Nov 28 2022 at 02:34):

Update please!

Scott Morrison (Nov 28 2022 at 02:35):

Ideally the port_status.py script would tell us something about the status of PRs (e.g. merged, help-wanted, awaiting-review).

Heather Macbeth (Nov 28 2022 at 02:37):

Maybe ideally the wiki would record the hash and the PR number and the port_status.pyscript would work out everything else (no Yes or No to fall out of date)

port-progress bot (Nov 28 2022 at 02:42):

mathlib port progress algebra.order.field.defs
Ported files: 51/78 (65.4% of total)
Ported lines: 20957/35064 (59.8% of total)
Longest unported chain: 5/19 (73.7% progress)

port-progress bot (Nov 28 2022 at 02:45):

mathlib port progress data.rat.order
Ported files: 68/127 (53.5% of total)
Ported lines: 24374/52775 (46.2% of total)
Longest unported chain: 11/25 (56.0% progress)

port-progress bot (Nov 28 2022 at 02:49):

mathlib port progress data.nat.choose.basic
Ported files: 64/124 (51.6% of total)
Ported lines: 23498/52349 (44.9% of total)
Longest unported chain: 11/25 (56.0% progress)

port-progress bot (Nov 28 2022 at 02:52):

mathlib port progress category_theory.limits.yoneda
Ported files: 34/90 (37.8% of total)
Ported lines: 13815/32890 (42.0% of total)
Longest unported chain: 25/36 (30.6% progress)

port-progress bot (Nov 28 2022 at 02:56):

mathlib port progress data.fintype.basic
Ported files: 70/183 (38.3% of total)
Ported lines: 25078/85608 (29.3% of total)
Longest unported chain: 24/38 (36.8% progress)

port-progress bot (Nov 28 2022 at 03:00):

mathlib port progress topology.metric_space.basic
Ported files: 79/507 (15.6% of total)
Ported lines: 26518/225094 (11.8% of total)
Longest unported chain: 57/71 (19.7% progress)

port-progress bot (Nov 28 2022 at 03:37):

mathlib port progress all
Ported files: 94/2779 (3.4% of total)
Ported lines: 28259/961139 (2.9% of total)
Longest unported chain: 108/122 (11.5% progress)

Jireh Loreaux (Nov 28 2022 at 03:41):

Scott Morrison said:

We're blazing along today.

algebra.group_with_zero.commute

is now available.

PRed with a green tick as mathlib4#762, it should be easy to review, there were virtually no issues.

Eric Wieser (Nov 28 2022 at 12:51):

Note that the "ported to mathlib4" comment bot will be inactive until #17737 is merged

port-progress bot (Nov 28 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 54/80 (67.5% of total)
Ported lines: 22085/35053 (63.0% of total)
Longest unported chain: 5/19 (73.7% progress)

port-progress bot (Nov 28 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 71/130 (54.6% of total)
Ported lines: 25519/52867 (48.3% of total)
Longest unported chain: 11/26 (57.7% progress)

port-progress bot (Nov 28 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 67/127 (52.8% of total)
Ported lines: 24643/52441 (47.0% of total)
Longest unported chain: 11/26 (57.7% progress)

port-progress bot (Nov 28 2022 at 18:15):

mathlib port progress category_theory.limits.yoneda
Ported files: 35/90 (38.9% of total)
Ported lines: 14428/31569 (45.7% of total)
Longest unported chain: 25/36 (30.6% progress)

port-progress bot (Nov 28 2022 at 18:18):

mathlib port progress data.fintype.basic
Ported files: 75/186 (40.3% of total)
Ported lines: 26333/85700 (30.7% of total)
Longest unported chain: 24/39 (38.5% progress)

port-progress bot (Nov 28 2022 at 18:22):

mathlib port progress topology.metric_space.basic
Ported files: 84/510 (16.5% of total)
Ported lines: 27773/225208 (12.3% of total)
Longest unported chain: 57/72 (20.8% progress)

port-progress bot (Nov 28 2022 at 18:59):

mathlib port progress all
Ported files: 100/2782 (3.6% of total)
Ported lines: 29612/961374 (3.1% of total)
Longest unported chain: 108/123 (12.2% progress)

Scott Morrison (Nov 28 2022 at 21:52):

Exciting, there are quite a few files ready to port:

order.heyting.basic
algebra.order.monoid.cancel.defs
algebra.order.monoid.canonical.defs
data.prod.lex
data.sigma.order
data.psigma.order

Scott Morrison (Nov 28 2022 at 21:54):

If it goes well, order.heyting.basic, order.boolean_algebra, order.symm_diff and data.set.basic form a chain than potentially can be ported in one go.

port-progress bot (Nov 28 2022 at 23:03):

mathlib port progress algebra.order.field.defs
Ported files: 57/80 (71.2% of total)
Ported lines: 22708/35053 (64.8% of total)
Longest unported chain: 5/19 (73.7% progress)

port-progress bot (Nov 28 2022 at 23:07):

mathlib port progress data.rat.order
Ported files: 75/130 (57.7% of total)
Ported lines: 26210/52867 (49.6% of total)
Longest unported chain: 11/26 (57.7% progress)

Heather Macbeth (Nov 28 2022 at 23:07):

Is there an off-by-one error in the port progress bot? The longest unported chain for algebra.order.field.defs shows as containing six files.

Scott Morrison (Nov 28 2022 at 23:19):

I think it's measuring the length of the path in edges, rather than vertices.

Scott Morrison (Nov 28 2022 at 23:19):

I can easily add one to both numbers. :-)

Heather Macbeth (Nov 28 2022 at 23:22):

The real progress is having a chain short enough to count.

port-progress bot (Nov 29 2022 at 18:03):

mathlib port progress algebra.order.field.defs
Ported files: 57/80 (71.2% of total)
Ported lines: 22708/34896 (65.1% of total)
Longest unported chain: 5/19 (73.7% progress)

port-progress bot (Nov 29 2022 at 18:07):

mathlib port progress data.rat.order
Ported files: 75/130 (57.7% of total)
Ported lines: 26210/52644 (49.8% of total)
Longest unported chain: 11/26 (57.7% progress)

Eric Wieser (Nov 30 2022 at 10:53):

Could someone take a quick look at #17756 (warning: python code)? The bot that adds synchronized labels still has some teething issues, but I'm hoping this will be the last one for a while

Eric Rodriguez (Nov 30 2022 at 12:02):

seems fine; I do worry about this approach of adding comments, though, as it means that we have to do extra verification every time these comments are added

Eric Wieser (Nov 30 2022 at 13:41):

I feel the same way, but we've already started down that path...

Eric Wieser (Nov 30 2022 at 13:41):

At any rate, it's easy to build a tool that removes the comment again before asking git if anything has changed

port-progress bot (Nov 30 2022 at 18:03):

mathlib port progress algebra.order.field.defs
Ported files: 58/80 (72.5% of total)
Ported lines: 23644/34953 (67.6% of total)
Longest unported chain: 5/19 (73.7% progress)

port-progress bot (Nov 30 2022 at 18:07):

mathlib port progress data.rat.order
Ported files: 79/130 (60.8% of total)
Ported lines: 27636/52657 (52.5% of total)
Longest unported chain: 11/26 (57.7% progress)

port-progress bot (Nov 30 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 74/127 (58.3% of total)
Ported lines: 26445/52251 (50.6% of total)
Longest unported chain: 11/26 (57.7% progress)

port-progress bot (Nov 30 2022 at 18:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 35/90 (38.9% of total)
Ported lines: 14428/31569 (45.7% of total)
Longest unported chain: 25/36 (30.6% progress)

port-progress bot (Nov 30 2022 at 18:18):

mathlib port progress data.fintype.basic
Ported files: 83/186 (44.6% of total)
Ported lines: 28307/85581 (33.1% of total)
Longest unported chain: 24/39 (38.5% progress)

port-progress bot (Nov 30 2022 at 18:22):

mathlib port progress topology.metric_space.basic
Ported files: 97/511 (19.0% of total)
Ported lines: 30464/225026 (13.5% of total)
Longest unported chain: 57/72 (20.8% progress)

port-progress bot (Nov 30 2022 at 18:26):

mathlib port progress all
Ported files: 112/2786 (4.0% of total)
Ported lines: 32205/962434 (3.3% of total)
Longest unported chain: 108/123 (12.2% progress)

Scott Morrison (Nov 30 2022 at 18:30):

@Yakov Pechersky, the code that is meant to outline nodes in red if there is an existing ad-hoc port in mathlib4 seems to have gone out of control, and is highlighting lots of already ported nodes. Could you look into this? Not super high priority.

Scott Morrison (Nov 30 2022 at 18:35):

If anyone is looking for something easy to do to contribute to the port, I left a bunch of review comments on https://github.com/leanprover-community/mathlib4/pull/772.

Scott Morrison (Nov 30 2022 at 18:35):

Getting that merged would open up several files.

Yakov Pechersky (Nov 30 2022 at 19:37):

https://github.com/leanprover-community/mathlib-tools/blob/master/mathlibtools/lib.py#L1077
That should be

if node["status"].ported:
  continue
if node_name in existing_files:
  node["color"] = "red"

Scott Morrison (Nov 30 2022 at 20:07):

Could you PR that?

Ruben Van de Velde (Nov 30 2022 at 20:18):

@Scott Morrison I think mathlib4#772 is ready to merge, if you want

Scott Morrison (Nov 30 2022 at 20:21):

If anyone would like to adopt https://github.com/leanprover-community/mathlib4/pull/804, which ports Order.Hom.Basic, that would be great.

Scott Morrison (Nov 30 2022 at 20:21):

That one seems to have some weird typeclass issues, however. (Note sure if they are related to those on the "instance loop?" thread here.)

Scott Morrison (Nov 30 2022 at 20:22):

Another easy PR to take over is https://github.com/leanprover-community/mathlib4/pull/793, which ports Order.Heyting, and I think only needs linting but is otherwise pretty good.

Scott Morrison (Nov 30 2022 at 20:23):

Oh, no, it has other problems too. :-) There are a few failing proofs.

Scott Morrison (Nov 30 2022 at 20:23):

And we need to comment out the pi_instance and refine_struct proofs and do them by hand.

Scott Morrison (Nov 30 2022 at 20:23):

These tactics are coming soon, so we should keep the proofs in as comments, but to make sure we get through these files quickly I think it's best if we just work around the absence of these tactics for now.

Yakov Pechersky (Nov 30 2022 at 20:30):

mathlib-tools#154

Ruben Van de Velde (Nov 30 2022 at 20:42):

Scott Morrison said:

If anyone would like to adopt https://github.com/leanprover-community/mathlib4/pull/804, which ports Order.Hom.Basic, that would be great.

Uh, is that supposed to error with PANIC at Lean.Meta.whnfEasyCases Lean.Meta.WHNF:305:22: unreachable code has been reached?

Scott Morrison (Nov 30 2022 at 20:43):

If you feel like producing a #mwe that demonstrates that PANIC, it will definitely be a Lean 4 bug. :-)

Scott Morrison (Nov 30 2022 at 20:44):

(Often these PANICs in half ported files disappear mysteriously once you fix a few errors earlier in the file, but nevertheless they are bugs, and deserve to be squashed. Producing the #mwe can be a bit trial-and-error when starting with a big file full of other errors, however!)

Ruben Van de Velde (Nov 30 2022 at 21:02):

I started poking at mathlib4#804, but most of the errors gave me a headache, so I just fixed the simplest ones

Scott Morrison (Nov 30 2022 at 22:05):

Currently reading for porting are:

data.int.units
data.nat.bits
algebra.order.sub.canonical
order.rel_iso.group
data.psigma.order

There are also two PRs that could use attention:

combinatorics.quiver.basic    -- mathlib4#749 needs review; this has the start of category theory as well
order.heyting.basic    -- mathlib4#793 needs documentation

Yaël Dillies (Nov 30 2022 at 22:29):

Wait, did someone port data.sigma.order without porting data.psigma.order simultaneously?

Yaël Dillies (Nov 30 2022 at 22:30):

@Jireh Loreaux, I think you just got one file ported, one free :grinning_face_with_smiling_eyes:

Eric Rodriguez (Dec 01 2022 at 00:15):

I'd really appreciate some docstrings on mathlib4#665 - it should be easy for someone who knows streams!

Arien Malec (Dec 01 2022 at 02:30):

Looking at data.nat.bits, it depends on nat.bit that used to be defined in core in init.data.nat.bitwise but Lean 4 doesn't have a Nat.bit equivalent.

Sky Wilshaw (Dec 01 2022 at 10:43):

It looks like algebra.order.sub.canonical is incorrectly marked as ready, it requires algebra.order.monoid.canonical.defs which I don't think has been ported.

Ruben Van de Velde (Dec 01 2022 at 10:53):

It's ported in https://github.com/leanprover-community/mathlib4/pull/778, which failed to merge a few hours ago

Ruben Van de Velde (Dec 01 2022 at 10:59):

Ah, Scott fixed the issue but then didn't kick it on the queue again. Anyone around who can?

Riccardo Brasca (Dec 01 2022 at 11:00):

I kicked on the queue.

Sky Wilshaw (Dec 01 2022 at 11:06):

Thank you, I think I'll try to port algebra.order.sub.canonical once mathlib4#778 is merged.

Riccardo Brasca (Dec 01 2022 at 11:09):

It's merged.

Scott Morrison (Dec 01 2022 at 14:35):

It's also completely fine to branch off an existing PR, and start work before that PR has been merged.

Scott Morrison (Dec 01 2022 at 14:35):

In fact, we're still seeing lots of bottle-necking (because of our typeclass issues in algebra.hom.group), so getting ahead of the curve by porting stuff based on open PRs could be really helpful.

port-progress bot (Dec 01 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 61/80 (76.2% of total)
Ported lines: 24781/35033 (70.7% of total)
Longest unported chain: 5/19 (73.7% progress)

port-progress bot (Dec 01 2022 at 18:07):

mathlib port progress data.rat.order
Ported files: 83/130 (63.8% of total)
Ported lines: 29565/52701 (56.1% of total)
Longest unported chain: 11/26 (57.7% progress)

port-progress bot (Dec 01 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 77/127 (60.6% of total)
Ported lines: 28148/52164 (54.0% of total)
Longest unported chain: 11/26 (57.7% progress)

port-progress bot (Dec 01 2022 at 18:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 35/90 (38.9% of total)
Ported lines: 14444/31585 (45.7% of total)
Longest unported chain: 25/36 (30.6% progress)

Eric Wieser (Dec 01 2022 at 18:15):

Eric Wieser said:

Could someone take a quick look at #17756 (warning: python code)? The bot that adds synchronized labels still has some teething issues, but I'm hoping this will be the last one for a while

:ping_pong:; I've already merged the PR generated by this PR!

port-progress bot (Dec 01 2022 at 18:17):

mathlib port progress data.fintype.basic
Ported files: 86/186 (46.2% of total)
Ported lines: 30022/85506 (35.1% of total)
Longest unported chain: 24/39 (38.5% progress)

port-progress bot (Dec 01 2022 at 18:21):

mathlib port progress topology.metric_space.basic
Ported files: 103/513 (20.1% of total)
Ported lines: 32567/225297 (14.5% of total)
Longest unported chain: 57/72 (20.8% progress)

port-progress bot (Dec 01 2022 at 18:25):

mathlib port progress all
Ported files: 119/2791 (4.3% of total)
Ported lines: 34397/963743 (3.6% of total)
Longest unported chain: 108/123 (12.2% progress)

Jireh Loreaux (Dec 01 2022 at 19:29):

Eric Wieser said:

Eric Wieser said:

Could someone take a quick look at #17756 (warning: python code)? The bot that adds synchronized labels still has some teething issues, but I'm hoping this will be the last one for a while

:ping_pong:; I've already merged the PR generated by this PR!

I placed this on the maintainer queue. It seemed fine to me, and even if there is some problem, we'll find out about it when reviewing the PRs it generates.

Riccardo Brasca (Dec 02 2022 at 11:50):

I don't see data.nat.even_odd_rec in the port-status.. what happened to it?

Riccardo Brasca (Dec 02 2022 at 12:29):

It has probably been removed in #17759 or because of that

Eric Rodriguez (Dec 02 2022 at 13:56):

I think the yaml would have to get copy pasted in

Scott Morrison (Dec 02 2022 at 15:12):

Actually, this is broken at the moment! scripts/port_status.py produces port_status.yaml locally, which you used to be able to copy and paste into #port-wiki.

Scott Morrison (Dec 02 2022 at 15:13):

However it now produces yaml in a different format, and which moreover is broken:

topology.algebra.order.filter: !!python/object:mathlibtools.file_status.FileStatus
  comments: ''
  mathlib3_hash: null
  mathlib4_pr: null
  ported: false

Scott Morrison (Dec 02 2022 at 15:13):

We should sort this out sooner rather than later, as mathlib3 refactoring efforts are generating new files.

Scott Morrison (Dec 02 2022 at 15:14):

(Some of which we will want to port in the next week or so.)

Jakob von Raumer (Dec 02 2022 at 15:15):

I noticed that port_status.py is not picking up some dependencies. For example, data.string.basic indirectly depends on data.string.defs but it's still marked as ready to port.

Scott Morrison (Dec 02 2022 at 15:16):

This is (probably) a known problem where the import is transitive via a tactic file.

Scott Morrison (Dec 02 2022 at 15:17):

Solutions:

  1. add the import explicitly in mathlib3
  2. hope this problem becomes irrelevant soon, once we're done with the files that are imported by tactics files.

Jakob von Raumer (Dec 02 2022 at 15:23):

In this case, the only missing requirement for data.string.defs is already PRed so it's going go pop up soon anyway.

Jireh Loreaux (Dec 02 2022 at 15:25):

@Scott Morrison what needs to happen to fix the new and broken yaml?

Scott Morrison (Dec 02 2022 at 15:27):

I'm not sure. At some point we still want (I think?) to switch to the "new" yaml format. But I've lost track of what is required to do that. @Yakov Pechersky?

There are two things that need doing:

  1. make sure the port_status.yaml that is output locally is correct for the new format.
  2. make sure all the tools that read #port-wiki can cope with the new format.

Yakov Pechersky (Dec 02 2022 at 15:28):

I have an example wiki page of how it'd be: https://github.com/leanprover-community/mathlib/wiki/mathlib4-port-status-new

Yakov Pechersky (Dec 02 2022 at 15:28):

And there is code to make the page look like that. The code exists for reading that new format.

Scott Morrison (Dec 02 2022 at 15:28):

Okay, so do we just have to press merge somewhere?

Scott Morrison (Dec 02 2022 at 15:29):

Presumably something in our fragile tooling will break, so it would be good to hit merge on a day when there is availability from you and/or Eric to patch up scripts. :-)

Yakov Pechersky (Dec 02 2022 at 15:29):

There's a little bit of a staging problem -- making sure that the defaults are updated in several places at the same time. So it is communication with @Eric Wieser on updating the mathlib scripts

Yakov Pechersky (Dec 02 2022 at 15:29):

Right!

Eric Wieser (Dec 02 2022 at 15:54):

Or we move everything into mathlib / into mathlibtools, so that the staging problem disappears

Eric Wieser (Dec 02 2022 at 15:55):

(where the latter option pushes the staging problem onto the users who has to remember to update mathlibtools)

port-progress bot (Dec 02 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 61/80 (76.2% of total)
Ported lines: 24781/35033 (70.7% of total)
Longest unported chain: 5/19 (73.7% progress)

port-progress bot (Dec 02 2022 at 18:07):

mathlib port progress data.rat.order
Ported files: 86/130 (66.2% of total)
Ported lines: 31458/52701 (59.7% of total)
Longest unported chain: 11/26 (57.7% progress)

port-progress bot (Dec 02 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 80/127 (63.0% of total)
Ported lines: 30041/52164 (57.6% of total)
Longest unported chain: 11/26 (57.7% progress)

port-progress bot (Dec 02 2022 at 18:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 42/90 (46.7% of total)
Ported lines: 15814/31585 (50.1% of total)
Longest unported chain: 20/36 (44.4% progress)

port-progress bot (Dec 02 2022 at 18:17):

mathlib port progress data.fintype.basic
Ported files: 89/186 (47.8% of total)
Ported lines: 31915/85511 (37.3% of total)
Longest unported chain: 24/39 (38.5% progress)

port-progress bot (Dec 02 2022 at 18:21):

mathlib port progress topology.metric_space.basic
Ported files: 106/517 (20.5% of total)
Ported lines: 34460/225572 (15.3% of total)
Longest unported chain: 57/72 (20.8% progress)

port-progress bot (Dec 02 2022 at 18:25):

mathlib port progress all
Ported files: 136/2795 (4.9% of total)
Ported lines: 38223/964090 (4.0% of total)
Longest unported chain: 111/126 (11.9% progress)

port-progress bot (Dec 02 2022 at 21:52):

mathlib port progress algebra.order.field.defs
Ported files: 58/73 (79.5% of total)
Ported lines: 23999/31812 (75.4% of total)
Longest unported chain: 4/19 (78.9% progress)

port-progress bot (Dec 02 2022 at 21:56):

mathlib port progress data.rat.order
Ported files: 86/131 (65.6% of total)
Ported lines: 31458/52633 (59.8% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 02 2022 at 22:00):

mathlib port progress data.nat.choose.basic
Ported files: 80/128 (62.5% of total)
Ported lines: 30041/52093 (57.7% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 02 2022 at 22:04):

mathlib port progress data.real.basic
Ported files: 100/307 (32.6% of total)
Ported lines: 33921/120374 (28.2% of total)
Longest unported chain: 31/48 (35.4% progress)

port-progress bot (Dec 02 2022 at 22:07):

mathlib port progress category_theory.limits.yoneda
Ported files: 42/90 (46.7% of total)
Ported lines: 15814/31585 (50.1% of total)
Longest unported chain: 20/36 (44.4% progress)

port-progress bot (Dec 02 2022 at 22:11):

mathlib port progress data.fintype.basic
Ported files: 89/187 (47.6% of total)
Ported lines: 31915/85440 (37.4% of total)
Longest unported chain: 22/39 (43.6% progress)

Scott Morrison (Dec 02 2022 at 23:38):

Hot off the press ready for porting:

order.symm_diff
algebra.group.with_one.defs
combinatorics.quiver.connected_component
order.heyting.boundary

The first two are pretty important, the second two not so important (but great if you want something low pressure to practice on :-)

Scott Morrison (Dec 02 2022 at 23:40):

I think the most pressing task at the moment is someone having a good look at https://github.com/leanprover-community/mathlib4/pull/804, porting Order.Hom.Basic. It is very much not working at the moment, and typeclass inferences involving FunLike are failing. I haven't had a chance to look much, so I don't know if this is just instances set up badly, or deeper problems that will involve extracting a #mwe to send to the Lean 4 devs.

Scott Morrison (Dec 02 2022 at 23:41):

I'm pretty close to offline for the next 48 hours, and likely won't have a chance to look at this.

Kevin Buzzard (Dec 02 2022 at 23:46):

Having already started on the now-not-existing algebra.group.with_one I'd like to claim algebra.group.with_one.defs :-)

Moritz Doll (Dec 02 2022 at 23:59):

hopefully the porting opens up a bit more once we have a good chunk of the basic algebra done.

Scott Morrison (Dec 03 2022 at 00:04):

And here it comes: freshly available for porting:

algebra.divisibility.basic
algebra.ring.basic
algebra.hom.commute

Scott Morrison (Dec 03 2022 at 00:07):

Also just checking in on

algebra.group.type_tags    -- WIP by @Vtec234 6eb334bd8f3433d5b08ba156b8ec3e6af47e1904
algebra.hom.equiv.basic    -- WIP @winstonyin 76171581280d5b5d1e2d1f4f37e5420357bdc636

@Wojciech Nawrocki and @Winston Yin, if you want to put up PRs for these, even if they are nothing more than the output of mathport and marked as WIP, it's probably easier for us to track and/or help out with problems.

Moritz Doll (Dec 03 2022 at 01:24):

Scott Morrison said:

And here it comes: freshly available for porting:

algebra.divisibility.basic
algebra.ring.basic
algebra.hom.commute

algebra.ring.basic was very easy - I have no idea what to do with the ad-hoc version. If someone wants to take a look: mathlib4#830

Winston Yin (Dec 03 2022 at 01:41):

I’ll PR algebra.hom.equiv.basic in a few hours. There was a broken type class issue there a couple days ago that was traced back to algebra.hom.group. Hopefully it’s fixed by recent Lean4 patches.

Scott Morrison (Dec 03 2022 at 02:17):

@Moritz Doll, if everything compiles and tests correctly without the ad hoc file, you can just drop it.

Scott Morrison (Dec 03 2022 at 02:17):

It's possible that some of it is needed for tactic files, however.

Jireh Loreaux (Dec 03 2022 at 03:47):

Moritz, if there is stuff in the ad hoc version which is necessary, I would just put them in a temporary file which will later be removed once we port that material.

Scott Morrison (Dec 03 2022 at 03:48):

@Jireh Loreaux, there's a separate thread about this, title "Algebra.Ring.Basic". Since there are now duplicated instances, we probably better fix it sooner rather than later.

Jireh Loreaux (Dec 03 2022 at 03:49):

Yeah sorry, I was just reading it.

Matej Penciak (Dec 03 2022 at 04:06):

Scott Morrison said:

And here it comes: freshly available for porting:

algebra.divisibility.basic
algebra.ring.basic
algebra.hom.commute

I just finished up a port of algebra.divisibility.basic, there were very few fixes it needed so it went very quick.

Can I get non-master pushing rights to mathlib4? My github username is mpenciak

Wojciech Nawrocki (Dec 03 2022 at 04:18):

Scott Morrison said:

Also just checking in on

algebra.group.type_tags    -- WIP by @Vtec234 6eb334bd8f3433d5b08ba156b8ec3e6af47e1904
algebra.hom.equiv.basic    -- WIP @winstonyin 76171581280d5b5d1e2d1f4f37e5420357bdc636

Wojciech Nawrocki and Winston Yin, if you want to put up PRs for these, even if they are nothing more than the output of mathport and marked as WIP, it's probably easier for us to track and/or help out with problems.

Done! I initially parked it on the wiki before beginning to fixup the port. Would you rather people always make a PR as soon as possible with just the mathport outputs and do the fixups afterwards?

Arien Malec (Dec 03 2022 at 05:53):

I can report that combinatorics.quiver.connected_component is ugly

Arien Malec (Dec 03 2022 at 05:54):

I have an initial cleanup but suspect the typing and other issues here are going to be beyond my capabilities.

Arien Malec (Dec 03 2022 at 05:57):

happy to push the PR as is (I've cleaned up naming and fixed some of the obvious issues) but I'll have to pass on to someone to address the ugly.

Kevin Buzzard (Dec 03 2022 at 07:46):

@Wojciech Nawrocki I've been making PRs immediately when I start to port, and marking them WIP. This has several advantages as far as I can see. Firstly you can do the boring job of noting the mathlib3 commit immediately, and not a few days later when you've forgotten which commit it was. Secondly it's a powerful way of making it known that you're working on the file, it's easier to spot because there are far fewer mathlib4 PRs than there are lines of code in the horrible port status wiki file. Thirdly while you're at it you can make the mathlib3 PR freezing the file and cross reference the PR and now you've done pretty much all the admin work necessary. I copy the autopprted file over, fix the imports, add set_option autoImplicit false -- **TODO** remove this and just push and PR and then get going and keep pushing as I go.

Scott Morrison (Dec 03 2022 at 12:47):

@Kevin Buzzard, there's no need to make PRs to mathlib freezing files anymore. This is taken care of by a bot.

Eric Wieser (Dec 03 2022 at 13:01):

Unfortunately the bot is still slightly broken... Fix is at #17797, hopefully the last one for a while. Every time I make an assumption about the format of our docstrings, I end up being wrong!

Kevin Buzzard (Dec 03 2022 at 13:01):

Oh so that's now the default way to do this? I thought the bot was just angrily picking up the pieces when the humans didn't do what they were told.

Eric Wieser (Dec 03 2022 at 13:01):

The bot is better because it doesn't even run a CI job (why bother checking comments compile?)

Kevin Buzzard (Dec 03 2022 at 13:03):

Well one synch comment PR I made didn't compile ;-) (#17082)

Eric Wieser (Dec 03 2022 at 13:05):

Bors will still run CI on it before the merge actually goes through.

Eric Wieser (Dec 03 2022 at 13:06):

The bot is already mentioned at https://github.com/leanprover-community/mathlib4/wiki/Porting-wiki, but I've removed the comment that asks you to replace the SHA with the one after the comment was added now that port_status knows to ignore it

port-progress bot (Dec 03 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 58/73 (79.5% of total)
Ported lines: 23999/31812 (75.4% of total)
Longest unported chain: 4/19 (78.9% progress)

port-progress bot (Dec 03 2022 at 18:07):

mathlib port progress data.rat.order
Ported files: 89/131 (67.9% of total)
Ported lines: 33160/52648 (63.0% of total)
Longest unported chain: 9/26 (65.4% progress)

Heather Macbeth (Dec 03 2022 at 18:08):

The true "longest unported chain" for algebra.order.field.defs,

algebra.group_with_one.defs
algebra.order.monoid_with_zero.defs
algebra.order.ring.defs
algebra.order.field.defs

is now shorter than some unported chain involving base material which is not actually needed:

- data.rbtree.init
- data.rbmap.basic
  data.list.defs
  data.string.defs
  tactic.core

Is it possible to modify the "longest unported chain" script so that it requires that the chain actually end at the target file?

port-progress bot (Dec 03 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 83/128 (64.8% of total)
Ported lines: 31743/52108 (60.9% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 03 2022 at 18:14):

mathlib port progress data.real.basic
Ported files: 96/232 (41.4% of total)
Ported lines: 34432/92135 (37.4% of total)
Longest unported chain: 15/33 (54.5% progress)

port-progress bot (Dec 03 2022 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 45/90 (50.0% of total)
Ported lines: 16286/31612 (51.5% of total)
Longest unported chain: 19/36 (47.2% progress)

Scott Morrison (Dec 03 2022 at 18:21):

https://github.com/leanprover-community/mathlib-tools/pull/155

port-progress bot (Dec 03 2022 at 18:21):

mathlib port progress data.fintype.basic
Ported files: 92/187 (49.2% of total)
Ported lines: 33617/85495 (39.3% of total)
Longest unported chain: 22/39 (43.6% progress)

port-progress bot (Dec 03 2022 at 18:25):

mathlib port progress topology.metric_space.basic
Ported files: 110/520 (21.2% of total)
Ported lines: 36190/225594 (16.0% of total)
Longest unported chain: 55/72 (23.6% progress)

port-progress bot (Dec 03 2022 at 18:29):

mathlib port progress all
Ported files: 143/2803 (5.1% of total)
Ported lines: 40449/964761 (4.2% of total)
Longest unported chain: 109/126 (13.5% progress)

Heather Macbeth (Dec 03 2022 at 18:44):

The port-progress pdfs for some porting targets (eg topology.metric_space.basic) aren't being generated, and when I run the command locally I get the error

Node names and attributes should not contain ":" unless they are quoted with "".
For example the string 'attribute:data1' should be written as '"attribute:data1"'.
Please refer https://github.com/pydot/pydot/issues/258

Is this due to incorrectly-formatted lines in the porting status wiki? If so, any idea what it would be?

Eric Wieser (Dec 03 2022 at 18:51):

Sounds like it's an escaping bug in our graph output generation

Frédéric Dupuis (Dec 03 2022 at 19:43):

I'm currently working on porting order.symm_diff, and I'm running into something that should probably be fixed in mathport: the syntax for calc blocks seems to be systematically broken. This shows up, for example, in the proof of docs#symm_diff_symm_diff_left. I can fix it by putting braces around the rw statement, but I don't actually know what style we are going for here.

The PR is mathlib4#842.

Scott Morrison (Dec 04 2022 at 01:19):

I conjecture it is
algebra.order.absolute_value: 'No: incorrectly marked as ready: needs algebra.hom.group'

Scott Morrison (Dec 04 2022 at 01:19):

and it is the colon after 'ready' that is somehow ending up in an attribute

Scott Morrison (Dec 04 2022 at 01:20):

There are also a Yes : and a No : that could be the problem.

Scott Morrison (Dec 04 2022 at 01:20):

I will just clean up all of them and hope for the best.

Kevin Buzzard (Dec 04 2022 at 01:21):

I think we have algebra.hom.group now anyway :-)

Scott Morrison (Dec 04 2022 at 01:28):

Okay, I deleted that comment.

Dan Velleman (Dec 04 2022 at 01:59):

@Frédéric Dupuis : I assume the problem you are running into is the one discussed in this issue:
#1844
The comments at the end seem to indicate that no final decision has been made about how calc proofs should be formatted.

Frédéric Dupuis (Dec 04 2022 at 02:20):

@Dan Velleman Thanks! In that case I'll just go ahead and do something that works to avoid holding up the port over this.

port-progress bot (Dec 04 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 58/73 (79.5% of total)
Ported lines: 24042/31867 (75.4% of total)
Longest unported chain: 4/19 (78.9% progress)

port-progress bot (Dec 04 2022 at 18:07):

mathlib port progress data.rat.order
Ported files: 89/131 (67.9% of total)
Ported lines: 33203/52716 (63.0% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 04 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 83/128 (64.8% of total)
Ported lines: 31786/52176 (60.9% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 04 2022 at 18:14):

mathlib port progress data.real.basic
Ported files: 96/229 (41.9% of total)
Ported lines: 34475/91237 (37.8% of total)
Longest unported chain: 15/33 (54.5% progress)

port-progress bot (Dec 04 2022 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 45/90 (50.0% of total)
Ported lines: 16329/31655 (51.6% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 04 2022 at 18:21):

mathlib port progress data.fintype.basic
Ported files: 92/187 (49.2% of total)
Ported lines: 33660/85563 (39.3% of total)
Longest unported chain: 22/39 (43.6% progress)

port-progress bot (Dec 04 2022 at 18:25):

mathlib port progress topology.metric_space.basic
Ported files: 110/519 (21.2% of total)
Ported lines: 36233/225647 (16.1% of total)
Longest unported chain: 55/72 (23.6% progress)

port-progress bot (Dec 04 2022 at 19:02):

mathlib port progress all
Ported files: 143/2804 (5.1% of total)
Ported lines: 40492/965201 (4.2% of total)
Longest unported chain: 109/126 (13.5% progress)

port-progress bot (Dec 05 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 59/73 (80.8% of total)
Ported lines: 24393/31900 (76.5% of total)
Longest unported chain: 4/19 (78.9% progress)

port-progress bot (Dec 05 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 90/131 (68.7% of total)
Ported lines: 33610/52810 (63.6% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 05 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 84/128 (65.6% of total)
Ported lines: 32189/52267 (61.6% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 05 2022 at 18:14):

mathlib port progress data.real.basic
Ported files: 97/229 (42.4% of total)
Ported lines: 34882/91340 (38.2% of total)
Longest unported chain: 15/33 (54.5% progress)

port-progress bot (Dec 05 2022 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 45/90 (50.0% of total)
Ported lines: 16329/31655 (51.6% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 05 2022 at 18:21):

mathlib port progress data.fintype.basic
Ported files: 93/187 (49.7% of total)
Ported lines: 34063/85684 (39.8% of total)
Longest unported chain: 22/39 (43.6% progress)

port-progress bot (Dec 05 2022 at 18:25):

mathlib port progress topology.metric_space.basic
Ported files: 111/519 (21.4% of total)
Ported lines: 36640/225864 (16.2% of total)
Longest unported chain: 55/72 (23.6% progress)

port-progress bot (Dec 05 2022 at 19:02):

mathlib port progress all
Ported files: 144/2804 (5.1% of total)
Ported lines: 40899/965905 (4.2% of total)
Longest unported chain: 109/126 (13.5% progress)

Scott Morrison (Dec 06 2022 at 04:00):

(deleted)

Siddhartha Gadgil (Dec 06 2022 at 06:56):

Would it be possible to track also data.nat.prime?

Ruben Van de Velde (Dec 06 2022 at 09:01):

Scott Morrison said:

The current list of immediate porting candidates is:

High priority:

  • group_theory.group_action.defs -- just some naming issues to clean up in mathlib4#854

Ready for review again

port-progress bot (Dec 06 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 63/75 (84.0% of total)
Ported lines: 27450/31938 (85.9% of total)
Longest unported chain: 3/19 (84.2% progress)

port-progress bot (Dec 06 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 101/133 (75.9% of total)
Ported lines: 39022/52864 (73.8% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 06 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 96/130 (73.8% of total)
Ported lines: 37667/52321 (72.0% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 06 2022 at 18:15):

mathlib port progress data.nat.prime
Ported files: 115/286 (40.2% of total)
Ported lines: 40746/111562 (36.5% of total)
Longest unported chain: 32/49 (34.7% progress)

port-progress bot (Dec 06 2022 at 18:18):

mathlib port progress data.real.basic
Ported files: 110/231 (47.6% of total)
Ported lines: 40395/91394 (44.2% of total)
Longest unported chain: 15/33 (54.5% progress)

port-progress bot (Dec 06 2022 at 18:22):

mathlib port progress category_theory.limits.yoneda
Ported files: 46/90 (51.1% of total)
Ported lines: 17419/31687 (55.0% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 06 2022 at 18:25):

mathlib port progress data.fintype.basic
Ported files: 105/189 (55.6% of total)
Ported lines: 39541/85738 (46.1% of total)
Longest unported chain: 22/39 (43.6% progress)

port-progress bot (Dec 06 2022 at 18:29):

mathlib port progress topology.metric_space.basic
Ported files: 124/521 (23.8% of total)
Ported lines: 42157/225922 (18.7% of total)
Longest unported chain: 55/72 (23.6% progress)

port-progress bot (Dec 06 2022 at 19:16):

mathlib port progress all
Ported files: 159/2809 (5.7% of total)
Ported lines: 46618/966941 (4.8% of total)
Longest unported chain: 113/130 (13.1% progress)

Scott Morrison (Dec 06 2022 at 20:44):

@Siddhartha Gadgil, I added data.nat.prime to the output of the port progress bot. As you can see from looking at the graph or the "longest unported chain", there is a lot of import reduction that could be done on the mathlib3 side to reduce this dependency graph. data.nat.prime is still far enough off that there's time if someone wants to do some of this refactoring now.

port-progress bot (Dec 06 2022 at 22:52):

mathlib port progress algebra.order.field.defs
Ported files: 63/75 (84.0% of total)
Ported lines: 27450/31938 (85.9% of total)
Longest unported chain: 3/19 (84.2% progress)

port-progress bot (Dec 06 2022 at 22:58):

mathlib port progress data.rat.order
Ported files: 102/133 (76.7% of total)
Ported lines: 39568/52864 (74.8% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 06 2022 at 23:02):

mathlib port progress data.nat.choose.basic
Ported files: 97/130 (74.6% of total)
Ported lines: 38213/52321 (73.0% of total)
Longest unported chain: 9/26 (65.4% progress)

port-progress bot (Dec 06 2022 at 23:06):

mathlib port progress data.nat.prime
Ported files: 116/286 (40.6% of total)
Ported lines: 41292/111562 (37.0% of total)
Longest unported chain: 32/49 (34.7% progress)

port-progress bot (Dec 06 2022 at 23:10):

mathlib port progress data.real.basic
Ported files: 111/231 (48.1% of total)
Ported lines: 40941/91394 (44.8% of total)
Longest unported chain: 15/33 (54.5% progress)

port-progress bot (Dec 06 2022 at 23:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 46/90 (51.1% of total)
Ported lines: 17419/31687 (55.0% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 06 2022 at 23:18):

mathlib port progress data.fintype.basic
Ported files: 106/189 (56.1% of total)
Ported lines: 40087/85738 (46.8% of total)
Longest unported chain: 22/39 (43.6% progress)

port-progress bot (Dec 06 2022 at 23:22):

mathlib port progress topology.metric_space.basic
Ported files: 126/521 (24.2% of total)
Ported lines: 42757/225987 (18.9% of total)
Longest unported chain: 55/72 (23.6% progress)

Siddhartha Gadgil (Dec 07 2022 at 00:38):

Scott Morrison said:

Siddhartha Gadgil, I added data.nat.prime to the output of the port progress bot. As you can see from looking at the graph or the "longest unported chain", there is a lot of import reduction that could be done on the mathlib3 side to reduce this dependency graph. data.nat.prime is still far enough off that there's time if someone wants to do some of this refactoring now.

Thanks. It would be nice if this lands before my course starts (beginning of January) and this is also my milestone for switching from binport for a couple of things.

Never having contributed to mathlib3 I am hesitant to reduce imports myself as I may mess things up.

Scott Morrison (Dec 07 2022 at 00:44):

I think it is very unlikely data.nat.prime will be done by the end of December. I haven't looked to see how much the requirements could be shrunk by refactoring, but as is I don't see all of the finiteness stuff done until at least late January. (Pinging @Sarah Smith as I know she wants to keep track of requirements for people who are teaching.)

Heather Macbeth (Dec 07 2022 at 00:48):

Siddhartha Gadgil said:

Never having contributed to mathlib3 I am hesitant to reduce imports myself as I may mess things up.

There's no danger of a rogue proposal breaking mathlib, if this is what you are worried about -- there are a number of automated checks that get run before a proposed change is accepted!

Sarah Smith (Dec 07 2022 at 00:51):

Scott Morrison said:

(Pinging Sarah Smith as I know she wants to keep track of requirements for people who are teaching.)

@Scott Morrison You continue to read my mind from across the globe, thank you Scott

port-progress bot (Dec 07 2022 at 01:12):

mathlib port progress all
Ported files: 163/2811 (5.8% of total)
Ported lines: 47547/967324 (4.9% of total)
Longest unported chain: 111/130 (14.6% progress)

Siddhartha Gadgil (Dec 07 2022 at 02:09):

Thanks for the information. I will work around this. I just need good examples of basic mathematics (including algorithms) and since Nat.gcd and its basic properties are in Lean 4 itself I can just define primes and use them.

Scott Morrison (Dec 07 2022 at 03:19):

I've opened a PR for Data.Set.Basic at https://github.com/leanprover-community/mathlib4/pull/892

Scott Morrison (Dec 07 2022 at 03:20):

It has many errors, but skimming through what remains it seems they are for a great variety of reasons. This is good news, because it means anyone who wants to can work on it. Please feel free to scroll down to a random point in the file and start work. :-)

Matej Penciak (Dec 07 2022 at 04:45):

This is not particularly important, but trying to run the port progress script locally I'm running into some issues:

~/MathlibPort/mathlib/src ❯ leanproject import-graph --to ring_theory.mv_polynomial.basic --port-status --exclude-tactics out.pdf
while parsing a block mapping
  in "<byte string>", line 19, column 1:
    algebra.abs: Yes mathlib4#477 c4 ...
    ^
expected <block end>, but found '<scalar>'
  in "<byte string>", line 322, column 28:
    algebra.order.group.prod: 'No'
                               ^

It seems like the script is running into issues parsing the port-status YAML file.

The following runs fine: leanproject import-graph --to ring_theory.mv_polynomial.basic out.pdf, but it'd be nice to have some coloration :(

EDIT: I may have totally borked something, because now even the port_status.py script is breaking with a yaml parsing error

(Weirdly, running with --exclude-tactics also returns an error: 'algebra.order.monoid.units')

EDIT2: This may be related to the added algebra.order.group.order_iso line?
https://github.com/leanprover-community/mathlib/wiki/mathlib4-port-status/_compare/9c2bc022783594980df80f786404a0dbf452c487...20a5d7d9a87647c3cd50697d34b9d086b0fff92b

Kevin Buzzard (Dec 07 2022 at 06:59):

Right -- that line doesn't end in a '

Mario Carneiro (Dec 07 2022 at 07:01):

looks like it was typoed for a ;

Scott Morrison (Dec 07 2022 at 07:05):

Fixed.

Ruben Van de Velde (Dec 07 2022 at 09:52):

Siddhartha Gadgil said:

Scott Morrison said:

Siddhartha Gadgil, I added data.nat.prime to the output of the port progress bot. As you can see from looking at the graph or the "longest unported chain", there is a lot of import reduction that could be done on the mathlib3 side to reduce this dependency graph. data.nat.prime is still far enough off that there's time if someone wants to do some of this refactoring now.

Thanks. It would be nice if this lands before my course starts (beginning of January) and this is also my milestone for switching from binport for a couple of things.

Never having contributed to mathlib3 I am hesitant to reduce imports myself as I may mess things up.

I'm removing the dependency on finite stuff in #17840

Ruben Van de Velde (Dec 07 2022 at 09:52):

Or most of it - it still depends on a bunch of list stuff

Ruben Van de Velde (Dec 07 2022 at 10:49):

I've also got a branch that removes the list dependencies at the expense of moving nat.factors and the norm_num extension out of data.nat.prime, but that's for after I get #17840 compiling

Ruben Van de Velde (Dec 07 2022 at 16:04):

https://github.com/leanprover-community/mathlib4/pull/898 is ready to land after the merge conflicts got fixed - just needs someone to tell bors

Heather Macbeth (Dec 07 2022 at 16:07):

I took it upon myself (I've never been sure whether the author officially has the right to do this ...)

Heather Macbeth (Dec 07 2022 at 16:38):

Hmm, maybe bors is stuck.

Ruben Van de Velde (Dec 07 2022 at 16:44):

Seems like it's building now

port-progress bot (Dec 07 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 66/75 (88.0% of total)
Ported lines: 27842/31954 (87.1% of total)
Longest unported chain: 1/19 (94.7% progress)

port-progress bot (Dec 07 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 107/133 (80.5% of total)
Ported lines: 40246/52635 (76.5% of total)
Longest unported chain: 7/26 (73.1% progress)

port-progress bot (Dec 07 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 106/131 (80.9% of total)
Ported lines: 39110/52386 (74.7% of total)
Longest unported chain: 7/27 (74.1% progress)

port-progress bot (Dec 07 2022 at 18:15):

mathlib port progress data.nat.prime
Ported files: 127/287 (44.3% of total)
Ported lines: 42536/111631 (38.1% of total)
Longest unported chain: 30/50 (40.0% progress)

port-progress bot (Dec 07 2022 at 18:18):

mathlib port progress data.real.basic
Ported files: 121/232 (52.2% of total)
Ported lines: 41981/91463 (45.9% of total)
Longest unported chain: 14/34 (58.8% progress)

port-progress bot (Dec 07 2022 at 18:22):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17673/31691 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 07 2022 at 18:25):

mathlib port progress data.fintype.basic
Ported files: 115/190 (60.5% of total)
Ported lines: 40984/85803 (47.8% of total)
Longest unported chain: 20/40 (50.0% progress)

port-progress bot (Dec 07 2022 at 18:29):

mathlib port progress topology.metric_space.basic
Ported files: 137/522 (26.2% of total)
Ported lines: 44005/226076 (19.5% of total)
Longest unported chain: 53/73 (27.4% progress)

port-progress bot (Dec 07 2022 at 19:16):

mathlib port progress all
Ported files: 177/2817 (6.3% of total)
Ported lines: 49585/968556 (5.1% of total)
Longest unported chain: 111/131 (15.3% progress)

Scott Morrison (Dec 07 2022 at 23:02):

We are very very close to our first goal!

  • algebra.order.ring.defs is open and ready for porting
  • algebra.order.field.defs has no other prerequisites, so potentially can be done at the same time
  • algebra.order.ring.canonical and then data.nat.order.basic can also be done immediately once algebra.order.ring.defs is ready.

Scott Morrison (Dec 07 2022 at 23:08):

There is lots of stuff available for porting today:

data.set.basic                   -- contributions welcome mathlib4#892
algebra.order.ring.defs
algebra.order.with_zero
algebra.order.group.abs          -- just needs a merge? mathlib4#896
algebra.hom.group_instances
algebra.order.monoid.with_top    -- WIP Jon Eugster
algebra.group.opposite
algebra.group_with_zero.units.lemmas
algebra.order.group.inj_surj
algebra.group.ulift
ring_theory.coprime.basic        -- mathlib4#899
algebra.ring.idempotents
order.hom.bounded                -- mathlib4#888
algebra.euclidean_domain.basic
algebra.order.group.type_tags
algebra.hom.equiv.type_tags
algebra.order.hom.monoid
algebra.group.with_one.basic
combinatorics.quiver.cast
algebra.order.sub.basic

We may be through the bottleneck now, so please invite your friends along. :-)

Kevin Buzzard (Dec 07 2022 at 23:32):

What is our second goal? I've been using the pdfs for inspiration rather than the port status script.

Eric Wieser (Dec 07 2022 at 23:45):

mathlib4#892 would be best left until a new mathport output is available

Scott Morrison (Dec 08 2022 at 00:23):

@Kevin Buzzard, data.rat.order is the primary short term goal. It will be very helpful for people teaching next semester in Lean 4 if that is done by the new year. It feels completely plausible.

Scott Morrison (Dec 08 2022 at 01:04):

I made a start on algebra.order.ring.defs at mathlib4#905. Anyone is welcome to work on it.

Scott Morrison (Dec 08 2022 at 04:32):

It's now ready for review.

Scott Morrison (Dec 08 2022 at 04:40):

and includes algebra.order.field.defs, since it is trivial.

Scott Morrison (Dec 08 2022 at 04:45):

and algebra.order.ring.canonical.

Arien Malec (Dec 08 2022 at 04:48):

algebra.group.ulift was super trivial -- feels good!

Scott Morrison (Dec 08 2022 at 04:59):

@Arien Malec, could you add the additive versions of the #aligns? This will be automated soon.

Arien Malec (Dec 08 2022 at 05:05):

Don't see instructions on the wiki -- what's the Zulip thread?

Arien Malec (Dec 08 2022 at 05:11):

This? https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/.23align.20and.20to_additive/near/314364635

Scott Morrison (Dec 08 2022 at 05:16):

Would you be able to add this to the wiki?

Arien Malec (Dec 08 2022 at 05:26):

Done -- is there a way to interrogate Lean to see the exact naming? Or does it require knowledge of the to_additive algorithm? It's clear when mul_foo gets renamed to add_foo, but I see inv, smul, pow attributes & I don't have a clear mental model for what to_additive does there.

Scott Morrison (Dec 08 2022 at 05:39):

You can hover over the to_additive keyword to find the additivized name on the Lean 4 side.

Scott Morrison (Dec 08 2022 at 05:40):

There is not a trivial way to look it up on the Lean 3 side. Usually you can quickly guess it from the other three names, however. Also, if you're really stuck you can go the mathlib itself and add a ? to to_additive, and it will print the name it is choosing.

This will all go away soon when mathport gains the ability to do it automatically.

Arien Malec (Dec 08 2022 at 06:24):

Also found:

private def nameDict : String  List String
| "one"         => ["zero"]
| "mul"         => ["add"]
| "smul"        => ["vadd"]
| "inv"         => ["neg"]
| "div"         => ["sub"]
| "prod"        => ["sum"]
| "hmul"        => ["hadd"]
| "hsmul"       => ["hvadd"]
| "hdiv"        => ["hsub"]
| "hpow"        => ["hsmul"]
| "finprod"     => ["finsum"]
| "pow"         => ["smul"]
| "npow"        => ["nsmul"]
| "zpow"        => ["zsmul"]
| "monoid"      => ["add", "Monoid"]
| "submonoid"   => ["add", "Submonoid"]
| "group"       => ["add", "Group"]
| "subgroup"    => ["add", "Subgroup"]
| "semigroup"   => ["add", "Semigroup"]
| "magma"       => ["add", "Magma"]
| "haar"        => ["add", "Haar"]
| "prehaar"     => ["add", "Prehaar"]
| "unit"        => ["add", "Unit"]
| "units"       => ["add", "Units"]
| x             => [x]

Johan Commelin (Dec 08 2022 at 07:21):

Scott Morrison said:

I made a start on algebra.order.ring.defs at mathlib4#905. Anyone is welcome to work on it.

This looks good to me! If one more person with a bit more porting experience then me can look it over, then I'm happy to kick it on the queue.

Ruben Van de Velde (Dec 08 2022 at 13:12):

Ruben Van de Velde said:

I've also got a branch that removes the list dependencies at the expense of moving nat.factors and the norm_num extension out of data.nat.prime, but that's for after I get #17840 compiling

This is now #17854

port-progress bot (Dec 08 2022 at 18:04):

mathlib port progress algebra.order.field.defs
Ported files: 68/75 (90.7% of total)
Ported lines: 28848/31966 (90.2% of total)
Longest unported chain: 1/19 (94.7% progress)

port-progress bot (Dec 08 2022 at 18:08):

mathlib port progress data.rat.order
Ported files: 112/134 (83.6% of total)
Ported lines: 41757/52684 (79.3% of total)
Longest unported chain: 7/27 (74.1% progress)

port-progress bot (Dec 08 2022 at 18:11):

mathlib port progress data.nat.choose.basic
Ported files: 110/132 (83.3% of total)
Ported lines: 40618/52456 (77.4% of total)
Longest unported chain: 8/28 (71.4% progress)

port-progress bot (Dec 08 2022 at 18:15):

mathlib port progress data.nat.prime
Ported files: 128/221 (57.9% of total)
Ported lines: 43595/89069 (48.9% of total)
Longest unported chain: 14/34 (58.8% progress)

port-progress bot (Dec 08 2022 at 18:18):

mathlib port progress data.real.basic
Ported files: 128/233 (54.9% of total)
Ported lines: 43780/91550 (47.8% of total)
Longest unported chain: 15/35 (57.1% progress)

port-progress bot (Dec 08 2022 at 18:22):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17677/31695 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 08 2022 at 18:26):

mathlib port progress data.fintype.basic
Ported files: 120/191 (62.8% of total)
Ported lines: 42510/85882 (49.5% of total)
Longest unported chain: 21/41 (48.8% progress)

Winston Yin (Dec 08 2022 at 18:27):

@Scott Morrison I ported order.ring.defs yesterday (it compiles) but the tricky thing is removing the ad hoc port order.ring

Winston Yin (Dec 08 2022 at 18:27):

(deleted)

Winston Yin (Dec 08 2022 at 18:29):

Oops never mind, looks like you’ve merged your PR already

port-progress bot (Dec 08 2022 at 18:29):

mathlib port progress topology.metric_space.basic
Ported files: 145/524 (27.7% of total)
Ported lines: 45974/226176 (20.3% of total)
Longest unported chain: 54/74 (27.0% progress)

port-progress bot (Dec 08 2022 at 19:14):

mathlib port progress all
Ported files: 186/2822 (6.6% of total)
Ported lines: 51637/969537 (5.3% of total)
Longest unported chain: 112/132 (15.2% progress)

port-progress bot (Dec 09 2022 at 03:55):

mathlib port progress data.rat.order
Ported files: 113/134 (84.3% of total)
Ported lines: 42049/52695 (79.8% of total)
Longest unported chain: 7/27 (74.1% progress)

Scott Morrison (Dec 09 2022 at 03:59):

The port progress bot now produces graphs that omit all files which have been ported, and all their children have been ported.

This now makes the graphs much less cluttered (we're making progress!) and easier to see what we need to be working on to achieve the next targets.

port-progress bot (Dec 09 2022 at 04:02):

mathlib port progress data.rat.order
Ported files: 113/134 (84.3% of total)
Ported lines: 42049/52695 (79.8% of total)
Longest unported chain: 7/27 (74.1% progress)

port-progress bot (Dec 09 2022 at 04:05):

mathlib port progress data.nat.choose.basic
Ported files: 111/132 (84.1% of total)
Ported lines: 40898/52455 (78.0% of total)
Longest unported chain: 8/28 (71.4% progress)

port-progress bot (Dec 09 2022 at 04:09):

mathlib port progress data.nat.prime
Ported files: 119/156 (76.3% of total)
Ported lines: 42043/61245 (68.6% of total)
Longest unported chain: 10/30 (66.7% progress)

port-progress bot (Dec 09 2022 at 04:13):

mathlib port progress data.real.basic
Ported files: 130/233 (55.8% of total)
Ported lines: 44251/91549 (48.3% of total)
Longest unported chain: 15/35 (57.1% progress)

port-progress bot (Dec 09 2022 at 04:16):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17677/31695 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 09 2022 at 04:20):

mathlib port progress data.fintype.basic
Ported files: 121/192 (63.0% of total)
Ported lines: 42790/85921 (49.8% of total)
Longest unported chain: 22/42 (47.6% progress)

port-progress bot (Dec 09 2022 at 04:24):

mathlib port progress topology.metric_space.basic
Ported files: 149/524 (28.4% of total)
Ported lines: 46585/225456 (20.7% of total)
Longest unported chain: 55/75 (26.7% progress)

port-progress bot (Dec 09 2022 at 05:21):

mathlib port progress all
Ported files: 192/2827 (6.8% of total)
Ported lines: 52472/969650 (5.4% of total)
Longest unported chain: 114/134 (14.9% progress)

Ruben Van de Velde (Dec 09 2022 at 06:34):

port-progress bot said:

mathlib port progress data.nat.prime
Ported files: 127/287 (44.3% of total)
Ported lines: 42536/111631 (38.1% of total)
Longest unported chain: 30/50 (40.0% progress)

port-progress bot said:

mathlib port progress data.nat.prime
Ported files: 119/156 (76.3% of total)
Ported lines: 42043/61245 (68.6% of total)
Longest unported chain: 10/30 (66.7% progress)

That looks a bit more attainable now. I don't see much remaining that would obviously help reduce dependencies

port-progress bot (Dec 09 2022 at 18:04):

mathlib port progress data.rat.order
Ported files: 113/134 (84.3% of total)
Ported lines: 42049/52695 (79.8% of total)
Longest unported chain: 7/27 (74.1% progress)

port-progress bot (Dec 09 2022 at 18:08):

mathlib port progress data.nat.choose.basic
Ported files: 111/132 (84.1% of total)
Ported lines: 40898/52455 (78.0% of total)
Longest unported chain: 8/28 (71.4% progress)

port-progress bot (Dec 09 2022 at 18:11):

mathlib port progress data.nat.prime
Ported files: 120/156 (76.9% of total)
Ported lines: 42532/61245 (69.4% of total)
Longest unported chain: 10/30 (66.7% progress)

port-progress bot (Dec 09 2022 at 18:15):

mathlib port progress data.real.basic
Ported files: 131/233 (56.2% of total)
Ported lines: 44740/91588 (48.8% of total)
Longest unported chain: 15/35 (57.1% progress)

port-progress bot (Dec 09 2022 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17677/31695 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 09 2022 at 18:21):

mathlib port progress data.fintype.basic
Ported files: 121/192 (63.0% of total)
Ported lines: 42790/85973 (49.8% of total)
Longest unported chain: 22/42 (47.6% progress)

port-progress bot (Dec 09 2022 at 18:25):

mathlib port progress topology.metric_space.basic
Ported files: 152/525 (29.0% of total)
Ported lines: 47313/224644 (21.1% of total)
Longest unported chain: 55/75 (26.7% progress)

port-progress bot (Dec 09 2022 at 19:10):

mathlib port progress all
Ported files: 195/2831 (6.9% of total)
Ported lines: 53200/969836 (5.5% of total)
Longest unported chain: 115/135 (14.8% progress)

Yuyang Zhao (Dec 10 2022 at 12:47):

I have made some PRs to reduce the dependencies of data.fintype.basic
#17880: data.set.lattice and its dependencies (also reduces the longest unported chain of mathlib)
#17886: int.order.basic
#17887: data.list.of_fn and its dependencies
#17888: data.multiset.powerset and data.list.sublists (also reduces the longest unported chain of mathlib)

port-progress bot (Dec 10 2022 at 18:04):

mathlib port progress data.rat.order
Ported files: 113/134 (84.3% of total)
Ported lines: 42052/52698 (79.8% of total)
Longest unported chain: 7/27 (74.1% progress)

port-progress bot (Dec 10 2022 at 18:08):

mathlib port progress data.nat.choose.basic
Ported files: 111/132 (84.1% of total)
Ported lines: 40898/52455 (78.0% of total)
Longest unported chain: 8/28 (71.4% progress)

port-progress bot (Dec 10 2022 at 18:11):

mathlib port progress data.nat.prime
Ported files: 120/156 (76.9% of total)
Ported lines: 42532/61245 (69.4% of total)
Longest unported chain: 10/30 (66.7% progress)

port-progress bot (Dec 10 2022 at 18:15):

mathlib port progress data.real.basic
Ported files: 131/233 (56.2% of total)
Ported lines: 44743/91593 (48.8% of total)
Longest unported chain: 15/35 (57.1% progress)

port-progress bot (Dec 10 2022 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17677/31695 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 10 2022 at 18:22):

mathlib port progress data.fintype.basic
Ported files: 121/192 (63.0% of total)
Ported lines: 42790/85973 (49.8% of total)
Longest unported chain: 22/42 (47.6% progress)

port-progress bot (Dec 10 2022 at 18:25):

mathlib port progress topology.metric_space.basic
Ported files: 152/525 (29.0% of total)
Ported lines: 47316/224685 (21.1% of total)
Longest unported chain: 55/75 (26.7% progress)

port-progress bot (Dec 10 2022 at 19:08):

mathlib port progress all
Ported files: 195/2832 (6.9% of total)
Ported lines: 53203/969953 (5.5% of total)
Longest unported chain: 115/135 (14.8% progress)

Winston Yin (Dec 11 2022 at 03:18):

Do I understand this correctly: grey nodes suggest room for improvement in the way these files are imported by other files, not that there's something wrong with these files themselves?

Scott Morrison (Dec 11 2022 at 09:21):

Yes. A node is marked grey is no declarations in it are used in the target file. This usually means we have something like:

  • Three files, A, B, C, with C the "target file".
  • B imports A
  • C imports B
  • but C only depends on parts of B which did not depend on A.
    Then A will be marked in gray.

It suggests that it may be possible to split B into B and B', with B importing A and C importing B'. This may not necessarily be a good idea, but fairly often is.

Scott Morrison (Dec 11 2022 at 09:22):

Long strings of gray files (which are displayed as long strings of files prefixed with - in the "longest unported chain" links) are particularly suspicious.

port-progress bot (Dec 11 2022 at 18:04):

mathlib port progress data.rat.order
Ported files: 113/134 (84.3% of total)
Ported lines: 42066/52712 (79.8% of total)
Longest unported chain: 7/27 (74.1% progress)

port-progress bot (Dec 11 2022 at 18:08):

mathlib port progress data.nat.choose.basic
Ported files: 111/132 (84.1% of total)
Ported lines: 40904/52461 (78.0% of total)
Longest unported chain: 8/28 (71.4% progress)

port-progress bot (Dec 11 2022 at 18:12):

mathlib port progress data.nat.prime
Ported files: 120/156 (76.9% of total)
Ported lines: 42550/61263 (69.5% of total)
Longest unported chain: 10/30 (66.7% progress)

port-progress bot (Dec 11 2022 at 18:16):

mathlib port progress data.real.basic
Ported files: 131/233 (56.2% of total)
Ported lines: 44765/91650 (48.8% of total)
Longest unported chain: 15/35 (57.1% progress)

port-progress bot (Dec 11 2022 at 18:19):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17677/31695 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 11 2022 at 18:23):

mathlib port progress data.fintype.basic
Ported files: 121/183 (66.1% of total)
Ported lines: 42800/82721 (51.7% of total)
Longest unported chain: 21/41 (48.8% progress)

port-progress bot (Dec 11 2022 at 18:27):

mathlib port progress topology.metric_space.basic
Ported files: 152/525 (29.0% of total)
Ported lines: 47358/224698 (21.1% of total)
Longest unported chain: 54/74 (27.0% progress)

port-progress bot (Dec 11 2022 at 19:20):

mathlib port progress all
Ported files: 195/2834 (6.9% of total)
Ported lines: 53253/970192 (5.5% of total)
Longest unported chain: 114/134 (14.9% progress)

port-progress bot (Dec 12 2022 at 02:11):

mathlib port progress data.rat.order
Ported files: 115/134 (85.8% of total)
Ported lines: 44237/52712 (83.9% of total)
Longest unported chain: 6/27 (77.8% progress)

Johan Commelin (Dec 12 2022 at 06:45):

Did the bot die?

Scott Morrison (Dec 12 2022 at 07:10):

Oops, didn't realise I'd cause confusion. I asked for a one-off run as I wanted to see the new graph. :-)

Scott Morrison (Dec 12 2022 at 07:11):

Maybe I'll update the bot to update the graphs more often, but only post once a day.

Scott Morrison (Dec 12 2022 at 09:53):

Suggestions for anyone looking for a porting task, and who would like advice for identifying the highest priority work:

  1. Click on the latest link to data.rat.order posted by the port-progress-bot, and

    • Help out with any open PRs (you can just click on a dark blue node)
    • Start the port of any open file (those nodes in light blue)
      • in particular anyone can start on data.nat.gcd.basic.
  2. repeat the same for the other targets that port-progress-bot posts about, e.g. data.fintype.basic.

  3. review the output of scripts/port_status.sh and work on something from that.

    • In particular data.list.basic and data.set.n_ary (possibly also data.set.prod and data.set.function in the same PR) are now ready to port, and high priority.

Ruben Van de Velde (Dec 12 2022 at 10:11):

Could someone give bors another kick on https://github.com/leanprover-community/mathlib4/pull/955?

Patrick Massot (Dec 12 2022 at 10:37):

Tomorrow we'll have a mathlib4 afternoon in Orsay with Floris, Joël, Riccardo and I. Hopefully we'll find useful things to try.

Scott Morrison (Dec 12 2022 at 10:41):

Hopefully the graphs now update every two hours (but only get a new URL each day), so are usable to find out what's coming up next.

Kevin Buzzard (Dec 12 2022 at 10:59):

Re Data.Int.Order.Basic: as far as I can see the main decision to make right now is whether we are going to ask the Lean 4 devs to change their definition of div and mod on Int, or whether we are going to work around this ourselves. Looks like Leo is still on vacation.

Yaël Dillies (Dec 12 2022 at 11:05):

What difference is there?

Ruben Van de Velde (Dec 12 2022 at 11:08):

See https://leanprover-community.github.io/mathlib4_docs/Std/Data/Int/Basic.html

Yaël Dillies (Dec 12 2022 at 11:09):

One or more equations did not get rendered due to their size. :upside_down:

Kevin Buzzard (Dec 12 2022 at 11:10):

-- lean 3
#eval (-5 : ) / -2 -- 3
-- lean 4
#eval -5 / -2 -- 2

Yaël Dillies (Dec 12 2022 at 11:10):

Oh no

Yaël Dillies (Dec 12 2022 at 11:11):

Lean 4 is on the right side of history here, right? We want a + b / c = (a * c + b) / c, or am I wrong?

Kevin Buzzard (Dec 12 2022 at 11:15):

See https://leanprover.zulipchat.com/#narrow/stream/341532-lean4-dev/topic/.5BRFC.5D.20Int.2Ediv.20convention/near/296956937 for an in-depth discussion.

Yaël Dillies (Dec 12 2022 at 11:19):

Oh no, I see

Kevin Buzzard (Dec 12 2022 at 11:25):

Re Algebra.Hom.Ring : right now this seems to be a file which has been half-ported. I am scared to just start at the first error and press on -- this file has just been advertised as needing help, so for all I know someone else has already fixed up the next 100 lines and is about to push. I far prefer trying to fix up the last few errors in a file which are causing problems, when I'm leaping into a file which someone else has claimed.

Kevin Buzzard (Dec 12 2022 at 11:26):

My Lean time has been rather fragmented for the last few days and this is precisely why I didn't claim a file during that time -- I didn't want to fix the capitalisation in half the file and then have to stop for 2 days and then fix 1/2 of the remainder and then stop for another day whilst other people look on thinking "we need this file and it's still hugely broken". When Imperial's term is over in 4 days' time I'll be able to go back to claiming files.

port-progress bot (Dec 12 2022 at 18:04):

mathlib port progress data.rat.order
Ported files: 118/134 (88.1% of total)
Ported lines: 46281/52718 (87.8% of total)
Longest unported chain: 5/27 (81.5% progress)

port-progress bot (Dec 12 2022 at 18:08):

mathlib port progress data.nat.choose.basic
Ported files: 116/132 (87.9% of total)
Ported lines: 44821/52467 (85.4% of total)
Longest unported chain: 6/28 (78.6% progress)

port-progress bot (Dec 12 2022 at 18:11):

mathlib port progress data.nat.prime
Ported files: 128/156 (82.1% of total)
Ported lines: 47428/61269 (77.4% of total)
Longest unported chain: 8/30 (73.3% progress)

port-progress bot (Dec 12 2022 at 18:15):

mathlib port progress data.real.basic
Ported files: 140/233 (60.1% of total)
Ported lines: 49724/91666 (54.2% of total)
Longest unported chain: 13/35 (62.9% progress)

port-progress bot (Dec 12 2022 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17677/31695 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 12 2022 at 18:22):

mathlib port progress data.fintype.basic
Ported files: 126/183 (68.9% of total)
Ported lines: 46717/82740 (56.5% of total)
Longest unported chain: 19/41 (53.7% progress)

port-progress bot (Dec 12 2022 at 18:26):

mathlib port progress topology.metric_space.basic
Ported files: 162/525 (30.9% of total)
Ported lines: 52370/224722 (23.3% of total)
Longest unported chain: 52/74 (29.7% progress)

port-progress bot (Dec 12 2022 at 19:09):

mathlib port progress all
Ported files: 212/2835 (7.5% of total)
Ported lines: 58840/970763 (6.1% of total)
Longest unported chain: 112/134 (16.4% progress)

Winston Yin (Dec 13 2022 at 02:03):

@Kevin Buzzard Algebra.Hom.Ring is completely ported except for two simp lint errors. Would anyone like to take a crack at them? mathlib4#958

Scott Morrison (Dec 13 2022 at 11:26):

We're getting very close to data.rat.order now; hopefully in the next day or two.

If anyone wants to take a look at data.nat.cast.basic, it is open for porting.

Patrick Massot (Dec 13 2022 at 12:53):

We are starting our mathlib4 hackaton in Orsay.

Moritz Doll (Dec 13 2022 at 12:54):

so tomorrow we have filters in mathlib4?

Patrick Massot (Dec 13 2022 at 12:54):

We want to tackle:

  • Floris: data.nat.cast.basic
  • Riccardo: algebra.field.basic
  • Joël: algebra.group_power.ring
  • Patrick: data.set.prod

Ruben Van de Velde (Dec 13 2022 at 12:55):

Ah, I was just starting on data.set.prod, @Patrick Massot

Patrick Massot (Dec 13 2022 at 12:55):

No problem, I can switch

Patrick Massot (Dec 13 2022 at 12:57):

I'll do algebra.ring.opposite then

Patrick Massot (Dec 13 2022 at 14:59):

algebra.ring.opposite is currently blocked by an issue with the simps attribute so I'll start on data.set.sigma

Patrick Massot (Dec 13 2022 at 16:27):

data.set.basic is waiting for an answer to https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/referring.20to.20namespace.20in.20theorem.20name so I'll start on logic.embedding.set

Patrick Massot (Dec 13 2022 at 17:15):

I'll do data.set.bool_indicator now.

Patrick Massot (Dec 13 2022 at 17:50):

The first Orsay mathlib4 hackaton is now over. We ported 10 files!

Riccardo Brasca (Dec 13 2022 at 17:51):

We wait for all the people in the Paris area!

port-progress bot (Dec 13 2022 at 18:04):

mathlib port progress data.rat.order
Ported files: 120/134 (89.6% of total)
Ported lines: 47452/52727 (90.0% of total)
Longest unported chain: 4/27 (85.2% progress)

port-progress bot (Dec 13 2022 at 18:08):

mathlib port progress data.nat.choose.basic
Ported files: 118/132 (89.4% of total)
Ported lines: 45687/52545 (86.9% of total)
Longest unported chain: 5/28 (82.1% progress)

port-progress bot (Dec 13 2022 at 18:11):

mathlib port progress data.nat.prime
Ported files: 131/156 (84.0% of total)
Ported lines: 48889/61347 (79.7% of total)
Longest unported chain: 7/30 (76.7% progress)

port-progress bot (Dec 13 2022 at 18:15):

mathlib port progress data.real.basic
Ported files: 147/233 (63.1% of total)
Ported lines: 52022/91744 (56.7% of total)
Longest unported chain: 12/35 (65.7% progress)

port-progress bot (Dec 13 2022 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17677/31695 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 13 2022 at 18:22):

mathlib port progress data.fintype.basic
Ported files: 131/183 (71.6% of total)
Ported lines: 47859/82818 (57.8% of total)
Longest unported chain: 18/41 (56.1% progress)

port-progress bot (Dec 13 2022 at 18:26):

mathlib port progress topology.metric_space.basic
Ported files: 169/525 (32.2% of total)
Ported lines: 54668/224783 (24.3% of total)
Longest unported chain: 51/74 (31.1% progress)

port-progress bot (Dec 13 2022 at 19:09):

mathlib port progress all
Ported files: 219/2843 (7.7% of total)
Ported lines: 61138/971375 (6.3% of total)
Longest unported chain: 113/136 (16.9% progress)

Rémy Degenne (Dec 13 2022 at 19:37):

Patrick Massot said:

The first Orsay mathlib4 hackaton is now over. We ported 10 files!

I saw your message about starting the hackaton, got motivated and installed lean 4 for the first time. I verified my installation by porting my first (very small) file. Overall, the installation was smooth and mathport did all the porting work. The porting wiki is great :+1:

Scott Morrison (Dec 13 2022 at 21:09):

@Patrick Massot (and others) please remember to include the mathlib3 sha that you are using as the basis for your port in the PR description. This sha is available (amongst other places) in the README of mathport.

https://github.com/leanprover-community/mathlib4/pull/988 is currently missing a sha

Scott Morrison (Dec 13 2022 at 21:10):

Further, please remember to include your PR number, in the format mathlib4#nnn, in the #port-status wiki page.

If the file is not already there (e.g. for https://github.com/leanprover-community/mathlib4/pull/988, which ports data.set.bool_indicator), please add the line yourself. This will happen for newly introduced files in mathlib.

Scott Morrison (Dec 13 2022 at 21:32):

Sent 8 PRs to bors, delegated another 4, and sent a few back to authors!

Scott Morrison (Dec 14 2022 at 00:54):

Data.Int.Cast.Lemmas is up as a PR mathlib4#995. I've done most of the cleanup, but there are few broken proofs that need attention. This is on the critical path to Data.Rat.Order.

Scott Morrison (Dec 14 2022 at 01:40):

I've started on Data.Rat.Defs as mathlib4#998. I've done the first pass, but many many proofs are still broken. I think this is probably the highest priority file for now, and could use multiple eyes. Just start somewhere and fix errors. :-)

Winston Yin (Dec 14 2022 at 01:47):

One of you lucky ducks is going to get mathlib4#1000 soon

Scott Morrison (Dec 14 2022 at 12:35):

Today's advice about what to work on:

  • We are super close to Data.Rat.Order, but mathlib4#998 for Data.Rat.Defs still needs a lot of work. There are many independent problems, so I would encourage anyone with some time today to have a look at this and push any fixes you can.
  • After that, I think Data.List.Basic is an important target, which Chris has started in mathlib4#996. Again, it has many problems, and could do with many helpers!
  • Otherwise, please look at the port-progress-bot graphs for your favourite file, and either:

    1. ideally, go help out with an open PR (shaded dark blue)
    2. otherwise, open a new PR (light blue files)

Ruben Van de Velde (Dec 14 2022 at 14:23):

Taking a look at Data.Rat.Defs for the next 15 mins or so

Mario Carneiro (Dec 14 2022 at 14:31):

note that Data.Rat.Defs is expected to be harder than the usual port since Rat has been redefined

Mario Carneiro (Dec 14 2022 at 14:32):

or actually maybe Data.Rat.Defs is easy, just #aligns and Data.Rat.Basic is the hard one

Yaël Dillies (Dec 14 2022 at 14:35):

Is Rat in Std now?

Mario Carneiro (Dec 14 2022 at 14:49):

yes

Ruben Van de Velde (Dec 14 2022 at 15:02):

Oh, is that why injection fails?

Kevin Buzzard (Dec 14 2022 at 17:17):

data.list.basic is mathlib4#966

port-progress bot (Dec 14 2022 at 18:04):

mathlib port progress data.rat.order
Ported files: 124/134 (92.5% of total)
Ported lines: 48762/52747 (92.4% of total)
Longest unported chain: 2/27 (92.6% progress)

port-progress bot (Dec 14 2022 at 18:08):

mathlib port progress data.nat.choose.basic
Ported files: 119/131 (90.8% of total)
Ported lines: 46260/52260 (88.5% of total)
Longest unported chain: 4/27 (85.2% progress)

port-progress bot (Dec 14 2022 at 18:11):

mathlib port progress data.nat.prime
Ported files: 137/156 (87.8% of total)
Ported lines: 51065/61376 (83.2% of total)
Longest unported chain: 6/29 (79.3% progress)

port-progress bot (Dec 14 2022 at 18:15):

mathlib port progress data.real.basic
Ported files: 158/233 (67.8% of total)
Ported lines: 55024/91803 (59.9% of total)
Longest unported chain: 11/34 (67.6% progress)

port-progress bot (Dec 14 2022 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17697/31715 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 14 2022 at 18:22):

mathlib port progress data.fintype.basic
Ported files: 135/183 (73.8% of total)
Ported lines: 49488/82863 (59.7% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Dec 14 2022 at 18:26):

mathlib port progress topology.metric_space.basic
Ported files: 191/525 (36.4% of total)
Ported lines: 58414/224862 (26.0% of total)
Longest unported chain: 50/73 (31.5% progress)

port-progress bot (Dec 14 2022 at 19:07):

mathlib port progress all
Ported files: 253/2843 (8.9% of total)
Ported lines: 66687/971624 (6.9% of total)
Longest unported chain: 112/135 (17.0% progress)

port-progress bot (Dec 15 2022 at 18:03):

mathlib port progress data.rat.order
Ported files: 124/134 (92.5% of total)
Ported lines: 48823/52808 (92.5% of total)
Longest unported chain: 2/27 (92.6% progress)

port-progress bot (Dec 15 2022 at 18:07):

mathlib port progress data.nat.choose.basic
Ported files: 120/131 (91.6% of total)
Ported lines: 47665/52309 (91.1% of total)
Longest unported chain: 3/27 (88.9% progress)

Ruben Van de Velde (Dec 15 2022 at 18:08):

These graphs are getting ridiculously small now

port-progress bot (Dec 15 2022 at 18:11):

mathlib port progress data.nat.prime
Ported files: 138/156 (88.5% of total)
Ported lines: 52506/61461 (85.4% of total)
Longest unported chain: 5/29 (82.8% progress)

port-progress bot (Dec 15 2022 at 18:14):

mathlib port progress data.real.basic
Ported files: 165/233 (70.8% of total)
Ported lines: 58572/91940 (63.7% of total)
Longest unported chain: 10/34 (70.6% progress)

port-progress bot (Dec 15 2022 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17722/31740 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 15 2022 at 18:21):

mathlib port progress data.fintype.basic
Ported files: 137/183 (74.9% of total)
Ported lines: 52172/82949 (62.9% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Dec 15 2022 at 18:25):

mathlib port progress topology.metric_space.basic
Ported files: 200/525 (38.1% of total)
Ported lines: 62272/225123 (27.7% of total)
Longest unported chain: 50/73 (31.5% progress)

port-progress bot (Dec 15 2022 at 19:10):

mathlib port progress all
Ported files: 266/2844 (9.4% of total)
Ported lines: 71430/972360 (7.3% of total)
Longest unported chain: 112/135 (17.0% progress)

Heather Macbeth (Dec 15 2022 at 20:12):

Ruben Van de Velde said:

These graphs are getting ridiculously small now

When data.rat.order and data.nat.choose.basic are ported, we need more targets to track! Maybe linear_algebra.basic?

Riccardo Brasca (Dec 15 2022 at 20:55):

What is the command to generate say data.real.basic.pdf? Using leanproject I always get huge graphs (and with less colors).

Scott Morrison (Dec 15 2022 at 21:15):

The bot is running:

leanproject import-graph --to $target --exclude-tactics --reduce --port-status --exclude-ported --show-unused --mathlib4 $tmp_dir/mathlib4 $graph_dir/$today/$target.pdf

Riccardo Brasca (Dec 15 2022 at 21:30):

I get

Error: no such option: --exclude-ported

I have leanproject version 1.3.1, that I think is the last one, so this is maybe only in the github repo.

Scott Morrison (Dec 15 2022 at 21:36):

This option removes everything that has been ported, and whose children have been ported. It is what is making the graphs for targets we're almost done with small.

Scott Morrison (Dec 15 2022 at 21:37):

You can

git clone git@github.com:leanprover-community/mathlib-tools.git
cd mathlib-tools
pip3 install .

to get master. (Perhaps pip install ., depending on your system.)

Patrick Massot (Dec 15 2022 at 21:55):

Should I release a new version?

Riccardo Brasca (Dec 15 2022 at 22:01):

I think it's a good idea. There is discussion somewhere about not forcing people to manually update mathlib-tools (I mean, even more manually than via pip), and the graph is now way better than the file, especially if one has a target in mind.

Patrick Massot (Dec 15 2022 at 22:07):

Please enjoy version 1.3.2

port-progress bot (Dec 16 2022 at 01:52):

mathlib port progress data.rat.order
Ported files: 124/134 (92.5% of total)
Ported lines: 48823/52808 (92.5% of total)
Longest unported chain: 2/27 (92.6% progress)

port-progress bot (Dec 16 2022 at 01:56):

mathlib port progress data.nat.choose.basic
Ported files: 121/131 (92.4% of total)
Ported lines: 48244/52309 (92.2% of total)
Longest unported chain: 2/27 (92.6% progress)

port-progress bot (Dec 16 2022 at 02:00):

mathlib port progress data.nat.prime
Ported files: 140/156 (89.7% of total)
Ported lines: 54274/61461 (88.3% of total)
Longest unported chain: 4/29 (86.2% progress)

port-progress bot (Dec 16 2022 at 02:03):

mathlib port progress data.real.basic
Ported files: 169/233 (72.5% of total)
Ported lines: 61013/91940 (66.4% of total)
Longest unported chain: 8/34 (76.5% progress)

port-progress bot (Dec 16 2022 at 02:07):

mathlib port progress data.fintype.basic
Ported files: 141/183 (77.0% of total)
Ported lines: 54613/82949 (65.8% of total)
Longest unported chain: 17/40 (57.5% progress)

Siddhartha Gadgil (Dec 16 2022 at 02:08):

Patrick Massot said:

Please enjoy version 1.3.2

I still get an error for --exclude-ported

port-progress bot (Dec 16 2022 at 02:11):

mathlib port progress algebra.big_operators.basic
Ported files: 153/215 (71.2% of total)
Ported lines: 57393/94179 (60.9% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Dec 16 2022 at 02:15):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17722/31740 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 16 2022 at 02:19):

mathlib port progress topology.metric_space.basic
Ported files: 203/525 (38.7% of total)
Ported lines: 64564/225113 (28.7% of total)
Longest unported chain: 50/73 (31.5% progress)

Scott Morrison (Dec 16 2022 at 02:23):

@Siddhartha Gadgil, can you show us your command line?

Siddhartha Gadgil (Dec 16 2022 at 02:24):

$ leanproject import-graph --to data.nat.prime --exclude-tactics --reduce --port-status --exclude-ported --show-unused --mathlib4 ~/dev/mathlib4 data.nat.prime.pdf
Usage: leanproject import-graph [OPTIONS] [OUTPUT]
Try 'leanproject import-graph -h' for help.

Error: No such option: --exclude-ported Did you mean --exclude-tactics?

Scott Morrison (Dec 16 2022 at 02:26):

Hmm, I freshly reinstall mathlibtools and it is working for me.

Scott Morrison (Dec 16 2022 at 02:26):

What does leanproject --version give you?

Siddhartha Gadgil (Dec 16 2022 at 02:28):

It gives 1.3.0. This seems to be pip vs pipx problem at my end

Siddhartha Gadgil (Dec 16 2022 at 02:45):

Thanks. Upgrading with pip seems to have fixed it (seems because I ran out of RAM and should get-cache etc first).

port-progress bot (Dec 16 2022 at 03:17):

mathlib port progress all
Ported files: 270/2844 (9.5% of total)
Ported lines: 73717/972514 (7.6% of total)
Longest unported chain: 112/135 (17.0% progress)

Riccardo Brasca (Dec 16 2022 at 09:33):

Is there a reason why docs4#coe_nat_zsmul is not tagged simp?

Kevin Buzzard (Dec 16 2022 at 09:37):

docs#coe_nat_zsmul

Kevin Buzzard (Dec 16 2022 at 09:42):

Interesting! Because of the way attributes have changed I think it could in theory be the case that the lemma is tagged @[simp] later on and the docs don't notice. It's unfortunately really hard to see the attributes on a declaration in lean 4, for some reason. But I would guess that it's more likely that either it was forgotten or it didn't work (eg simp could already prove it). Did you try adding it and linting, or proving it with simp?

Riccardo Brasca (Dec 16 2022 at 09:47):

The linter does not complain, at least the one at the end of the file. I don't know it it's tagged simp somewhere, but in Algebra.GroupPower.Lemmas it's not (and a proof broke because of this).

Riccardo Brasca (Dec 16 2022 at 09:57):

Also, what am I supposed to do with lemmas like docs#zpow_bit0? Should I just remove them or they should be ported anyway? There is a warning saying thy're deprecated. (This has surely been already discussed, sorry)

Kevin Buzzard (Dec 16 2022 at 09:58):

My instinct is just to not port them (and make a porting note saying you skipped them). I don't really see any reason for the functions bit0 and bit1 to exist any more. Re the simp, just add @[simp], I've got no idea why it isn't there.

Riccardo Brasca (Dec 16 2022 at 10:00):

That's also my instict, but I see that a bunch of them are there, like docs4#bit0_add (but no bit0_neg :thinking: ).

Kevin Buzzard (Dec 16 2022 at 10:02):

I personally would like to see bit0 and bit1 removed, they are just there for historical reasons and they confuse new users, so I don't see any reason to port them.

Ruben Van de Velde (Dec 16 2022 at 10:03):

It's a lot easier to throw them all out later than figure out which ones were ported and which ones weren't and restoring them manually if they turn out useful

Scott Morrison (Dec 16 2022 at 10:05):

Please keep them!

Scott Morrison (Dec 16 2022 at 10:06):

We've already had at least one round of adding back in omitted bit0/bit1 lemmas that turned out needed by other lemmas.

Riccardo Brasca (Dec 16 2022 at 10:08):

OK :)

Moritz Doll (Dec 16 2022 at 10:09):

What happens to data.nat.bits? It is one of the two topmost dependencies for order.filter.basic

Siddhartha Gadgil (Dec 16 2022 at 10:42):

Moritz Doll said:

What happens to data.nat.bits? It is one of the two topmost dependencies for order.filter.basic

It is also heading on one of the paths of data.nat.prime(which is getting close)

Scott Morrison (Dec 16 2022 at 10:47):

I think we just port it?

Siddhartha Gadgil (Dec 16 2022 at 11:12):

I believe @Shreyas Srinivas wanted to port this at some point.

Shreyas Srinivas (Dec 16 2022 at 11:13):

Siddhartha Gadgil said:

I believe Shreyas Srinivas wanted to port this at some point.

Yes. However I was told that due to changes in the meaning of 0 and 1 and a bunch of other reasons, this was not to be ported.

Shreyas Srinivas (Dec 16 2022 at 11:16):

Siddhartha Gadgil said:

I believe Shreyas Srinivas wanted to port this at some point.

Relevant threads:

  1. https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/data.2Enat.2Ebits/near/314112248
  2. https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/status.20of.20data.2Enat.2Ebits/near/313758255

Siddhartha Gadgil (Dec 16 2022 at 11:17):

Yes, I saw those. The conclusion was eventually port to Std. But it seems that porting now to Mathlib will be useful.

Shreyas Srinivas (Dec 16 2022 at 11:30):

okay, in that case I will get onto it this Saturday.

Jireh Loreaux (Dec 16 2022 at 13:41):

I think the appropriate way to deal with bit0 and bit1 lemmas is to port them, but also mark them as deprecated.

Riccardo Brasca (Dec 16 2022 at 13:43):

They're already marked deprecated I think.

Shreyas Srinivas (Dec 16 2022 at 13:48):

Quick question: On what branch should i open the PR on mathlib4?

Riccardo Brasca (Dec 16 2022 at 13:49):

You can chose the name you want.

Siddhartha Gadgil (Dec 16 2022 at 13:49):

@Shreyas Srinivas remember to update the wiki from 'No' to 'No WIP ...' if you are working on this.

Shreyas Srinivas (Dec 16 2022 at 13:51):

Riccardo Brasca said:

You can chose the name you want.

Github does not let me create a new branch when creating my pull request. I need to choose one of the existing branches. Screenshot below
image.png

Yaël Dillies (Dec 16 2022 at 13:52):

You should create the branch from the mathlib4 repository, not from your clone of it.

Johan Commelin (Dec 16 2022 at 13:52):

Or push your local work (on a branch) to the ml4 repo

Shreyas Srinivas (Dec 16 2022 at 13:57):

Got it. PR link (https://github.com/leanprover-community/mathlib4/pull/1075)

Siddhartha Gadgil (Dec 16 2022 at 14:05):

You should be pushing directly to the branch on mathlib4, and making a PR to master. For example, you can merge your PR into the mathlib4 branch and then make a PR to master from that.

Jireh Loreaux (Dec 16 2022 at 14:05):

Riccardo, I mean mark the new lemmas involving them as deprecated.

Siddhartha Gadgil (Dec 16 2022 at 14:06):

Jireh Loreaux said:

Riccardo, I mean mark the new lemmas involving them as deprecated.

Sometimes useful lemmas about parity are proved indirectly using bits. We will want to retain these.

Siddhartha Gadgil (Dec 16 2022 at 14:07):

And the proofs of the new lemmas are fine. Just with terminology that should be changed.

Siddhartha Gadgil (Dec 16 2022 at 14:08):

For example, theorem sq_pos_iff (a : R) : 0 < a ^ 2 ↔ a ≠ 0 is something that should remain. The present proof goes via bit0.

Jireh Loreaux (Dec 16 2022 at 14:09):

Right, what I mean is that if bit0 or bit1 appear in the statements, then those lemmas should be deprecated. Appearing in the proofs only is fine.

Shreyas Srinivas (Dec 16 2022 at 14:11):

Siddhartha Gadgil said:

You should be pushing directly to the branch on mathlib4, and making a PR to master. For example, you can merge your PR into the mathlib4 branch and then make a PR to master from that.

Ah okay, for now I have followed the safe option of not directly sending a PR to master. I push to my fork and then send a pull request from github. The PR is on a branch data_nat_bits following a pattern I observed on the mathlib4 repo

Siddhartha Gadgil (Dec 16 2022 at 14:27):

Two PRs will work fine too, but you should merge the first (i.e., the one onto your branch in mathlib4) yourself when you are ready and ask for a review of the second (onto master) when you are ready for that.

port-progress bot (Dec 16 2022 at 18:04):

mathlib port progress data.rat.order
Ported files: 124/134 (92.5% of total)
Ported lines: 48823/52808 (92.5% of total)
Longest unported chain: 2/27 (92.6% progress)

port-progress bot (Dec 16 2022 at 18:08):

mathlib port progress data.nat.choose.basic
Ported files: 123/131 (93.9% of total)
Ported lines: 48830/52309 (93.3% of total)
Longest unported chain: 1/27 (96.3% progress)

port-progress bot (Dec 16 2022 at 18:12):

mathlib port progress data.nat.prime
Ported files: 142/156 (91.0% of total)
Ported lines: 54860/61461 (89.3% of total)
Longest unported chain: 3/29 (89.7% progress)

port-progress bot (Dec 16 2022 at 18:16):

mathlib port progress data.real.basic
Ported files: 174/233 (74.7% of total)
Ported lines: 61957/91940 (67.4% of total)
Longest unported chain: 8/34 (76.5% progress)

port-progress bot (Dec 16 2022 at 18:20):

mathlib port progress data.fintype.basic
Ported files: 143/183 (78.1% of total)
Ported lines: 55199/82949 (66.5% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Dec 16 2022 at 18:24):

mathlib port progress algebra.big_operators.basic
Ported files: 156/215 (72.6% of total)
Ported lines: 58238/94179 (61.8% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Dec 16 2022 at 18:27):

mathlib port progress category_theory.limits.yoneda
Ported files: 47/90 (52.2% of total)
Ported lines: 17722/31740 (55.8% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 16 2022 at 18:32):

mathlib port progress topology.metric_space.basic
Ported files: 212/525 (40.4% of total)
Ported lines: 66543/225113 (29.6% of total)
Longest unported chain: 50/73 (31.5% progress)

port-progress bot (Dec 16 2022 at 19:22):

mathlib port progress all
Ported files: 282/2844 (9.9% of total)
Ported lines: 76135/972603 (7.8% of total)
Longest unported chain: 112/135 (17.0% progress)

Thomas Murrills (Dec 16 2022 at 21:06):

Should grey files be ported? For example, if you see a grey file kind of high up in the graph with all its dependencies ported and not at the top of a long grey chain, should you just try to port it instead of waiting for/coming up with a refactor?

Jireh Loreaux (Dec 16 2022 at 21:07):

I would say that it depends on the utility of the refactor. So, perhaps, but not necessarily.

Thomas Murrills (Dec 16 2022 at 21:10):

Hmm. Is there a way for me as a person unfamiliar with the lay of the land of mathlib dependencies to judge that? (Should I ask somewhere on a per-file basis?)

Thomas Murrills (Dec 16 2022 at 21:10):

If not I'll just stick to attacking cyan bubbles :)

Jireh Loreaux (Dec 16 2022 at 21:13):

If you have a refactor in mind for a series of grey bubbles, I would suggest it here and see what people think.

Thomas Murrills (Dec 16 2022 at 21:15):

If I don't have one in mind, but think that I can port a grey bubble without too much trouble, should I go for it?

Jireh Loreaux (Dec 16 2022 at 21:23):

Yes, I would. (Unless grey means that not all dependencies have been satisfied; does cyan override grey?)

Scott Morrison (Dec 16 2022 at 23:03):

Siddhartha Gadgil said:

Shreyas Srinivas remember to update the wiki from 'No' to 'No WIP ...' if you are working on this.

Actually, I think people probably shouldn't be doing this. Just open a preliminary PR asap. We're soon not going to be using the #port-status wiki at all, and it causes endless problems that people edit it in new and exciting ways that the tool can't understand. :-) For now I'd prefer the transitions to simply be:

No---> No mathlib4#nnn abcdef1234 ---> Yes mathlib4#nnn abcdef1234.

Scott Morrison (Dec 16 2022 at 23:05):

Thomas Murrills said:

If I don't have one in mind, but think that I can port a grey bubble without too much trouble, should I go for it?

Yes, unless you are a mathlib3 expert who likes to refactor, you should just ignore the gray shading and port these files as you would any other.

Moritz Doll (Dec 17 2022 at 00:45):

If the refactors are too close to the porting wave, then they might cause more delays. In the end we have to port all files, so we don't really gain anything by refactoring (for the port at least). If the split/refactor is good regardless of the port, then it can be done before the porting wave hits it or afterwards.

Moritz Doll (Dec 17 2022 at 00:47):

Can we have order.filter.basic as a new port progress target when the natural numbers targets are reached?

Shreyas Srinivas (Dec 17 2022 at 01:23):

Moritz Doll said:

If the refactors are too close to the porting wave, then they might cause more delays. In the end we have to port all files, so we don't really gain anything by refactoring (for the port at least). If the split/refactor is good regardless of the port, then it can be done before the porting wave hits it or afterwards.

I am working on data.nat.bits and some of its dependencies. I don't expect to be finished until tomorrow night. I apologise if I am holding things up.

Scott Morrison (Dec 17 2022 at 08:02):

Just a heads up to everyone about current top priorities for the port.

  1. Data.Rat.Defs: @Mario Carneiro is working on add_def'. Anyone could have a look at mul_def and inv_def, and either fix the proofs or ask Mario to do them too.
  2. Data.List.Basic: this file is huge, and broken all over, and is the biggest blocker to important progress. Pick a random section and hack away, please. This one will take a lot of work.
  3. Order.CompleteLattice is also blocking lots of important ports, however this one is nearly done: if someone could lint, and double check names, we should be close to merging this one.
  4. We have a lot on the #queue4, which I'll try to get to tonight, but if other maintainers could try to clear this a bit that would be great.

Kevin Buzzard (Dec 17 2022 at 09:00):

I do not like this approach of "fix data.list.basic". I find it very depressing to work on something and then to discover that someone else did it too -- I value my time and don't like seeing it wasted, and it's happened twice before to me. What is a better workflow? This is all moot today because I'm at a family do all day but in general I'm interested in better ways to manage situations like this because term is over now and I really want to help. Can we perhaps have a dedicated thread for every "active" file and people working on it should post to the thread saying things like "ok I've just pulled and I'm looking at lines 1234-2000 for the next hour"?

Kevin Buzzard (Dec 17 2022 at 09:01):

The #queue4 job is of course certainly something I could do; my comments above don't apply to this important task

Scott Morrison (Dec 17 2022 at 09:17):

@Kevin Buzzard, okay, lets use https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/Data.2EList.2EBasic.

Scott Morrison (Dec 17 2022 at 09:21):

Another approach to this problem is to commit really often (like every error you fix). We squash merge, so there's no downside to having a complicated git history. Whoever commits more frequently wins. :-)

Reid Barton (Dec 17 2022 at 09:40):

Then you also need to pull the branch every time you are about to fix an error

Scott Morrison (Dec 17 2022 at 09:48):

Or just notice that someone pushed after fixing at most one error (because you get notified when you try to push).

Patrick Massot (Dec 17 2022 at 10:06):

Then it would be nice if people learn to type git pull --rebase.

Patrick Massot (Dec 17 2022 at 10:06):

So that the history isn't needlessly awful.

Scott Morrison (Dec 17 2022 at 10:13):

I have to admit I've never understood why people care about histories when we are just squashing the PR immediately afterwards.

Scott Morrison (Dec 17 2022 at 10:13):

Rewriting history when multiple people are working is just making life miserable, no?

Scott Morrison (Dec 17 2022 at 10:14):

The only downside I've ever felt was that it takes up space on the PR page when there are lots of commits.

Johan Commelin (Dec 17 2022 at 10:14):

git pull --rebase only rewrites local history.

Johan Commelin (Dec 17 2022 at 10:14):

So it doesn't make the life of other people miserable

Scott Morrison (Dec 17 2022 at 10:15):

But the whole point of my suggestion was that you push your branch after fixing each individual lemma. So there is never any "local history".

Johan Commelin (Dec 17 2022 at 10:15):

There is one commit of local history.

Johan Commelin (Dec 17 2022 at 10:16):

And with git pull --rebase you make the commit appear at the end of the current global history.

Scott Morrison (Dec 17 2022 at 10:16):

And what does the --rebase do? Oh, you mean it avoids having a little diamond in the history.

Scott Morrison (Dec 17 2022 at 10:16):

I'm still unsure how that could be worth having to type --rebase... :-)

Johan Commelin (Dec 17 2022 at 10:17):

Well, at least with my config, the alternative is that I have to agree to a merge commit.

Scott Morrison (Dec 17 2022 at 10:17):

Ah, sure, I guess that is two extra keystrokes.

Scott Morrison (Dec 17 2022 at 10:18):

(for me, an editor pops up, and I hit cmd-w to make it go away again)

Scott Morrison (Dec 17 2022 at 10:19):

I have mul_def in the Data.Rat.Defs down to the following gory goal:

 Int.div n₁ (Nat.gcd (Int.natAbs n₁) d₂) * Int.div n₂ (Nat.gcd d₁ (Int.natAbs n₂)) * (d₁ * d₂) =
  n₁ * n₂ * (d₂ / (Nat.gcd (Int.natAbs n₁) d₂) * (d₁ / (Nat.gcd d₁ (Int.natAbs n₂))))

Scott Morrison (Dec 17 2022 at 10:19):

It is "just" commutativity and associativity of multiplication and exact division in .

Patrick Massot (Dec 17 2022 at 10:22):

You can teach git that git p means git pull --rebase.

Scott Morrison (Dec 17 2022 at 10:24):

Okay, I'll try :-)

Sebastian Ullrich (Dec 17 2022 at 10:30):

There's also

git config pull.rebase true

Sebastian Ullrich (Dec 17 2022 at 10:31):

Add --global to affect all repos

Scott Morrison (Dec 17 2022 at 10:47):

Okay, I've finished mul_def and inv_def in Data.Rat.Defs.

port-progress bot (Dec 17 2022 at 18:05):

mathlib port progress data.rat.order
Ported files: 124/134 (92.5% of total)
Ported lines: 48823/52808 (92.5% of total)
Longest unported chain: 2/27 (92.6% progress)

port-progress bot (Dec 17 2022 at 18:08):

mathlib port progress data.nat.choose.basic
Ported files: 124/131 (94.7% of total)
Ported lines: 49191/52309 (94.0% of total)
Longest unported chain: 1/27 (96.3% progress)

port-progress bot (Dec 17 2022 at 18:11):

mathlib port progress data.nat.prime
Ported files: 142/156 (91.0% of total)
Ported lines: 54860/61461 (89.3% of total)
Longest unported chain: 3/29 (89.7% progress)

port-progress bot (Dec 17 2022 at 18:15):

mathlib port progress data.real.basic
Ported files: 174/233 (74.7% of total)
Ported lines: 61957/91940 (67.4% of total)
Longest unported chain: 8/34 (76.5% progress)

port-progress bot (Dec 17 2022 at 18:19):

mathlib port progress data.fintype.basic
Ported files: 143/183 (78.1% of total)
Ported lines: 55199/82949 (66.5% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Dec 17 2022 at 18:23):

mathlib port progress algebra.big_operators.basic
Ported files: 157/215 (73.0% of total)
Ported lines: 58599/94179 (62.2% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Dec 17 2022 at 18:27):

mathlib port progress category_theory.limits.yoneda
Ported files: 48/92 (52.2% of total)
Ported lines: 17705/31944 (55.4% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 17 2022 at 18:31):

mathlib port progress topology.metric_space.basic
Ported files: 213/525 (40.6% of total)
Ported lines: 66904/225113 (29.7% of total)
Longest unported chain: 50/73 (31.5% progress)

port-progress bot (Dec 17 2022 at 19:21):

mathlib port progress all
Ported files: 286/2845 (10.1% of total)
Ported lines: 76956/972853 (7.9% of total)
Longest unported chain: 112/135 (17.0% progress)

Arien Malec (Dec 17 2022 at 20:53):

Looking at the distance to data.complex.basic from data.real.basic, is there a good reason that data.real.sqrt imports so much of topology?

Mario Carneiro (Dec 17 2022 at 20:54):

it's defined in terms of exp most likely

Mario Carneiro (Dec 17 2022 at 20:56):

oh, it looks like I made an abortive attempt to do it direct from cau_seq but others made it there in the meantime and defined it using abstract nonsense

Mario Carneiro (Dec 17 2022 at 20:57):

see the comments around src#real.sqrt

Mario Carneiro (Dec 17 2022 at 21:00):

looks like it used to be in data.real.basic and it got moved in https://github.com/leanprover-community/mathlib/commit/461865b

Kevin Buzzard (Dec 17 2022 at 21:01):

/-- `x ↦ x ^ n` as an order isomorphism of `ℝ≥0`. -/
def pow_order_iso (n : ) (hn : n  0) : 0 o 0 :=
strict_mono.order_iso_of_surjective (λ x, x ^ n)
  (λ x y h, strict_mono_on_pow hn.bot_lt (zero_le x) (zero_le y) h) $
  (continuous_id.pow _).surjective (tendsto_pow_at_top hn) $
    by simpa [order_bot.at_bot_eq, pos_iff_ne_zero]

is in topology.nnreal.instances (so imports a lot of topology, and as you can see the proof uses continuity) and sqrt on nnreal is now defined to be the inverse of x \mapsto x^2, and then sqrt on real is defined using this.

Mario Carneiro (Dec 17 2022 at 21:02):

I'm inclined to revert 461865b just to take the dependencies out of real.sqrt and use the order_iso thing to prove continuity

Patrick Massot (Dec 17 2022 at 21:58):

port-progress bot said:

mathlib port progress all
Ported files: 286/2845 (10.1% of total)
Ported lines: 76956/972853 (7.9% of total)
Longest unported chain: 112/135 (17.0% progress)

We reached the 10% files milestone! :tada:

Chris Hughes (Dec 18 2022 at 00:35):

data.nat.choose.basic is already ported but it appears on all of these progress reports.

Scott Morrison (Dec 18 2022 at 09:45):

I'll take data.nat.choose.basic off the list.

Kevin Buzzard (Dec 18 2022 at 10:10):

Why don't you add data.complex.basic? Not for any particular reason (so if there is a file which should be added for a good reason then add that instead). The reason I suggest it is that it was pointed out yesterday that this file unnecessarily imports a shedload of topology, so it will focus the mind.

Moritz Doll (Dec 18 2022 at 10:25):

but then the import tree looks horrible. it might be better to have files that have tractable import trees

Kevin Buzzard (Dec 18 2022 at 13:00):

I wondered whether instead it would inspire people to pull the topology out :-)

Kevin Buzzard (Dec 18 2022 at 13:00):

Or even better, work on topology!

port-progress bot (Dec 18 2022 at 18:04):

mathlib port progress data.rat.order
Ported files: 124/134 (92.5% of total)
Ported lines: 48823/52808 (92.5% of total)
Longest unported chain: 2/27 (92.6% progress)

port-progress bot (Dec 18 2022 at 18:08):

mathlib port progress data.nat.prime
Ported files: 142/156 (91.0% of total)
Ported lines: 54860/61461 (89.3% of total)
Longest unported chain: 3/29 (89.7% progress)

port-progress bot (Dec 18 2022 at 18:12):

mathlib port progress data.real.basic
Ported files: 176/233 (75.5% of total)
Ported lines: 63420/91940 (69.0% of total)
Longest unported chain: 8/34 (76.5% progress)

port-progress bot (Dec 18 2022 at 18:16):

mathlib port progress data.fintype.basic
Ported files: 144/183 (78.7% of total)
Ported lines: 56564/82949 (68.2% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Dec 18 2022 at 18:19):

mathlib port progress algebra.big_operators.basic
Ported files: 158/215 (73.5% of total)
Ported lines: 59964/94179 (63.7% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Dec 18 2022 at 18:23):

mathlib port progress order.filter.basic
Ported files: 177/279 (63.4% of total)
Ported lines: 62898/110912 (56.7% of total)
Longest unported chain: 24/47 (48.9% progress)

port-progress bot (Dec 18 2022 at 18:27):

mathlib port progress category_theory.limits.yoneda
Ported files: 48/92 (52.2% of total)
Ported lines: 17705/31944 (55.4% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 18 2022 at 18:31):

mathlib port progress topology.metric_space.basic
Ported files: 215/525 (41.0% of total)
Ported lines: 68367/225126 (30.4% of total)
Longest unported chain: 50/73 (31.5% progress)

port-progress bot (Dec 18 2022 at 19:24):

mathlib port progress all
Ported files: 288/2845 (10.1% of total)
Ported lines: 78419/973149 (8.1% of total)
Longest unported chain: 112/135 (17.0% progress)

Scott Morrison (Dec 18 2022 at 20:49):

If anyone feels like doing it, it looks quite straightforward to remove the finiteness import from order.filter.basic (of course you need to move all the lemmas mentioning finiteness out to order.filter.finite, but there is no collateral damage).

Heather Macbeth (Dec 18 2022 at 22:32):

FWIW, Patrick previously argued against removing the finiteness import from order.filter.basic.

Patrick Massot (Dec 19 2022 at 01:07):

I also don't see the point of trying to make the path to filter.basic shorter. We'll need to port finiteness anyway and, as far as I can tell, having filters sooner won't give us anything since they are not needed for any tactic or urgent teaching. As far as I can tell, getting general purposes tactics and teaching are the only urgent targets.

port-progress bot (Dec 19 2022 at 18:05):

mathlib port progress data.rat.order
Ported files: 124/134 (92.5% of total)
Ported lines: 48823/52808 (92.5% of total)
Longest unported chain: 2/27 (92.6% progress)

port-progress bot (Dec 19 2022 at 18:08):

mathlib port progress data.nat.prime
Ported files: 144/156 (92.3% of total)
Ported lines: 56055/61461 (91.2% of total)
Longest unported chain: 3/29 (89.7% progress)

port-progress bot (Dec 19 2022 at 18:12):

mathlib port progress data.real.basic
Ported files: 180/233 (77.3% of total)
Ported lines: 65503/91940 (71.2% of total)
Longest unported chain: 8/34 (76.5% progress)

port-progress bot (Dec 19 2022 at 18:16):

mathlib port progress data.fintype.basic
Ported files: 144/183 (78.7% of total)
Ported lines: 56564/82976 (68.2% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Dec 19 2022 at 18:20):

mathlib port progress algebra.big_operators.basic
Ported files: 160/215 (74.4% of total)
Ported lines: 61289/94221 (65.0% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Dec 19 2022 at 18:24):

mathlib port progress order.filter.basic
Ported files: 180/279 (64.5% of total)
Ported lines: 64561/110939 (58.2% of total)
Longest unported chain: 24/47 (48.9% progress)

port-progress bot (Dec 19 2022 at 18:28):

mathlib port progress category_theory.limits.yoneda
Ported files: 48/92 (52.2% of total)
Ported lines: 17705/31944 (55.4% of total)
Longest unported chain: 19/36 (47.2% progress)

port-progress bot (Dec 19 2022 at 18:32):

mathlib port progress topology.metric_space.basic
Ported files: 219/525 (41.7% of total)
Ported lines: 70450/225203 (31.3% of total)
Longest unported chain: 50/73 (31.5% progress)

port-progress bot (Dec 19 2022 at 19:22):

mathlib port progress all
Ported files: 295/2846 (10.4% of total)
Ported lines: 81013/973772 (8.3% of total)
Longest unported chain: 112/135 (17.0% progress)

Heather Macbeth (Dec 20 2022 at 01:07):

data.real.cau_seq is now available for porting! It should be a fun one.

Scott Morrison (Dec 20 2022 at 12:00):

If anyone is looking for suggestions about high priority work at this moment:

  • Data.Rat.Order in mathlib4#1116 appears to have just one more sorry, which I think is just a matter of basic logic.
  • Data.Nat.Bits in mathlib4#1095 needs polishing/review/merging
  • Data.List.Basic still needs a fair bit of work (I think?)

Mario Carneiro (Dec 20 2022 at 12:00):

I'm going to work on Data.Rat.Order now

Scott Morrison (Dec 20 2022 at 12:02):

After those:

Moritz Doll (Dec 20 2022 at 12:29):

Data.Fin.Basic is extremely long (~3000 loc) and has lots of errors still

Johan Commelin (Dec 20 2022 at 13:05):

I pushed some stuff to

feat: port Algebra.Hom.Aut #1111

cc @Antoine Labelle

port-progress bot (Dec 20 2022 at 18:04):

mathlib port progress data.rat.order
Ported files: 126/134 (94.0% of total)
Ported lines: 49464/52808 (93.7% of total)
Longest unported chain: 1/27 (96.3% progress)

port-progress bot (Dec 20 2022 at 18:08):

mathlib port progress data.nat.prime
Ported files: 145/156 (92.9% of total)
Ported lines: 57089/61461 (92.9% of total)
Longest unported chain: 3/29 (89.7% progress)

port-progress bot (Dec 20 2022 at 18:12):

mathlib port progress data.real.basic
Ported files: 186/233 (79.8% of total)
Ported lines: 68256/91940 (74.2% of total)
Longest unported chain: 8/34 (76.5% progress)

port-progress bot (Dec 20 2022 at 18:16):

mathlib port progress data.fintype.basic
Ported files: 146/183 (79.8% of total)
Ported lines: 57663/82976 (69.5% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Dec 20 2022 at 18:19):

mathlib port progress algebra.big_operators.basic
Ported files: 162/215 (75.3% of total)
Ported lines: 62388/94221 (66.2% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Dec 20 2022 at 18:23):

mathlib port progress order.filter.basic
Ported files: 186/279 (66.7% of total)
Ported lines: 67314/110939 (60.7% of total)
Longest unported chain: 24/47 (48.9% progress)

port-progress bot (Dec 20 2022 at 18:27):

mathlib port progress category_theory.limits.yoneda
Ported files: 49/92 (53.3% of total)
Ported lines: 18038/31944 (56.5% of total)
Longest unported chain: 18/36 (50.0% progress)

port-progress bot (Dec 20 2022 at 18:31):

mathlib port progress topology.metric_space.basic
Ported files: 229/525 (43.6% of total)
Ported lines: 74858/225203 (33.2% of total)
Longest unported chain: 50/73 (31.5% progress)

port-progress bot (Dec 20 2022 at 19:21):

mathlib port progress all
Ported files: 309/2846 (10.9% of total)
Ported lines: 86118/973772 (8.8% of total)
Longest unported chain: 112/135 (17.0% progress)

Johan Commelin (Dec 20 2022 at 19:45):

port-progress bot said:

| mathlib port progress | data.rat.order | |

I just kicked this one on the queue. Not sure why it's listed as 126/134.

Kevin Buzzard (Dec 20 2022 at 19:57):

Is it to do with some random early files which are in Std and are not being ported, or something?

Mario Carneiro (Dec 20 2022 at 20:22):

We hit our first second milestone, data.rat.order :tada: :tada: :tada:

Johan Commelin (Dec 20 2022 at 20:25):

What are the milestones? (It's not the first item on Scott's list of targets... he's already removed others before.)

Mario Carneiro (Dec 20 2022 at 20:26):

oh, I guess I missed that / forgot

Mario Carneiro (Dec 20 2022 at 20:27):

ah right, algebra.order.field.defs is a previous major milestone, so this is our second

Johan Commelin (Dec 20 2022 at 20:30):

Chris Hughes said:

data.nat.choose.basic is already ported but it appears on all of these progress reports.

This one was ticked of recently as well.

Mario Carneiro (Dec 20 2022 at 20:30):

Oh, I thought that one was still ahead

Mario Carneiro (Dec 20 2022 at 20:31):

even better

Scott Morrison (Dec 21 2022 at 05:24):

Thanks to some great work by @Mario Carneiro and @David Renshaw, polyrith and tauto are now available in mathlib4!

Scott Morrison (Dec 21 2022 at 05:24):

tauto will see some further improvements after lean4#1963 is resolved, so please don't rush off to restore all the -- Porting note: tautos quite yet. :-)

Johan Commelin (Dec 21 2022 at 11:06):

@Scott Morrison Could you please add algebra.order.floor as a target? It's a node with high in-degree.

David Renshaw (Dec 21 2022 at 12:27):

and tauto are now available in mathlib4!

And note that mathlib4's tauto does not try to apply symmetry lemmas, so it's not yet quite as powerful as mathlib3's tauto. Once the solve_by_elim improvements in https://github.com/leanprover-community/mathlib4/pull/856 land, the gap will be closed somewhat.

port-progress bot (Dec 21 2022 at 12:31):

mathlib port progress algebra.order.floor
Ported files: 176/196 (89.8% of total)
Ported lines: 65501/75353 (86.9% of total)
Longest unported chain: 3/31 (90.3% progress)

port-progress bot (Dec 21 2022 at 18:05):

mathlib port progress data.nat.prime
Ported files: 147/156 (94.2% of total)
Ported lines: 57609/61673 (93.4% of total)
Longest unported chain: 1/29 (96.6% progress)

port-progress bot (Dec 21 2022 at 18:08):

mathlib port progress data.real.basic
Ported files: 192/235 (81.7% of total)
Ported lines: 69575/92386 (75.3% of total)
Longest unported chain: 8/34 (76.5% progress)

Ruben Van de Velde (Dec 21 2022 at 18:12):

port-progress bot said:

mathlib port progress data.nat.prime
Ported files: 147/156 (94.2% of total)
Ported lines: 57609/61673 (93.4% of total)
Longest unported chain: 1/29 (96.6% progress)

Does this mean the only remaining blocker is nat.sqrt?

port-progress bot (Dec 21 2022 at 18:12):

mathlib port progress data.fintype.basic
Ported files: 146/183 (79.8% of total)
Ported lines: 57909/83012 (69.8% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Dec 21 2022 at 18:16):

mathlib port progress algebra.order.floor
Ported files: 176/196 (89.8% of total)
Ported lines: 65747/75389 (87.2% of total)
Longest unported chain: 3/31 (90.3% progress)

port-progress bot (Dec 21 2022 at 18:20):

mathlib port progress algebra.big_operators.basic
Ported files: 162/215 (75.3% of total)
Ported lines: 62634/94257 (66.5% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Dec 21 2022 at 18:24):

mathlib port progress order.filter.basic
Ported files: 189/279 (67.7% of total)
Ported lines: 68094/110975 (61.4% of total)
Longest unported chain: 24/47 (48.9% progress)

port-progress bot (Dec 21 2022 at 18:28):

mathlib port progress category_theory.limits.yoneda
Ported files: 50/92 (54.3% of total)
Ported lines: 18263/31944 (57.2% of total)
Longest unported chain: 18/36 (50.0% progress)

port-progress bot (Dec 21 2022 at 18:32):

mathlib port progress data.complex.basic
Ported files: 237/576 (41.1% of total)
Ported lines: 76807/243115 (31.6% of total)
Longest unported chain: 56/79 (29.1% progress)

Kevin Buzzard (Dec 21 2022 at 18:34):

port-progress bot said:

mathlib port progress data.complex.basic
Ported files: 237/576 (41.1% of total)
Ported lines: 76807/243115 (31.6% of total)
Longest unported chain: 56/79 (29.1% progress)

A new challenge appeared!

port-progress bot (Dec 21 2022 at 18:36):

mathlib port progress topology.metric_space.basic
Ported files: 235/525 (44.8% of total)
Ported lines: 76140/225283 (33.8% of total)
Longest unported chain: 50/73 (31.5% progress)

Ruben Van de Velde (Dec 21 2022 at 18:43):

port-progress bot said:

mathlib port progress topology.metric_space.basic
Ported files: 235/525 (44.8% of total)
Ported lines: 76140/225283 (33.8% of total)
Longest unported chain: 50/73 (31.5% progress)

Two new challenges!

Heather Macbeth (Dec 21 2022 at 18:45):

Can I put in a request (again) for linear_algebra.basic as another new challenge?

port-progress bot (Dec 21 2022 at 19:30):

mathlib port progress all
Ported files: 319/2847 (11.2% of total)
Ported lines: 88221/975125 (9.0% of total)
Longest unported chain: 112/135 (17.0% progress)

port-progress bot (Dec 21 2022 at 22:48):

mathlib port progress linear_algebra.basic
Ported files: 213/386 (55.2% of total)
Ported lines: 72918/153439 (47.5% of total)
Longest unported chain: 37/60 (38.3% progress)

Scott Morrison (Dec 21 2022 at 22:51):

Just a heads up to everyone that the port-progress-bot will not be running between the 23rd and 30th.

Kevin Buzzard (Dec 21 2022 at 22:51):

is it going skiing?

Scott Morrison (Dec 21 2022 at 22:52):

If someone would like to adopt it, the necessary steps are:

  • have someplace that can host the PDF files, that a script running in cron can push to without interaction.
  • a server that can run a script from cron, on which leanproject import-graph works properly (some people report getting low-resolution images).

Kevin Buzzard (Dec 21 2022 at 22:52):

Maybe it's time for another doomed attempt at my end to actually get my computer to produce these graphs myself.

Eric Wieser (Dec 21 2022 at 22:53):

I can likely get this working on GitHub actions when I get some time

Kevin Buzzard (Dec 21 2022 at 23:03):

Ok so I've got closer than ever before:

buzzard@brutus:~/lean-projects/mathlib/scripts$ leanproject --version
leanproject, version 1.3.2
buzzard@brutus:~/lean-projects/mathlib/scripts$ leanproject import-graph --to algebra.order.floor --exclude-tactics --reduce --port-status --exclude-ported --show-unused --mathlib4 ~/dev/mathlib4 algebra.order.floor.pdf

works but gives me the attached pdf algebra.order.floor.pdf which has far more nodes in it than the pdf file posted a few hours ago. What am I doing wrong?

Scott Morrison (Dec 21 2022 at 23:06):

Are you running on an ancient mathlib?

Scott Morrison (Dec 21 2022 at 23:06):

algebra.group.with_one doesn't exist anymore, it was split a while back.

Kevin Buzzard (Dec 21 2022 at 23:19):

ha ha I'm on a branch (I was reviewing mathlib3 PRs earlier) and the branch was coming off a super-old master :-)

Kevin Buzzard (Dec 21 2022 at 23:24):

It works! :tada: Have a nice holiday port-progress-bot! And thanks Scott!

Sarah Smith (Dec 22 2022 at 00:41):

Mario Carneiro said:

We hit our first second milestone, data.rat.order :tada: :tada: :tada:

We had to pause on positivity and norm_num(still needs division) until data.rat.order ported :smile: but they can be completed now! Would anyone @mathlib mentees be interested in finishing these? Here are placeholder issues: 1100, 1101, and 1102

Eric Rodriguez (Dec 22 2022 at 00:42):

when trying to run the port status script, I get this error a lot:

image.png

do people know why this is? @Eric Wieser I think you wrote this

Eric Wieser (Dec 22 2022 at 00:44):

Your git is more than a year old

Eric Rodriguez (Dec 22 2022 at 01:00):

yikes

Eric Rodriguez (Dec 22 2022 at 01:02):

wait no, it's on 2.39.0

Eric Wieser (Dec 22 2022 at 01:04):

Oh hmm

Eric Wieser (Dec 22 2022 at 01:05):

What OS?

Eric Rodriguez (Dec 22 2022 at 01:05):

macos

Eric Wieser (Dec 22 2022 at 01:05):

Does it work for you on gitpod?

Eric Rodriguez (Dec 22 2022 at 01:06):

how can I run the script on gitpod? i pretty much just edit lean on gitpod

Eric Rodriguez (Dec 22 2022 at 01:06):

and lean3 at that

Eric Wieser (Dec 22 2022 at 01:07):

You can open the vscode terminal in gitpod and then you have a command line

Eric Wieser (Dec 22 2022 at 01:09):

And at least for the mathlib3 gitpod that will already have everything installed

Eric Rodriguez (Dec 22 2022 at 01:11):

yeah okay it did work (although i did need to pip3 install mathlibtools)

Eric Rodriguez (Dec 22 2022 at 01:12):

tracking down a changelog for git itself is challenging as well :/

Eric Wieser (Dec 22 2022 at 01:12):

Is the git version there older or newer?

Eric Wieser (Dec 22 2022 at 01:13):

(I'll split this zulip thread when I'm on my laptop tomorrow)

Eric Rodriguez (Dec 22 2022 at 01:13):

2.37.2

Eric Wieser (Dec 22 2022 at 01:15):

Can you downgrade on your Mac / install a newer version on gitpod? Just to check if it's a git change or some weird platform thing

Eric Rodriguez (Dec 22 2022 at 01:23):

gitpod's apt-get doesn't have a new version and brew doesn't have an old one :) what a happy state of affairs. let me ask to see if other people can repro

Eric Wieser (Dec 22 2022 at 01:28):

Git 2.39 release notes say

  • With a bit of header twiddling, use the native regexp library on
    macOS instead of the compat/ one.

Eric Wieser (Dec 22 2022 at 01:29):

Which makes me think it's a platform thing

Eric Rodriguez (Dec 22 2022 at 01:30):

well this is fun... now scripts have to deal with two different styles of regex

Notification Bot (Dec 22 2022 at 01:41):

26 messages were moved from this topic to #mathlib4 > git error from port_status on macOS by Eric Wieser.

David Michael Roberts (Dec 22 2022 at 05:49):

Kevin Buzzard said:

is it going skiing?

Waveski, maybe...

Johan Commelin (Dec 22 2022 at 08:34):

Eric Wieser said:

I can likely get this working on GitHub actions when I get some time

If it doesn't work, I can probably run a cronjob on my server.

Heather Macbeth (Dec 22 2022 at 18:01):

Sarah Smith said:

We had to pause on positivity and norm_num(still needs division) until data.rat.order ported :smile: but they can be completed now! Would anyone mathlib mentees be interested in finishing these? Here are placeholder issues: 1100, 1101, and 1102

For anyone interested in doing the newly-available positivity extensions, let me record what I know. They are harder than the corresponding Lean 3 extensions, because instead of using mk_app you have to work with Qq. For example, compare the positivity extensions for addition in Lean 3:
https://github.com/leanprover-community/mathlib/blob/2f3994e1b117b1e1da49bcfb67334f33460c3ce4/src/tactic/positivity.lean#L417
and in Lean 4:
https://github.com/leanprover-community/mathlib4/blob/master/Mathlib/Tactic/Positivity/Basic.lean#L62

So it would be great if someone who understands Qq can take this on.

port-progress bot (Dec 22 2022 at 18:03):

mathlib port progress data.nat.prime
Ported files: 148/156 (94.9% of total)
Ported lines: 57850/61663 (93.8% of total)
Longest unported chain: 1/29 (96.6% progress)

port-progress bot (Dec 22 2022 at 18:07):

mathlib port progress algebra.order.floor
Ported files: 178/196 (90.8% of total)
Ported lines: 67438/75372 (89.5% of total)
Longest unported chain: 3/31 (90.3% progress)

Johan Commelin (Dec 22 2022 at 18:08):

I just kicked data.nat.prime on the queue. Another target in the bag.

port-progress bot (Dec 22 2022 at 18:11):

mathlib port progress data.real.basic
Ported files: 194/227 (85.5% of total)
Ported lines: 71374/85421 (83.6% of total)
Longest unported chain: 6/34 (82.4% progress)

port-progress bot (Dec 22 2022 at 18:14):

mathlib port progress linear_algebra.basic
Ported files: 220/386 (57.0% of total)
Ported lines: 76083/153413 (49.6% of total)
Longest unported chain: 37/60 (38.3% progress)

port-progress bot (Dec 22 2022 at 18:18):

mathlib port progress data.fintype.basic
Ported files: 147/183 (80.3% of total)
Ported lines: 59540/83002 (71.7% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Dec 22 2022 at 18:22):

mathlib port progress algebra.big_operators.basic
Ported files: 163/215 (75.8% of total)
Ported lines: 64264/94246 (68.2% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Dec 22 2022 at 18:25):

mathlib port progress order.filter.basic
Ported files: 192/279 (68.8% of total)
Ported lines: 70181/110957 (63.3% of total)
Longest unported chain: 24/47 (48.9% progress)

port-progress bot (Dec 22 2022 at 18:29):

mathlib port progress category_theory.limits.yoneda
Ported files: 50/92 (54.3% of total)
Ported lines: 18263/31944 (57.2% of total)
Longest unported chain: 18/36 (50.0% progress)

port-progress bot (Dec 22 2022 at 18:33):

mathlib port progress data.complex.basic
Ported files: 246/576 (42.7% of total)
Ported lines: 80325/243099 (33.0% of total)
Longest unported chain: 56/79 (29.1% progress)

Kevin Buzzard (Dec 22 2022 at 18:35):

For people who are looking for things to port I would urge them to look at the pdfs rather than the output of the port script. Creating PRs which depend on other PRs is fine here, and some of the pdfs represent important goals which we want done sooner rather than later so that more people can use Lean 4 in their work.

port-progress bot (Dec 22 2022 at 18:36):

mathlib port progress topology.metric_space.basic
Ported files: 244/525 (46.5% of total)
Ported lines: 79658/225267 (35.4% of total)
Longest unported chain: 50/73 (31.5% progress)

Johan Commelin (Dec 22 2022 at 18:44):

Aren't files at the top of #port-status very likely to also be in those pdfs?

Johan Commelin (Dec 22 2022 at 18:46):

Anybody with a vague enthusiasm for porting the finiteness hierarchy is very welcome to pour in a lot of energy there. I think it's going to be one of the major next hurdles.

Kevin Buzzard (Dec 22 2022 at 19:23):

Johan Commelin said:

Aren't files at the top of #port-status very likely to also be in those pdfs?

You would have thought so, wouldn't you! But sometimes the porting program can throw up some pretty random things.

port-progress bot (Dec 22 2022 at 19:28):

mathlib port progress all
Ported files: 333/2849 (11.7% of total)
Ported lines: 92744/975641 (9.5% of total)
Longest unported chain: 112/135 (17.0% progress)

David Renshaw (Dec 22 2022 at 21:15):

@Heather Macbeth I can look at positivity tomorrow, if Mario or someone else has not already jumped on it.

Heather Macbeth (Dec 22 2022 at 21:15):

Awesome!!

Heather Macbeth (Dec 22 2022 at 21:15):

I will double-check which extensions are high-priority for me personally, but definitely division, inversion and absolute values.

Heather Macbeth (Dec 23 2022 at 15:35):

I think algebra.order.floor might be ready to port. It shows up with all sorts of crazy imports on

port-progress bot said:

| mathlib port progress | algebra.order.floor | |

like

data.tree
algebra.order.field_power
data.rat.cast
data.meta_defs

but its actual import list is only

import data.int.lemmas
import data.set.intervals.group
import data.set.lattice
import tactic.abel
import tactic.linarith
import tactic.positivity

I think those other imports are transitive imports via the tactic files. So they may well not be needed.

Heather Macbeth (Dec 23 2022 at 15:38):

Or, at least, maybe it's blocked by data.int.lemmas (which itself is blocked by mathlib4#1159), but not by all those other files.

port progress bot (jmc) (Dec 23 2022 at 16:47):

mathlib port progress algebra.order.floor
Ported files: 178/196 (90.8% of total)
Ported lines: 67438/75372 (89.5% of total)
Longest unported chain: 3/31 (90.3% progress)

port progress bot (jmc) (Dec 23 2022 at 16:50):

mathlib port progress data.real.basic
Ported files: 195/227 (85.9% of total)
Ported lines: 71554/85421 (83.8% of total)
Longest unported chain: 6/34 (82.4% progress)

port progress bot (jmc) (Dec 23 2022 at 16:52):

mathlib port progress linear_algebra.basic
Ported files: 223/386 (57.8% of total)
Ported lines: 76721/153413 (50.0% of total)
Longest unported chain: 37/60 (38.3% progress)

port progress bot (jmc) (Dec 23 2022 at 16:54):

mathlib port progress data.fintype.basic
Ported files: 147/183 (80.3% of total)
Ported lines: 59540/83002 (71.7% of total)
Longest unported chain: 17/40 (57.5% progress)

port progress bot (jmc) (Dec 23 2022 at 16:56):

mathlib port progress algebra.big_operators.basic
Ported files: 163/215 (75.8% of total)
Ported lines: 64264/94246 (68.2% of total)
Longest unported chain: 21/44 (52.3% progress)

port progress bot (jmc) (Dec 23 2022 at 16:59):

mathlib port progress order.filter.basic
Ported files: 193/279 (69.2% of total)
Ported lines: 70343/110957 (63.4% of total)
Longest unported chain: 24/47 (48.9% progress)

port progress bot (jmc) (Dec 23 2022 at 17:01):

mathlib port progress category_theory.limits.yoneda
Ported files: 50/92 (54.3% of total)
Ported lines: 18263/31944 (57.2% of total)
Longest unported chain: 18/36 (50.0% progress)

port progress bot (jmc) (Dec 23 2022 at 17:03):

mathlib port progress data.complex.basic
Ported files: 251/577 (43.5% of total)
Ported lines: 81876/243311 (33.7% of total)
Longest unported chain: 56/79 (29.1% progress)

port progress bot (jmc) (Dec 23 2022 at 17:05):

mathlib port progress topology.metric_space.basic
Ported files: 249/525 (47.4% of total)
Ported lines: 81209/225267 (36.1% of total)
Longest unported chain: 50/73 (31.5% progress)

Johan Commelin (Dec 23 2022 at 17:12):

The graphs will start working in an hour or two, once another cron job kicks in.

port progress bot (jmc) (Dec 24 2022 at 06:53):

mathlib port progress algebra.order.floor
Ported files: 178/196 (90.8% of total)
Ported lines: 67438/75372 (89.5% of total)
Longest unported chain: 3/31 (90.3% progress)

port progress bot (jmc) (Dec 24 2022 at 06:55):

mathlib port progress data.real.basic
Ported files: 195/227 (85.9% of total)
Ported lines: 71554/85421 (83.8% of total)
Longest unported chain: 6/34 (82.4% progress)

port progress bot (jmc) (Dec 24 2022 at 06:58):

mathlib port progress linear_algebra.basic
Ported files: 223/386 (57.8% of total)
Ported lines: 76721/153413 (50.0% of total)
Longest unported chain: 37/60 (38.3% progress)

port progress bot (jmc) (Dec 24 2022 at 07:00):

mathlib port progress data.fintype.basic
Ported files: 147/183 (80.3% of total)
Ported lines: 59540/83002 (71.7% of total)
Longest unported chain: 17/40 (57.5% progress)

port progress bot (jmc) (Dec 24 2022 at 07:02):

mathlib port progress algebra.big_operators.basic
Ported files: 163/215 (75.8% of total)
Ported lines: 64264/94246 (68.2% of total)
Longest unported chain: 21/44 (52.3% progress)

port progress bot (jmc) (Dec 24 2022 at 07:04):

mathlib port progress order.filter.basic
Ported files: 193/279 (69.2% of total)
Ported lines: 70343/110969 (63.4% of total)
Longest unported chain: 24/47 (48.9% progress)

port progress bot (jmc) (Dec 24 2022 at 07:07):

mathlib port progress category_theory.limits.yoneda
Ported files: 50/92 (54.3% of total)
Ported lines: 18263/31944 (57.2% of total)
Longest unported chain: 18/36 (50.0% progress)

port progress bot (jmc) (Dec 24 2022 at 07:09):

mathlib port progress data.complex.basic
Ported files: 251/577 (43.5% of total)
Ported lines: 81876/243323 (33.6% of total)
Longest unported chain: 56/79 (29.1% progress)

port progress bot (jmc) (Dec 24 2022 at 07:11):

mathlib port progress topology.metric_space.basic
Ported files: 249/525 (47.4% of total)
Ported lines: 81209/225279 (36.0% of total)
Longest unported chain: 50/73 (31.5% progress)

port progress bot (jmc) (Dec 24 2022 at 07:14):

mathlib port progress all
Ported files: 339/2851 (11.9% of total)
Ported lines: 94267/976193 (9.7% of total)
Longest unported chain: 112/135 (17.0% progress)

Reid Barton (Dec 24 2022 at 07:42):

The graphs don't appear to exist yet.

Johan Commelin (Dec 24 2022 at 07:44):

Hmm, there was a hiccup with the switch to lean 3.50.2

Johan Commelin (Dec 24 2022 at 07:44):

I'll run the graph script again

Riccardo Brasca (Dec 24 2022 at 10:12):

The list The following files are marked as ported, but do not have a SYNCHRONIZED WITH MATHLIB4 label is now huge. What happened to the script?

Eric Wieser (Dec 24 2022 at 10:19):

The yaml file PR numbers are now "wrong", so I'm wary of merging its output

Reid Barton (Dec 24 2022 at 10:20):

Ideally it would not modify existing headers, but it's a pain to work on this script

Eric Wieser (Dec 24 2022 at 10:20):

The script was designed to make the mathlib3 headers match the yaml file

Eric Wieser (Dec 24 2022 at 10:22):

If the yaml file no longer contains the information we want in the headers, we should either add the information back or stop wanting it in the headers

Johan Commelin (Dec 24 2022 at 10:25):

I would be happy with just SYNCHRONIZED WITH MATHLIB4 in a comment in the Lean 3 files.

Johan Commelin (Dec 24 2022 at 10:25):

I don't think the pointers to ml4 PRs are very important.

Riccardo Brasca (Dec 24 2022 at 10:27):

I agree. Sooner or later the PR that ported the file will be obsolete.

Eric Wieser (Dec 24 2022 at 10:32):

Let's update the script then to do that

Eric Wieser (Dec 24 2022 at 10:34):

That should be as simple as removing a line from the inserted comment, and removing the list of PRs from stdout

port progress bot (jmc) (Dec 25 2022 at 08:18):

mathlib port progress algebra.order.floor
Ported files: 180/196 (91.8% of total)
Ported lines: 67933/75372 (90.1% of total)
Longest unported chain: 3/31 (90.3% progress)

port progress bot (jmc) (Dec 25 2022 at 08:20):

mathlib port progress data.real.basic
Ported files: 198/227 (87.2% of total)
Ported lines: 73306/85421 (85.8% of total)
Longest unported chain: 6/34 (82.4% progress)

port progress bot (jmc) (Dec 25 2022 at 08:22):

mathlib port progress linear_algebra.basic
Ported files: 230/386 (59.6% of total)
Ported lines: 79474/153413 (51.8% of total)
Longest unported chain: 37/60 (38.3% progress)

port progress bot (jmc) (Dec 25 2022 at 08:24):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59979/83002 (72.3% of total)
Longest unported chain: 17/40 (57.5% progress)

port progress bot (jmc) (Dec 25 2022 at 08:27):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64703/94246 (68.7% of total)
Longest unported chain: 21/44 (52.3% progress)

port progress bot (jmc) (Dec 25 2022 at 08:29):

mathlib port progress order.filter.basic
Ported files: 198/279 (71.0% of total)
Ported lines: 72588/110969 (65.4% of total)
Longest unported chain: 24/47 (48.9% progress)

port progress bot (jmc) (Dec 25 2022 at 08:31):

mathlib port progress category_theory.limits.yoneda
Ported files: 50/92 (54.3% of total)
Ported lines: 18263/31944 (57.2% of total)
Longest unported chain: 18/36 (50.0% progress)

port progress bot (jmc) (Dec 25 2022 at 08:33):

mathlib port progress data.complex.basic
Ported files: 259/577 (44.9% of total)
Ported lines: 84791/243323 (34.8% of total)
Longest unported chain: 56/79 (29.1% progress)

port progress bot (jmc) (Dec 25 2022 at 08:36):

mathlib port progress topology.metric_space.basic
Ported files: 256/525 (48.8% of total)
Ported lines: 83962/225279 (37.3% of total)
Longest unported chain: 50/73 (31.5% progress)

port progress bot (jmc) (Dec 25 2022 at 08:39):

mathlib port progress all
Ported files: 348/2851 (12.2% of total)
Ported lines: 97300/976224 (10.0% of total)
Longest unported chain: 112/135 (17.0% progress)

Reid Barton (Dec 25 2022 at 10:29):

The graphs don't exist, again--was it supposed to be fixed in general?

Johan Commelin (Dec 25 2022 at 12:16):

Maybe something is wrong with the cronjob...

port progress bot (jmc) (Dec 26 2022 at 09:40):

mathlib port progress algebra.order.floor
Ported files: 180/196 (91.8% of total)
Ported lines: 67933/75372 (90.1% of total)
Longest unported chain: 3/31 (90.3% progress)

port progress bot (jmc) (Dec 26 2022 at 09:42):

mathlib port progress data.real.basic
Ported files: 198/227 (87.2% of total)
Ported lines: 73306/85421 (85.8% of total)
Longest unported chain: 6/34 (82.4% progress)

port progress bot (jmc) (Dec 26 2022 at 09:44):

mathlib port progress linear_algebra.basic
Ported files: 230/386 (59.6% of total)
Ported lines: 79474/153413 (51.8% of total)
Longest unported chain: 37/60 (38.3% progress)

port progress bot (jmc) (Dec 26 2022 at 09:46):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59979/83002 (72.3% of total)
Longest unported chain: 17/40 (57.5% progress)

port progress bot (jmc) (Dec 26 2022 at 09:49):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64703/94246 (68.7% of total)
Longest unported chain: 21/44 (52.3% progress)

port progress bot (jmc) (Dec 26 2022 at 09:51):

mathlib port progress order.filter.basic
Ported files: 198/279 (71.0% of total)
Ported lines: 72588/110969 (65.4% of total)
Longest unported chain: 24/47 (48.9% progress)

port progress bot (jmc) (Dec 26 2022 at 09:53):

mathlib port progress category_theory.limits.yoneda
Ported files: 50/92 (54.3% of total)
Ported lines: 18263/31944 (57.2% of total)
Longest unported chain: 18/36 (50.0% progress)

port progress bot (jmc) (Dec 26 2022 at 09:55):

mathlib port progress data.complex.basic
Ported files: 260/577 (45.1% of total)
Ported lines: 84837/243323 (34.9% of total)
Longest unported chain: 56/79 (29.1% progress)

port progress bot (jmc) (Dec 26 2022 at 09:58):

mathlib port progress topology.metric_space.basic
Ported files: 257/525 (49.0% of total)
Ported lines: 84008/225279 (37.3% of total)
Longest unported chain: 50/73 (31.5% progress)

port progress bot (jmc) (Dec 26 2022 at 10:01):

mathlib port progress all
Ported files: 349/2851 (12.2% of total)
Ported lines: 97346/976237 (10.0% of total)
Longest unported chain: 112/135 (17.0% progress)

Henrik Böving (Dec 26 2022 at 11:31):

If someone want's to tell me whether I did Vector3 right here: https://github.com/leanprover-community/mathlib4/pull/1204 I'll happily start ramping up more PRs, the only reason I haven't yet is because I'm not sure whether what I did is what is expected so I didn't want to do lots of work that I have to revise later again because of a general mistake I'm making.

port progress bot (jmc) (Dec 27 2022 at 07:43):

mathlib port progress algebra.order.floor
Ported files: 180/196 (91.8% of total)
Ported lines: 67950/75389 (90.1% of total)
Longest unported chain: 3/31 (90.3% progress)

port progress bot (jmc) (Dec 27 2022 at 07:46):

mathlib port progress data.real.basic
Ported files: 200/227 (88.1% of total)
Ported lines: 74042/85438 (86.7% of total)
Longest unported chain: 6/34 (82.4% progress)

port progress bot (jmc) (Dec 27 2022 at 07:48):

mathlib port progress linear_algebra.basic
Ported files: 236/386 (61.1% of total)
Ported lines: 81513/153430 (53.1% of total)
Longest unported chain: 37/60 (38.3% progress)

port progress bot (jmc) (Dec 27 2022 at 07:50):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59996/83019 (72.3% of total)
Longest unported chain: 17/40 (57.5% progress)

port progress bot (jmc) (Dec 27 2022 at 07:53):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64720/94263 (68.7% of total)
Longest unported chain: 21/44 (52.3% progress)

port progress bot (jmc) (Dec 27 2022 at 07:55):

mathlib port progress order.filter.basic
Ported files: 199/279 (71.3% of total)
Ported lines: 72748/110986 (65.5% of total)
Longest unported chain: 24/47 (48.9% progress)

port progress bot (jmc) (Dec 27 2022 at 07:57):

mathlib port progress category_theory.limits.yoneda
Ported files: 50/92 (54.3% of total)
Ported lines: 18263/31944 (57.2% of total)
Longest unported chain: 18/36 (50.0% progress)

port progress bot (jmc) (Dec 27 2022 at 07:59):

mathlib port progress data.complex.basic
Ported files: 269/577 (46.6% of total)
Ported lines: 87360/243478 (35.9% of total)
Longest unported chain: 56/79 (29.1% progress)

port progress bot (jmc) (Dec 28 2022 at 10:03):

mathlib port progress algebra.order.floor
Ported files: 180/196 (91.8% of total)
Ported lines: 67950/75389 (90.1% of total)
Longest unported chain: 3/31 (90.3% progress)

port progress bot (jmc) (Dec 28 2022 at 10:05):

mathlib port progress data.real.basic
Ported files: 200/227 (88.1% of total)
Ported lines: 74042/85438 (86.7% of total)
Longest unported chain: 6/34 (82.4% progress)

port progress bot (jmc) (Dec 28 2022 at 10:08):

mathlib port progress linear_algebra.basic
Ported files: 236/386 (61.1% of total)
Ported lines: 81513/153430 (53.1% of total)
Longest unported chain: 37/60 (38.3% progress)

port progress bot (jmc) (Dec 28 2022 at 10:10):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59996/83019 (72.3% of total)
Longest unported chain: 17/40 (57.5% progress)

port progress bot (jmc) (Dec 28 2022 at 10:12):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64720/94263 (68.7% of total)
Longest unported chain: 21/44 (52.3% progress)

port progress bot (jmc) (Dec 28 2022 at 10:14):

mathlib port progress order.filter.basic
Ported files: 199/279 (71.3% of total)
Ported lines: 72748/110986 (65.5% of total)
Longest unported chain: 24/47 (48.9% progress)

port progress bot (jmc) (Dec 28 2022 at 10:16):

mathlib port progress category_theory.limits.yoneda
Ported files: 50/92 (54.3% of total)
Ported lines: 18263/31944 (57.2% of total)
Longest unported chain: 18/36 (50.0% progress)

port progress bot (jmc) (Dec 28 2022 at 10:19):

mathlib port progress data.complex.basic
Ported files: 269/577 (46.6% of total)
Ported lines: 87360/243478 (35.9% of total)
Longest unported chain: 56/79 (29.1% progress)

port progress bot (jmc) (Dec 28 2022 at 10:21):

mathlib port progress topology.metric_space.basic
Ported files: 266/525 (50.7% of total)
Ported lines: 86531/225434 (38.4% of total)
Longest unported chain: 50/73 (31.5% progress)

port progress bot (jmc) (Dec 28 2022 at 10:24):

mathlib port progress all
Ported files: 360/2852 (12.6% of total)
Ported lines: 99942/976704 (10.2% of total)
Longest unported chain: 112/135 (17.0% progress)

Ruben Van de Velde (Dec 28 2022 at 11:54):

Who's getting us to 100,000 lines ported?

Johan Commelin (Dec 28 2022 at 12:04):

Whoever fixes the final linting errors in data.list.basic?

Johan Commelin (Dec 28 2022 at 12:04):

(I'm offline for the next ~4 hrs.)

Riccardo Brasca (Dec 28 2022 at 12:08):

I am having a look

Riccardo Brasca (Dec 28 2022 at 13:57):

I've done a couple of them, but I am stuck on the others. Most of them about the LHS that can be simplified using results in core/std. In all cases replacing the LHS with the simplified version seems a bad idea, but using priority doesn't work (maybe results always apply first?).

Chris Hughes (Dec 28 2022 at 14:00):

simp priority in Lean3 was not that useful, maybe it changed in Lean4, but in Lean3 it applied simp lemmas in order of the depth of the subexpression they applied to first, and then priority second or something like that

Riccardo Brasca (Dec 28 2022 at 14:03):

To give a precise example, in std there is

@[simp] theorem getLast_eq_getLastD (a l h) : @getLast α (a::l) h = getLastD l a := by

And this breaks

@[simp]
theorem getLast_cons {a : α} {l : List α} :
     h : l  nil, getLast (a :: l) (cons_ne_nil a l) = getLast l h := by

with

#check @List.getLast_cons /- Left-hand side simplifies from
  List.getLast (a :: l) (_ : a :: l ≠ [])
to
  List.getLastD l a
using
  simp only [List.getLast_eq_getLastD]
Try to change the left-hand side to the simplified term!

Riccardo Brasca (Dec 28 2022 at 14:04):

I don' think changing the LHS is a good idea

Chris Hughes (Dec 28 2022 at 14:08):

But when does getLast_cons apply as a simp lemma anyway. How would you infer h : l ne nil?

Reid Barton (Dec 28 2022 at 14:19):

I guess with some kind of simp [h] or simp [*]

Reid Barton (Dec 28 2022 at 14:37):

I feel like we don't have a clear path forward with this simp stuff. Is it unreasonable to hope that the simp set will be basically the same between mathlib 3 and mathlib 4? Are there too many other changes to how simp works for instance?

Reid Barton (Dec 28 2022 at 14:38):

Obviously all we really care about is that simp still closes all the goals it used to close... but it's hard to know what effect removing specific simp lemmas would have.

Riccardo Brasca (Dec 28 2022 at 14:45):

Here the difference is the result in std I guess. We now have List.getLastD, and I think the Lean3 analogue is docs#list.ilast', but there is no simp lemma analogue to getLast_eq_getLastD. So I think that is't not because simp is different, there is a new simp lemma.

Reid Barton (Dec 28 2022 at 14:46):

Right. It's tempting to say: just get rid of all the new simp lemmas. But maybe it's not the right answer

Mario Carneiro (Dec 28 2022 at 14:48):

in the presence of the new simp lemma, the equivalent of getLast_cons is \all h : l != [], getLastD a l = getLast l h

Mario Carneiro (Dec 28 2022 at 14:51):

which does not look like a good global simp lemma, since while not properly looping would still fight against getLast_eq_getLastD when l is of the form b :: l' since b :: l' != [] is simp-provable. I think this should just be used as a local simp lemma

Reid Barton (Dec 28 2022 at 14:54):

What about removing simp from getLast_eq_getLastD?

Reid Barton (Dec 28 2022 at 14:54):

It seems like while there's a huge amount of porting remaining to be done is the wrong time to try to make large changes to the simp set?

Mario Carneiro (Dec 28 2022 at 14:56):

I would like to discuss this in the context of concrete breakage, rather than adding any blanket rules along the lines of "no new simp lemmas"

Mario Carneiro (Dec 28 2022 at 14:57):

I don't think this is a large change to the simp set. list.last is a rarely used function

Reid Barton (Dec 28 2022 at 14:57):

I was going to say just the opposite--these questions are going to come up over and over (I think in Data.List.Basic there were already like 50 of these simp_nf linter errors?) and we need a way to make progress on them that doesn't depend on a fine analysis of each one individually

Mario Carneiro (Dec 28 2022 at 14:58):

again, we can't make those judgments without staring at a few broken simp calls first

Mario Carneiro (Dec 28 2022 at 14:58):

we can roll things back if the fallout of some change looks to be too bad

Reid Barton (Dec 28 2022 at 14:58):

I agree a policy like "no new simp lemmas" is the wrong approach, but there has to be some kind of general goal

Reid Barton (Dec 28 2022 at 14:59):

because otherwise I think we will waste a lot of time now contemplating what to do about simp lemmas, and also a lot of time later when all the simps break

Reid Barton (Dec 28 2022 at 14:59):

I'd rather avoid at least one of those!

Mario Carneiro (Dec 28 2022 at 15:01):

I think it's fine to lean toward keeping all the old annotations (in mathlib), and reverting changes in core/std that cause breakage, but std should not be explicitly backward compatibly tied to mathlib in the same way as mathlib4

Mario Carneiro (Dec 28 2022 at 15:01):

that's why #align directives are in mathlib4, not std, even for files that have been basically completely moved over

Mario Carneiro (Dec 28 2022 at 15:06):

Reid Barton said:

(I think in Data.List.Basic there were already like 50 of these simp_nf linter errors?)

By the way I have noticed this generally in lean 4, the simp_nf linter seems to fire a lot even when there have been no significant changes. I think it's detecting non-confluence in the original lean 3 simp set

Mario Carneiro (Dec 28 2022 at 15:11):

Mario Carneiro said:

in the presence of the new simp lemma, the equivalent of getLast_cons is \all h : l != [], getLastD a l = getLast l h

thinking about this some more, I think it's not even a good simp lemma if you set aside the confluence issues - if I were in the middle of a proof I would rather have the LHS in the goal than the RHS, unless I wanted to specifically prove that the expression does not depend on a. The h argument is more problematic because it will block further rewrites

Reid Barton (Dec 28 2022 at 15:11):

In the normalize thread it sounded like that might be due in part to simp no longer applying the most recent simp lemmas first

Mario Carneiro (Dec 28 2022 at 15:12):

it uses a discrimination tree instead of going over everything in order. This is a huge performance win, one of the main reasons we think lean 4 will be faster on mathlib, but it means you can't rely on declaration order as priority

Reid Barton (Dec 28 2022 at 15:13):

How hard would it be to collect the data of all simp lemmas that are actually used by a simp (without only) in mathlib 3?

Mario Carneiro (Dec 28 2022 at 15:13):

as usual, that's the kind of thing that lean 4 makes trivial but requires heroic effort to extract in lean 3

Mario Carneiro (Dec 28 2022 at 15:14):

which is annoying when it's needed for a port

Mario Carneiro (Dec 28 2022 at 15:14):

we could squeeze all simps in mathlib by regex...?

Reid Barton (Dec 28 2022 at 15:14):

maybe with lean -D trace.simplify.rewrite=true and processing a few GBs of text?

Mario Carneiro (Dec 28 2022 at 15:15):

The squeeze_simp tactic already implements most of that functionality, so it's just a matter of calling it everywhere

Mario Carneiro (Dec 28 2022 at 15:16):

unfortunately I think the error rate is too high for it to be applied at scale

Reid Barton (Dec 28 2022 at 15:16):

Ah yeah because you want to exclude explicitly-requested simp lemmas anyways

Mario Carneiro (Dec 28 2022 at 15:16):

specifically, it often produces unparsable terms

Mario Carneiro (Dec 28 2022 at 15:17):

which is not really its fault, lean 3 has a roundtripping issue in general

port progress bot (jmc) (Dec 29 2022 at 08:05):

mathlib port progress algebra.order.floor
Ported files: 180/196 (91.8% of total)
Ported lines: 67950/75389 (90.1% of total)
Longest unported chain: 3/31 (90.3% progress)

port progress bot (jmc) (Dec 29 2022 at 08:08):

mathlib port progress data.real.basic
Ported files: 202/227 (89.0% of total)
Ported lines: 74252/85438 (86.9% of total)
Longest unported chain: 6/34 (82.4% progress)

port progress bot (jmc) (Dec 29 2022 at 08:10):

mathlib port progress linear_algebra.basic
Ported files: 238/386 (61.7% of total)
Ported lines: 82208/153441 (53.6% of total)
Longest unported chain: 37/60 (38.3% progress)

port progress bot (jmc) (Dec 29 2022 at 08:12):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59996/83019 (72.3% of total)
Longest unported chain: 17/40 (57.5% progress)

port progress bot (jmc) (Dec 29 2022 at 08:14):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64720/94263 (68.7% of total)
Longest unported chain: 21/44 (52.3% progress)

port progress bot (jmc) (Dec 29 2022 at 08:16):

mathlib port progress order.filter.basic
Ported files: 199/279 (71.3% of total)
Ported lines: 72748/110997 (65.5% of total)
Longest unported chain: 24/47 (48.9% progress)

port progress bot (jmc) (Dec 29 2022 at 08:19):

mathlib port progress category_theory.limits.yoneda
Ported files: 50/92 (54.3% of total)
Ported lines: 18263/31944 (57.2% of total)
Longest unported chain: 18/36 (50.0% progress)

port progress bot (jmc) (Dec 29 2022 at 08:21):

mathlib port progress data.complex.basic
Ported files: 274/577 (47.5% of total)
Ported lines: 88552/243489 (36.4% of total)
Longest unported chain: 56/79 (29.1% progress)

port progress bot (jmc) (Dec 29 2022 at 08:23):

mathlib port progress topology.metric_space.basic
Ported files: 271/525 (51.6% of total)
Ported lines: 87723/225445 (38.9% of total)
Longest unported chain: 50/73 (31.5% progress)

port progress bot (jmc) (Dec 29 2022 at 08:26):

mathlib port progress all
Ported files: 367/2852 (12.9% of total)
Ported lines: 101497/976826 (10.4% of total)
Longest unported chain: 112/135 (17.0% progress)

port progress bot (jmc) (Dec 30 2022 at 06:57):

mathlib port progress algebra.order.floor
Ported files: 180/196 (91.8% of total)
Ported lines: 67950/75389 (90.1% of total)
Longest unported chain: 3/31 (90.3% progress)

port progress bot (jmc) (Dec 30 2022 at 07:00):

mathlib port progress data.real.basic
Ported files: 203/227 (89.4% of total)
Ported lines: 74353/85438 (87.0% of total)
Longest unported chain: 6/34 (82.4% progress)

port progress bot (jmc) (Dec 30 2022 at 07:02):

mathlib port progress linear_algebra.basic
Ported files: 241/386 (62.4% of total)
Ported lines: 82739/153423 (53.9% of total)
Longest unported chain: 37/60 (38.3% progress)

port progress bot (jmc) (Dec 30 2022 at 07:04):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59996/83019 (72.3% of total)
Longest unported chain: 17/40 (57.5% progress)

port progress bot (jmc) (Dec 30 2022 at 07:06):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64720/94263 (68.7% of total)
Longest unported chain: 21/44 (52.3% progress)

port progress bot (jmc) (Dec 30 2022 at 07:09):

mathlib port progress order.filter.basic
Ported files: 199/279 (71.3% of total)
Ported lines: 72748/110997 (65.5% of total)
Longest unported chain: 24/47 (48.9% progress)

port progress bot (jmc) (Dec 30 2022 at 07:11):

mathlib port progress category_theory.limits.yoneda
Ported files: 51/92 (55.4% of total)
Ported lines: 18439/31944 (57.7% of total)
Longest unported chain: 17/36 (52.8% progress)

port progress bot (jmc) (Dec 30 2022 at 07:13):

mathlib port progress data.complex.basic
Ported files: 279/577 (48.4% of total)
Ported lines: 89279/243471 (36.7% of total)
Longest unported chain: 56/79 (29.1% progress)

port progress bot (jmc) (Dec 30 2022 at 07:16):

mathlib port progress topology.metric_space.basic
Ported files: 276/525 (52.6% of total)
Ported lines: 88450/225427 (39.2% of total)
Longest unported chain: 50/73 (31.5% progress)

port progress bot (jmc) (Dec 30 2022 at 07:19):

mathlib port progress all
Ported files: 377/2852 (13.2% of total)
Ported lines: 102591/976808 (10.5% of total)
Longest unported chain: 112/135 (17.0% progress)

port progress bot (jmc) (Dec 31 2022 at 06:29):

mathlib port progress algebra.order.floor
Ported files: 180/196 (91.8% of total)
Ported lines: 67950/75389 (90.1% of total)
Longest unported chain: 3/31 (90.3% progress)

port progress bot (jmc) (Dec 31 2022 at 06:31):

mathlib port progress data.real.basic
Ported files: 203/227 (89.4% of total)
Ported lines: 74353/85438 (87.0% of total)
Longest unported chain: 6/34 (82.4% progress)

port progress bot (jmc) (Dec 31 2022 at 06:33):

mathlib port progress linear_algebra.basic
Ported files: 242/386 (62.7% of total)
Ported lines: 83491/153423 (54.4% of total)
Longest unported chain: 37/60 (38.3% progress)

port progress bot (jmc) (Dec 31 2022 at 06:36):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59996/83019 (72.3% of total)
Longest unported chain: 17/40 (57.5% progress)

port progress bot (jmc) (Dec 31 2022 at 06:38):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64720/94263 (68.7% of total)
Longest unported chain: 21/44 (52.3% progress)

port progress bot (jmc) (Dec 31 2022 at 06:40):

mathlib port progress order.filter.basic
Ported files: 199/279 (71.3% of total)
Ported lines: 72748/110997 (65.5% of total)
Longest unported chain: 24/47 (48.9% progress)

port progress bot (jmc) (Dec 31 2022 at 06:42):

mathlib port progress category_theory.limits.yoneda
Ported files: 51/92 (55.4% of total)
Ported lines: 18439/31944 (57.7% of total)
Longest unported chain: 17/36 (52.8% progress)

port progress bot (jmc) (Dec 31 2022 at 06:45):

mathlib port progress data.complex.basic
Ported files: 281/577 (48.7% of total)
Ported lines: 90156/243469 (37.0% of total)
Longest unported chain: 56/79 (29.1% progress)

port progress bot (jmc) (Dec 31 2022 at 06:47):

mathlib port progress topology.metric_space.basic
Ported files: 278/525 (53.0% of total)
Ported lines: 89327/225425 (39.6% of total)
Longest unported chain: 50/73 (31.5% progress)

port progress bot (jmc) (Dec 31 2022 at 06:50):

mathlib port progress all
Ported files: 382/2852 (13.4% of total)
Ported lines: 103777/976783 (10.6% of total)
Longest unported chain: 112/135 (17.0% progress)

Eric Wieser (Dec 31 2022 at 16:56):

Eric Wieser said:

That should be as simple as removing a line from the inserted comment, and removing the list of PRs from stdout

Done in #18030.

port-progress bot (Dec 31 2022 at 18:03):

mathlib port progress data.nat.prime
Ported files: 149/156 (95.5% of total)
Ported lines: 58545/61663 (94.9% of total)
Longest unported chain: 1/29 (96.6% progress)

port-progress bot (Dec 31 2022 at 18:06):

mathlib port progress algebra.order.floor
Ported files: 180/196 (91.8% of total)
Ported lines: 67950/75389 (90.1% of total)
Longest unported chain: 3/31 (90.3% progress)

port-progress bot (Dec 31 2022 at 18:10):

mathlib port progress data.real.basic
Ported files: 203/227 (89.4% of total)
Ported lines: 74353/85438 (87.0% of total)
Longest unported chain: 6/34 (82.4% progress)

port-progress bot (Dec 31 2022 at 18:13):

mathlib port progress linear_algebra.basic
Ported files: 243/386 (63.0% of total)
Ported lines: 84230/153423 (54.9% of total)
Longest unported chain: 37/60 (38.3% progress)

port-progress bot (Dec 31 2022 at 18:17):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59996/83019 (72.3% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Dec 31 2022 at 18:21):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64720/94263 (68.7% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Dec 31 2022 at 18:24):

mathlib port progress order.filter.basic
Ported files: 199/279 (71.3% of total)
Ported lines: 72748/110997 (65.5% of total)
Longest unported chain: 24/47 (48.9% progress)

port-progress bot (Dec 31 2022 at 18:28):

mathlib port progress category_theory.limits.yoneda
Ported files: 51/92 (55.4% of total)
Ported lines: 18439/31944 (57.7% of total)
Longest unported chain: 17/36 (52.8% progress)

port-progress bot (Dec 31 2022 at 18:31):

mathlib port progress data.complex.basic
Ported files: 282/577 (48.9% of total)
Ported lines: 90895/243461 (37.3% of total)
Longest unported chain: 56/79 (29.1% progress)

port-progress bot (Dec 31 2022 at 18:35):

mathlib port progress topology.metric_space.basic
Ported files: 279/525 (53.1% of total)
Ported lines: 90066/225417 (40.0% of total)
Longest unported chain: 50/73 (31.5% progress)

port-progress bot (Dec 31 2022 at 19:27):

mathlib port progress all
Ported files: 383/2853 (13.4% of total)
Ported lines: 104516/977206 (10.7% of total)
Longest unported chain: 112/135 (17.0% progress)

Scott Morrison (Jan 01 2023 at 03:22):

@Johan Commelin, my bot came back online this morning when this computer was plugged back in. We should turn one of the bots off --- I don't know that there's any reason to prefer one or the other?

Johan Commelin (Jan 01 2023 at 09:11):

I'll turn mine off

Yaël Dillies (Jan 01 2023 at 10:17):

Can Scott's bot get a nice profile picture?

Notification Bot (Jan 01 2023 at 10:32):

A message was moved from this topic to #mathlib4 > synchronization label bot by Eric Wieser.

port-progress bot (Jan 01 2023 at 18:03):

mathlib port progress algebra.order.floor
Ported files: 180/196 (91.8% of total)
Ported lines: 67950/75389 (90.1% of total)
Longest unported chain: 3/31 (90.3% progress)

port-progress bot (Jan 01 2023 at 18:07):

mathlib port progress data.real.basic
Ported files: 203/227 (89.4% of total)
Ported lines: 74353/85438 (87.0% of total)
Longest unported chain: 6/34 (82.4% progress)

port-progress bot (Jan 01 2023 at 18:11):

mathlib port progress linear_algebra.basic
Ported files: 246/386 (63.7% of total)
Ported lines: 85069/153423 (55.4% of total)
Longest unported chain: 37/60 (38.3% progress)

port-progress bot (Jan 01 2023 at 18:14):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59996/83019 (72.3% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Jan 01 2023 at 18:18):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64720/94263 (68.7% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Jan 01 2023 at 18:21):

mathlib port progress order.filter.basic
Ported files: 199/279 (71.3% of total)
Ported lines: 72748/110997 (65.5% of total)
Longest unported chain: 24/47 (48.9% progress)

port-progress bot (Jan 01 2023 at 18:25):

mathlib port progress category_theory.limits.yoneda
Ported files: 52/92 (56.5% of total)
Ported lines: 18571/31944 (58.1% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 01 2023 at 18:29):

mathlib port progress data.complex.basic
Ported files: 286/577 (49.6% of total)
Ported lines: 92160/243461 (37.9% of total)
Longest unported chain: 56/79 (29.1% progress)

port-progress bot (Jan 01 2023 at 18:32):

mathlib port progress topology.metric_space.basic
Ported files: 282/525 (53.7% of total)
Ported lines: 90905/225417 (40.3% of total)
Longest unported chain: 50/73 (31.5% progress)

port-progress bot (Jan 01 2023 at 19:19):

mathlib port progress all
Ported files: 388/2853 (13.6% of total)
Ported lines: 105913/977206 (10.8% of total)
Longest unported chain: 112/135 (17.0% progress)

port-progress bot (Jan 02 2023 at 18:03):

mathlib port progress algebra.order.floor
Ported files: 181/196 (92.3% of total)
Ported lines: 68053/75239 (90.4% of total)
Longest unported chain: 2/31 (93.5% progress)

port-progress bot (Jan 02 2023 at 18:07):

mathlib port progress data.real.basic
Ported files: 204/227 (89.9% of total)
Ported lines: 74449/85281 (87.3% of total)
Longest unported chain: 5/34 (85.3% progress)

port-progress bot (Jan 02 2023 at 18:11):

mathlib port progress linear_algebra.basic
Ported files: 247/386 (64.0% of total)
Ported lines: 85148/153249 (55.6% of total)
Longest unported chain: 37/60 (38.3% progress)

port-progress bot (Jan 02 2023 at 18:15):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59862/82885 (72.2% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Jan 02 2023 at 18:18):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64575/94118 (68.6% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Jan 02 2023 at 18:22):

mathlib port progress order.filter.basic
Ported files: 200/279 (71.7% of total)
Ported lines: 72841/110837 (65.7% of total)
Longest unported chain: 24/47 (48.9% progress)

port-progress bot (Jan 02 2023 at 18:25):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18739/31897 (58.7% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 02 2023 at 18:29):

mathlib port progress data.complex.basic
Ported files: 289/577 (50.1% of total)
Ported lines: 93599/243287 (38.5% of total)
Longest unported chain: 56/79 (29.1% progress)

port-progress bot (Jan 02 2023 at 18:33):

mathlib port progress topology.metric_space.basic
Ported files: 285/525 (54.3% of total)
Ported lines: 92344/225227 (41.0% of total)
Longest unported chain: 50/73 (31.5% progress)

port-progress bot (Jan 02 2023 at 19:19):

mathlib port progress all
Ported files: 400/2853 (14.0% of total)
Ported lines: 108648/976956 (11.1% of total)
Longest unported chain: 112/135 (17.0% progress)

Riccardo Brasca (Jan 03 2023 at 16:45):

What is the strategy concerning changing the hash when we modify a ported file? Of course one is supposed to open a mathlib4 PR, but when should we modify the hash?

I have maybe misunderstood something, but I think we should try to keep the list "The following files have been modified since the commit at which they were verified" not too long, otherwise it will become a mess.

Eric Wieser (Jan 03 2023 at 16:58):

I think we should build some better tooling to verify that there is no diff before changing those SHAs

Eric Wieser (Jan 03 2023 at 17:00):

Of course one is supposed to open a mathlib4 PR

Are people doing this manually or with one-shot mode?

Eric Wieser (Jan 03 2023 at 17:00):

cc @Yaël Dillies?

Riccardo Brasca (Jan 03 2023 at 17:00):

Is this is even possible? The current files have really been modified (sometimes with new theorems), so I am afraid a human check is needed.

Eric Wieser (Jan 03 2023 at 17:00):

You can have git construct a three-way merge between the commit that was ported and the most recent port

Eric Wieser (Jan 03 2023 at 17:01):

And then a human can review that diff in the form of a PR

Riccardo Brasca (Jan 03 2023 at 17:01):

I think people are doing it by hand (or maybe they've just forgot to do it and nobody noticed)

Eric Wieser (Jan 03 2023 at 17:01):

If so then I think our workflow is wrong; making people create the mathlib4 PR before merging the 3 PR means that we're doing things manually and likely to make a mess where mathport wouldn't.

Eric Wieser (Jan 03 2023 at 17:02):

Maybe having a gitpod container with mathport and mathlib4 preconfigured would encourage the use of one-shot mode?

Reid Barton (Jan 03 2023 at 17:05):

I definitely agree that we should have better tooling for this process. I'm also not sure it is very urgent to do anything about it for now.
It would be nice if we could distinguish cases where the mathlib 3 change really affects downstream modules, so that we can take care of just those promptly.

Riccardo Brasca (Jan 03 2023 at 17:05):

The current workflow seems to be opening both PR at the same time. Usually the mathlib4 got accepted first, with a comment like "merge once the mathlib3 PR is accepted". Then I think people just merge the mathlib4 PR, without changing the hash, and now the file is listed as modified, even if it's in sync.

port-progress bot (Jan 03 2023 at 18:03):

mathlib port progress algebra.order.floor
Ported files: 184/196 (93.9% of total)
Ported lines: 68605/75350 (91.0% of total)
Longest unported chain: 2/31 (93.5% progress)

port-progress bot (Jan 03 2023 at 18:07):

mathlib port progress data.real.basic
Ported files: 207/227 (91.2% of total)
Ported lines: 75049/85440 (87.8% of total)
Longest unported chain: 5/34 (85.3% progress)

port-progress bot (Jan 03 2023 at 18:11):

mathlib port progress linear_algebra.basic
Ported files: 252/386 (65.3% of total)
Ported lines: 87108/153490 (56.8% of total)
Longest unported chain: 37/60 (38.3% progress)

port-progress bot (Jan 03 2023 at 18:15):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59913/82936 (72.2% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Jan 03 2023 at 18:19):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64641/94185 (68.6% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Jan 03 2023 at 18:22):

mathlib port progress order.filter.basic
Ported files: 203/279 (72.8% of total)
Ported lines: 73420/110975 (66.2% of total)
Longest unported chain: 24/47 (48.9% progress)

port-progress bot (Jan 03 2023 at 18:26):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18754/31912 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 03 2023 at 18:30):

mathlib port progress data.complex.basic
Ported files: 296/577 (51.3% of total)
Ported lines: 95818/243612 (39.3% of total)
Longest unported chain: 56/79 (29.1% progress)

port-progress bot (Jan 03 2023 at 18:33):

mathlib port progress topology.metric_space.basic
Ported files: 292/525 (55.6% of total)
Ported lines: 94551/225540 (41.9% of total)
Longest unported chain: 50/73 (31.5% progress)

Eric Wieser (Jan 03 2023 at 18:35):

I also think this thread is a bad place to have these discussions

image.png

port-progress bot (Jan 03 2023 at 19:22):

mathlib port progress all
Ported files: 414/2854 (14.5% of total)
Ported lines: 111848/977679 (11.4% of total)
Longest unported chain: 112/135 (17.0% progress)

Yaël Dillies (Jan 03 2023 at 20:26):

Eric Wieser said:

Of course one is supposed to open a mathlib4 PR

Are people doing this manually or with one-shot mode?

I've never used mathport. All the PRs I opened to mathlib4 were done manually.

Notification Bot (Jan 03 2023 at 22:01):

30 messages were moved from this topic to #mathlib4 > mathport and forward-porting by Eric Wieser.

port-progress bot (Jan 04 2023 at 18:04):

mathlib port progress algebra.order.floor
Ported files: 185/196 (94.4% of total)
Ported lines: 68946/75350 (91.5% of total)
Longest unported chain: 2/31 (93.5% progress)

port-progress bot (Jan 04 2023 at 18:08):

mathlib port progress data.real.basic
Ported files: 208/227 (91.6% of total)
Ported lines: 75390/85440 (88.2% of total)
Longest unported chain: 5/34 (85.3% progress)

Ruben Van de Velde (Jan 04 2023 at 18:10):

I kept waiting for data.fin.basic, but apparently that's only used in a single line in tactic.ring (re: floor)

Heather Macbeth (Jan 04 2023 at 18:11):

However, data.int.lemmas was genuinely a blocker for that, and it was only merged a few days ago.

port-progress bot (Jan 04 2023 at 18:12):

mathlib port progress linear_algebra.basic
Ported files: 256/386 (66.3% of total)
Ported lines: 88789/153490 (57.8% of total)
Longest unported chain: 37/60 (38.3% progress)

port-progress bot (Jan 04 2023 at 18:15):

mathlib port progress data.fintype.basic
Ported files: 148/183 (80.9% of total)
Ported lines: 59913/82936 (72.2% of total)
Longest unported chain: 17/40 (57.5% progress)

port-progress bot (Jan 04 2023 at 18:19):

mathlib port progress algebra.big_operators.basic
Ported files: 164/215 (76.3% of total)
Ported lines: 64641/94185 (68.6% of total)
Longest unported chain: 21/44 (52.3% progress)

port-progress bot (Jan 04 2023 at 18:23):

mathlib port progress order.filter.basic
Ported files: 204/279 (73.1% of total)
Ported lines: 73761/110975 (66.5% of total)
Longest unported chain: 24/47 (48.9% progress)

port-progress bot (Jan 04 2023 at 18:27):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18754/31912 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 04 2023 at 18:31):

mathlib port progress data.complex.basic
Ported files: 300/577 (52.0% of total)
Ported lines: 97499/243612 (40.0% of total)
Longest unported chain: 56/79 (29.1% progress)

port-progress bot (Jan 04 2023 at 18:35):

mathlib port progress topology.metric_space.basic
Ported files: 296/525 (56.4% of total)
Ported lines: 96232/225540 (42.7% of total)
Longest unported chain: 50/73 (31.5% progress)

Kevin Buzzard (Jan 04 2023 at 18:50):

I started thinking about the port the day Scott's video was announced on this Zulip, and the scale of the job became apparent to me very quickly. But now we are over half way towards many fundamental files; these figures are really exciting. It's also great to see #mathlib4 being one of the most popular streams right now. I firmly believe that as the material gets more advanced, more people will start to help -- the idea being that a good way to read a random mathlib file about stuff you're interested in is to port it, and you'll learn a bit about Lean 4 along the way. Has anyone considered making a revision of the video?

port-progress bot (Jan 04 2023 at 19:27):

mathlib port progress all
Ported files: 423/2857 (14.8% of total)
Ported lines: 114607/978052 (11.7% of total)
Longest unported chain: 112/135 (17.0% progress)

Moritz Doll (Jan 04 2023 at 22:26):

I've been not in the loop for a week now, but it seems to me that we need to get data.list.basic and data.fin.basic ported before it makes sense to convince more people to join the porting effort. The idea of updating has been discussed (on the porting meeting if I remember correctly), but someone has to put in the work.

Johan Commelin (Jan 05 2023 at 15:07):

See #port-status for some fresh files all the way at the top of the queue.

Henrik Böving (Jan 05 2023 at 15:09):

Data.List.Lemmas could have a conflict with std4/core I presume?

Johan Commelin (Jan 05 2023 at 15:11):

I dunno, but I'm afraid that it will

Henrik Böving (Jan 05 2023 at 15:12):

/me proceeds to cleverly avoid that file and ports infix instead

port-progress bot (Jan 05 2023 at 18:04):

mathlib port progress algebra.order.floor
Ported files: 185/196 (94.4% of total)
Ported lines: 68972/75376 (91.5% of total)
Longest unported chain: 2/31 (93.5% progress)

port-progress bot (Jan 05 2023 at 18:07):

mathlib port progress data.real.basic
Ported files: 208/227 (91.6% of total)
Ported lines: 75422/85472 (88.2% of total)
Longest unported chain: 5/34 (85.3% progress)

port-progress bot (Jan 05 2023 at 18:11):

mathlib port progress linear_algebra.basic
Ported files: 258/386 (66.8% of total)
Ported lines: 93103/153552 (60.6% of total)
Longest unported chain: 36/60 (40.0% progress)

port-progress bot (Jan 05 2023 at 18:15):

mathlib port progress data.fintype.basic
Ported files: 150/183 (82.0% of total)
Ported lines: 64206/82962 (77.4% of total)
Longest unported chain: 16/40 (60.0% progress)

port-progress bot (Jan 05 2023 at 18:19):

mathlib port progress algebra.big_operators.basic
Ported files: 166/215 (77.2% of total)
Ported lines: 68934/94211 (73.2% of total)
Longest unported chain: 20/44 (54.5% progress)

port-progress bot (Jan 05 2023 at 18:22):

mathlib port progress order.filter.basic
Ported files: 206/279 (73.8% of total)
Ported lines: 78057/111004 (70.3% of total)
Longest unported chain: 23/47 (51.1% progress)

port-progress bot (Jan 05 2023 at 18:26):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18754/31912 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 05 2023 at 18:30):

mathlib port progress data.complex.basic
Ported files: 302/577 (52.3% of total)
Ported lines: 101813/243700 (41.8% of total)
Longest unported chain: 55/79 (30.4% progress)

Eric Wieser (Jan 05 2023 at 18:30):

@Henrik Böving said:

/me proceeds to cleverly avoid that file and ports infix instead

Can we get #18067 in first?

Johan Commelin (Jan 05 2023 at 18:32):

I'm sure we can. I kicked it on the queue.

Henrik Böving (Jan 05 2023 at 18:32):

I'm done with the port modulo 1 theorem, 2 confusing things and 1 thing that's probably a bug so that's going to take a while still :D

port-progress bot (Jan 05 2023 at 18:34):

mathlib port progress topology.metric_space.basic
Ported files: 298/525 (56.8% of total)
Ported lines: 100546/225628 (44.6% of total)
Longest unported chain: 49/73 (32.9% progress)

Johan Commelin (Jan 05 2023 at 18:34):

Eric's PR adds 3 decls. Should be easy to port them (even manually, if we're in a hurry).

port-progress bot (Jan 05 2023 at 19:26):

mathlib port progress all
Ported files: 428/2857 (15.0% of total)
Ported lines: 119812/978436 (12.2% of total)
Longest unported chain: 111/135 (17.8% progress)

Henrik Böving (Jan 05 2023 at 21:51):

Eric Wieser said:

Henrik Böving said:

/me proceeds to cleverly avoid that file and ports infix instead

Can we get #18067 in first?

so now that this is merged and I got my PR ready, how do I port your changes as well? Do I manually translate?

Johan Commelin (Jan 05 2023 at 21:52):

Or you wait till tomorrow, and grab them out of the nightly mathport file.

Henrik Böving (Jan 05 2023 at 21:57):

I shall do that.

Johan Commelin (Jan 06 2023 at 11:56):

mathlib4#1380 is for Data.List.BigOperators.Basic

port-progress bot (Jan 06 2023 at 18:03):

mathlib port progress algebra.order.floor
Ported files: 185/196 (94.4% of total)
Ported lines: 68991/75395 (91.5% of total)
Longest unported chain: 2/31 (93.5% progress)

port-progress bot (Jan 06 2023 at 18:07):

mathlib port progress data.real.basic
Ported files: 209/228 (91.7% of total)
Ported lines: 75725/85775 (88.3% of total)
Longest unported chain: 5/34 (85.3% progress)

port-progress bot (Jan 06 2023 at 18:11):

mathlib port progress linear_algebra.basic
Ported files: 264/387 (68.2% of total)
Ported lines: 94934/153881 (61.7% of total)
Longest unported chain: 34/60 (43.3% progress)

port-progress bot (Jan 06 2023 at 18:15):

mathlib port progress data.fintype.basic
Ported files: 152/183 (83.1% of total)
Ported lines: 65060/82995 (78.4% of total)
Longest unported chain: 14/40 (65.0% progress)

port-progress bot (Jan 06 2023 at 18:18):

mathlib port progress algebra.big_operators.basic
Ported files: 169/215 (78.6% of total)
Ported lines: 70144/94253 (74.4% of total)
Longest unported chain: 18/44 (59.1% progress)

port-progress bot (Jan 06 2023 at 18:22):

mathlib port progress order.filter.basic
Ported files: 209/279 (74.9% of total)
Ported lines: 79267/111046 (71.4% of total)
Longest unported chain: 21/47 (55.3% progress)

port-progress bot (Jan 06 2023 at 18:25):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18754/31912 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 06 2023 at 18:29):

mathlib port progress data.complex.basic
Ported files: 307/577 (53.2% of total)
Ported lines: 103426/243811 (42.4% of total)
Longest unported chain: 53/79 (32.9% progress)

port-progress bot (Jan 06 2023 at 18:33):

mathlib port progress topology.metric_space.basic
Ported files: 303/525 (57.7% of total)
Ported lines: 102155/225735 (45.3% of total)
Longest unported chain: 47/73 (35.6% progress)

port-progress bot (Jan 06 2023 at 19:20):

mathlib port progress all
Ported files: 439/2857 (15.4% of total)
Ported lines: 122214/978606 (12.5% of total)
Longest unported chain: 109/135 (19.3% progress)

Heather Macbeth (Jan 07 2023 at 17:13):

mathlib4#1304 Algebra.Order.Floor is on the critical path to Data.Real.Basic. It is now ready for review, modulo mathlib4#1392 and mathlib4#1394, both also awaiting review. If anyone has review time today, they are worthy targets!

Note mathlib4#1394 is meta code.

Ruben Van de Velde (Jan 07 2023 at 17:17):

1392 looks good to me :innocent:

Johan Commelin (Jan 07 2023 at 17:20):

@Ruben Van de Velde But you are only porting a part of a file there, do I understand that right?

Johan Commelin (Jan 07 2023 at 17:27):

If so, I'm wondering whether we should remove the porting header, so that it gets qualified as "ad hoc" port.

Ruben Van de Velde (Jan 07 2023 at 17:35):

The rest is meta code, so I'm not sure if we'd ever port it, but either way is fine by me

Johan Commelin (Jan 07 2023 at 17:45):

What does the meta code do? I don't know this file.

Johan Commelin (Jan 07 2023 at 17:45):

If we decide that it doesn't need to be ported, we should record that decision in a comment.

Johan Commelin (Jan 07 2023 at 17:47):

@Mario Carneiro Is this a clear case?

Mario Carneiro (Jan 07 2023 at 17:48):

which meta code?

Mario Carneiro (Jan 07 2023 at 17:50):

there is a positivity extension for floor/ceil in algebra.order.floor, if that's what you're talking about. It should be ignored for the purpose of the port, and an issue should be made on mathlib4 to track it

Johan Commelin (Jan 07 2023 at 17:50):

https://github.com/leanprover-community/mathlib4/pull/1392/commits/0a38ad8c57b9f734e5b57524caca665cd57fc380

Mario Carneiro (Jan 07 2023 at 17:51):

oh that. This is all subsumed by stuff in lean 4 core

Mario Carneiro (Jan 07 2023 at 17:52):

so unless you are using the theorems (and you really shouldn't, they are intended for tactic use only) the whole file can be skipped

Johan Commelin (Jan 07 2023 at 17:52):

Ok, let's add that as a big fat comment

Johan Commelin (Jan 07 2023 at 18:00):

Done, and merge-queued.

port-progress bot (Jan 07 2023 at 18:04):

mathlib port progress algebra.order.floor
Ported files: 185/196 (94.4% of total)
Ported lines: 69124/75528 (91.5% of total)
Longest unported chain: 2/31 (93.5% progress)

port-progress bot (Jan 07 2023 at 18:07):

mathlib port progress data.real.basic
Ported files: 209/228 (91.7% of total)
Ported lines: 75858/85908 (88.3% of total)
Longest unported chain: 5/34 (85.3% progress)

port-progress bot (Jan 07 2023 at 18:11):

mathlib port progress linear_algebra.basic
Ported files: 264/387 (68.2% of total)
Ported lines: 95073/154095 (61.7% of total)
Longest unported chain: 34/60 (43.3% progress)

port-progress bot (Jan 07 2023 at 18:14):

mathlib port progress data.fintype.basic
Ported files: 152/183 (83.1% of total)
Ported lines: 65196/83155 (78.4% of total)
Longest unported chain: 14/40 (65.0% progress)

port-progress bot (Jan 07 2023 at 18:18):

mathlib port progress algebra.big_operators.basic
Ported files: 169/215 (78.6% of total)
Ported lines: 70280/94413 (74.4% of total)
Longest unported chain: 18/44 (59.1% progress)

Kevin Buzzard (Jan 07 2023 at 18:20):

Heather Macbeth said:

mathlib4#1304 Algebra.Order.Floor is on the critical path to Data.Real.Basic. It is now ready for review, modulo mathlib4#1392 and mathlib4#1394, both also awaiting review. If anyone has review time today, they are worthy targets!

Note mathlib4#1394 is meta code.

mathlib4#1304 has merge conflicts apparently :-/

port-progress bot (Jan 07 2023 at 18:22):

mathlib port progress order.filter.basic
Ported files: 209/279 (74.9% of total)
Ported lines: 79403/111257 (71.4% of total)
Longest unported chain: 21/47 (55.3% progress)

port-progress bot (Jan 07 2023 at 18:25):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18757/31915 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

Ruben Van de Velde (Jan 07 2023 at 18:26):

Kevin Buzzard said:

Heather Macbeth said:

mathlib4#1304 Algebra.Order.Floor is on the critical path to Data.Real.Basic. It is now ready for review, modulo mathlib4#1392 and mathlib4#1394, both also awaiting review. If anyone has review time today, they are worthy targets!

Note mathlib4#1394 is meta code.

mathlib4#1304 has merge conflicts apparently :-/

Probably because 1392 merged?

port-progress bot (Jan 07 2023 at 18:29):

mathlib port progress data.complex.basic
Ported files: 307/577 (53.2% of total)
Ported lines: 103565/244035 (42.4% of total)
Longest unported chain: 53/79 (32.9% progress)

port-progress bot (Jan 07 2023 at 18:33):

mathlib port progress topology.metric_space.basic
Ported files: 303/525 (57.7% of total)
Ported lines: 102294/225959 (45.3% of total)
Longest unported chain: 47/73 (35.6% progress)

Chris Hughes (Jan 07 2023 at 18:45):

Kevin Buzzard said:

Heather Macbeth said:

mathlib4#1304 Algebra.Order.Floor is on the critical path to Data.Real.Basic. It is now ready for review, modulo mathlib4#1392 and mathlib4#1394, both also awaiting review. If anyone has review time today, they are worthy targets!

Note mathlib4#1394 is meta code.

mathlib4#1304 has merge conflicts apparently :-/

The merge conflicts are usually Mathlib.lean

Heather Macbeth (Jan 07 2023 at 18:56):

It was the conflicts from review changes to mathlib4#1392. Fixed.

port-progress bot (Jan 07 2023 at 19:07):

mathlib port progress all
Ported files: 440/2857 (15.4% of total)
Ported lines: 123168/979576 (12.6% of total)
Longest unported chain: 109/135 (19.3% progress)

Henrik Böving (Jan 08 2023 at 11:13):

https://math.commelin.net/files/port_status.html marks algebra.hom.group_action as portable so I just started it over here: https://github.com/leanprover-community/mathlib4/pull/1424 but it is missing a dependency to Mathlib.Algebra.GroupRingAction.Invariant, did that thing move somewhere else or is this a bug in the port_status detector?

David Loeffler (Jan 08 2023 at 11:19):

Henrik Böving said:

https://math.commelin.net/files/port_status.html marks algebra.hom.group_action as portable so I just started it over here: https://github.com/leanprover-community/mathlib4/pull/1424 but it is missing a dependency to Mathlib.Algebra.GroupRingAction.Invariant, did that thing move somewhere else or is this a bug in the port_status detector?

I'm guessing this is to do with #18092?

Henrik Böving (Jan 08 2023 at 11:21):

Ah so the issue is that mathport did not run through yet? Can I run it locally for this single file somehow? Or shall I just wait until tomorrow then.

Eric Wieser (Jan 08 2023 at 11:29):

Mathport now runs twice a day, so you only need to wait till 6 hours or so from now

Ruben Van de Velde (Jan 08 2023 at 12:15):

Or manually remove the last 15 or so lines and the import from the mathported file

port-progress bot (Jan 08 2023 at 18:03):

mathlib port progress algebra.order.floor
Ported files: 185/196 (94.4% of total)
Ported lines: 69128/75532 (91.5% of total)
Longest unported chain: 2/31 (93.5% progress)

port-progress bot (Jan 08 2023 at 18:07):

mathlib port progress data.real.basic
Ported files: 209/228 (91.7% of total)
Ported lines: 75862/85912 (88.3% of total)
Longest unported chain: 5/34 (85.3% progress)

port-progress bot (Jan 08 2023 at 18:11):

mathlib port progress linear_algebra.basic
Ported files: 258/366 (70.5% of total)
Ported lines: 94224/147738 (63.8% of total)
Longest unported chain: 26/52 (50.0% progress)

port-progress bot (Jan 08 2023 at 18:14):

mathlib port progress data.fintype.basic
Ported files: 152/183 (83.1% of total)
Ported lines: 65200/83197 (78.4% of total)
Longest unported chain: 14/40 (65.0% progress)

port-progress bot (Jan 08 2023 at 18:18):

mathlib port progress algebra.big_operators.basic
Ported files: 169/215 (78.6% of total)
Ported lines: 70284/94471 (74.4% of total)
Longest unported chain: 18/44 (59.1% progress)

port-progress bot (Jan 08 2023 at 18:22):

mathlib port progress order.filter.basic
Ported files: 209/279 (74.9% of total)
Ported lines: 79407/111315 (71.3% of total)
Longest unported chain: 21/47 (55.3% progress)

port-progress bot (Jan 08 2023 at 18:25):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18765/31923 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 08 2023 at 18:29):

mathlib port progress data.complex.basic
Ported files: 308/574 (53.7% of total)
Ported lines: 103667/243781 (42.5% of total)
Longest unported chain: 53/79 (32.9% progress)

port-progress bot (Jan 08 2023 at 18:33):

mathlib port progress topology.metric_space.basic
Ported files: 304/522 (58.2% of total)
Ported lines: 102396/225705 (45.4% of total)
Longest unported chain: 47/73 (35.6% progress)

port-progress bot (Jan 08 2023 at 19:03):

mathlib port progress all
Ported files: 441/2857 (15.4% of total)
Ported lines: 123270/979965 (12.6% of total)
Longest unported chain: 101/127 (20.5% progress)

port-progress bot (Jan 09 2023 at 18:03):

mathlib port progress algebra.order.floor
Ported files: 185/196 (94.4% of total)
Ported lines: 69184/75588 (91.5% of total)
Longest unported chain: 2/31 (93.5% progress)

port-progress bot (Jan 09 2023 at 18:07):

mathlib port progress data.real.basic
Ported files: 210/228 (92.1% of total)
Ported lines: 76433/85968 (88.9% of total)
Longest unported chain: 5/34 (85.3% progress)

port-progress bot (Jan 09 2023 at 18:11):

mathlib port progress linear_algebra.basic
Ported files: 260/366 (71.0% of total)
Ported lines: 94850/147794 (64.2% of total)
Longest unported chain: 26/52 (50.0% progress)

port-progress bot (Jan 09 2023 at 18:14):

mathlib port progress data.fintype.basic
Ported files: 152/183 (83.1% of total)
Ported lines: 65256/83253 (78.4% of total)
Longest unported chain: 14/40 (65.0% progress)

port-progress bot (Jan 09 2023 at 18:18):

mathlib port progress algebra.big_operators.basic
Ported files: 169/215 (78.6% of total)
Ported lines: 70340/94527 (74.4% of total)
Longest unported chain: 18/44 (59.1% progress)

port-progress bot (Jan 09 2023 at 18:22):

mathlib port progress order.filter.basic
Ported files: 209/279 (74.9% of total)
Ported lines: 79463/111371 (71.3% of total)
Longest unported chain: 21/47 (55.3% progress)

port-progress bot (Jan 09 2023 at 18:25):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18765/31923 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 09 2023 at 18:29):

mathlib port progress data.complex.basic
Ported files: 312/574 (54.4% of total)
Ported lines: 104409/243842 (42.8% of total)
Longest unported chain: 53/79 (32.9% progress)

port-progress bot (Jan 09 2023 at 18:33):

mathlib port progress topology.metric_space.basic
Ported files: 306/522 (58.6% of total)
Ported lines: 103022/225761 (45.6% of total)
Longest unported chain: 47/73 (35.6% progress)

port-progress bot (Jan 09 2023 at 19:04):

mathlib port progress all
Ported files: 447/2857 (15.6% of total)
Ported lines: 124395/980055 (12.7% of total)
Longest unported chain: 101/127 (20.5% progress)

Ruben Van de Velde (Jan 10 2023 at 13:27):

port-progress bot said:

mathlib port progress data.real.basic
Ported files: 210/228 (92.1% of total)
Ported lines: 76433/85968 (88.9% of total)
Longest unported chain: 5/34 (85.3% progress)

Now at 2 unported dependencies and five in progress: mathlib4#1447 (needs review); mathlib4#1188; mathlib4#1304 (needs review); mathlib4#1418; mathlib4#1440 (needs help)

Eric Wieser (Jan 10 2023 at 13:38):

Note that #8146 was intended to help with the port of data/real/basic.lean itself by removing the refine_struct

Eric Wieser (Jan 10 2023 at 13:38):

Although it's hitting some odd typeclass problems I haven't yet had a chance to debug

Eric Wieser (Jan 10 2023 at 16:40):

#18118 is the first half of #8146 and passes CI

port-progress bot (Jan 10 2023 at 18:03):

mathlib port progress algebra.order.floor
Ported files: 186/196 (94.9% of total)
Ported lines: 70554/75786 (93.1% of total)
Longest unported chain: 1/31 (96.8% progress)

port-progress bot (Jan 10 2023 at 18:06):

mathlib port progress data.real.basic
Ported files: 212/228 (93.0% of total)
Ported lines: 78645/86205 (91.2% of total)
Longest unported chain: 2/34 (94.1% progress)

port-progress bot (Jan 10 2023 at 18:10):

mathlib port progress linear_algebra.basic
Ported files: 271/366 (74.0% of total)
Ported lines: 98294/148021 (66.4% of total)
Longest unported chain: 23/52 (55.8% progress)

port-progress bot (Jan 10 2023 at 18:14):

mathlib port progress data.fintype.basic
Ported files: 160/183 (87.4% of total)
Ported lines: 67985/83264 (81.6% of total)
Longest unported chain: 11/40 (72.5% progress)

port-progress bot (Jan 10 2023 at 18:17):

mathlib port progress algebra.big_operators.basic
Ported files: 178/215 (82.8% of total)
Ported lines: 73224/94537 (77.5% of total)
Longest unported chain: 15/44 (65.9% progress)

port-progress bot (Jan 10 2023 at 18:21):

mathlib port progress order.filter.basic
Ported files: 217/279 (77.8% of total)
Ported lines: 82379/111569 (73.8% of total)
Longest unported chain: 18/47 (61.7% progress)

port-progress bot (Jan 10 2023 at 18:25):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18765/31923 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 10 2023 at 18:28):

mathlib port progress data.complex.basic
Ported files: 325/574 (56.6% of total)
Ported lines: 109838/244093 (45.0% of total)
Longest unported chain: 50/79 (36.7% progress)

port-progress bot (Jan 10 2023 at 18:32):

mathlib port progress topology.metric_space.basic
Ported files: 319/522 (61.1% of total)
Ported lines: 108451/226012 (48.0% of total)
Longest unported chain: 44/73 (39.7% progress)

port-progress bot (Jan 10 2023 at 19:03):

mathlib port progress all
Ported files: 464/2857 (16.2% of total)
Ported lines: 130603/980453 (13.3% of total)
Longest unported chain: 97/127 (23.6% progress)

Johan Commelin (Jan 10 2023 at 19:06):

Bam! 0.6% lines ported in one day.

Ruben Van de Velde (Jan 10 2023 at 19:13):

Or reviewed :)

Heather Macbeth (Jan 10 2023 at 19:14):

I have proposed this before, but if a scripting wizard wants to put together a %-of-mathlib-ported timeseries graph that updates every day, I think it would be very motivational.

Eric Wieser (Jan 10 2023 at 19:15):

Where does the script that generates the current output live?

Ruben Van de Velde (Jan 10 2023 at 19:23):

@Lukas Miaskiwskyi are you actively working on mathlib4#1462 still?

Heather Macbeth (Jan 10 2023 at 19:23):

Eric Wieser said:

Where does the script that generates the current output live?

I believe it's leanproject port-progress, but it would also be nice to scrape this stream for the history.

Lukas Miaskiwskyi (Jan 10 2023 at 19:25):

Ruben Van de Velde said:

Lukas Miaskiwskyi are you actively working on mathlib4#1462 still?

Yep, this very moment, but I'm still at the very beginning with it

Ruben Van de Velde (Jan 10 2023 at 19:31):

Lukas Miaskiwskyi said:

Ruben Van de Velde said:

Lukas Miaskiwskyi are you actively working on mathlib4#1462 still?

Yep, this very moment, but I'm still at the very beginning with it

Then I'll stop :)

Should I push the changes I made locally?

Lukas Miaskiwskyi (Jan 10 2023 at 19:34):

Sure, go for it! Sorry for swiping it from you :D

Eric Wieser (Jan 10 2023 at 19:34):

Heather Macbeth said:

Eric Wieser said:

Where does the script that generates the current output live?

I believe it's leanproject port-progress, but it would also be nice to scrape this stream for the history.

My thinking was that if port-progress is just scraping the repo in some way, then it might be easier than scraping the stream

Johan Commelin (Jan 10 2023 at 19:35):

~/data/math/port_progress/mathlib$ cat ~/bin/port-progress-bot.sh
# You'd need the zulip command line client installed via `pip install zulip`
# and credentials for an account in `$TMP_DIR/zuliprc`.

TARGETS="algebra.order.floor data.real.basic linear_algebra.basic data.fintype.basic algebra.big_operators.basic order.filter.basic category_theory.limits.yoneda data.complex.basic topology.metric_space.basic all"
BASE_URL=https://math.commelin.net/files/mathlib4
TMP_DIR=/home/jmc/data/math/port_progress
GRAPH_DIR=/home/jmc/sites/math/files/mathlib4

mkdir -p $TMP_DIR
today=$(date -I)
mkdir -p $GRAPH_DIR/$today/

cd $TMP_DIR
cd mathlib
git clean -xfd
git pull
leanpkg configure
leanproject get-cache
scripts/mk_all.sh

cd $GRAPH_DIR
ln -sfn $today latest

cd $TMP_DIR/mathlib
for target in $TARGETS; do

    leanproject port-progress --to $target > $target.out
    cat $target.out | tail -n +6 > $GRAPH_DIR/$today/$target
    cat $target.out | \
      head -n 5 | \
      sed -e "s%\(mathlib port progress *| \)\([0-9a-z_\.]*\)%\1[\2]($BASE_URL/$today/\2.pdf)%" | \
      sed -e "s|\(Longest unported chain\)|[\1]($BASE_URL/$today/$target)|" | \
      zulip-send -s mathlib4 --subject "port progress" --config-file $TMP_DIR/zuliprc

done

Ruben Van de Velde (Jan 10 2023 at 19:36):

Pushed - over to you. Should have checked for the PR first :)

Eric Wieser (Jan 10 2023 at 19:45):

Thanks @Johan Commelin, I've uploaded that at https://github.com/leanprover-community/mathlib-port-status/blob/main/scripts/port-progress-bot.sh so that it doesn't get lost

Yaël Dillies (Jan 10 2023 at 19:53):

Heather Macbeth said:

I have proposed this before, but if a scripting wizard wants to put together a %-of-mathlib-ported timeseries graph that updates every day, I think it would be very motivational.

Could these graphs be overlayed with the existing ones for number of files and number of lines on the stats page?

Ruben Van de Velde (Jan 10 2023 at 20:10):

If people are around to review, I think we might be able to start on data.real.basic tomorrow. (I'm off for the night now, in any case)

Eric Wieser (Jan 10 2023 at 20:12):

Eric Wieser said:

Note that #8146 was intended to help with the port of data/real/basic.lean itself by removing the refine_struct

@Ruben Van de Velde , did you see this?

Heather Macbeth (Jan 10 2023 at 22:34):

Yaël Dillies said:

Heather Macbeth said:

I have proposed this before, but if a scripting wizard wants to put together a %-of-mathlib-ported timeseries graph that updates every day, I think it would be very motivational.

Could these graphs be overlayed with the existing ones for number of files and number of lines on the stats page?

@Yaël Dillies Indeed.

Ruben Van de Velde (Jan 11 2023 at 08:16):

Johan Commelin (Jan 11 2023 at 08:19):

@Eric Wieser is planning to touch up the final prereq.

Ruben Van de Velde (Jan 11 2023 at 08:20):

Yeah, looks like another 9 hours before mathport picks up the parameter change

Eric Wieser (Jan 11 2023 at 09:32):

Can we trigger mathport CI manually?

Johan Commelin (Jan 11 2023 at 09:32):

Probably, but it's quite heavy I think.

Johan Commelin (Jan 11 2023 at 09:33):

But in this case, it's probably justified

Eric Wieser (Jan 11 2023 at 09:33):

On the other hand, I had one more data/real/basic refactor queued up

Ruben Van de Velde (Jan 11 2023 at 09:34):

Then better do it quick :)

Eric Wieser (Jan 11 2023 at 09:34):

So I guess I have 6 hours or so to wrap that up

Eric Wieser (Jan 11 2023 at 10:46):

Optimistically #8146 is now on track to pass CI, after working around an annoying norm_num bug

Johan Commelin (Jan 11 2023 at 16:46):

#port-status updated after List.Perm got merged. Looking forward to the new graphs.

Ruben Van de Velde (Jan 11 2023 at 16:53):

data.list.sublists and data.multiset.basic are probably good targets

Heather Macbeth (Jan 11 2023 at 17:06):

Ruben Van de Velde said:

Yeah, looks like another 9 hours before mathport picks up the parameter change

Mathport updated!

port-progress bot (Jan 11 2023 at 18:04):

mathlib port progress data.real.basic
Ported files: 216/228 (94.7% of total)
Ported lines: 79993/86236 (92.8% of total)
Longest unported chain: 1/34 (97.1% progress)

Eric Wieser (Jan 11 2023 at 18:04):

I'll do the merge now

port-progress bot (Jan 11 2023 at 18:07):

mathlib port progress linear_algebra.basic
Ported files: 277/366 (75.7% of total)
Ported lines: 101278/148082 (68.4% of total)
Longest unported chain: 20/52 (61.5% progress)

Ruben Van de Velde (Jan 11 2023 at 18:08):

Heather Macbeth said:

Ruben Van de Velde said:

Yeah, looks like another 9 hours before mathport picks up the parameter change

Mathport updated!

I'd propose that we just port data.real.basic now (unless something is fundamentally broken), rather than wait for more refactoring

port-progress bot (Jan 11 2023 at 18:11):

mathlib port progress data.fintype.basic
Ported files: 164/183 (89.6% of total)
Ported lines: 70097/83297 (84.2% of total)
Longest unported chain: 8/40 (80.0% progress)

port-progress bot (Jan 11 2023 at 18:15):

mathlib port progress algebra.big_operators.basic
Ported files: 182/215 (84.7% of total)
Ported lines: 75339/94573 (79.7% of total)
Longest unported chain: 12/44 (72.7% progress)

port-progress bot (Jan 11 2023 at 18:18):

mathlib port progress order.filter.basic
Ported files: 222/279 (79.6% of total)
Ported lines: 84638/111609 (75.8% of total)
Longest unported chain: 15/47 (68.1% progress)

port-progress bot (Jan 11 2023 at 18:22):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18765/31923 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 11 2023 at 18:26):

mathlib port progress data.complex.basic
Ported files: 335/574 (58.4% of total)
Ported lines: 113550/244209 (46.5% of total)
Longest unported chain: 47/79 (40.5% progress)

port-progress bot (Jan 11 2023 at 18:30):

mathlib port progress topology.metric_space.basic
Ported files: 328/522 (62.8% of total)
Ported lines: 112069/226122 (49.6% of total)
Longest unported chain: 41/73 (43.8% progress)

Eric Wieser (Jan 11 2023 at 18:33):

Eric Wieser said:

I'll do the merge now

Done in https://github.com/leanprover-community/mathlib4/pull/1469. There's one bug I caught in the original PR regarding a rename that isn't reflected in the #align. What should docs#cau_seq.is_complete.is_complete be called?

Eric Wieser (Jan 11 2023 at 18:35):

Ruben Van de Velde said:

I'd propose that we just port data.real.basic now (unless something is fundamentally broken), rather than wait for more refactoring

I think I now agree; #8146 is proving more troublesome than expected, and the fallout in real.lean is now tiny. You'll have an annoying refine_struct which I recommend you replace with a regular structure and sorry all the proof fields. That will give you enough to port the rest of the file, and then hopefully by the time you have that I'll have #8146 ready and can save you from the sorries

port-progress bot (Jan 11 2023 at 19:01):

mathlib port progress all
Ported files: 474/2858 (16.6% of total)
Ported lines: 134018/980816 (13.7% of total)
Longest unported chain: 95/127 (25.2% progress)

Johan Commelin (Jan 11 2023 at 19:05):

+ 0.4%

More than I expected, frankly!

Heather Macbeth (Jan 11 2023 at 21:30):

Can someone please remind me how to generate the longest unported chain in mathlib, like this page:
https://tqft.net/mathlib4/2023-01-12/all
I tried leanproject port-progress but after giving the length of the longest unported chain it hangs indefinitely (is it still working?).

Scott Morrison (Jan 11 2023 at 21:31):

Are all the oleans built? Even with them, it should be very slow.

Scott Morrison (Jan 11 2023 at 21:32):

~30 minutes on my machine (you can see the gaps between the port-progress-bot posting: it is working full-time in between posts).

Heather Macbeth (Jan 11 2023 at 21:32):

Ah, no they're not. I was trying some speculative import-rearrangement to see what it would do to the chain.

Heather Macbeth (Jan 11 2023 at 21:33):

I think it used not to need the oleans? A couple of months ago I was able to play this game and inspect what the new longest chain was:
https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/port.20progress/near/310105496

Scott Morrison (Jan 11 2023 at 21:42):

Maybe computing the longest chain to a particular target, rather than all, will be faster?

Heather Macbeth (Jan 11 2023 at 21:42):

No, same behaviour with leanproject port-progress --to analysis.normed_space.star.gelfand_duality.

Heather Macbeth (Jan 11 2023 at 21:43):

Is there functionality just to compute the longest chain, without inspecting its port progress? Maybe that's what I was using before.

Scott Morrison (Jan 11 2023 at 21:44):

Doesn't seem to be.

James Gallicchio (Jan 11 2023 at 22:00):

one thing i noticed was that leanproject port-progress is re-using the tooling that lints for unnecessary imports... which seems like an odd choice, since presumably going through the entire AST is much more intensive than just parsing each file's imports and doing it based on that graph

Eric Wieser (Jan 11 2023 at 22:01):

If you don't care about the - markers then I would guess removing this line would speed it up a lot

Heather Macbeth (Jan 11 2023 at 22:19):

Aha! And indeed that line was added since last time I experimented.

Eric Wieser (Jan 11 2023 at 22:22):

Hiding it behind a flag is probably a reasonable compromise

Eric Wieser (Jan 11 2023 at 22:23):

I also wonder if we can construct this information faster from the tlean export we hand to trepplein

port-progress bot (Jan 12 2023 at 18:04):

mathlib port progress data.real.basic
Ported files: 216/228 (94.7% of total)
Ported lines: 79993/86267 (92.7% of total)
Longest unported chain: 1/34 (97.1% progress)

port-progress bot (Jan 12 2023 at 18:08):

mathlib port progress data.fintype.basic
Ported files: 164/183 (89.6% of total)
Ported lines: 70103/83329 (84.1% of total)
Longest unported chain: 8/40 (80.0% progress)

port-progress bot (Jan 12 2023 at 18:12):

mathlib port progress algebra.big_operators.basic
Ported files: 182/215 (84.7% of total)
Ported lines: 75345/94605 (79.6% of total)
Longest unported chain: 12/44 (72.7% progress)

port-progress bot (Jan 12 2023 at 18:16):

mathlib port progress order.filter.basic
Ported files: 222/279 (79.6% of total)
Ported lines: 84644/111641 (75.8% of total)
Longest unported chain: 15/47 (68.1% progress)

port-progress bot (Jan 12 2023 at 18:19):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18765/31923 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 12 2023 at 18:23):

mathlib port progress linear_algebra.basic
Ported files: 277/366 (75.7% of total)
Ported lines: 101298/148135 (68.4% of total)
Longest unported chain: 20/52 (61.5% progress)

port-progress bot (Jan 12 2023 at 18:27):

mathlib port progress data.complex.basic
Ported files: 336/574 (58.5% of total)
Ported lines: 113649/244345 (46.5% of total)
Longest unported chain: 47/79 (40.5% progress)

port-progress bot (Jan 12 2023 at 18:31):

mathlib port progress topology.metric_space.basic
Ported files: 328/522 (62.8% of total)
Ported lines: 112089/226189 (49.6% of total)
Longest unported chain: 41/73 (43.8% progress)

port-progress bot (Jan 12 2023 at 18:59):

mathlib port progress all
Ported files: 478/2860 (16.7% of total)
Ported lines: 135104/981191 (13.8% of total)
Longest unported chain: 94/126 (25.4% progress)

Ruben Van de Velde (Jan 13 2023 at 14:32):

@Johan Commelin mathlib4#1539 can be reviewed again, if you want to

Johan Commelin (Jan 13 2023 at 19:20):

https://math.commelin.net/files/mathlib4/latest/data.fintype.basic.pdf

Johan Commelin (Jan 13 2023 at 19:20):

The stats will follow soon :shout: :bird:

Johan Commelin (Jan 13 2023 at 19:27):

This one is now quite fascinating: https://math.commelin.net/files/mathlib4/latest/order.filter.basic.pdf

Johan Commelin (Jan 13 2023 at 19:27):

Lots of green scattered all over the place

Arien Malec (Jan 13 2023 at 19:29):

I thought there was a strategy for de-topologizing data.complex.basic but still shows in the graph?

port progress bot (jmc) (Jan 13 2023 at 19:32):

mathlib port progress data.real.basic
Ported files: 218/228 (95.6% of total)
Ported lines: 82253/86267 (95.3% of total)
Longest unported chain: 1/34 (97.1% progress)

port progress bot (jmc) (Jan 13 2023 at 19:35):

mathlib port progress linear_algebra.basic
Ported files: 294/366 (80.3% of total)
Ported lines: 109542/148160 (73.9% of total)
Longest unported chain: 15/52 (71.2% progress)

port progress bot (jmc) (Jan 13 2023 at 19:37):

mathlib port progress data.fintype.basic
Ported files: 172/183 (94.0% of total)
Ported lines: 75638/83342 (90.8% of total)
Longest unported chain: 3/40 (92.5% progress)

port progress bot (jmc) (Jan 13 2023 at 19:39):

mathlib port progress algebra.big_operators.basic
Ported files: 195/215 (90.7% of total)
Ported lines: 81810/94618 (86.5% of total)
Longest unported chain: 7/44 (84.1% progress)

port progress bot (jmc) (Jan 13 2023 at 19:42):

mathlib port progress order.filter.basic
Ported files: 235/279 (84.2% of total)
Ported lines: 91198/111654 (81.7% of total)
Longest unported chain: 10/47 (78.7% progress)

port progress bot (jmc) (Jan 13 2023 at 19:44):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18765/31923 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port progress bot (jmc) (Jan 13 2023 at 19:46):

mathlib port progress data.complex.basic
Ported files: 355/574 (61.8% of total)
Ported lines: 122860/244382 (50.3% of total)
Longest unported chain: 42/79 (46.8% progress)

port progress bot (jmc) (Jan 13 2023 at 19:49):

mathlib port progress topology.metric_space.basic
Ported files: 347/522 (66.5% of total)
Ported lines: 121300/226226 (53.6% of total)
Longest unported chain: 36/73 (50.7% progress)

port progress bot (jmc) (Jan 13 2023 at 19:52):

mathlib port progress all
Ported files: 502/2859 (17.6% of total)
Ported lines: 145153/981157 (14.8% of total)
Longest unported chain: 89/126 (29.4% progress)

Johan Commelin (Jan 13 2023 at 19:57):

1% 1% 1%
:octopus: :octopus: :octopus:

James Gallicchio (Jan 14 2023 at 21:43):

(does the port-bot only have a 5 day working week?)

Chris Hughes (Jan 14 2023 at 22:25):

In France I once visited a website that closed after 6pm.

port-progress bot (Jan 15 2023 at 18:03):

mathlib port progress data.real.basic
Ported files: 219/229 (95.6% of total)
Ported lines: 82424/86438 (95.4% of total)
Longest unported chain: 1/34 (97.1% progress)

port-progress bot (Jan 15 2023 at 18:07):

mathlib port progress data.fintype.basic
Ported files: 173/184 (94.0% of total)
Ported lines: 75810/83514 (90.8% of total)
Longest unported chain: 3/40 (92.5% progress)

port-progress bot (Jan 15 2023 at 18:11):

mathlib port progress algebra.big_operators.basic
Ported files: 197/216 (91.2% of total)
Ported lines: 82092/94771 (86.6% of total)
Longest unported chain: 7/44 (84.1% progress)

port-progress bot (Jan 15 2023 at 18:14):

mathlib port progress order.filter.basic
Ported files: 236/278 (84.9% of total)
Ported lines: 91446/111657 (81.9% of total)
Longest unported chain: 10/47 (78.7% progress)

port-progress bot (Jan 15 2023 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18773/31931 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 15 2023 at 18:21):

mathlib port progress linear_algebra.basic
Ported files: 296/365 (81.1% of total)
Ported lines: 110315/148186 (74.4% of total)
Longest unported chain: 15/52 (71.2% progress)

port-progress bot (Jan 15 2023 at 18:25):

mathlib port progress data.complex.basic
Ported files: 359/573 (62.7% of total)
Ported lines: 123759/244474 (50.6% of total)
Longest unported chain: 42/79 (46.8% progress)

port-progress bot (Jan 15 2023 at 18:29):

mathlib port progress topology.metric_space.basic
Ported files: 349/521 (67.0% of total)
Ported lines: 122080/226275 (54.0% of total)
Longest unported chain: 36/73 (50.7% progress)

port-progress bot (Jan 15 2023 at 18:56):

mathlib port progress all
Ported files: 511/2863 (17.8% of total)
Ported lines: 146142/982653 (14.9% of total)
Longest unported chain: 89/126 (29.4% progress)

Ruben Van de Velde (Jan 16 2023 at 08:22):

Anyone up for data.finset.image?

Johan Commelin (Jan 16 2023 at 08:23):

Go ahead!

Johan Commelin (Jan 16 2023 at 08:23):

That one will unblock 4 or 5 other things, I think

Johan Commelin (Jan 16 2023 at 08:24):

If you pick data.finset.image then I'll start on data.finset.order.

Johan Commelin (Jan 16 2023 at 08:26):

ooh, that one is tiny

Johan Commelin (Jan 16 2023 at 08:32):

done

Johan Commelin (Jan 16 2023 at 09:03):

@Scott Morrison Now that real.basic and fintype.basic are almost done, could you please add number_theory.legendre_symbol.quadratic_reciprocity to the list?

Ruben Van de Velde (Jan 16 2023 at 09:38):

Ruben Van de Velde said:

Anyone up for data.finset.image?

@Chris Hughes did - can you make the PR?

Ruben Van de Velde (Jan 16 2023 at 10:43):

Ruben Van de Velde said:

Ruben Van de Velde said:

Anyone up for data.finset.image?

Chris Hughes did - can you make the PR?

mathlib4#1586 should be good to go and unblock data.finset.{pi,card,fold}, I think

Johan Commelin (Jan 16 2023 at 12:20):

#port-status has some juicy stuff available!

Ruben Van de Velde (Jan 16 2023 at 12:22):

Claiming data.finset.fold

Eric Rodriguez (Jan 16 2023 at 12:26):

why is everything these days in "Earlier items in the list are required in more places in mathlib." as opposed to "The following files have all dependencies ported already, and should be ready to port:"?

Ruben Van de Velde (Jan 16 2023 at 12:41):

I think "Earlier items" shouldn't be a header

Mario Carneiro (Jan 16 2023 at 12:43):

it's not, here's the port_status.py code:

print('# The following files have all dependencies ported already, and should be ready to port:')
print('# Earlier items in the list are required in more places in mathlib.')
allDone = dict(sorted(allDone.items(), key=lambda item: -item[1][0]))
for k, v in allDone.items():
    if v[1] == "":
        print(k)
    else:
        print(k + "    -- " + v[1])

print()

this is translated to HTML by johan's bot, which I guess results in multiple headers for the two lines

Anne Baanen (Jan 16 2023 at 12:45):

I'm claiming algebra.module.linear_map :)

Ruben Van de Velde (Jan 16 2023 at 12:52):

I'm guessing the # is treated as a markdown header

Ruben Van de Velde (Jan 16 2023 at 12:53):

Moving on to card

Ruben Van de Velde (Jan 16 2023 at 13:29):

Could someone take a look at the termination_by issues in mathlib4#1589? I never manage to get those right

Kevin Buzzard (Jan 16 2023 at 14:06):

If I type

leanproject import-graph --to group_theory.monoid_localization --exclude-tactics --reduce --port-status --exclude-ported --show-unused group_theory.monoid_localization.pdf

into my home PC I get a graph. If I type it into my laptop I get

The node group_theory.monoid_localization is not in the digraph.

Is this something to do with not having enough graph library installed?

Ruben Van de Velde (Jan 16 2023 at 14:35):

Chris finished Data.Finset.Card mathlib4#1589 which should unblock data.finset.{option,prod,sum}

Eric Wieser (Jan 16 2023 at 14:51):

Is this something to do with not having enough graph library installed?

Sounds like they have different versions of mathlib checked out

port-progress bot (Jan 16 2023 at 18:04):

mathlib port progress data.real.basic
Ported files: 219/229 (95.6% of total)
Ported lines: 82430/86444 (95.4% of total)
Longest unported chain: 1/34 (97.1% progress)

port-progress bot (Jan 16 2023 at 18:07):

mathlib port progress data.fintype.basic
Ported files: 175/184 (95.1% of total)
Ported lines: 78991/83547 (94.5% of total)
Longest unported chain: 1/40 (97.5% progress)

port-progress bot (Jan 16 2023 at 18:11):

mathlib port progress algebra.big_operators.basic
Ported files: 202/216 (93.5% of total)
Ported lines: 86229/94822 (90.9% of total)
Longest unported chain: 3/44 (93.2% progress)

Reid Barton (Jan 16 2023 at 18:12):

data.real.basic is also almost done

port-progress bot (Jan 16 2023 at 18:15):

mathlib port progress order.filter.basic
Ported files: 242/278 (87.1% of total)
Ported lines: 95698/111708 (85.7% of total)
Longest unported chain: 8/47 (83.0% progress)

port-progress bot (Jan 16 2023 at 18:19):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18773/31931 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 16 2023 at 18:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 395/1016 (38.9% of total)
Ported lines: 134016/436048 (30.7% of total)
Longest unported chain: 64/103 (37.9% progress)

Ruben Van de Velde (Jan 16 2023 at 18:24):

395/1016, ouch

port-progress bot (Jan 16 2023 at 18:27):

mathlib port progress linear_algebra.basic
Ported files: 303/365 (83.0% of total)
Ported lines: 114924/148252 (77.5% of total)
Longest unported chain: 13/52 (75.0% progress)

port-progress bot (Jan 16 2023 at 18:31):

mathlib port progress data.complex.basic
Ported files: 367/573 (64.0% of total)
Ported lines: 128414/244560 (52.5% of total)
Longest unported chain: 40/79 (49.4% progress)

port-progress bot (Jan 16 2023 at 18:34):

mathlib port progress topology.metric_space.basic
Ported files: 358/521 (68.7% of total)
Ported lines: 127736/226347 (56.4% of total)
Longest unported chain: 34/73 (53.4% progress)

port-progress bot (Jan 16 2023 at 19:02):

mathlib port progress all
Ported files: 525/2863 (18.3% of total)
Ported lines: 152170/982925 (15.5% of total)
Longest unported chain: 87/126 (31.0% progress)

Michael Stoll (Jan 16 2023 at 19:34):

Ruben Van de Velde said:

395/1016, ouch

Meaningful number theory uses a lot of other stuff :smile:

Kevin Buzzard (Jan 16 2023 at 20:11):

I definitely second that, and it's one of the reasons I've been vocally behind one repository containing lots of pure maths since 2017. The proof of FLT uses topology, geometry, algebra, analysis, ...

Jason Rute (Jan 17 2023 at 04:16):

I was just curious how fast the port is going over time, so I wrote a simple (and brittle) web scrapping script to get the progress from this thread for the "all" tables and here is the resulting plot: Screen-Shot-2023-01-16-at-11.13.41-PM.png

James Gallicchio (Jan 17 2023 at 04:23):

Y'know part of me was hoping it would look less linear :sweat_smile:

Heather Macbeth (Jan 17 2023 at 04:25):

This is great! We should add it to the stats page
https://leanprover-community.github.io/mathlib_stats.html

James Gallicchio (Jan 17 2023 at 04:32):

Where are the mathlib3 stats calculated? Can we just do the same calculation for the mathlib4 repo and overlay it? (I mean quite literally the same calculation, just total number of files and lines)

James Gallicchio (Jan 17 2023 at 05:04):

Ah, here: https://github.com/leanprover-community/mathlib_stats

Eric Wieser (Jan 17 2023 at 11:20):

Note that if we measure lines in mathlib4, the graphs will cross before the port is done

Johan Commelin (Jan 17 2023 at 13:21):

algebra.big_operators.basic is ready!

Johan Commelin (Jan 17 2023 at 13:22):

Let's knock down those targets!

Ruben Van de Velde (Jan 17 2023 at 13:30):

Already > 30 PRs landed today - how many can we manage? :)

Johan Commelin (Jan 17 2023 at 13:32):

Top of #port-status currently looks like

data.fin.tuple.basic  mathlib4#1516 7c523cb78f4153682c2929e3006c863bfef463d0 if possible please wait for mathlib#10346
algebra.big_operators.basic
data.fintype.sigma
order.sup_indep
algebra.module.linear_map  mathlib4#1587 9003f28797c0664a49e4179487267c494477d853
order.omega_complete_partial_order  mathlib4#1168 9116dd6709f303dcf781632e15fdef382b0fc579
data.enat.basic  mathlib4#1531 9003f28797c0664a49e4179487267c494477d853
ring_theory.congruence
data.fintype.list
control.traversable.instances  mathlib4#1393 18a5306c091183ac90884daa9373fa3b178e8607
order.hom.lattice

Johan Commelin (Jan 17 2023 at 13:32):

I think data.fintype.sigma is already done

Johan Commelin (Jan 17 2023 at 13:35):

I'm going to start algebra.big_operators.basic.

Johan Commelin (Jan 17 2023 at 13:36):

(If someone else did, please ping here.)

Ruben Van de Velde (Jan 17 2023 at 13:37):

Looking at sup_indep

port-progress bot (Jan 17 2023 at 18:03):

mathlib port progress data.real.basic
Ported files: 220/229 (96.1% of total)
Ported lines: 83112/86454 (96.1% of total)
Longest unported chain: 1/34 (97.1% progress)

port-progress bot (Jan 17 2023 at 18:07):

mathlib port progress algebra.big_operators.basic
Ported files: 207/216 (95.8% of total)
Ported lines: 89374/94832 (94.2% of total)
Longest unported chain: 1/44 (97.7% progress)

port-progress bot (Jan 17 2023 at 18:10):

mathlib port progress order.filter.basic
Ported files: 251/278 (90.3% of total)
Ported lines: 100086/111813 (89.5% of total)
Longest unported chain: 7/47 (85.1% progress)

port-progress bot (Jan 17 2023 at 18:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18783/31941 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

Johan Commelin (Jan 17 2023 at 18:16):

The links to the graphs are broken for me.

port-progress bot (Jan 17 2023 at 18:19):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 418/1018 (41.1% of total)
Ported lines: 143140/436989 (32.8% of total)
Longest unported chain: 63/103 (38.8% progress)

port-progress bot (Jan 17 2023 at 18:22):

mathlib port progress linear_algebra.basic
Ported files: 315/365 (86.3% of total)
Ported lines: 120003/148383 (80.9% of total)
Longest unported chain: 11/52 (78.8% progress)

port-progress bot (Jan 17 2023 at 18:26):

mathlib port progress data.complex.basic
Ported files: 386/573 (67.4% of total)
Ported lines: 136531/244691 (55.8% of total)
Longest unported chain: 38/79 (51.9% progress)

port-progress bot (Jan 17 2023 at 18:30):

mathlib port progress topology.metric_space.basic
Ported files: 374/521 (71.8% of total)
Ported lines: 134430/226478 (59.4% of total)
Longest unported chain: 32/73 (56.2% progress)

Kevin Buzzard (Jan 17 2023 at 18:36):

Johan Commelin said:

The links to the graphs are broken for me.

They're working for me.

Johan Commelin (Jan 17 2023 at 18:36):

Aah, now they also work on my side

port-progress bot (Jan 17 2023 at 19:00):

mathlib port progress all
Ported files: 553/2865 (19.3% of total)
Ported lines: 161763/983915 (16.4% of total)
Longest unported chain: 85/126 (32.5% progress)

Johan Commelin (Jan 17 2023 at 19:02):

0.9%

Kevin Buzzard (Jan 17 2023 at 19:05):

We have ported almost 20% of mathlib!

Chris Hughes (Jan 17 2023 at 19:14):

Johan Commelin said:

The links to the graphs are broken for me.

The graphs for already ported files don't work

Johan Commelin (Jan 17 2023 at 19:29):

@Kevin Buzzard I think #{ported lines} is a better measure than #{ported files}

Chris Hughes (Jan 17 2023 at 19:47):

Johan Commelin said:

Kevin Buzzard I think #{ported lines} is a better measure than #{ported files}

I think ported files is better because the number is bigger

Yaël Dillies (Jan 17 2023 at 20:48):

No, ported lines is better. But you have to count the number of ported lines in mathlib, as mathlib4 inflates that number.

Johan Commelin (Jan 17 2023 at 20:49):

@Yaël Dillies I thought that's already what is happening?

Yaël Dillies (Jan 17 2023 at 20:51):

Then why did @Eric Wieser claim that we couldn't overlay the graphs because they would cross before the port was over?

Eric Wieser (Jan 17 2023 at 20:52):

Because mathlib3 files often end up bigger when ported into mathlib4 files.

Yaël Dillies (Jan 17 2023 at 20:53):

... which is why I'm suggesting counting the number of mathlib3 lines ported, rather than the number of lines in mathlib4

Yaël Dillies (Jan 17 2023 at 20:55):

Namely, finset.sum ported_files (\lambda file, file.number_of_lines)

Patrick Massot (Jan 17 2023 at 20:56):

We are already counting lines in mathlib3.

Damiano Testa (Jan 17 2023 at 20:56):

golf:

ported_files.sum (\lambda file, file.number_of_lines)

Yaël Dillies (Jan 17 2023 at 20:57):

Then I see no problem with the current approach

Yaël Dillies (Jan 17 2023 at 20:58):

Damiano, I didn't want to look obscure, but ported_files.sum number_of_lines is the golfest.

Eric Wieser (Jan 17 2023 at 21:09):

Yaël Dillies said:

... which is why I'm suggesting counting the number of mathlib3 lines ported, rather than the number of lines in mathlib4

Well, you asked why i said they would cross, and if you look at my message I was talking about counting mathlib4 lines. Indeed, if you are counting mathlib3 lines everything is fine :)

port-progress bot (Jan 18 2023 at 18:04):

mathlib port progress algebra.big_operators.basic
Ported files: 208/216 (96.3% of total)
Ported lines: 91313/94856 (96.3% of total)
Longest unported chain: 1/44 (97.7% progress)

Johan Commelin (Jan 18 2023 at 18:07):

@Scott Morrison :this: can be removed from your list of targets

port-progress bot (Jan 18 2023 at 18:08):

mathlib port progress order.filter.basic
Ported files: 254/278 (91.4% of total)
Ported lines: 100799/111852 (90.1% of total)
Longest unported chain: 5/47 (89.4% progress)

port-progress bot (Jan 18 2023 at 18:12):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18783/31941 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 18 2023 at 18:17):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 428/1020 (42.0% of total)
Ported lines: 146423/437212 (33.5% of total)
Longest unported chain: 61/103 (40.8% progress)

port-progress bot (Jan 18 2023 at 18:22):

mathlib port progress linear_algebra.basic
Ported files: 319/365 (87.4% of total)
Ported lines: 122479/148425 (82.5% of total)
Longest unported chain: 10/52 (80.8% progress)

port-progress bot (Jan 18 2023 at 18:26):

mathlib port progress data.complex.basic
Ported files: 390/573 (68.1% of total)
Ported lines: 139013/244739 (56.8% of total)
Longest unported chain: 37/79 (53.2% progress)

port-progress bot (Jan 18 2023 at 18:30):

mathlib port progress topology.metric_space.basic
Ported files: 378/521 (72.6% of total)
Ported lines: 136912/226526 (60.4% of total)
Longest unported chain: 31/73 (57.5% progress)

port-progress bot (Jan 18 2023 at 19:05):

mathlib port progress all
Ported files: 564/2871 (19.6% of total)
Ported lines: 164795/984604 (16.7% of total)
Longest unported chain: 84/126 (33.3% progress)

Johan Commelin (Jan 18 2023 at 19:09):

0.3%

Johan Commelin (Jan 19 2023 at 11:56):

data.array.lemmas
data.fintype.lattice
data.fintype.prod
data.fintype.sum
data.fintype.powerset
data.sym.basic  mathlib4#1672 509de852e1de55e1efa8eacfa11df0823f26f226
data.fin.vec_notation  Waiting for forward port of mathlib#10346
data.finset.noncomm_prod
data.fintype.option
algebra.big_operators.order
algebra.big_operators.pi
data.finite.set

Top of #port-status

Eric Wieser (Jan 19 2023 at 11:59):

file#data/array/lemmas is surely a false positive? Did we even port Array?

Johan Commelin (Jan 19 2023 at 12:04):

@Eric Wieser Nope, it's not.

Johan Commelin (Jan 19 2023 at 12:04):

It's imported by legit low-level files

Eric Wieser (Jan 19 2023 at 12:07):

Let's not port it yet

Eric Wieser (Jan 19 2023 at 12:07):

I think we should try and shuffle dependencies so that it's not needed (edit: starting with #18226)

Notification Bot (Jan 19 2023 at 12:10):

8 messages were moved from this topic to #mathlib4 > Updating SHAs for modified files by Eric Wieser.

Johan Commelin (Jan 19 2023 at 12:12):

@Eric Wieser Do you think we can have a separate section of "longest unported chain of deps = 1" files?

Reid Barton (Jan 19 2023 at 12:12):

Seems reasonable.

Johan Commelin (Jan 19 2023 at 12:12):

Then we can detect such files that need a ml3 reshuffle a bit earlier.

Johan Commelin (Jan 19 2023 at 12:13):

Again, that section should be sorted by "importancy", like #port-status is

Eric Wieser (Jan 19 2023 at 12:14):

That's not that different from the table at https://leanprover-community.github.io/mathlib-port-status, is it? Scrolling to the yellow and uncolored rows gives a good estimate of that information

Johan Commelin (Jan 19 2023 at 12:16):

Aah, fair enough

Johan Commelin (Jan 19 2023 at 12:16):

Eric Wieser said:

I think we should try and shuffle dependencies so that it's not needed (edit: starting with #18226)

Thanks for starting the PR

Johan Commelin (Jan 19 2023 at 12:16):

Do you think you can break this edge as well?

src/logic/equiv/list.lean
6:import data.array.lemmas

Eric Wieser (Jan 19 2023 at 12:24):

Yes, I'll put that in the same PR

Eric Wieser (Jan 19 2023 at 12:28):

Done, lets see what CI has to say

Eric Wieser (Jan 19 2023 at 12:34):

Also added a comment to #port-wiki, but I guess that propagates slowly

Ruben Van de Velde (Jan 19 2023 at 12:37):

@Eric Wieser, in case you weren't watching CI closely :)

Error: /home/lean/actions-runner/_work/mathlib/mathlib/src/computability/primrec.lean:1043:12:
unknown identifier 'equiv.array_equiv_fin'

Eric Wieser (Jan 19 2023 at 12:38):

Seems you weren't watching CI closely, already fixed :)

Johan Commelin (Jan 19 2023 at 12:39):

Eric Wieser said:

Also added a comment to #port-wiki, but I guess that propagates slowly

It's on #port-status already :wink:

Eric Wieser (Jan 19 2023 at 12:39):

Eric Wieser said:

Also added a comment to #port-wiki, but I guess that propagates slowly

@Johan Commelin, could you modify start_port.sh to include any comments from the yaml file in the commit message when people make PRs? Sometimes people don't read the comments before starting, and that way the reviewers would see them.

Kevin Buzzard (Jan 19 2023 at 14:31):

If we're looking for something new to track, polynomials would be an interesting one. It needs finsupp but it's the key to a lot of algebra.

port-progress bot (Jan 19 2023 at 18:03):

mathlib port progress order.filter.basic
Ported files: 262/278 (94.2% of total)
Ported lines: 103242/111870 (92.3% of total)
Longest unported chain: 5/47 (89.4% progress)

port-progress bot (Jan 19 2023 at 18:07):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18783/31941 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 19 2023 at 18:12):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 445/1020 (43.6% of total)
Ported lines: 149982/437246 (34.3% of total)
Longest unported chain: 61/103 (40.8% progress)

port-progress bot (Jan 19 2023 at 18:15):

mathlib port progress linear_algebra.basic
Ported files: 329/365 (90.1% of total)
Ported lines: 125426/148449 (84.5% of total)
Longest unported chain: 10/52 (80.8% progress)

port-progress bot (Jan 19 2023 at 18:19):

mathlib port progress data.complex.basic
Ported files: 404/573 (70.5% of total)
Ported lines: 142358/244833 (58.1% of total)
Longest unported chain: 37/79 (53.2% progress)

port-progress bot (Jan 19 2023 at 18:23):

mathlib port progress topology.metric_space.basic
Ported files: 391/521 (75.0% of total)
Ported lines: 140179/226562 (61.9% of total)
Longest unported chain: 31/73 (57.5% progress)

Johan Commelin (Jan 19 2023 at 18:48):

Eric Wieser said:

I think we should try and shuffle dependencies so that it's not needed (edit: starting with #18226)

Hooray! array.lemmas is gone from #port-status

port-progress bot (Jan 19 2023 at 18:50):

mathlib port progress all
Ported files: 581/2874 (20.2% of total)
Ported lines: 168694/984966 (17.1% of total)
Longest unported chain: 84/126 (33.3% progress)

Johan Commelin (Jan 19 2023 at 18:52):

0.4%

Eric Rodriguez (Jan 20 2023 at 00:13):

is there a #queue4?

Eric Rodriguez (Jan 20 2023 at 00:13):

nice

Johan Commelin (Jan 20 2023 at 12:40):

I merged Data.Sym.Basic. So now Data.Fintype.Vector is up for grabs. It's on the critical path to https://tqft.net/mathlib4/latest/order.filter.basic.pdf

I'm afk for ~45m, so I will not claim Data.Fintype.Vector yet.

Johan Commelin (Jan 20 2023 at 13:27):

Started the PR at mathlib4#1716

port progress bot (jmc) (Jan 20 2023 at 20:48):

mathlib port progress order.filter.basic
Ported files: 265/276 (96.0% of total)
Ported lines: 103885/111444 (93.2% of total)
Longest unported chain: 1/47 (97.9% progress)

Johan Commelin (Jan 20 2023 at 20:49):

Almost there!

port progress bot (jmc) (Jan 20 2023 at 20:50):

mathlib port progress linear_algebra.basic
Ported files: 336/363 (92.6% of total)
Ported lines: 128402/147731 (86.9% of total)
Longest unported chain: 8/52 (84.6% progress)

port progress bot (jmc) (Jan 20 2023 at 20:53):

mathlib port progress topology.metric_space.basic
Ported files: 402/522 (77.0% of total)
Ported lines: 144610/226133 (63.9% of total)
Longest unported chain: 28/73 (61.6% progress)

port progress bot (jmc) (Jan 20 2023 at 20:55):

mathlib port progress data.polynomial.basic
Ported files: 355/399 (89.0% of total)
Ported lines: 131997/161864 (81.5% of total)
Longest unported chain: 14/58 (75.9% progress)

Johan Commelin (Jan 20 2023 at 20:56):

Oooh! We are closer to polynomials than to metric spaces! Maybe not so surprising after all.

port progress bot (jmc) (Jan 20 2023 at 20:57):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18783/31941 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

Ruben Van de Velde (Jan 20 2023 at 21:00):

That's a looot of gray nodes for polynomials too

port progress bot (jmc) (Jan 20 2023 at 21:00):

mathlib port progress data.complex.basic
Ported files: 416/574 (72.5% of total)
Ported lines: 147075/244405 (60.2% of total)
Longest unported chain: 34/79 (57.0% progress)

port progress bot (jmc) (Jan 20 2023 at 21:03):

mathlib port progress all
Ported files: 609/2881 (21.1% of total)
Ported lines: 174607/985636 (17.7% of total)
Longest unported chain: 82/126 (34.9% progress)

Johan Commelin (Jan 20 2023 at 21:08):

0.6%

Xavier Roblot (Jan 21 2023 at 05:52):

I updated the list of targets on the wiki page. All the targets listed there have been already completed :)

Reid Barton (Jan 21 2023 at 06:55):

Can I vote for replacing topology.metric_space.basic by topology.basic? the metric space one is still basically infinitely far away

Johan Commelin (Jan 21 2023 at 08:24):

@Reid Barton Voila: https://math.commelin.net/files/mathlib4/2023-01-21/topology.basic.pdf

port progress bot (jmc) (Jan 21 2023 at 19:49):

mathlib port progress order.filter.basic
Ported files: 266/276 (96.4% of total)
Ported lines: 105194/111500 (94.3% of total)
Longest unported chain: 1/47 (97.9% progress)

port progress bot (jmc) (Jan 21 2023 at 19:51):

mathlib port progress linear_algebra.basic
Ported files: 337/361 (93.4% of total)
Ported lines: 129689/147179 (88.1% of total)
Longest unported chain: 8/52 (84.6% progress)

port progress bot (jmc) (Jan 21 2023 at 19:54):

mathlib port progress topology.basic
Ported files: 308/332 (92.8% of total)
Ported lines: 117597/132069 (89.0% of total)
Longest unported chain: 8/53 (84.9% progress)

port progress bot (jmc) (Jan 21 2023 at 19:56):

mathlib port progress data.polynomial.basic
Ported files: 360/399 (90.2% of total)
Ported lines: 134041/161791 (82.8% of total)
Longest unported chain: 14/58 (75.9% progress)

port progress bot (jmc) (Jan 21 2023 at 19:58):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18783/31941 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port progress bot (jmc) (Jan 21 2023 at 20:01):

mathlib port progress data.complex.basic
Ported files: 422/575 (73.4% of total)
Ported lines: 149374/244576 (61.1% of total)
Longest unported chain: 34/79 (57.0% progress)

port progress bot (jmc) (Jan 21 2023 at 20:04):

mathlib port progress all
Ported files: 619/2884 (21.5% of total)
Ported lines: 177377/986150 (18.0% of total)
Longest unported chain: 80/125 (36.0% progress)

James Gallicchio (Jan 21 2023 at 22:00):

0.3% :}

Eric Rodriguez (Jan 21 2023 at 22:08):

what are these numbers meant to represent?

James Gallicchio (Jan 21 2023 at 22:10):

Johan has been posting the daily delta for % of lines ported. Good measure for progress.

Johan Commelin (Jan 21 2023 at 22:10):

percentage of total number of lines ported in the past day.

port-progress bot (Jan 22 2023 at 18:03):

mathlib port progress order.filter.basic
Ported files: 266/276 (96.4% of total)
Ported lines: 105194/111494 (94.3% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Jan 22 2023 at 18:07):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18783/31941 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

Trebor Huang (Jan 22 2023 at 18:08):

We might let the bot do the difference calculation. Or is doing arithmetic once a day not really worth the hassle of maintaining stateful bots?

port-progress bot (Jan 22 2023 at 18:11):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 470/1022 (46.0% of total)
Ported lines: 157103/436013 (36.0% of total)
Longest unported chain: 59/103 (42.7% progress)

port-progress bot (Jan 22 2023 at 18:14):

mathlib port progress linear_algebra.basic
Ported files: 336/359 (93.6% of total)
Ported lines: 129216/145986 (88.5% of total)
Longest unported chain: 8/52 (84.6% progress)

port-progress bot (Jan 22 2023 at 18:18):

mathlib port progress data.complex.basic
Ported files: 421/573 (73.5% of total)
Ported lines: 148901/243379 (61.2% of total)
Longest unported chain: 34/79 (57.0% progress)

port-progress bot (Jan 22 2023 at 18:21):

mathlib port progress topology.metric_space.basic
Ported files: 407/521 (78.1% of total)
Ported lines: 146436/225105 (65.1% of total)
Longest unported chain: 28/73 (61.6% progress)

port-progress bot (Jan 22 2023 at 18:46):

mathlib port progress all
Ported files: 622/2886 (21.6% of total)
Ported lines: 178141/986471 (18.1% of total)
Longest unported chain: 80/125 (36.0% progress)

Anand Rao (Jan 23 2023 at 04:41):

Would it be possible to add combinatorics.simple_graph.basic as a porting target?

Johan Commelin (Jan 23 2023 at 05:18):

cc @Scott Morrison

James Gallicchio (Jan 23 2023 at 13:11):

Anand Rao said:

Would it be possible to add combinatorics.simple_graph.basic as a porting target?

unless i'm mistaken it looks like we just need to port data.sym.sym2 and then it's able to be ported

Patrick Massot (Jan 23 2023 at 14:09):

I wanted to know the current porting speed so I just spent half an hour playing with python. For curious people, I'll let the code here. First we need to download messages, assuming you have the zulip python package and a .zuliprc in your home, first use this script:

from pathlib import Path
import pickle
import zulip

# Pass the path to your zuliprc file here.
client = zulip.Client(config_file="~/.zuliprc")

request = {
    "anchor": "newest",
    "num_before": 1500,
    "num_after": 0,
    "narrow": [
        {"operator": "stream", "operand": "mathlib4"},
        {"operator": "sender", "operand": "port-progress-bot@leanprover.zulipchat.com "}
    ],
    "apply_markdown": False
}
results = client.get_messages(request)

# Let's save the result to avoid hitting an API rate limit while testing
pickle.dump(results, open('progress.pickle', 'wb'))

This will create a file progress.pickle with raw output. Then you can play with it in another script (if you don't split this in download then play and play too much then you'll hit some API rate limit).

  from pathlib import Path
  from datetime import datetime
  import re
import pickle

results = pickle.load(open('progress.pickle', "rb"))

reg = re.compile(r'\(([^%]*)')

stats = open('stats.csv', 'w')
prev = 1.2

for msg in results['messages']:
    content = msg['content']
    if not "all.pdf" in content:
        continue
    stamp = int(msg['timestamp'])
    lines = content.split('\n')
    cols = lines[3].split('|')
    m = reg.match(cols[3].strip())
    if not m:
        continue
    stat = float(m.group(1))
    stats.write(f"{datetime.fromtimestamp(stamp).date()}, {stat}, {stat - prev}\n")
    prev = stat

This will create stats.csv with three columns: date, proportion of ported lines, progress since previous data point. Be careful that the bot has been slightly chaotic, don't assume there is one line per day.


Patrick Massot (Jan 23 2023 at 14:11):

The current output is

Johan Commelin (Jan 23 2023 at 14:12):

Thanks for putting this together!

Johan Commelin (Jan 23 2023 at 14:15):

@Patrick Massot Maybe you can teach it to also scrape output from my bot? That would fill in some of the gaps.

Patrick Massot (Jan 23 2023 at 14:19):

How is your bot called?

Reid Barton (Jan 23 2023 at 14:19):

port progress bot (jmc)

Johan Commelin (Jan 23 2023 at 14:22):

@Patrick Massot And maybe use {stat - prev:.1f}to print the final column? That way you print only 1 decimal place.

Patrick Massot (Jan 23 2023 at 14:31):

Updated scripts:

from pathlib import Path
import pickle
import zulip

# Pass the path to your zuliprc file here.
client = zulip.Client(config_file="~/.zuliprc")

request = {
    "anchor": "newest",
    "num_before": 1500,
    "num_after": 0,
    "narrow": [
        {"operator": "stream", "operand": "mathlib4"},
        {"operator": "sender", "operand": "port-progress-bot@leanprover.zulipchat.com"}
    ],
    "apply_markdown": False
}
results = client.get_messages(request)

request = {
    "anchor": "newest",
    "num_before": 1500,
    "num_after": 0,
    "narrow": [
        {"operator": "stream", "operand": "mathlib4"},
        {"operator": "sender", "operand": "port-progress-jmc-bot@leanprover.zulipchat.com"}
    ],
    "apply_markdown": False
}
results['messages'].extend(client.get_messages(request)['messages'])

# Let's save the result to avoid hitting an API rate limit while testing
pickle.dump(results, open('progress.pickle', 'wb'))

msgs = [msg for msg in results['messages'] if "all.pdf" in msg]
Path('portmsgs').write_text(str(msgs))

and

from pathlib import Path
from datetime import datetime
import re
import pickle

results = pickle.load(open('progress.pickle', "rb"))

reg = re.compile(r'\(([^%]*)')

stats = open('stats.csv', 'w')
prev = 1.2

for msg in sorted(results['messages'], key=lambda msg: msg['timestamp']):
    content = msg['content']
    if not "all.pdf" in content:
        continue
    stamp = int(msg['timestamp'])
    lines = content.split('\n')
    cols = lines[3].split('|')
    m = reg.match(cols[3].strip())
    if not m:
        continue
    stat = float(m.group(1))
    stats.write(f"{datetime.fromtimestamp(stamp).date()}, {stat}, {stat - prev:.1f}\n")
    prev = stat

Patrick Massot (Jan 23 2023 at 14:32):

Updated output

Yakov Pechersky (Jan 23 2023 at 16:21):

I assume the bot works by checking out the repository, then running some script to get the graphs and the values. You could add a step where you check out a commit at a previous date like git checkout 'master@{1979-02-26 18:30:00}' but with the time a day ago (https://stackoverflow.com/a/6990682), calculate the stats, and do the delta calculation

Eric Wieser (Jan 23 2023 at 16:23):

I think it's messier than that because the bot works by scraping the wiki page and checking out mathlib HEAD

Eric Wieser (Jan 23 2023 at 16:23):

The wiki page is just generated by another bot though!

Johan Commelin (Jan 23 2023 at 16:23):

I think we're mostly interested in seeing trends, so maybe it's not worth the effort.
Calculating the stats is quite expensive. The bot usually runs for ~30 mins to do the calculations for a single day.

Eric Wieser (Jan 23 2023 at 16:26):

Isn't 95% of that work producing the chains though?

Eric Wieser (Jan 23 2023 at 16:26):

Computing the number of ported lines/files should be super cheap

Adam Topaz (Jan 23 2023 at 17:15):

Today is the first time I'm trying to port something since before the start_port script was created. Do we need to manually change the port status page like in the olden days, or is this automatic now?

Eric Wieser (Jan 23 2023 at 17:22):

#port-status is generated automatically (on GitHub every half hour) from #port-wiki which is generated automatically (on Reid's server every ???) by reading the mathlib4 history, the open mathlib4 PRs, and https://github.com/leanprover-community/mathlib4/wiki/port-comments/_edit

Eric Wieser (Jan 23 2023 at 17:24):

So it's automatic once you create the PR I think

Adam Topaz (Jan 23 2023 at 17:24):

okay great. Thanks

Johan Commelin (Jan 23 2023 at 17:30):

#port-wiki is also generated every half hour, on my server.

Johan Commelin (Jan 23 2023 at 17:31):

@Eric Wieser it runs 0 mod 30.

Eric Wieser (Jan 23 2023 at 17:31):

When does it usually complete?

Johan Commelin (Jan 23 2023 at 17:31):

Should I make that -5 mod 30?

Johan Commelin (Jan 23 2023 at 17:32):

Done

Eric Wieser (Jan 23 2023 at 17:32):

Yes, because the webpage is running at 0 mod 30 also :)

Eric Wieser (Jan 23 2023 at 17:33):

Although in practice it seems the github cron job is running 5 minutes behind anyway

port-progress bot (Jan 23 2023 at 18:02):

mathlib port progress order.filter.basic
Ported files: 263/272 (96.7% of total)
Ported lines: 107451/111134 (96.7% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Jan 23 2023 at 18:06):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18793/31951 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 23 2023 at 18:10):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 476/1027 (46.3% of total)
Ported lines: 161907/436701 (37.1% of total)
Longest unported chain: 58/103 (43.7% progress)

port-progress bot (Jan 23 2023 at 18:13):

mathlib port progress linear_algebra.basic
Ported files: 333/355 (93.8% of total)
Ported lines: 129313/145683 (88.8% of total)
Longest unported chain: 7/52 (86.5% progress)

port-progress bot (Jan 23 2023 at 18:17):

mathlib port progress data.complex.basic
Ported files: 425/573 (74.2% of total)
Ported lines: 153547/243584 (63.0% of total)
Longest unported chain: 33/79 (58.2% progress)

port-progress bot (Jan 23 2023 at 18:21):

mathlib port progress topology.metric_space.basic
Ported files: 411/521 (78.9% of total)
Ported lines: 151076/225304 (67.1% of total)
Longest unported chain: 27/73 (63.0% progress)

port-progress bot (Jan 23 2023 at 18:45):

mathlib port progress all
Ported files: 636/2887 (22.0% of total)
Ported lines: 185138/986704 (18.8% of total)
Longest unported chain: 79/125 (36.8% progress)

James Gallicchio (Jan 23 2023 at 20:17):

+0.7% lines :0 y'all are cruising

Johan Commelin (Jan 24 2023 at 06:40):

@porters I added #port-comments as linkifier to the wiki page where you can add comments about files.

Yury G. Kudryashov (Jan 24 2023 at 06:52):

Can you add me to @ porters?

Johan Commelin (Jan 24 2023 at 06:52):

It doesn't actually exist. But I guess it makes sense to make it.

port-progress bot (Jan 24 2023 at 18:03):

mathlib port progress order.filter.basic
Ported files: 263/272 (96.7% of total)
Ported lines: 107461/111144 (96.7% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Jan 24 2023 at 18:07):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18793/31951 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

Patrick Massot (Jan 24 2023 at 18:07):

@Scott Morrison order.filter.basic should be removed, it has been ported. Also it may be nice to tweak the computation to remove files that typically won't be ported, so that a ported file hits 100% porting.

port-progress bot (Jan 24 2023 at 18:11):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 492/1020 (48.2% of total)
Ported lines: 168174/435032 (38.7% of total)
Longest unported chain: 57/103 (44.7% progress)

port-progress bot (Jan 24 2023 at 18:14):

mathlib port progress linear_algebra.basic
Ported files: 335/355 (94.4% of total)
Ported lines: 129875/145704 (89.1% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Jan 24 2023 at 18:18):

mathlib port progress data.complex.basic
Ported files: 436/571 (76.4% of total)
Ported lines: 158979/243261 (65.4% of total)
Longest unported chain: 28/79 (64.6% progress)

port-progress bot (Jan 24 2023 at 18:21):

mathlib port progress topology.metric_space.basic
Ported files: 423/521 (81.2% of total)
Ported lines: 156851/225350 (69.6% of total)
Longest unported chain: 22/73 (69.9% progress)

port-progress bot (Jan 24 2023 at 18:43):

mathlib port progress all
Ported files: 656/2889 (22.7% of total)
Ported lines: 192930/987461 (19.5% of total)
Longest unported chain: 74/125 (40.8% progress)

Johan Commelin (Jan 24 2023 at 20:32):

0.8%

port-progress bot (Jan 25 2023 at 18:02):

mathlib port progress order.filter.basic
Ported files: 263/272 (96.7% of total)
Ported lines: 107496/111179 (96.7% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Jan 25 2023 at 18:06):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18794/31952 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 25 2023 at 18:10):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 493/1017 (48.5% of total)
Ported lines: 168754/434160 (38.9% of total)
Longest unported chain: 57/103 (44.7% progress)

port-progress bot (Jan 25 2023 at 18:13):

mathlib port progress linear_algebra.basic
Ported files: 335/355 (94.4% of total)
Ported lines: 129998/145841 (89.1% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Jan 25 2023 at 18:17):

mathlib port progress data.complex.basic
Ported files: 437/568 (76.9% of total)
Ported lines: 159545/242337 (65.8% of total)
Longest unported chain: 26/79 (67.1% progress)

port-progress bot (Jan 25 2023 at 18:21):

mathlib port progress topology.metric_space.basic
Ported files: 423/518 (81.7% of total)
Ported lines: 157189/224434 (70.0% of total)
Longest unported chain: 20/73 (72.6% progress)

port-progress bot (Jan 25 2023 at 18:42):

mathlib port progress all
Ported files: 660/2892 (22.8% of total)
Ported lines: 194105/988585 (19.6% of total)
Longest unported chain: 74/125 (40.8% progress)

Johan Commelin (Jan 25 2023 at 18:43):

0.1%

Kevin Buzzard (Jan 25 2023 at 18:46):

There is still progress behind the scenes though!

Jireh Loreaux (Jan 25 2023 at 20:36):

For a slightly different perspective, we can consider our progress year-to-date. I'll say this is a reasonable proxy for our porting speed because:

  1. it's after the port really got off the ground and many people got involved.
  2. it's after the holidays, so we're not averaging over an unnatural gap
  3. it's a decent enough chunk of time to smooth out noise.

On 2022-12-31 we had 104516/977206 and on 2023-01-25 we had 194105/988585. Assuming linear growth for mathlib3 and for lines ported (not necessarily a valid assumption) we arrive at a completion date of 2023-10-06 (October 6).

James Gallicchio (Jan 26 2023 at 00:01):

That does put into perspective how worth it is to make mathport better. Worth spending a few days to learn how mathport works in order to implement improvements to it.

port progress bot (jmc) (Jan 26 2023 at 14:02):

mathlib port progress order.filter.basic
Ported files: 263/272 (96.7% of total)
Ported lines: 107505/111188 (96.7% of total)
Longest unported chain: 1/47 (97.9% progress)

port progress bot (jmc) (Jan 26 2023 at 14:06):

mathlib port progress analysis.calculus.fderiv
Ported files: 475/703 (67.6% of total)
Ported lines: 171504/310369 (55.3% of total)
Longest unported chain: 35/89 (60.7% progress)

port progress bot (jmc) (Jan 26 2023 at 14:08):

mathlib port progress measure_theory.integral.bochner
Ported files: 506/994 (50.9% of total)
Ported lines: 177128/455935 (38.8% of total)
Longest unported chain: 53/106 (50.0% progress)

port progress bot (jmc) (Jan 26 2023 at 14:11):

mathlib port progress data.complex.exponential
Ported files: 448/570 (78.6% of total)
Ported lines: 166810/244559 (68.2% of total)
Longest unported chain: 26/80 (67.5% progress)

port progress bot (jmc) (Jan 26 2023 at 14:13):

mathlib port progress linear_algebra.determinant
Ported files: 443/633 (70.0% of total)
Ported lines: 156878/259563 (60.4% of total)
Longest unported chain: 33/81 (59.3% progress)

port progress bot (jmc) (Jan 26 2023 at 14:16):

mathlib port progress data.polynomial.basic
Ported files: 365/397 (91.9% of total)
Ported lines: 137736/160908 (85.6% of total)
Longest unported chain: 10/58 (82.8% progress)

port progress bot (jmc) (Jan 26 2023 at 14:18):

mathlib port progress ring_theory.polynomial.basic
Ported files: 430/557 (77.2% of total)
Ported lines: 153865/226467 (67.9% of total)
Longest unported chain: 26/74 (64.9% progress)

port progress bot (jmc) (Jan 26 2023 at 14:20):

mathlib port progress linear_algebra.basis
Ported files: 394/441 (89.3% of total)
Ported lines: 146299/177476 (82.4% of total)
Longest unported chain: 11/59 (81.4% progress)

port progress bot (jmc) (Jan 26 2023 at 14:23):

mathlib port progress topology.continuous_function.bounded
Ported files: 476/703 (67.7% of total)
Ported lines: 172114/306359 (56.2% of total)
Longest unported chain: 33/87 (62.1% progress)

Johan Commelin (Jan 26 2023 at 14:24):

:up: contains Arzela-Ascoli

port progress bot (jmc) (Jan 26 2023 at 14:26):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 495/876 (56.5% of total)
Ported lines: 175783/385692 (45.6% of total)
Longest unported chain: 41/93 (55.9% progress)

port progress bot (jmc) (Jan 26 2023 at 14:28):

mathlib port progress probability.independence
Ported files: 507/1008 (50.3% of total)
Ported lines: 177247/463003 (38.3% of total)
Longest unported chain: 58/111 (47.7% progress)

port-progress bot (Jan 26 2023 at 18:02):

mathlib port progress order.filter.basic
Ported files: 263/272 (96.7% of total)
Ported lines: 107505/111188 (96.7% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Jan 26 2023 at 18:06):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18794/31952 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 26 2023 at 18:10):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 511/1017 (50.2% of total)
Ported lines: 176992/434211 (40.8% of total)
Longest unported chain: 54/103 (47.6% progress)

port-progress bot (Jan 26 2023 at 18:13):

mathlib port progress linear_algebra.basic
Ported files: 337/355 (94.9% of total)
Ported lines: 133032/145850 (91.2% of total)
Longest unported chain: 3/52 (94.2% progress)

port-progress bot (Jan 26 2023 at 18:17):

mathlib port progress data.complex.basic
Ported files: 451/568 (79.4% of total)
Ported lines: 167291/242346 (69.0% of total)
Longest unported chain: 25/79 (68.4% progress)

Johan Commelin (Jan 26 2023 at 18:20):

We need to tackle those (d)finsupp files. Then linear algebra will be "in the pocket".

port-progress bot (Jan 26 2023 at 18:21):

mathlib port progress topology.metric_space.basic
Ported files: 434/518 (83.8% of total)
Ported lines: 164346/224443 (73.2% of total)
Longest unported chain: 19/73 (74.0% progress)

port-progress bot (Jan 26 2023 at 18:42):

mathlib port progress all
Ported files: 685/2893 (23.7% of total)
Ported lines: 204248/989420 (20.6% of total)
Longest unported chain: 71/125 (43.2% progress)

Johan Commelin (Jan 26 2023 at 18:49):

1.0%

Johan Commelin (Jan 27 2023 at 08:41):

During the meeting yesterday there were two suggestions/feature requests concerning these progress reports:

  • we could remove all green nodes (aka ported files) from the graphs; they clutter the pdfs, and don't really add much
  • the tables could display the number of blue (dark and light) nodes in the graph (aka in progress/ready to be ported)

port progress bot (jmc) (Jan 27 2023 at 15:50):

mathlib port progress linear_algebra.basic
Ported files: 339/355 (95.5% of total)
Ported lines: 134772/145884 (92.4% of total)
Longest unported chain: 3/52 (94.2% progress)

Johan Commelin (Jan 27 2023 at 15:51):

Patrick fixed the first bullet point.

Johan Commelin (Jan 27 2023 at 15:51):

Except that my bot didn't switch over yet :face_palm:

port progress bot (jmc) (Jan 27 2023 at 15:52):

mathlib port progress data.polynomial.basic
Ported files: 368/397 (92.7% of total)
Ported lines: 139831/160942 (86.9% of total)
Longest unported chain: 9/58 (84.5% progress)

port progress bot (jmc) (Jan 27 2023 at 15:55):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18794/31952 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port progress bot (jmc) (Jan 27 2023 at 15:57):

mathlib port progress data.complex.basic
Ported files: 460/568 (81.0% of total)
Ported lines: 170968/242380 (70.5% of total)
Longest unported chain: 25/79 (68.4% progress)

port progress bot (jmc) (Jan 27 2023 at 15:59):

mathlib port progress analysis.calculus.fderiv
Ported files: 489/703 (69.6% of total)
Ported lines: 175843/310403 (56.6% of total)
Longest unported chain: 35/89 (60.7% progress)

port progress bot (jmc) (Jan 27 2023 at 16:02):

mathlib port progress measure_theory.integral.bochner
Ported files: 521/994 (52.4% of total)
Ported lines: 181940/455969 (39.9% of total)
Longest unported chain: 52/106 (50.9% progress)

port progress bot (jmc) (Jan 27 2023 at 16:05):

mathlib port progress data.complex.exponential
Ported files: 461/570 (80.9% of total)
Ported lines: 171267/244593 (70.0% of total)
Longest unported chain: 26/80 (67.5% progress)

port progress bot (jmc) (Jan 27 2023 at 16:07):

mathlib port progress linear_algebra.determinant
Ported files: 453/633 (71.6% of total)
Ported lines: 161089/259597 (62.1% of total)
Longest unported chain: 31/81 (61.7% progress)

Anne Baanen (Jan 27 2023 at 16:08):

I'd like to claim algebra.module.submodule.

Ruben Van de Velde (Jan 27 2023 at 16:09):

Anne Baanen said:

I'd like to claim algebra.module.submodule.

As in !4#1888?

Ruben Van de Velde (Jan 27 2023 at 16:09):

Feel free to take over

port progress bot (jmc) (Jan 27 2023 at 16:10):

mathlib port progress ring_theory.polynomial.basic
Ported files: 438/557 (78.6% of total)
Ported lines: 157434/226501 (69.5% of total)
Longest unported chain: 24/74 (67.6% progress)

Anne Baanen (Jan 27 2023 at 16:11):

Ruben Van de Velde said:

Anne Baanen said:

I'd like to claim algebra.module.submodule.

As in !4#1888?

Oops, didn't see that you already started. Would it be OK if I pushed a few fixes?

Ruben Van de Velde (Jan 27 2023 at 16:11):

Yeah, go ahead. I need to focus on other things for a while

port progress bot (jmc) (Jan 27 2023 at 16:12):

mathlib port progress linear_algebra.basis
Ported files: 400/441 (90.7% of total)
Ported lines: 148977/177510 (83.9% of total)
Longest unported chain: 9/59 (84.7% progress)

port progress bot (jmc) (Jan 27 2023 at 16:14):

mathlib port progress topology.continuous_function.bounded
Ported files: 491/703 (69.8% of total)
Ported lines: 176752/306393 (57.7% of total)
Longest unported chain: 33/87 (62.1% progress)

port progress bot (jmc) (Jan 27 2023 at 16:17):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 511/876 (58.3% of total)
Ported lines: 180894/385726 (46.9% of total)
Longest unported chain: 39/93 (58.1% progress)

port progress bot (jmc) (Jan 27 2023 at 16:19):

mathlib port progress probability.independence
Ported files: 523/1008 (51.9% of total)
Ported lines: 182358/463037 (39.4% of total)
Longest unported chain: 57/111 (48.6% progress)

Anne Baanen (Jan 27 2023 at 17:05):

Ruben Van de Velde said:

Yeah, go ahead. I need to focus on other things for a while

I'm going in 10 to 15 minutes. Everything should build and lint correctly, we need to run the other fixing scripts and check the names and docstrings.

Johan Commelin (Jan 27 2023 at 17:52):

The graphs now exlude all green nodes.

Johan Commelin (Jan 27 2023 at 17:53):

@Scott Morrison If you want the same behaviour for your bot, then you need to use the --really-exclude-ported flag (after updating leanproject)

port-progress bot (Jan 27 2023 at 18:02):

mathlib port progress order.filter.basic
Ported files: 263/272 (96.7% of total)
Ported lines: 107539/111222 (96.7% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Jan 27 2023 at 18:06):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18794/31952 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 27 2023 at 18:10):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 529/1017 (52.0% of total)
Ported lines: 185546/434306 (42.7% of total)
Longest unported chain: 53/103 (48.5% progress)

port-progress bot (Jan 27 2023 at 18:14):

mathlib port progress linear_algebra.basic
Ported files: 341/355 (96.1% of total)
Ported lines: 137076/145890 (94.0% of total)
Longest unported chain: 2/52 (96.2% progress)

port-progress bot (Jan 27 2023 at 18:17):

mathlib port progress data.complex.basic
Ported files: 463/568 (81.5% of total)
Ported lines: 173864/242428 (71.7% of total)
Longest unported chain: 25/79 (68.4% progress)

port-progress bot (Jan 27 2023 at 18:21):

mathlib port progress topology.metric_space.basic
Ported files: 445/518 (85.9% of total)
Ported lines: 170741/224516 (76.0% of total)
Longest unported chain: 19/73 (74.0% progress)

port-progress bot (Jan 27 2023 at 18:43):

mathlib port progress all
Ported files: 713/2894 (24.6% of total)
Ported lines: 215608/989810 (21.8% of total)
Longest unported chain: 71/125 (43.2% progress)

Johan Commelin (Jan 27 2023 at 18:43):

1.2%

Johan Commelin (Jan 27 2023 at 18:50):

#port-status claims that topology.tactic has 1 unported dependency. This must be something in the tactic.* directory, I guess. It's also the first file on the "longest unported chain".

Adam Topaz (Jan 27 2023 at 19:31):

I suppose it's tactic.tidy?

Adam Topaz (Jan 27 2023 at 19:32):

BTW, shouldn't it be very easy to implement something like continuity using aesop?

Heather Macbeth (Jan 27 2023 at 19:54):

In my opinion continuity (and similar tactics) should be implemented without backtracking, for performance reasons and also for ease of debugging: there's generally only one action that is sensible to do on the goal (like if the head symbol is + you want to apply continuous.add). The mathlib3 version gets this by implementing it over apply_rules (rather than over solve_by_elim, which does backtracking). I forget whether aesop has a no-backtracking option?

Heather Macbeth (Jan 27 2023 at 19:56):

More generally, I think aesop is a big improvement over solve_by_elim/apply_rules in problems where you do want to do backtracking (because it lets you set priorities to try the likely-better steps first). But in problems where you don't want to do backtracking it's about the same behaviour with a slightly more complicated setup.

Gabriel Ebner (Jan 27 2023 at 19:58):

aesop supports both backtrackable and nonbacktrackable rules. These are somewhat confusingly called safe and unsafe, resp.

Heather Macbeth (Jan 27 2023 at 20:00):

Do you mean that if you tag every lemma as safe then you will get no backtracking?

Heather Macbeth (Jan 27 2023 at 20:01):

In any case, that's still the same behaviour as apply_rules, right? It's not really the situation where aesop comes in to its own.

Sebastien Gouezel (Jan 28 2023 at 06:38):

Although continuity in mathlib3 is implemented on the basis of apply_rules, its performance is quite bad (much worse than applying the direct term), which I don't really understand because I had heard that apply was very cheap, so trying to apply lemmas where the head doesn't match should be pretty quick. It makes me wonder if it would be better to reimplement it by applying directly the right lemma: look at the head of the term, and choose the lemma to apply based on that. For instance, if you are proving that λ x, cos (sin (x + 3 * exp x)) is continuous, notice that the head is cos and apply directly continuous.cos. If we have n possible heads, it should be possible to choose the right lemma in log n steps and then I hope performance should be good. I'm curious if this would be easy to implement, and if the performance would indeed improve by an order of magnitude (which is what we need to make continuity really usable).

Of course, this kind of experimentation is for after the port!

Heather Macbeth (Jan 28 2023 at 06:41):

If aesop does this, that would definitely be a reason to use it!

Yury G. Kudryashov (Jan 28 2023 at 06:46):

I see that continuity has special handling for composition and in some cases we have, e.g., docs#continuous_fst instead of docs#continuous.fst marked with continuity. Would it be better to mandate that continuity lemmas should be of the form continuous.fst, not continuous_fst?

port-progress bot (Jan 28 2023 at 18:03):

mathlib port progress order.filter.basic
Ported files: 263/272 (96.7% of total)
Ported lines: 107544/111227 (96.7% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Jan 28 2023 at 18:06):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18794/31952 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 28 2023 at 18:11):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 534/1017 (52.5% of total)
Ported lines: 186455/434446 (42.9% of total)
Longest unported chain: 53/103 (48.5% progress)

port-progress bot (Jan 28 2023 at 18:14):

mathlib port progress linear_algebra.basic
Ported files: 342/355 (96.3% of total)
Ported lines: 137578/145932 (94.3% of total)
Longest unported chain: 2/52 (96.2% progress)

port-progress bot (Jan 28 2023 at 18:18):

mathlib port progress data.complex.basic
Ported files: 464/568 (81.7% of total)
Ported lines: 174378/242497 (71.9% of total)
Longest unported chain: 25/79 (68.4% progress)

port-progress bot (Jan 28 2023 at 18:22):

mathlib port progress topology.metric_space.basic
Ported files: 446/518 (86.1% of total)
Ported lines: 171252/224567 (76.3% of total)
Longest unported chain: 19/73 (74.0% progress)

port-progress bot (Jan 28 2023 at 18:45):

mathlib port progress all
Ported files: 717/2898 (24.7% of total)
Ported lines: 216449/990757 (21.8% of total)
Longest unported chain: 71/125 (43.2% progress)

Johan Commelin (Jan 28 2023 at 20:46):

0.0%

Yury G. Kudryashov (Jan 28 2023 at 21:52):

It would be nice if someone reviews ##18312. I have a bunch of files from Topology ported but they depend on a version of Topology.Order from #18312, not from master.

Kevin Buzzard (Jan 29 2023 at 00:21):

Johan Commelin said:

0.0%

Yeah but it's the weekend ;-)

port-progress bot (Jan 29 2023 at 18:04):

mathlib port progress linear_algebra.basic
Ported files: 343/355 (96.6% of total)
Ported lines: 137904/145932 (94.5% of total)
Longest unported chain: 2/52 (96.2% progress)

port-progress bot (Jan 29 2023 at 18:07):

mathlib port progress topology.basic
Ported files: 319/328 (97.3% of total)
Ported lines: 126879/130562 (97.2% of total)
Longest unported chain: 1/53 (98.1% progress)

port-progress bot (Jan 29 2023 at 18:11):

mathlib port progress data.polynomial.basic
Ported files: 373/397 (94.0% of total)
Ported lines: 143106/160993 (88.9% of total)
Longest unported chain: 8/58 (86.2% progress)

port-progress bot (Jan 29 2023 at 18:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18794/31952 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 29 2023 at 18:18):

mathlib port progress data.complex.basic
Ported files: 467/568 (82.2% of total)
Ported lines: 175117/242497 (72.2% of total)
Longest unported chain: 25/79 (68.4% progress)

port-progress bot (Jan 29 2023 at 18:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 541/1017 (53.2% of total)
Ported lines: 188381/434446 (43.4% of total)
Longest unported chain: 53/103 (48.5% progress)

port-progress bot (Jan 29 2023 at 18:32):

mathlib port progress all
Ported files: 730/2898 (25.2% of total)
Ported lines: 219874/990757 (22.2% of total)
Longest unported chain: 71/125 (43.2% progress)

Johan Commelin (Jan 29 2023 at 19:16):

0.4%

Kevin Buzzard (Jan 29 2023 at 22:41):

I remember being happy recently when we were 1/8 of the way there and now it's 1/4!

Yaël Dillies (Jan 29 2023 at 22:43):

Soon 2n2^n of the way!

Notification Bot (Jan 30 2023 at 17:28):

24 messages were moved from this topic to #PR reviews > #18312 review topology/order by Yury G. Kudryashov.

port-progress bot (Jan 30 2023 at 18:04):

mathlib port progress linear_algebra.basic
Ported files: 344/355 (96.9% of total)
Ported lines: 138431/145932 (94.9% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Jan 30 2023 at 18:06):

mathlib port progress topology.basic
Ported files: 319/328 (97.3% of total)
Ported lines: 126879/130562 (97.2% of total)
Longest unported chain: 1/53 (98.1% progress)

port-progress bot (Jan 30 2023 at 18:10):

mathlib port progress data.polynomial.basic
Ported files: 375/397 (94.5% of total)
Ported lines: 144777/160993 (89.9% of total)
Longest unported chain: 7/58 (87.9% progress)

port-progress bot (Jan 30 2023 at 18:14):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18794/31952 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 30 2023 at 18:18):

mathlib port progress data.complex.basic
Ported files: 469/568 (82.6% of total)
Ported lines: 176788/242497 (72.9% of total)
Longest unported chain: 25/79 (68.4% progress)

port-progress bot (Jan 30 2023 at 18:22):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 547/1017 (53.8% of total)
Ported lines: 192000/434446 (44.2% of total)
Longest unported chain: 52/103 (49.5% progress)

port-progress bot (Jan 30 2023 at 18:32):

mathlib port progress all
Ported files: 743/2898 (25.6% of total)
Ported lines: 224296/990756 (22.6% of total)
Longest unported chain: 71/125 (43.2% progress)

Johan Commelin (Jan 30 2023 at 18:34):

0.4%

Yury G. Kudryashov (Jan 30 2023 at 18:42):

You can drop topology.basic as a target (already ported) and add, say, topology.metric_space.basic.

Johan Commelin (Jan 30 2023 at 18:50):

This version of the bot runs on @Scott Morrison's hardware. I don't have access to that.

Yury G. Kudryashov (Jan 30 2023 at 18:53):

BTW, who runs mathport and how often?

Reid Barton (Jan 30 2023 at 18:54):

https://github.com/leanprover-community/mathport/blob/master/.github/workflows/build.yml#L11

Mario Carneiro (Jan 30 2023 at 18:54):

The mathport CI runs mathport, every 2 hours for mathlib4 changes and every 6 hours for mathlib3 changes (IIRC)

Jireh Loreaux (Jan 30 2023 at 18:55):

!4#1874 is GroupTheory.Coset and !4#1864 is GroupTheory.Subgroup.Finite. Both are ready for review (I think they should be relatively easy) and should unlock several files.

Reid Barton (Jan 30 2023 at 18:55):

https://github.com/leanprover-community/mathport/blob/master/.github/workflows/predata.yml#L9 seems to be once a day only, am I missing something? I thought it was more frequent also

Mario Carneiro (Jan 30 2023 at 18:58):

the CI history also indicates as much

Mario Carneiro (Jan 30 2023 at 18:58):

@Gabriel Ebner will know what the situation is

Gabriel Ebner (Jan 30 2023 at 19:01):

seems to be once a day only

Yes, it takes a couple of hours (i.e., uses a lot of CI resources) and there weren't many mathlib3 changes at the time. It used to run twice a day, and I downgraded it to once a day.

Gabriel Ebner (Jan 30 2023 at 19:02):

If you need it faster, you can click oin the "run workflow" button on https://github.com/leanprover-community/mathport/actions/workflows/predata.yml

Gabriel Ebner (Jan 30 2023 at 19:02):

But right now, mathport CI is completely borked.

Mario Carneiro (Jan 30 2023 at 19:03):

how hard is it to set up one of those "hey devs, mathport is borked" ping bots?

Gabriel Ebner (Jan 30 2023 at 19:04):

You'd need to ping different devs every time because it's different things every time. Right now half of the hoskinson machines are down.

Gabriel Ebner (Jan 30 2023 at 19:05):

Although github sends me "hey gabriel, mathport is borked" emails.

Yury G. Kudryashov (Jan 30 2023 at 19:31):

Any chances it will work again in the near future?

Mario Carneiro (Jan 30 2023 at 19:33):

it appears it is at least partially the fault of a breaking change in mathlib4

Yury G. Kudryashov (Jan 30 2023 at 19:36):

What kind of a breaking change? Can I help?

Kevin Buzzard (Jan 30 2023 at 19:39):

I'm assuming this message is the relevant one.

Mario Carneiro (Jan 30 2023 at 19:42):

!4#1951

Gabriel Ebner (Jan 30 2023 at 20:12):

near future

Yes. ETA for next mathlib4 update is 30 minutes, ETA for next mathlib3 update is 6 hours.

Yury G. Kudryashov (Jan 30 2023 at 23:53):

Which of the jobs builds mathlib3port from the Lean 3 mathlib master branch?

Gabriel Ebner (Jan 30 2023 at 23:55):

Two jobs are doing that. First predata needs to run (producing tlean/ast files from mathlib3), and then mathport (which uses this data to generate Lean 4 files).

Gabriel Ebner (Jan 30 2023 at 23:57):

A predata run finished 30 minutes ago, and the next mathport run is scheduled to start any minute now. We should see an update to mathlib3port in 45 minutes or so.

Yury G. Kudryashov (Jan 30 2023 at 23:59):

I see that the next predata is running. Do you mind if I restart it? I want to have a version of mathlib3port with #18312

Yury G. Kudryashov (Jan 31 2023 at 00:00):

Never mind. I'll just wait till tomorrow. It turns out, I have some other urgent things to do.

Gabriel Ebner (Jan 31 2023 at 00:09):

Waiting, restarting, starting a new one. All three are fine with me.

Jakob von Raumer (Jan 31 2023 at 12:10):

Having the PR tags on mathlib-port-status would be a cool feature, to quickly see where help is needed

Eric Wieser (Jan 31 2023 at 12:32):

Jakob von Raumer said:

Having the PR tags on mathlib-port-status would be a cool feature, to quickly see where help is needed

PRs to https://github.com/leanprover-community/mathlib-port-status are welcome :).

Eric Wieser (Jan 31 2023 at 12:35):

Although I suspect the path to what you're asking is to merge make_port_status.py with that repo

Jakob von Raumer (Jan 31 2023 at 12:46):

I'll have a look

port-progress bot (Jan 31 2023 at 18:03):

mathlib port progress linear_algebra.basic
Ported files: 344/355 (96.9% of total)
Ported lines: 138443/145944 (94.9% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Jan 31 2023 at 18:07):

mathlib port progress topology.metric_space.basic
Ported files: 455/518 (87.8% of total)
Ported lines: 176481/224522 (78.6% of total)
Longest unported chain: 17/73 (76.7% progress)

port-progress bot (Jan 31 2023 at 18:11):

mathlib port progress data.polynomial.basic
Ported files: 375/397 (94.5% of total)
Ported lines: 144795/161011 (89.9% of total)
Longest unported chain: 7/58 (87.9% progress)

port-progress bot (Jan 31 2023 at 18:15):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18794/31952 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Jan 31 2023 at 18:19):

mathlib port progress data.complex.basic
Ported files: 474/568 (83.5% of total)
Ported lines: 179883/242367 (74.2% of total)
Longest unported chain: 23/79 (70.9% progress)

port-progress bot (Jan 31 2023 at 18:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 553/1017 (54.4% of total)
Ported lines: 195534/434346 (45.0% of total)
Longest unported chain: 52/103 (49.5% progress)

port-progress bot (Jan 31 2023 at 18:32):

mathlib port progress all
Ported files: 752/2898 (25.9% of total)
Ported lines: 228181/990688 (23.0% of total)
Longest unported chain: 69/125 (44.8% progress)

Johan Commelin (Jan 31 2023 at 18:35):

0.4%

Notification Bot (Feb 01 2023 at 10:51):

24 messages were moved from this topic to #mathlib4 > Suggestions for #port-status by Eric Wieser.

Johan Commelin (Feb 01 2023 at 11:21):

Order.CompactlyGenerated !4#1976

at the top of #port-status is ready for review

port-progress bot (Feb 01 2023 at 18:04):

mathlib port progress linear_algebra.basic
Ported files: 345/355 (97.2% of total)
Ported lines: 139991/145889 (96.0% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 01 2023 at 18:09):

mathlib port progress topology.metric_space.basic
Ported files: 469/515 (91.1% of total)
Ported lines: 187806/222235 (84.5% of total)
Longest unported chain: 12/73 (83.6% progress)

port-progress bot (Feb 01 2023 at 18:12):

mathlib port progress data.polynomial.basic
Ported files: 377/397 (95.0% of total)
Ported lines: 146885/160956 (91.3% of total)
Longest unported chain: 6/58 (89.7% progress)

port-progress bot (Feb 01 2023 at 18:16):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18800/31958 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Feb 01 2023 at 18:20):

mathlib port progress data.complex.basic
Ported files: 488/565 (86.4% of total)
Ported lines: 191208/240087 (79.6% of total)
Longest unported chain: 18/79 (77.2% progress)

port-progress bot (Feb 01 2023 at 18:25):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 572/1018 (56.2% of total)
Ported lines: 209066/434738 (48.1% of total)
Longest unported chain: 51/103 (50.5% progress)

port-progress bot (Feb 01 2023 at 18:33):

mathlib port progress all
Ported files: 775/2904 (26.7% of total)
Ported lines: 242377/992169 (24.4% of total)
Longest unported chain: 68/126 (46.0% progress)

Johan Commelin (Feb 01 2023 at 18:41):

1.4%

Jireh Loreaux (Feb 01 2023 at 19:10):

Fun fact: that's 4.8% in the last week alone.

Ruben Van de Velde (Feb 01 2023 at 19:11):

So four months left

Matthew Ballard (Feb 02 2023 at 12:17):

1/4

port-progress bot (Feb 02 2023 at 18:04):

mathlib port progress linear_algebra.basic
Ported files: 345/355 (97.2% of total)
Ported lines: 139994/145892 (96.0% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 02 2023 at 18:09):

mathlib port progress topology.metric_space.basic
Ported files: 477/515 (92.6% of total)
Ported lines: 194953/222265 (87.7% of total)
Longest unported chain: 7/73 (90.4% progress)

port-progress bot (Feb 02 2023 at 18:14):

mathlib port progress data.polynomial.basic
Ported files: 377/397 (95.0% of total)
Ported lines: 146891/160962 (91.3% of total)
Longest unported chain: 6/58 (89.7% progress)

port-progress bot (Feb 02 2023 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18800/31958 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Feb 02 2023 at 18:23):

mathlib port progress data.complex.basic
Ported files: 497/565 (88.0% of total)
Ported lines: 198837/240117 (82.8% of total)
Longest unported chain: 13/79 (83.5% progress)

port-progress bot (Feb 02 2023 at 18:29):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 583/1018 (57.3% of total)
Ported lines: 216833/434783 (49.9% of total)
Longest unported chain: 51/103 (50.5% progress)

port-progress bot (Feb 02 2023 at 18:34):

mathlib port progress combinatorics.additive.behrend
Ported files: 573/953 (60.1% of total)
Ported lines: 215992/423104 (51.0% of total)
Longest unported chain: 45/103 (56.3% progress)

port-progress bot (Feb 02 2023 at 18:48):

mathlib port progress all
Ported files: 794/2905 (27.3% of total)
Ported lines: 252053/993119 (25.4% of total)
Longest unported chain: 68/126 (46.0% progress)

Johan Commelin (Feb 02 2023 at 18:59):

1.0%

Kevin Buzzard (Feb 02 2023 at 19:56):

The 1% days are good days

port progress bot (jmc) (Feb 03 2023 at 19:48):

mathlib port progress linear_algebra.basic
Ported files: 345/355 (97.2% of total)
Ported lines: 139995/145840 (96.0% of total)
Longest unported chain: 1/52 (98.1% progress)

port progress bot (jmc) (Feb 03 2023 at 19:50):

mathlib port progress data.polynomial.basic
Ported files: 377/397 (95.0% of total)
Ported lines: 146892/160910 (91.3% of total)
Longest unported chain: 6/58 (89.7% progress)

port progress bot (jmc) (Feb 03 2023 at 19:52):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18800/31958 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port progress bot (jmc) (Feb 03 2023 at 19:55):

mathlib port progress data.complex.basic
Ported files: 499/566 (88.2% of total)
Ported lines: 200022/240116 (83.3% of total)
Longest unported chain: 12/77 (84.4% progress)

port progress bot (jmc) (Feb 03 2023 at 19:57):

mathlib port progress analysis.calculus.fderiv
Ported files: 538/706 (76.2% of total)
Ported lines: 209088/310774 (67.3% of total)
Longest unported chain: 30/89 (66.3% progress)

port progress bot (jmc) (Feb 03 2023 at 20:00):

mathlib port progress measure_theory.integral.bochner
Ported files: 579/997 (58.1% of total)
Ported lines: 218386/456623 (47.8% of total)
Longest unported chain: 49/106 (53.8% progress)

port progress bot (jmc) (Feb 03 2023 at 20:03):

mathlib port progress data.complex.exponential
Ported files: 500/568 (88.0% of total)
Ported lines: 200579/242332 (82.8% of total)
Longest unported chain: 13/78 (83.3% progress)

port progress bot (jmc) (Feb 03 2023 at 20:05):

mathlib port progress linear_algebra.determinant
Ported files: 483/634 (76.2% of total)
Ported lines: 176755/259903 (68.0% of total)
Longest unported chain: 29/81 (64.2% progress)

port progress bot (jmc) (Feb 03 2023 at 20:08):

mathlib port progress ring_theory.polynomial.basic
Ported files: 464/557 (83.3% of total)
Ported lines: 172359/226717 (76.0% of total)
Longest unported chain: 22/74 (70.3% progress)

port progress bot (jmc) (Feb 03 2023 at 20:10):

mathlib port progress linear_algebra.basis
Ported files: 416/441 (94.3% of total)
Ported lines: 159286/177544 (89.7% of total)
Longest unported chain: 7/59 (88.1% progress)

port progress bot (jmc) (Feb 03 2023 at 20:13):

mathlib port progress topology.continuous_function.bounded
Ported files: 538/706 (76.2% of total)
Ported lines: 209141/306762 (68.2% of total)
Longest unported chain: 28/87 (67.8% progress)

port progress bot (jmc) (Feb 03 2023 at 20:15):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 566/879 (64.4% of total)
Ported lines: 216416/386268 (56.0% of total)
Longest unported chain: 37/93 (60.2% progress)

port progress bot (jmc) (Feb 03 2023 at 20:18):

mathlib port progress probability.independence
Ported files: 580/1011 (57.4% of total)
Ported lines: 218505/463691 (47.1% of total)
Longest unported chain: 54/111 (51.4% progress)

Arien Malec (Feb 03 2023 at 21:01):

We are closer to Data.Complex.Exponential than to Data.Complex.Basic

Arien Malec (Feb 03 2023 at 21:02):

There's some deep mathematical truth there.

Arien Malec (Feb 03 2023 at 21:03):

(this must have been a timing thing).

Yury G. Kudryashov (Feb 04 2023 at 02:59):

How do you generate an import graph that ignores already ported files?

Yury G. Kudryashov (Feb 04 2023 at 03:01):

Answer: upgrade mathlibtools

Johan Commelin (Feb 06 2023 at 09:01):

Here's a different heuristic to measure progress:

mathlib on master$ git ls-files | rg "basic.lean" | xargs rg -l "SYNCH" | wc -l
107

mathlib on master$ git ls-files | rg "basic.lean" | wc -l
264

Johan Commelin (Feb 06 2023 at 09:01):

This suggests we are ~40% done with the "hard" files.

Ruben Van de Velde (Feb 06 2023 at 10:09):

Welcome to mathlib, where "basic" means "hard" :)

Patrick Massot (Feb 06 2023 at 13:13):

Don't you say "basic sciences" in English? In French this is translated as "hard sciences".

Jason Rute (Feb 06 2023 at 13:15):

Just curious. Is the port progress bot down? I admit I like watching the progress from afar.

Chris Hughes (Feb 06 2023 at 13:16):

You can see the progress here if you like https://leanprover-community.github.io/mathlib-port-status/

Johan Commelin (Feb 06 2023 at 13:17):

I pinged Scott already, about the bot.

Johan Commelin (Feb 06 2023 at 13:17):

If it doesn't show up ~ 5 hrs from now, then I'll revive my copy of the bot.

Eric Wieser (Feb 06 2023 at 14:06):

Chris Hughes said:

You can see the progress here if you like https://leanprover-community.github.io/mathlib-port-status/

It would be trivial to add longest chain information to this page for a fixed list of targets, if that's useful

Eric Wieser (Feb 06 2023 at 14:06):

It would slightly less trivial to add a page that lets you type in any module you like and generates that longest chain client-side

Eric Wieser (Feb 06 2023 at 14:06):

I don't know how happy CI would be if I generate 3000 pages with the longest chain for every file

Johan Commelin (Feb 06 2023 at 14:10):

I don't think that's worth the CI overhead to compute this

Eric Wieser (Feb 06 2023 at 14:15):

The overhead should be small, we already have the graph built

Eric Wieser (Feb 06 2023 at 14:15):

The bot on this thread is really slow because it also tries to work out which files aren't really needed, which requires invoking lean

Johan Commelin (Feb 06 2023 at 14:17):

Well, I'll leave it up to you then.

Johan Commelin (Feb 06 2023 at 14:17):

I would rather run CI 6x per hour and leave out those 3000 pages.

Lukas Miaskiwskyi (Feb 06 2023 at 14:46):

I thought the port progress bot was just taking the weekends off. At least that was a thing previously. But I'd also like it to work seven days a week, yeah

Jason Rute said:

Just curious. Is the port progress bot down? I admit I like watching the progress from afar.

Eric Wieser (Feb 06 2023 at 16:19):

Johan Commelin said:

I would rather run CI 6x per hour and leave out those 3000 pages.

CI takes about a minute but we now have 3000 pages, such as https://leanprover-community.github.io/mathlib-port-status/file/algebra/big_operators/basic

Johan Commelin (Feb 06 2023 at 17:23):

port-status#topology/basic

port-progress bot (Feb 06 2023 at 18:04):

mathlib port progress linear_algebra.basic
Ported files: 345/355 (97.2% of total)
Ported lines: 139995/145840 (96.0% of total)
Longest unported chain: 1/52 (98.1% progress)

Johan Commelin (Feb 06 2023 at 18:04):

Welcome back!

port-progress bot (Feb 06 2023 at 18:07):

mathlib port progress topology.metric_space.basic
Ported files: 457/480 (95.2% of total)
Ported lines: 190439/207337 (91.8% of total)
Longest unported chain: 6/67 (91.0% progress)

Tobias Grosser (Feb 06 2023 at 18:07):

port-status#all

Yury G. Kudryashov (Feb 06 2023 at 18:08):

I forgot to update SHA.

Yury G. Kudryashov (Feb 06 2023 at 18:08):

Is there a webpage with a list of all files with wrong SHA sums?

Eric Wieser (Feb 06 2023 at 18:09):

https://leanprover-community.github.io/mathlib-port-status/out-of-sync

Eric Wieser (Feb 06 2023 at 18:10):

Tobias Grosser said:

port-status#all

This doesn't exist, because it would just be a worse version of the homepage, #port-status

port-progress bot (Feb 06 2023 at 18:11):

mathlib port progress data.polynomial.basic
Ported files: 377/397 (95.0% of total)
Ported lines: 146892/160910 (91.3% of total)
Longest unported chain: 6/58 (89.7% progress)

Tobias Grosser (Feb 06 2023 at 18:14):

Eric Wieser said:

Tobias Grosser said:

port-status#all

This doesn't exist, because it would just be a worse version of the homepage, #port-status

I just tried to get the #all box printed. As the bot does sometimes at the end of the day when we all celebrate. Had hoped I can learn about how to use our bots.

port-progress bot (Feb 06 2023 at 18:15):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18800/31958 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

Yury G. Kudryashov (Feb 06 2023 at 18:16):

I see that the last section of #port-status is empty. Is it a bug?

Eric Wieser (Feb 06 2023 at 18:18):

That section is for files that have no SHA at all

Eric Wieser (Feb 06 2023 at 18:18):

Which I think there should be none of?

Yury G. Kudryashov (Feb 06 2023 at 18:19):

Which section lists files that were updated in mathlib3 after they were ported?

port-progress bot (Feb 06 2023 at 18:19):

mathlib port progress data.complex.basic
Ported files: 511/566 (90.3% of total)
Ported lines: 206971/240146 (86.2% of total)
Longest unported chain: 12/77 (84.4% progress)

Eric Wieser (Feb 06 2023 at 18:19):

Had hoped I can learn about how to use our bots.

I don't think we have any bots that response to messages

Eric Wieser (Feb 06 2023 at 18:19):

Yury G. Kudryashov said:

Which section lists files that were updated in mathlib3 after they were ported?

Eric Wieser said:

https://leanprover-community.github.io/mathlib-port-status/out-of-sync

port-progress bot (Feb 06 2023 at 18:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 609/1020 (59.7% of total)
Ported lines: 228465/434905 (52.5% of total)
Longest unported chain: 51/103 (50.5% progress)

port-progress bot (Feb 06 2023 at 18:27):

mathlib port progress combinatorics.additive.behrend
Ported files: 601/955 (62.9% of total)
Ported lines: 227900/423231 (53.8% of total)
Longest unported chain: 45/102 (55.9% progress)

port-progress bot (Feb 06 2023 at 18:35):

mathlib port progress all
Ported files: 858/2907 (29.5% of total)
Ported lines: 271990/993663 (27.4% of total)
Longest unported chain: 68/125 (45.6% progress)

Johan Commelin (Feb 06 2023 at 18:41):

2.0% (since Thursday, = 4 days)

Kevin Buzzard (Feb 06 2023 at 18:49):

(including a weekend)

Yury G. Kudryashov (Feb 06 2023 at 20:38):

Could you please add a hash sum to pages like https://leanprover-community.github.io/mathlib-port-status/file/algebra/big_operators/basic that we can copy+paste into mathlib4 files?

Yury G. Kudryashov (Feb 06 2023 at 20:39):

It can be either the hash sum of master, or the hash sum of the latest PR that touched this file.

Eric Wieser (Feb 06 2023 at 20:39):

You can use the hash of the top commit

Yury G. Kudryashov (Feb 06 2023 at 20:39):

I see a shortened hash sum but headers use full sums.

Eric Wieser (Feb 06 2023 at 20:39):

Clearly I should add back the comment that says "newest first"

Eric Wieser (Feb 06 2023 at 20:40):

The shortened hash is a link to the full hash

Eric Wieser (Feb 06 2023 at 20:40):

But I guess that's not ideal

Yury G. Kudryashov (Feb 06 2023 at 20:40):

Yes, it's just 1 click away but being able to copy+paste would be more convenient.

Eric Wieser (Feb 06 2023 at 20:41):

Would a "copy to clipboard" button be better or worse than just having the full SHA?

Yury G. Kudryashov (Feb 06 2023 at 20:41):

The same for me.

Eric Wieser (Feb 06 2023 at 20:46):

I'll add a full hash at the bottom along with instructions

Eric Wieser (Feb 06 2023 at 20:46):

port-status#algebra/big_operators/basic

port-progress bot (Feb 07 2023 at 18:04):

mathlib port progress linear_algebra.basic
Ported files: 345/355 (97.2% of total)
Ported lines: 140020/145865 (96.0% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 07 2023 at 18:07):

mathlib port progress topology.metric_space.basic
Ported files: 457/480 (95.2% of total)
Ported lines: 190470/207368 (91.9% of total)
Longest unported chain: 6/67 (91.0% progress)

port-progress bot (Feb 07 2023 at 18:11):

mathlib port progress data.polynomial.basic
Ported files: 377/397 (95.0% of total)
Ported lines: 146917/160935 (91.3% of total)
Longest unported chain: 6/58 (89.7% progress)

port-progress bot (Feb 07 2023 at 18:15):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18800/31958 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Feb 07 2023 at 18:19):

mathlib port progress data.complex.basic
Ported files: 513/566 (90.6% of total)
Ported lines: 207574/240192 (86.4% of total)
Longest unported chain: 12/77 (84.4% progress)

port-progress bot (Feb 07 2023 at 18:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 614/1020 (60.2% of total)
Ported lines: 230260/434975 (52.9% of total)
Longest unported chain: 51/103 (50.5% progress)

port-progress bot (Feb 07 2023 at 18:27):

mathlib port progress combinatorics.additive.behrend
Ported files: 607/955 (63.6% of total)
Ported lines: 229778/423298 (54.3% of total)
Longest unported chain: 45/102 (55.9% progress)

port-progress bot (Feb 07 2023 at 18:35):

mathlib port progress all
Ported files: 872/2907 (30.0% of total)
Ported lines: 275816/993851 (27.8% of total)
Longest unported chain: 68/125 (45.6% progress)

Johan Commelin (Feb 07 2023 at 20:29):

0.4%

Yury G. Kudryashov (Feb 08 2023 at 15:21):

https://leanprover-community.github.io/mathlib-port-status/old reports topology.fiber_bundle.is_homeomorphic_trivial_bundle as "Maybe ready to port" but it was ported.

Eric Wieser (Feb 08 2023 at 16:02):

Maybe #port-wiki doesn't have it yet?

Eric Wieser (Feb 08 2023 at 16:03):

topology.fiber_bundle.is_homeomorphic_trivial_bundle: 'No'

Eric Wieser (Feb 08 2023 at 16:04):

The problem is that the porting comment has been line-wrapped

Eric Wieser (Feb 08 2023 at 16:04):

https://github.com/leanprover-community/mathlib4/pull/2132#discussion_r1100356049

Reid Barton (Feb 08 2023 at 16:05):

ahaha

Reid Barton (Feb 08 2023 at 16:05):

to satisfy the linter probably

Eric Wieser (Feb 08 2023 at 16:05):

Do we fix the script to handle that, or fix the linter?

Eric Wieser (Feb 08 2023 at 16:06):

Do we have any module names that would have to be wrapped mid-name, which would really mess with things?

Reid Barton (Feb 08 2023 at 16:06):

fixing the linter sounds a lot easier

Reid Barton (Feb 08 2023 at 16:06):

just ignore lines starting with !

Eric Wieser (Feb 08 2023 at 16:07):

Changing the regex here is probably also easy

Eric Wieser (Feb 08 2023 at 16:07):

As long as the line wrap only ever happens after the word module

Reid Barton (Feb 08 2023 at 16:07):

I don't agree.

Reid Barton (Feb 08 2023 at 16:07):

Just change the linter

Eric Wieser (Feb 08 2023 at 16:07):

Oh you're right, because we match line by line

port-progress bot (Feb 08 2023 at 18:04):

mathlib port progress linear_algebra.basic
Ported files: 345/355 (97.2% of total)
Ported lines: 140020/145865 (96.0% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 08 2023 at 18:08):

mathlib port progress topology.metric_space.basic
Ported files: 457/480 (95.2% of total)
Ported lines: 190470/207368 (91.9% of total)
Longest unported chain: 6/67 (91.0% progress)

port-progress bot (Feb 08 2023 at 18:12):

mathlib port progress data.polynomial.basic
Ported files: 377/397 (95.0% of total)
Ported lines: 146917/160935 (91.3% of total)
Longest unported chain: 6/58 (89.7% progress)

port-progress bot (Feb 08 2023 at 18:16):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18800/31958 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Feb 08 2023 at 18:20):

mathlib port progress data.complex.basic
Ported files: 513/566 (90.6% of total)
Ported lines: 207580/240198 (86.4% of total)
Longest unported chain: 12/77 (84.4% progress)

port-progress bot (Feb 08 2023 at 18:24):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 619/1020 (60.7% of total)
Ported lines: 231233/435096 (53.1% of total)
Longest unported chain: 51/103 (50.5% progress)

port-progress bot (Feb 08 2023 at 18:29):

mathlib port progress combinatorics.additive.behrend
Ported files: 610/955 (63.9% of total)
Ported lines: 230535/423422 (54.4% of total)
Longest unported chain: 45/102 (55.9% progress)

port-progress bot (Feb 08 2023 at 18:37):

mathlib port progress all
Ported files: 885/2907 (30.4% of total)
Ported lines: 278998/994060 (28.1% of total)
Longest unported chain: 68/125 (45.6% progress)

Johan Commelin (Feb 08 2023 at 18:37):

0.3%

Moritz Doll (Feb 09 2023 at 04:39):

Could we get some more interesting goal in the analysis part (the other bot had fderiv which was pretty good)

port-progress bot (Feb 09 2023 at 18:04):

mathlib port progress linear_algebra.basic
Ported files: 345/355 (97.2% of total)
Ported lines: 140057/145902 (96.0% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 09 2023 at 18:08):

mathlib port progress topology.metric_space.basic
Ported files: 457/480 (95.2% of total)
Ported lines: 190523/207421 (91.9% of total)
Longest unported chain: 6/67 (91.0% progress)

Eric Wieser (Feb 09 2023 at 18:09):

@Moritz Firsching @Moritz Doll, note you can get a progress bar for any file by going to port-status#analysis/calculus/fderiv

Moritz Firsching (Feb 09 2023 at 18:09):

@Moritz Doll ... different Moritz

port-progress bot (Feb 09 2023 at 18:11):

mathlib port progress data.polynomial.basic
Ported files: 377/397 (95.0% of total)
Ported lines: 146954/160972 (91.3% of total)
Longest unported chain: 6/58 (89.7% progress)

port-progress bot (Feb 09 2023 at 18:15):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18800/31958 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Feb 09 2023 at 18:19):

mathlib port progress data.complex.basic
Ported files: 513/566 (90.6% of total)
Ported lines: 207633/240267 (86.4% of total)
Longest unported chain: 12/77 (84.4% progress)

port-progress bot (Feb 09 2023 at 18:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 619/1020 (60.7% of total)
Ported lines: 231301/435180 (53.2% of total)
Longest unported chain: 51/103 (50.5% progress)

port-progress bot (Feb 09 2023 at 18:27):

mathlib port progress combinatorics.additive.behrend
Ported files: 610/955 (63.9% of total)
Ported lines: 230597/423516 (54.4% of total)
Longest unported chain: 45/102 (55.9% progress)

port-progress bot (Feb 09 2023 at 18:35):

mathlib port progress all
Ported files: 884/2858 (30.9% of total)
Ported lines: 279083/994802 (28.1% of total)
Longest unported chain: 68/125 (45.6% progress)

Johan Commelin (Feb 09 2023 at 18:41):

0.0%

Yury G. Kudryashov (Feb 09 2023 at 22:41):

!4#2167 !4#2172 are ready for review

Moritz Doll (Feb 09 2023 at 23:27):

Eric Wieser said:

note you can get a progress bar for any file by going to port-status#analysis/calculus/fderiv

I am more interested in the graph, specifically to see which files should have priority and to find files that only depend on one (almost done) PR. At the moment it seems not to important since everything is blocked by LinearAlgebra.Basic.

Yury G. Kudryashov (Feb 09 2023 at 23:55):

!4#2163 !4#2157 are ready too

Eric Wieser (Feb 10 2023 at 00:16):

#18415 will remove linear_algebra.span from some of those graphs

Yury G. Kudryashov (Feb 10 2023 at 00:29):

!4#2160

Eric Wieser (Feb 10 2023 at 02:07):

Moritz Doll said:

I am more interested in the graph, specifically to see which files should have priority and to find files that only depend on one (almost done) PR. At the moment it seems not to important since everything is blocked by LinearAlgebra.Basic.

There's now a graph hiding on port-status#analysis/calculus/fderiv

Yury G. Kudryashov (Feb 10 2023 at 07:16):

Eric Wieser said:

Oh you're right, because we match line by line

Any progress? Port status still counts this file as unported.

Eric Wieser (Feb 10 2023 at 09:07):

Reid Barton said:

just ignore lines starting with !

No, someone needs to fix the mathlib4 linter

Johan Commelin (Feb 10 2023 at 11:25):

Done in https://github.com/leanprover-community/mathlib4/pull/2190

Johan Commelin (Feb 10 2023 at 11:32):

@Eric Wieser I fixed two files. Were there any others?

Eric Wieser (Feb 10 2023 at 11:32):

I have no idea, were those files found with regex?

Eric Wieser (Feb 10 2023 at 11:33):

I think probably searching for source file\s*\n is probably sufficient

Johan Commelin (Feb 10 2023 at 11:33):

yeah, they were found by regex

Eric Wieser (Feb 10 2023 at 12:25):

Merged! Hopefully port-status#topology/fiber_bundle/is_homeomorphic_trivial_bundle will update shortly

port-progress bot (Feb 10 2023 at 18:05):

mathlib port progress linear_algebra.basic
Ported files: 345/355 (97.2% of total)
Ported lines: 140057/145902 (96.0% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 10 2023 at 18:10):

mathlib port progress topology.metric_space.basic
Ported files: 457/480 (95.2% of total)
Ported lines: 190574/207472 (91.9% of total)
Longest unported chain: 6/67 (91.0% progress)

port-progress bot (Feb 10 2023 at 18:15):

mathlib port progress data.polynomial.basic
Ported files: 377/397 (95.0% of total)
Ported lines: 146954/160972 (91.3% of total)
Longest unported chain: 6/58 (89.7% progress)

port-progress bot (Feb 10 2023 at 18:20):

mathlib port progress category_theory.limits.yoneda
Ported files: 53/92 (57.6% of total)
Ported lines: 18800/31958 (58.8% of total)
Longest unported chain: 16/36 (55.6% progress)

port-progress bot (Feb 10 2023 at 18:25):

mathlib port progress data.complex.basic
Ported files: 513/566 (90.6% of total)
Ported lines: 207684/240339 (86.4% of total)
Longest unported chain: 12/77 (84.4% progress)

port-progress bot (Feb 10 2023 at 18:30):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 619/1020 (60.7% of total)
Ported lines: 231352/435353 (53.1% of total)
Longest unported chain: 51/103 (50.5% progress)

port-progress bot (Feb 10 2023 at 18:36):

mathlib port progress combinatorics.additive.behrend
Ported files: 610/955 (63.9% of total)
Ported lines: 230648/423689 (54.4% of total)
Longest unported chain: 45/102 (55.9% progress)

port-progress bot (Feb 10 2023 at 18:48):

mathlib port progress all
Ported files: 890/2860 (31.1% of total)
Ported lines: 279757/995851 (28.1% of total)
Longest unported chain: 68/125 (45.6% progress)

Johan Commelin (Feb 10 2023 at 19:01):

0.0%

Johan Commelin (Feb 11 2023 at 15:56):

Yay! Category theory is ready for porting! See "Unported files" in #port-dashboard

Eric Wieser (Feb 11 2023 at 17:16):

Eric Wieser said:

#18415 will remove linear_algebra.span from some of those graphs

Done. If linear_algebra.basic remains a blocker, we could consider removing the dependency from algebra.algebra.basic; only two lemmas in that file need the import, and one of them (docs#linear_map.ker_restrict_scalars) has a TODO comment saying "this result doesn't belong here". The other is docs#ker_algebra_map_End.

Johan Commelin (Feb 11 2023 at 17:24):

Sounds good to me

Eric Wieser (Feb 11 2023 at 17:40):

I'm not actively working on that at the moment

port-progress bot (Feb 11 2023 at 18:05):

mathlib port progress linear_algebra.basic
Ported files: 345/355 (97.2% of total)
Ported lines: 140063/145908 (96.0% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 11 2023 at 18:10):

mathlib port progress topology.metric_space.basic
Ported files: 450/468 (96.2% of total)
Ported lines: 189197/203317 (93.1% of total)
Longest unported chain: 5/67 (92.5% progress)

port-progress bot (Feb 11 2023 at 18:15):

mathlib port progress data.polynomial.basic
Ported files: 378/397 (95.2% of total)
Ported lines: 148134/160960 (92.0% of total)
Longest unported chain: 5/57 (91.2% progress)

port-progress bot (Feb 11 2023 at 18:19):

mathlib port progress category_theory.limits.yoneda
Ported files: 57/92 (62.0% of total)
Ported lines: 20261/31958 (63.4% of total)
Longest unported chain: 13/36 (63.9% progress)

port-progress bot (Feb 11 2023 at 18:24):

mathlib port progress data.complex.basic
Ported files: 519/566 (91.7% of total)
Ported lines: 210033/240327 (87.4% of total)
Longest unported chain: 12/77 (84.4% progress)

port-progress bot (Feb 11 2023 at 18:29):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 632/1020 (62.0% of total)
Ported lines: 236922/435339 (54.4% of total)
Longest unported chain: 50/102 (51.0% progress)

port-progress bot (Feb 11 2023 at 18:34):

mathlib port progress combinatorics.additive.behrend
Ported files: 622/955 (65.1% of total)
Ported lines: 236119/423675 (55.7% of total)
Longest unported chain: 44/102 (56.9% progress)

port-progress bot (Feb 11 2023 at 18:45):

mathlib port progress all
Ported files: 917/2863 (32.0% of total)
Ported lines: 290666/996168 (29.2% of total)
Longest unported chain: 67/125 (46.4% progress)

Johan Commelin (Feb 11 2023 at 18:51):

1.1%

port-progress bot (Feb 12 2023 at 18:05):

mathlib port progress linear_algebra.basic
Ported files: 345/355 (97.2% of total)
Ported lines: 140063/145908 (96.0% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 12 2023 at 18:10):

mathlib port progress topology.metric_space.basic
Ported files: 451/468 (96.4% of total)
Ported lines: 189294/203317 (93.1% of total)
Longest unported chain: 5/67 (92.5% progress)

Eric Wieser (Feb 12 2023 at 18:11):

(port-status#data/polynomial/basic#graph now has a slightly-interactive version of the graph below)

port-progress bot (Feb 12 2023 at 18:14):

mathlib port progress data.polynomial.basic
Ported files: 378/397 (95.2% of total)
Ported lines: 148134/160960 (92.0% of total)
Longest unported chain: 5/57 (91.2% progress)

port-progress bot (Feb 12 2023 at 18:19):

mathlib port progress category_theory.limits.yoneda
Ported files: 57/92 (62.0% of total)
Ported lines: 20261/31958 (63.4% of total)
Longest unported chain: 13/36 (63.9% progress)

port-progress bot (Feb 12 2023 at 18:24):

mathlib port progress data.complex.basic
Ported files: 521/566 (92.0% of total)
Ported lines: 210440/240327 (87.6% of total)
Longest unported chain: 12/77 (84.4% progress)

port-progress bot (Feb 12 2023 at 18:29):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 635/1020 (62.3% of total)
Ported lines: 237613/435339 (54.6% of total)
Longest unported chain: 50/102 (51.0% progress)

port-progress bot (Feb 12 2023 at 18:35):

mathlib port progress combinatorics.additive.behrend
Ported files: 626/955 (65.5% of total)
Ported lines: 236967/423675 (55.9% of total)
Longest unported chain: 44/102 (56.9% progress)

port-progress bot (Feb 12 2023 at 18:46):

mathlib port progress all
Ported files: 924/2863 (32.3% of total)
Ported lines: 291920/996169 (29.3% of total)
Longest unported chain: 67/125 (46.4% progress)

Johan Commelin (Feb 13 2023 at 07:14):

0.1%

port-progress bot (Feb 13 2023 at 18:03):

mathlib port progress linear_algebra.basic
Ported files: 346/355 (97.5% of total)
Ported lines: 142270/145953 (97.5% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 13 2023 at 18:08):

mathlib port progress topology.metric_space.basic
Ported files: 452/468 (96.6% of total)
Ported lines: 191516/203395 (94.2% of total)
Longest unported chain: 4/67 (94.0% progress)

port-progress bot (Feb 13 2023 at 18:12):

mathlib port progress data.polynomial.basic
Ported files: 379/397 (95.5% of total)
Ported lines: 150344/161026 (93.4% of total)
Longest unported chain: 4/57 (93.0% progress)

port-progress bot (Feb 13 2023 at 18:17):

mathlib port progress category_theory.limits.yoneda
Ported files: 57/92 (62.0% of total)
Ported lines: 20273/31970 (63.4% of total)
Longest unported chain: 13/36 (63.9% progress)

port-progress bot (Feb 13 2023 at 18:21):

mathlib port progress data.complex.basic
Ported files: 524/566 (92.6% of total)
Ported lines: 213192/240417 (88.7% of total)
Longest unported chain: 11/77 (85.7% progress)

port-progress bot (Feb 13 2023 at 18:27):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 639/1020 (62.6% of total)
Ported lines: 241481/435453 (55.5% of total)
Longest unported chain: 49/102 (52.0% progress)

port-progress bot (Feb 13 2023 at 18:32):

mathlib port progress combinatorics.additive.behrend
Ported files: 630/955 (66.0% of total)
Ported lines: 240835/423788 (56.8% of total)
Longest unported chain: 43/102 (57.8% progress)

port-progress bot (Feb 13 2023 at 18:42):

mathlib port progress all
Ported files: 934/2863 (32.6% of total)
Ported lines: 296910/996342 (29.8% of total)
Longest unported chain: 66/125 (47.2% progress)

Johan Commelin (Feb 13 2023 at 18:44):

0.5%

Chris Hughes (Feb 13 2023 at 18:48):

Why is it less than the percentage on https://leanprover-community.github.io/mathlib-port-status/

Oisin McGuinness (Feb 13 2023 at 18:51):

Daily increment, not total ported, I guess.

Chris Hughes (Feb 13 2023 at 18:56):

It says 29.8% lines ported here, but 30.0% on the website

Oisin McGuinness (Feb 13 2023 at 18:57):

Sorry, thought you were referring to Johan's number.

Jireh Loreaux (Feb 13 2023 at 19:27):

Were there several files merged while the bot was running?

Johan Commelin (Feb 13 2023 at 19:34):

I don't think so

Eric Wieser (Feb 13 2023 at 21:13):

I think some files might not have available line counts on the website?

Eric Wieser (Feb 13 2023 at 21:13):

The total number of _ported_ lines is the same, right?

Eric Wieser (Feb 13 2023 at 21:21):

I think it might be this try/catch: https://github.com/leanprover-community/mathlib-port-status/blob/0be459e429048ac2034760065d27330e2ba7c9fa/make_html.py#L232

Eric Wieser (Feb 13 2023 at 21:35):

I would guess it's due to default files not being handled correctly

port-progress bot (Feb 14 2023 at 18:03):

mathlib port progress linear_algebra.basic
Ported files: 346/355 (97.5% of total)
Ported lines: 142273/145956 (97.5% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 14 2023 at 18:08):

mathlib port progress topology.metric_space.basic
Ported files: 452/468 (96.6% of total)
Ported lines: 191519/203398 (94.2% of total)
Longest unported chain: 4/67 (94.0% progress)

port-progress bot (Feb 14 2023 at 18:12):

mathlib port progress data.polynomial.basic
Ported files: 381/397 (96.0% of total)
Ported lines: 151742/161029 (94.2% of total)
Longest unported chain: 4/57 (93.0% progress)

port-progress bot (Feb 14 2023 at 18:16):

mathlib port progress category_theory.limits.yoneda
Ported files: 60/92 (65.2% of total)
Ported lines: 20849/31970 (65.2% of total)
Longest unported chain: 13/36 (63.9% progress)

port-progress bot (Feb 14 2023 at 18:20):

mathlib port progress data.complex.basic
Ported files: 527/566 (93.1% of total)
Ported lines: 215280/240423 (89.5% of total)
Longest unported chain: 10/77 (87.0% progress)

port-progress bot (Feb 14 2023 at 18:25):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 647/1020 (63.4% of total)
Ported lines: 245258/435465 (56.3% of total)
Longest unported chain: 49/102 (52.0% progress)

port-progress bot (Feb 14 2023 at 18:30):

mathlib port progress combinatorics.additive.behrend
Ported files: 640/955 (67.0% of total)
Ported lines: 245072/423803 (57.8% of total)
Longest unported chain: 43/102 (57.8% progress)

port-progress bot (Feb 14 2023 at 18:39):

mathlib port progress all
Ported files: 952/2864 (33.2% of total)
Ported lines: 302920/996711 (30.4% of total)
Longest unported chain: 66/125 (47.2% progress)

Johan Commelin (Feb 14 2023 at 18:52):

0.6%

port-progress bot (Feb 15 2023 at 18:03):

mathlib port progress linear_algebra.basic
Ported files: 346/355 (97.5% of total)
Ported lines: 142274/145957 (97.5% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 15 2023 at 18:08):

mathlib port progress topology.metric_space.basic
Ported files: 452/468 (96.6% of total)
Ported lines: 191520/203399 (94.2% of total)
Longest unported chain: 4/67 (94.0% progress)

port-progress bot (Feb 15 2023 at 18:13):

mathlib port progress data.polynomial.basic
Ported files: 381/397 (96.0% of total)
Ported lines: 151749/161036 (94.2% of total)
Longest unported chain: 4/57 (93.0% progress)

port-progress bot (Feb 15 2023 at 18:17):

mathlib port progress category_theory.limits.yoneda
Ported files: 66/92 (71.7% of total)
Ported lines: 21874/31979 (68.4% of total)
Longest unported chain: 12/36 (66.7% progress)

port-progress bot (Feb 15 2023 at 18:22):

mathlib port progress data.complex.basic
Ported files: 528/566 (93.3% of total)
Ported lines: 215574/240433 (89.7% of total)
Longest unported chain: 10/77 (87.0% progress)

port-progress bot (Feb 15 2023 at 18:27):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 649/1022 (63.5% of total)
Ported lines: 245788/435737 (56.4% of total)
Longest unported chain: 49/102 (52.0% progress)

port-progress bot (Feb 15 2023 at 18:32):

mathlib port progress combinatorics.additive.behrend
Ported files: 642/957 (67.1% of total)
Ported lines: 245605/424078 (57.9% of total)
Longest unported chain: 43/102 (57.8% progress)

port-progress bot (Feb 15 2023 at 18:41):

mathlib port progress all
Ported files: 966/2865 (33.7% of total)
Ported lines: 307951/997153 (30.9% of total)
Longest unported chain: 66/125 (47.2% progress)

Jireh Loreaux (Feb 15 2023 at 19:09):

0.5%. That makes 6.5% in the past two weeks. On track for mid-July at that pace.

port-progress bot (Feb 16 2023 at 18:04):

mathlib port progress linear_algebra.basic
Ported files: 346/355 (97.5% of total)
Ported lines: 142290/145973 (97.5% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 16 2023 at 18:09):

mathlib port progress topology.metric_space.basic
Ported files: 452/468 (96.6% of total)
Ported lines: 191536/203415 (94.2% of total)
Longest unported chain: 4/67 (94.0% progress)

port-progress bot (Feb 16 2023 at 18:14):

mathlib port progress data.polynomial.basic
Ported files: 381/397 (96.0% of total)
Ported lines: 151765/161052 (94.2% of total)
Longest unported chain: 4/57 (93.0% progress)

port-progress bot (Feb 16 2023 at 18:18):

mathlib port progress category_theory.limits.yoneda
Ported files: 67/92 (72.8% of total)
Ported lines: 21930/31987 (68.6% of total)
Longest unported chain: 12/36 (66.7% progress)

port-progress bot (Feb 16 2023 at 18:23):

mathlib port progress data.complex.basic
Ported files: 528/568 (93.0% of total)
Ported lines: 215590/240375 (89.7% of total)
Longest unported chain: 9/76 (88.2% progress)

port-progress bot (Feb 16 2023 at 18:28):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 650/1025 (63.4% of total)
Ported lines: 247783/435788 (56.9% of total)
Longest unported chain: 49/102 (52.0% progress)

port-progress bot (Feb 16 2023 at 18:33):

mathlib port progress combinatorics.additive.behrend
Ported files: 643/960 (67.0% of total)
Ported lines: 247600/424129 (58.4% of total)
Longest unported chain: 43/102 (57.8% progress)

port-progress bot (Feb 16 2023 at 18:43):

mathlib port progress all
Ported files: 972/2868 (33.9% of total)
Ported lines: 310752/997327 (31.2% of total)
Longest unported chain: 66/125 (47.2% progress)

Johan Commelin (Feb 16 2023 at 18:50):

0.3%

port-progress bot (Feb 17 2023 at 18:03):

mathlib port progress linear_algebra.basic
Ported files: 346/355 (97.5% of total)
Ported lines: 142291/145974 (97.5% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 17 2023 at 18:08):

mathlib port progress topology.metric_space.basic
Ported files: 452/468 (96.6% of total)
Ported lines: 191635/203514 (94.2% of total)
Longest unported chain: 4/67 (94.0% progress)

port-progress bot (Feb 17 2023 at 18:13):

mathlib port progress data.polynomial.basic
Ported files: 381/397 (96.0% of total)
Ported lines: 151766/161053 (94.2% of total)
Longest unported chain: 4/57 (93.0% progress)

port-progress bot (Feb 17 2023 at 18:17):

mathlib port progress category_theory.limits.yoneda
Ported files: 68/92 (73.9% of total)
Ported lines: 22171/31987 (69.3% of total)
Longest unported chain: 11/36 (69.4% progress)

port-progress bot (Feb 17 2023 at 18:22):

mathlib port progress data.complex.basic
Ported files: 528/568 (93.0% of total)
Ported lines: 215689/240474 (89.7% of total)
Longest unported chain: 9/76 (88.2% progress)

port-progress bot (Feb 17 2023 at 18:27):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 651/1026 (63.5% of total)
Ported lines: 248176/436254 (56.9% of total)
Longest unported chain: 49/102 (52.0% progress)

port-progress bot (Feb 17 2023 at 18:32):

mathlib port progress combinatorics.additive.behrend
Ported files: 644/961 (67.0% of total)
Ported lines: 247993/424595 (58.4% of total)
Longest unported chain: 43/102 (57.8% progress)

port-progress bot (Feb 17 2023 at 18:43):

mathlib port progress all
Ported files: 973/2869 (33.9% of total)
Ported lines: 310892/997796 (31.2% of total)
Longest unported chain: 66/125 (47.2% progress)

Johan Commelin (Feb 17 2023 at 19:22):

0.0%

Jason Yuen (Feb 18 2023 at 03:53):

port-progress bot said:

mathlib port progress linear_algebra.basic
Ported files: 346/355 (97.5% of total)
Ported lines: 142291/145974 (97.5% of total)
Longest unported chain: 1/52 (98.1% progress)

This target is done. Can this target be removed?

port-progress bot (Feb 18 2023 at 18:04):

mathlib port progress linear_algebra.basic
Ported files: 346/355 (97.5% of total)
Ported lines: 142291/145974 (97.5% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 18 2023 at 18:10):

mathlib port progress topology.metric_space.basic
Ported files: 452/468 (96.6% of total)
Ported lines: 191635/203514 (94.2% of total)
Longest unported chain: 4/67 (94.0% progress)

port-progress bot (Feb 18 2023 at 18:15):

mathlib port progress data.polynomial.basic
Ported files: 381/397 (96.0% of total)
Ported lines: 151766/161053 (94.2% of total)
Longest unported chain: 4/57 (93.0% progress)

port-progress bot (Feb 18 2023 at 18:20):

mathlib port progress category_theory.limits.yoneda
Ported files: 68/92 (73.9% of total)
Ported lines: 22171/31987 (69.3% of total)
Longest unported chain: 11/36 (69.4% progress)

port-progress bot (Feb 18 2023 at 18:26):

mathlib port progress data.complex.basic
Ported files: 528/568 (93.0% of total)
Ported lines: 215689/240474 (89.7% of total)
Longest unported chain: 9/76 (88.2% progress)

port-progress bot (Feb 18 2023 at 18:32):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 651/1026 (63.5% of total)
Ported lines: 248176/436254 (56.9% of total)
Longest unported chain: 49/102 (52.0% progress)

port-progress bot (Feb 18 2023 at 18:38):

mathlib port progress combinatorics.additive.behrend
Ported files: 644/961 (67.0% of total)
Ported lines: 247993/424595 (58.4% of total)
Longest unported chain: 43/102 (57.8% progress)

port-progress bot (Feb 18 2023 at 18:50):

mathlib port progress all
Ported files: 979/2869 (34.1% of total)
Ported lines: 312164/997783 (31.3% of total)
Longest unported chain: 66/125 (47.2% progress)

Johan Commelin (Feb 18 2023 at 18:54):

0.1%

port-progress bot (Feb 19 2023 at 18:03):

mathlib port progress linear_algebra.basic
Ported files: 346/355 (97.5% of total)
Ported lines: 142291/145974 (97.5% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 19 2023 at 18:08):

mathlib port progress topology.metric_space.basic
Ported files: 453/468 (96.8% of total)
Ported lines: 192471/203514 (94.6% of total)
Longest unported chain: 3/67 (95.5% progress)

port-progress bot (Feb 19 2023 at 18:12):

mathlib port progress data.polynomial.basic
Ported files: 382/397 (96.2% of total)
Ported lines: 152602/161053 (94.8% of total)
Longest unported chain: 3/57 (94.7% progress)

port-progress bot (Feb 19 2023 at 18:17):

mathlib port progress category_theory.limits.yoneda
Ported files: 68/92 (73.9% of total)
Ported lines: 22195/32011 (69.3% of total)
Longest unported chain: 11/36 (69.4% progress)

port-progress bot (Feb 19 2023 at 18:21):

mathlib port progress data.complex.basic
Ported files: 531/568 (93.5% of total)
Ported lines: 217664/240477 (90.5% of total)
Longest unported chain: 9/76 (88.2% progress)

port-progress bot (Feb 19 2023 at 18:26):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 656/1026 (63.9% of total)
Ported lines: 251353/436260 (57.6% of total)
Longest unported chain: 48/102 (52.9% progress)

port-progress bot (Feb 19 2023 at 18:31):

mathlib port progress combinatorics.additive.behrend
Ported files: 649/961 (67.5% of total)
Ported lines: 251170/424601 (59.2% of total)
Longest unported chain: 42/102 (58.8% progress)

port-progress bot (Feb 19 2023 at 18:42):

mathlib port progress all
Ported files: 993/2869 (34.6% of total)
Ported lines: 317550/997843 (31.8% of total)
Longest unported chain: 65/125 (48.0% progress)

Johan Commelin (Feb 20 2023 at 07:45):

0.5%

port-progress bot (Feb 20 2023 at 18:03):

mathlib port progress linear_algebra.basic
Ported files: 346/355 (97.5% of total)
Ported lines: 142372/146055 (97.5% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 20 2023 at 18:08):

mathlib port progress topology.metric_space.basic
Ported files: 454/468 (97.0% of total)
Ported lines: 193427/203595 (95.0% of total)
Longest unported chain: 2/67 (97.0% progress)

port-progress bot (Feb 20 2023 at 18:12):

mathlib port progress data.polynomial.basic
Ported files: 382/397 (96.2% of total)
Ported lines: 152683/161134 (94.8% of total)
Longest unported chain: 3/57 (94.7% progress)

port-progress bot (Feb 20 2023 at 18:16):

mathlib port progress category_theory.limits.yoneda
Ported files: 69/92 (75.0% of total)
Ported lines: 22685/32092 (70.7% of total)
Longest unported chain: 11/36 (69.4% progress)

port-progress bot (Feb 20 2023 at 18:21):

mathlib port progress data.complex.basic
Ported files: 532/568 (93.7% of total)
Ported lines: 218620/240558 (90.9% of total)
Longest unported chain: 9/76 (88.2% progress)

port-progress bot (Feb 20 2023 at 18:26):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 658/1026 (64.1% of total)
Ported lines: 252742/436344 (57.9% of total)
Longest unported chain: 48/102 (52.9% progress)

port-progress bot (Feb 20 2023 at 18:31):

mathlib port progress combinatorics.additive.behrend
Ported files: 651/961 (67.7% of total)
Ported lines: 252559/424685 (59.5% of total)
Longest unported chain: 42/102 (58.8% progress)

port-progress bot (Feb 20 2023 at 18:40):

mathlib port progress all
Ported files: 1003/2869 (35.0% of total)
Ported lines: 320673/998208 (32.1% of total)
Longest unported chain: 65/125 (48.0% progress)

Johan Commelin (Feb 20 2023 at 18:53):

0.3%

port-progress bot (Feb 21 2023 at 18:03):

mathlib port progress linear_algebra.basic
Ported files: 346/355 (97.5% of total)
Ported lines: 142372/146055 (97.5% of total)
Longest unported chain: 1/52 (98.1% progress)

port-progress bot (Feb 21 2023 at 18:07):

mathlib port progress topology.metric_space.basic
Ported files: 454/468 (97.0% of total)
Ported lines: 193427/203595 (95.0% of total)
Longest unported chain: 2/67 (97.0% progress)

port-progress bot (Feb 21 2023 at 18:11):

mathlib port progress data.polynomial.basic
Ported files: 384/397 (96.7% of total)
Ported lines: 154145/161134 (95.7% of total)
Longest unported chain: 2/57 (96.5% progress)

port-progress bot (Feb 21 2023 at 18:15):

mathlib port progress category_theory.limits.yoneda
Ported files: 72/92 (78.3% of total)
Ported lines: 23602/32092 (73.5% of total)
Longest unported chain: 11/36 (69.4% progress)

port-progress bot (Feb 21 2023 at 18:19):

mathlib port progress data.complex.basic
Ported files: 534/568 (94.0% of total)
Ported lines: 220413/240558 (91.6% of total)
Longest unported chain: 8/76 (89.5% progress)

port-progress bot (Feb 21 2023 at 18:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 664/1026 (64.7% of total)
Ported lines: 256414/436344 (58.8% of total)
Longest unported chain: 45/102 (55.9% progress)

port-progress bot (Feb 21 2023 at 18:28):

mathlib port progress combinatorics.additive.behrend
Ported files: 657/961 (68.4% of total)
Ported lines: 256231/424685 (60.3% of total)
Longest unported chain: 39/102 (61.8% progress)

port-progress bot (Feb 21 2023 at 18:35):

mathlib port progress all
Ported files: 1020/2869 (35.6% of total)
Ported lines: 326621/998208 (32.7% of total)
Longest unported chain: 62/125 (50.4% progress)

Mario Carneiro (Feb 21 2023 at 18:37):

Ooh, 50% (by some metric...)

Eric Wieser (Feb 21 2023 at 18:44):

Seems that port-status#analysis/normed_space/star/gelfand_duality (at the end of that chain) is not willing to render such a large graph

Floris van Doorn (Feb 21 2023 at 19:00):

I like how we can celebrate reaching each percentage milestone 3 times :-)

Johan Commelin (Feb 21 2023 at 19:05):

0.6%

Johan Commelin (Feb 21 2023 at 20:56):

If I count correctly, there are only 15 unported files left that have more than 1000 dependents.

Johan Commelin (Feb 21 2023 at 20:57):

Of these, 3 are in progress, and 3 are ready to be ported.

Johan Commelin (Feb 21 2023 at 21:03):

I think that https://leanprover-community.github.io/mathlib-port-status/file/ring_theory/principal_ideal_domain is a nice target

Eric Wieser (Feb 21 2023 at 21:04):

This seems like a nice excuse to plug #18468, which will optimistically cut a bunch of files from the left side of that graph

before after
before after

Eric Wieser (Feb 21 2023 at 21:04):

Or at least, reduce the height of the graph by rearranging the nodes

Johan Commelin (Feb 22 2023 at 02:57):

We are 300 files away from the point where every unported file has ≤ 200 dependents. At that point, there will be ~1400 files left to be ported.

Eric Wieser (Feb 22 2023 at 13:20):

The new graph only ended up being shallower by two nodes, but it has more accessible root nodes now!

port-progress bot (Feb 22 2023 at 18:04):

mathlib port progress topology.metric_space.basic
Ported files: 454/468 (97.0% of total)
Ported lines: 193433/203601 (95.0% of total)
Longest unported chain: 2/67 (97.0% progress)

port-progress bot (Feb 22 2023 at 18:09):

mathlib port progress data.polynomial.basic
Ported files: 384/397 (96.7% of total)
Ported lines: 154154/161143 (95.7% of total)
Longest unported chain: 2/57 (96.5% progress)

port-progress bot (Feb 22 2023 at 18:13):

mathlib port progress category_theory.limits.yoneda
Ported files: 76/92 (82.6% of total)
Ported lines: 24273/32107 (75.6% of total)
Longest unported chain: 8/36 (77.8% progress)

port-progress bot (Feb 22 2023 at 18:18):

mathlib port progress data.complex.basic
Ported files: 536/568 (94.4% of total)
Ported lines: 222057/240579 (92.3% of total)
Longest unported chain: 8/76 (89.5% progress)

port-progress bot (Feb 22 2023 at 18:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 668/1027 (65.0% of total)
Ported lines: 259430/436413 (59.4% of total)
Longest unported chain: 43/98 (56.1% progress)

port-progress bot (Feb 22 2023 at 18:28):

mathlib port progress combinatorics.additive.behrend
Ported files: 661/962 (68.7% of total)
Ported lines: 259247/424754 (61.0% of total)
Longest unported chain: 37/102 (63.7% progress)

port-progress bot (Feb 22 2023 at 18:37):

mathlib port progress all
Ported files: 1039/2870 (36.2% of total)
Ported lines: 331437/998461 (33.2% of total)
Longest unported chain: 60/125 (52.0% progress)

Johan Commelin (Feb 22 2023 at 18:39):

0.5%

port-progress bot (Feb 23 2023 at 18:04):

mathlib port progress topology.metric_space.basic
Ported files: 456/470 (97.0% of total)
Ported lines: 194125/204293 (95.0% of total)
Longest unported chain: 2/69 (97.1% progress)

port-progress bot (Feb 23 2023 at 18:08):

mathlib port progress data.polynomial.basic
Ported files: 384/397 (96.7% of total)
Ported lines: 154197/161186 (95.7% of total)
Longest unported chain: 2/57 (96.5% progress)

port-progress bot (Feb 23 2023 at 18:12):

mathlib port progress category_theory.limits.yoneda
Ported files: 78/92 (84.8% of total)
Ported lines: 24650/32116 (76.8% of total)
Longest unported chain: 6/36 (83.3% progress)

port-progress bot (Feb 23 2023 at 18:16):

mathlib port progress data.complex.basic
Ported files: 537/568 (94.5% of total)
Ported lines: 222843/240662 (92.6% of total)
Longest unported chain: 8/77 (89.6% progress)

port-progress bot (Feb 23 2023 at 18:21):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 673/1027 (65.5% of total)
Ported lines: 263454/436569 (60.3% of total)
Longest unported chain: 43/98 (56.1% progress)

port-progress bot (Feb 23 2023 at 18:25):

mathlib port progress combinatorics.additive.behrend
Ported files: 665/962 (69.1% of total)
Ported lines: 262950/424910 (61.9% of total)
Longest unported chain: 37/102 (63.7% progress)

port-progress bot (Feb 23 2023 at 18:33):

mathlib port progress all
Ported files: 1054/2870 (36.7% of total)
Ported lines: 337721/998879 (33.8% of total)
Longest unported chain: 60/125 (52.0% progress)

Adam Topaz (Feb 23 2023 at 18:34):

Can we get Kan extensions ported before quadratic reciprocity? :race: :racecar:

Matthew Ballard (Feb 23 2023 at 18:35):

My class requested spending some time on the porting process

Johan Commelin (Feb 23 2023 at 18:50):

0.6%

Kevin Buzzard (Feb 23 2023 at 22:22):

Quadratic reciprocity is a nontrivial theorem so it wouldn't surprise me if Kan extensions got ported first

Adam Topaz (Feb 23 2023 at 22:38):

okay, so let's use docs#category_theory.presheaf_to_Sheaf as the benchmark ;)

Kevin Buzzard (Feb 23 2023 at 22:42):

I still reckon Gauss would have had a much easier time following his nose to sheafify a presheaf than to actually prove the hard theorem that is quadratic reciprocity

Adam Topaz (Feb 23 2023 at 22:43):

I agree. I think they're both nontrivial for entirely different reasons, so it would be interesting to see which one comes first.

port-progress bot (Feb 26 2023 at 18:05):

mathlib port progress topology.metric_space.basic
Ported files: 457/470 (97.2% of total)
Ported lines: 194229/204280 (95.1% of total)
Longest unported chain: 2/69 (97.1% progress)

port-progress bot (Feb 26 2023 at 18:08):

mathlib port progress data.polynomial.basic
Ported files: 384/397 (96.7% of total)
Ported lines: 154206/161195 (95.7% of total)
Longest unported chain: 2/57 (96.5% progress)

port-progress bot (Feb 26 2023 at 18:12):

mathlib port progress category_theory.limits.yoneda
Ported files: 79/92 (85.9% of total)
Ported lines: 25504/32122 (79.4% of total)
Longest unported chain: 5/36 (86.1% progress)

port-progress bot (Feb 26 2023 at 18:16):

mathlib port progress data.complex.basic
Ported files: 541/568 (95.2% of total)
Ported lines: 224542/240649 (93.3% of total)
Longest unported chain: 7/77 (90.9% progress)

port-progress bot (Feb 26 2023 at 18:20):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 679/1027 (66.1% of total)
Ported lines: 267039/436610 (61.2% of total)
Longest unported chain: 43/98 (56.1% progress)

port-progress bot (Feb 26 2023 at 18:24):

mathlib port progress combinatorics.additive.behrend
Ported files: 671/962 (69.8% of total)
Ported lines: 266532/424948 (62.7% of total)
Longest unported chain: 37/102 (63.7% progress)

Adam Topaz (Feb 26 2023 at 18:31):

port-progress bot said:

mathlib port progress category_theory.limits.yoneda
Ported files: 79/92 (85.9% of total)
Ported lines: 25504/32122 (79.4% of total)
Longest unported chain: 5/36 (86.1% progress)

Okay, I think we can kill this one off this week

port-progress bot (Feb 26 2023 at 18:31):

mathlib port progress all
Ported files: 1068/2875 (37.1% of total)
Ported lines: 344599/1000847 (34.4% of total)
Longest unported chain: 60/125 (52.0% progress)

Matthew Ballard (Feb 26 2023 at 18:54):

Adam Topaz said:

port-progress bot said:

mathlib port progress category_theory.limits.yoneda
Ported files: 79/92 (85.9% of total)
Ported lines: 25504/32122 (79.4% of total)
Longest unported chain: 5/36 (86.1% progress)

Okay, I think we can kill this one off this week

!4#2381

Matthew Ballard (Feb 26 2023 at 19:06):

Living life on the row

Yury G. Kudryashov (Feb 27 2023 at 04:34):

(deleted)

Johan Commelin (Feb 27 2023 at 07:40):

0.6%

port-progress bot (Feb 27 2023 at 18:04):

mathlib port progress topology.metric_space.basic
Ported files: 458/470 (97.4% of total)
Ported lines: 196227/204245 (96.1% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Feb 27 2023 at 18:08):

mathlib port progress data.polynomial.basic
Ported files: 384/397 (96.7% of total)
Ported lines: 154203/161192 (95.7% of total)
Longest unported chain: 2/57 (96.5% progress)

port-progress bot (Feb 27 2023 at 18:12):

mathlib port progress category_theory.limits.yoneda
Ported files: 80/92 (87.0% of total)
Ported lines: 26461/32122 (82.4% of total)
Longest unported chain: 4/36 (88.9% progress)

port-progress bot (Feb 27 2023 at 18:16):

mathlib port progress data.complex.basic
Ported files: 543/568 (95.6% of total)
Ported lines: 227417/240614 (94.5% of total)
Longest unported chain: 7/77 (90.9% progress)

port-progress bot (Feb 27 2023 at 18:20):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 684/1027 (66.6% of total)
Ported lines: 271333/436586 (62.1% of total)
Longest unported chain: 43/98 (56.1% progress)

port-progress bot (Feb 27 2023 at 18:24):

mathlib port progress combinatorics.additive.behrend
Ported files: 676/962 (70.3% of total)
Ported lines: 270826/424924 (63.7% of total)
Longest unported chain: 37/102 (63.7% progress)

port-progress bot (Feb 27 2023 at 18:31):

mathlib port progress all
Ported files: 1086/2877 (37.7% of total)
Ported lines: 354703/1001160 (35.4% of total)
Longest unported chain: 60/125 (52.0% progress)

Johan Commelin (Feb 27 2023 at 19:40):

1.0%

port-progress bot (Feb 28 2023 at 18:04):

mathlib port progress topology.metric_space.basic
Ported files: 458/470 (97.4% of total)
Ported lines: 196284/204229 (96.1% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Feb 28 2023 at 18:09):

mathlib port progress data.polynomial.basic
Ported files: 385/397 (97.0% of total)
Ported lines: 154559/161215 (95.9% of total)
Longest unported chain: 2/57 (96.5% progress)

port-progress bot (Feb 28 2023 at 18:13):

mathlib port progress category_theory.limits.yoneda
Ported files: 80/92 (87.0% of total)
Ported lines: 26461/32122 (82.4% of total)
Longest unported chain: 4/36 (88.9% progress)

Johan Commelin (Feb 28 2023 at 18:14):

wow, that's converging fast (-; Not so long ago it was only ~50% done.

port-progress bot (Feb 28 2023 at 18:18):

mathlib port progress data.complex.basic
Ported files: 543/568 (95.6% of total)
Ported lines: 227474/240598 (94.5% of total)
Longest unported chain: 7/77 (90.9% progress)

port-progress bot (Feb 28 2023 at 18:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 689/1027 (67.1% of total)
Ported lines: 272889/436606 (62.5% of total)
Longest unported chain: 41/98 (58.2% progress)

port-progress bot (Feb 28 2023 at 18:27):

mathlib port progress combinatorics.additive.behrend
Ported files: 682/962 (70.9% of total)
Ported lines: 272501/424944 (64.1% of total)
Longest unported chain: 35/102 (65.7% progress)

Eric Wieser (Feb 28 2023 at 18:28):

port-status#number_theory/legendre_symbol/quadratic_reciprocity can just about handle the graph for that now, if you leave it a while to think about the layout

port-progress bot (Feb 28 2023 at 18:36):

mathlib port progress all
Ported files: 1096/2879 (38.1% of total)
Ported lines: 358111/1001465 (35.8% of total)
Longest unported chain: 58/125 (53.6% progress)

Johan Commelin (Feb 28 2023 at 19:22):

0.4%

port-progress bot (Mar 01 2023 at 18:04):

mathlib port progress topology.metric_space.basic
Ported files: 458/470 (97.4% of total)
Ported lines: 196291/204236 (96.1% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Mar 01 2023 at 18:08):

mathlib port progress data.polynomial.basic
Ported files: 386/397 (97.2% of total)
Ported lines: 155091/161222 (96.2% of total)
Longest unported chain: 1/57 (98.2% progress)

port-progress bot (Mar 01 2023 at 18:12):

mathlib port progress category_theory.limits.yoneda
Ported files: 82/92 (89.1% of total)
Ported lines: 28322/32131 (88.1% of total)
Longest unported chain: 2/36 (94.4% progress)

port-progress bot (Mar 01 2023 at 18:16):

mathlib port progress data.complex.basic
Ported files: 543/568 (95.6% of total)
Ported lines: 227493/240617 (94.5% of total)
Longest unported chain: 7/77 (90.9% progress)

port-progress bot (Mar 01 2023 at 18:21):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 695/1031 (67.4% of total)
Ported lines: 276076/438450 (63.0% of total)
Longest unported chain: 40/98 (59.2% progress)

port-progress bot (Mar 01 2023 at 18:25):

mathlib port progress combinatorics.additive.behrend
Ported files: 688/966 (71.2% of total)
Ported lines: 275691/426791 (64.6% of total)
Longest unported chain: 34/102 (66.7% progress)

port-progress bot (Mar 01 2023 at 18:32):

mathlib port progress all
Ported files: 1108/2880 (38.5% of total)
Ported lines: 365606/1002344 (36.5% of total)
Longest unported chain: 58/126 (54.0% progress)

Johan Commelin (Mar 01 2023 at 18:36):

0.7%

Matthew Ballard (Mar 02 2023 at 03:58):

port-progress bot said:

mathlib port progress category_theory.limits.yoneda
Ported files: 82/92 (89.1% of total)
Ported lines: 28322/32131 (88.1% of total)
Longest unported chain: 2/36 (94.4% progress)

Can I suggest category_theory.adjunction.adjoint_functor_theorems next?

Adam Topaz (Mar 02 2023 at 04:01):

I think there are better reasons to make this the next category theory target:
https://leanprover-community.github.io/mathlib-port-status/file/category_theory/sites/dense_subsite

Matthew Ballard (Mar 02 2023 at 04:01):

Do you need it for the workshop?

Adam Topaz (Mar 02 2023 at 04:02):

Or this (or both :)):
https://leanprover-community.github.io/mathlib-port-status/file/category_theory/abelian/transfer

Matthew Ballard (Mar 02 2023 at 04:03):

https://leanprover-community.github.io/mathlib-port-status/file/category_theory/derived/exceptional_collection/beilinson ?

Adam Topaz (Mar 02 2023 at 04:03):

Matthew Ballard said:

Do you need it for the workshop?

Yeah, it would be nice to have this for the Copenhagen thing.

Matthew Ballard (Mar 02 2023 at 04:04):

Good enough for me

Adam Topaz (Mar 02 2023 at 04:05):

Another potential natural target:
https://leanprover-community.github.io/mathlib-port-status/file/category_theory/abelian/ext

Adam Topaz (Mar 02 2023 at 04:05):

https://leanprover-community.github.io/mathlib-port-status/file/category_theory/monoidal/tor

port-progress bot (Mar 02 2023 at 18:05):

mathlib port progress topology.metric_space.basic
Ported files: 459/471 (97.5% of total)
Ported lines: 196395/204312 (96.1% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Mar 02 2023 at 18:09):

mathlib port progress data.polynomial.basic
Ported files: 387/398 (97.2% of total)
Ported lines: 155184/161315 (96.2% of total)
Longest unported chain: 1/58 (98.3% progress)

port-progress bot (Mar 02 2023 at 18:13):

mathlib port progress category_theory.limits.yoneda
Ported files: 84/92 (91.3% of total)
Ported lines: 28859/32131 (89.8% of total)
Longest unported chain: 1/36 (97.2% progress)

port-progress bot (Mar 02 2023 at 18:18):

mathlib port progress data.complex.basic
Ported files: 529/551 (96.0% of total)
Ported lines: 221836/233014 (95.2% of total)
Longest unported chain: 6/77 (92.2% progress)

port-progress bot (Mar 02 2023 at 18:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 698/1033 (67.6% of total)
Ported lines: 277720/438584 (63.3% of total)
Longest unported chain: 39/99 (60.6% progress)

port-progress bot (Mar 02 2023 at 18:28):

mathlib port progress combinatorics.additive.behrend
Ported files: 692/969 (71.4% of total)
Ported lines: 277404/427061 (65.0% of total)
Longest unported chain: 33/102 (67.6% progress)

port-progress bot (Mar 02 2023 at 18:36):

mathlib port progress all
Ported files: 1125/2882 (39.0% of total)
Ported lines: 370858/1002582 (37.0% of total)
Longest unported chain: 57/126 (54.8% progress)

Johan Commelin (Mar 02 2023 at 18:50):

0.5%

Adam Topaz (Mar 03 2023 at 17:48):

Adam Topaz said:

Can we get Kan extensions ported before quadratic reciprocity? :race: :racecar:

!4#2601

Adam Topaz (Mar 03 2023 at 17:53):

Once the port is over (or over enough...) I'm going to try to clean up this Kan extension file. It was already a complete mess in mathlib3

Matthew Ballard (Mar 03 2023 at 17:58):

Khan!!!

port-progress bot (Mar 03 2023 at 18:04):

mathlib port progress topology.metric_space.basic
Ported files: 460/471 (97.7% of total)
Ported lines: 197504/204334 (96.7% of total)
Longest unported chain: 1/69 (98.6% progress)

Yury G. Kudryashov (Mar 03 2023 at 18:06):

This one is done :up:

port-progress bot (Mar 03 2023 at 18:08):

mathlib port progress data.polynomial.basic
Ported files: 387/398 (97.2% of total)
Ported lines: 155186/161317 (96.2% of total)
Longest unported chain: 1/58 (98.3% progress)

port-progress bot (Mar 03 2023 at 18:11):

mathlib port progress category_theory.limits.yoneda
Ported files: 85/92 (92.4% of total)
Ported lines: 29019/32137 (90.3% of total)
Longest unported chain: 1/36 (97.2% progress)

port-progress bot (Mar 03 2023 at 18:16):

mathlib port progress data.complex.basic
Ported files: 531/551 (96.4% of total)
Ported lines: 225968/232964 (97.0% of total)
Longest unported chain: 6/77 (92.2% progress)

port-progress bot (Mar 03 2023 at 18:20):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 702/1033 (68.0% of total)
Ported lines: 282581/438567 (64.4% of total)
Longest unported chain: 39/99 (60.6% progress)

port-progress bot (Mar 03 2023 at 18:25):

mathlib port progress combinatorics.additive.behrend
Ported files: 696/969 (71.8% of total)
Ported lines: 282265/427031 (66.1% of total)
Longest unported chain: 33/102 (67.6% progress)

port-progress bot (Mar 03 2023 at 18:32):

mathlib port progress all
Ported files: 1135/2882 (39.4% of total)
Ported lines: 378212/1002607 (37.7% of total)
Longest unported chain: 57/126 (54.8% progress)

Johan Commelin (Mar 03 2023 at 21:36):

0.7%

port-progress bot (Mar 04 2023 at 06:47):

mathlib port progress data.polynomial.basic
Ported files: 387/398 (97.2% of total)
Ported lines: 155187/161318 (96.2% of total)
Longest unported chain: 1/58 (98.3% progress)

port-progress bot (Mar 04 2023 at 06:51):

mathlib port progress data.complex.basic
Ported files: 531/551 (96.4% of total)
Ported lines: 225969/232965 (97.0% of total)
Longest unported chain: 6/77 (92.2% progress)

port-progress bot (Mar 04 2023 at 06:55):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 703/1035 (67.9% of total)
Ported lines: 282971/439428 (64.4% of total)
Longest unported chain: 39/99 (60.6% progress)

port-progress bot (Mar 04 2023 at 06:59):

mathlib port progress combinatorics.additive.behrend
Ported files: 697/969 (71.9% of total)
Ported lines: 282655/427032 (66.2% of total)
Longest unported chain: 33/102 (67.6% progress)

port-progress bot (Mar 04 2023 at 07:03):

mathlib port progress analysis.calculus.fderiv
Ported files: 624/717 (87.0% of total)
Ported lines: 260873/312910 (83.4% of total)
Longest unported chain: 19/89 (78.7% progress)

port-progress bot (Mar 04 2023 at 07:07):

mathlib port progress measure_theory.integral.bochner
Ported files: 707/1010 (70.0% of total)
Ported lines: 287562/460106 (62.5% of total)
Longest unported chain: 37/106 (65.1% progress)

port-progress bot (Mar 04 2023 at 07:11):

mathlib port progress data.complex.exponential
Ported files: 534/555 (96.2% of total)
Ported lines: 226985/235652 (96.3% of total)
Longest unported chain: 7/78 (91.0% progress)

port-progress bot (Mar 04 2023 at 07:15):

mathlib port progress linear_algebra.determinant
Ported files: 543/642 (84.6% of total)
Ported lines: 211575/263170 (80.4% of total)
Longest unported chain: 17/77 (77.9% progress)

port-progress bot (Mar 04 2023 at 07:19):

mathlib port progress ring_theory.polynomial.basic
Ported files: 507/564 (89.9% of total)
Ported lines: 197212/229823 (85.8% of total)
Longest unported chain: 11/70 (84.3% progress)

port-progress bot (Mar 04 2023 at 07:22):

mathlib port progress linear_algebra.basis
Ported files: 433/442 (98.0% of total)
Ported lines: 174312/177995 (97.9% of total)
Longest unported chain: 1/59 (98.3% progress)

port-progress bot (Mar 04 2023 at 07:26):

mathlib port progress topology.continuous_function.bounded
Ported files: 629/720 (87.4% of total)
Ported lines: 262138/310000 (84.6% of total)
Longest unported chain: 17/87 (80.5% progress)

port-progress bot (Mar 04 2023 at 07:30):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 677/894 (75.7% of total)
Ported lines: 279652/391595 (71.4% of total)
Longest unported chain: 25/93 (73.1% progress)

port-progress bot (Mar 04 2023 at 07:34):

mathlib port progress probability.independence
Ported files: 710/1025 (69.3% of total)
Ported lines: 287935/467811 (61.5% of total)
Longest unported chain: 42/111 (62.2% progress)

port-progress bot (Mar 04 2023 at 07:38):

mathlib port progress category_theory.abelian.basic
Ported files: 331/371 (89.2% of total)
Ported lines: 124064/142539 (87.0% of total)
Longest unported chain: 9/48 (81.2% progress)

port-progress bot (Mar 04 2023 at 07:42):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 334/398 (83.9% of total)
Ported lines: 125923/150311 (83.8% of total)
Longest unported chain: 15/54 (72.2% progress)

port-progress bot (Mar 04 2023 at 07:46):

mathlib port progress category_theory.monoidal.tor
Ported files: 593/751 (79.0% of total)
Ported lines: 221059/287962 (76.8% of total)
Longest unported chain: 23/82 (72.0% progress)

port-progress bot (Mar 04 2023 at 07:52):

mathlib port progress all
Ported files: 1137/2882 (39.5% of total)
Ported lines: 378830/1002698 (37.8% of total)
Longest unported chain: 57/126 (54.8% progress)

port-progress bot (Mar 04 2023 at 18:03):

mathlib port progress data.polynomial.basic
Ported files: 387/398 (97.2% of total)
Ported lines: 155187/161318 (96.2% of total)
Longest unported chain: 1/58 (98.3% progress)

port-progress bot (Mar 04 2023 at 18:07):

mathlib port progress data.complex.basic
Ported files: 534/551 (96.9% of total)
Ported lines: 226613/232965 (97.3% of total)
Longest unported chain: 5/77 (93.5% progress)

port-progress bot (Mar 04 2023 at 18:11):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 709/1035 (68.5% of total)
Ported lines: 285018/439428 (64.9% of total)
Longest unported chain: 38/99 (61.6% progress)

port-progress bot (Mar 04 2023 at 18:16):

mathlib port progress combinatorics.additive.behrend
Ported files: 703/969 (72.5% of total)
Ported lines: 284702/427032 (66.7% of total)
Longest unported chain: 32/102 (68.6% progress)

port-progress bot (Mar 04 2023 at 18:19):

mathlib port progress analysis.calculus.fderiv
Ported files: 629/717 (87.7% of total)
Ported lines: 262222/312910 (83.8% of total)
Longest unported chain: 18/89 (79.8% progress)

port-progress bot (Mar 04 2023 at 18:24):

mathlib port progress measure_theory.integral.bochner
Ported files: 713/1010 (70.6% of total)
Ported lines: 289609/460106 (62.9% of total)
Longest unported chain: 36/106 (66.0% progress)

port-progress bot (Mar 04 2023 at 18:27):

mathlib port progress data.complex.exponential
Ported files: 537/555 (96.8% of total)
Ported lines: 227629/235652 (96.6% of total)
Longest unported chain: 6/78 (92.3% progress)

port-progress bot (Mar 04 2023 at 18:31):

mathlib port progress linear_algebra.determinant
Ported files: 544/642 (84.7% of total)
Ported lines: 212211/263170 (80.6% of total)
Longest unported chain: 16/77 (79.2% progress)

port-progress bot (Mar 04 2023 at 18:35):

mathlib port progress ring_theory.polynomial.basic
Ported files: 508/564 (90.1% of total)
Ported lines: 197848/229823 (86.1% of total)
Longest unported chain: 11/70 (84.3% progress)

port-progress bot (Mar 04 2023 at 18:38):

mathlib port progress linear_algebra.basis
Ported files: 433/442 (98.0% of total)
Ported lines: 174312/177995 (97.9% of total)
Longest unported chain: 1/59 (98.3% progress)

Reid Barton (Mar 04 2023 at 18:39):

Is a .basis file any easier than a .basic file?

port-progress bot (Mar 04 2023 at 18:42):

mathlib port progress topology.continuous_function.bounded
Ported files: 635/720 (88.2% of total)
Ported lines: 264185/310000 (85.2% of total)
Longest unported chain: 16/87 (81.6% progress)

port-progress bot (Mar 04 2023 at 18:45):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 683/894 (76.4% of total)
Ported lines: 281699/391595 (71.9% of total)
Longest unported chain: 24/93 (74.2% progress)

port-progress bot (Mar 04 2023 at 18:49):

mathlib port progress probability.independence
Ported files: 716/1025 (69.9% of total)
Ported lines: 289982/467811 (62.0% of total)
Longest unported chain: 41/111 (63.1% progress)

port-progress bot (Mar 04 2023 at 18:53):

mathlib port progress category_theory.abelian.basic
Ported files: 332/371 (89.5% of total)
Ported lines: 125186/142539 (87.8% of total)
Longest unported chain: 8/48 (83.3% progress)

port-progress bot (Mar 04 2023 at 18:57):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 336/398 (84.4% of total)
Ported lines: 127096/150311 (84.6% of total)
Longest unported chain: 15/54 (72.2% progress)

port-progress bot (Mar 04 2023 at 19:00):

mathlib port progress category_theory.monoidal.tor
Ported files: 596/751 (79.4% of total)
Ported lines: 222868/287962 (77.4% of total)
Longest unported chain: 23/82 (72.0% progress)

Kevin Buzzard (Mar 04 2023 at 19:05):

Reid Barton said:

Is a .basis file any easier than a .basic file?

Heh, probably not right now at least, because it involves linear algebra.

port-progress bot (Mar 04 2023 at 19:07):

mathlib port progress all
Ported files: 1150/2882 (39.9% of total)
Ported lines: 383107/1002698 (38.2% of total)
Longest unported chain: 56/126 (55.6% progress)

Johan Commelin (Mar 04 2023 at 19:48):

0.5%

port-progress bot (Mar 06 2023 at 18:04):

mathlib port progress data.polynomial.basic
Ported files: 387/398 (97.2% of total)
Ported lines: 155187/161318 (96.2% of total)
Longest unported chain: 1/58 (98.3% progress)

port-progress bot (Mar 06 2023 at 18:07):

mathlib port progress data.complex.basic
Ported files: 538/551 (97.6% of total)
Ported lines: 227759/232967 (97.8% of total)
Longest unported chain: 2/77 (97.4% progress)

port-progress bot (Mar 06 2023 at 18:12):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 718/1035 (69.4% of total)
Ported lines: 287490/439430 (65.4% of total)
Longest unported chain: 38/99 (61.6% progress)

port-progress bot (Mar 06 2023 at 18:16):

mathlib port progress combinatorics.additive.behrend
Ported files: 711/969 (73.4% of total)
Ported lines: 286955/427034 (67.2% of total)
Longest unported chain: 32/102 (68.6% progress)

port-progress bot (Mar 06 2023 at 18:19):

mathlib port progress analysis.calculus.fderiv
Ported files: 635/717 (88.6% of total)
Ported lines: 264105/312912 (84.4% of total)
Longest unported chain: 18/89 (79.8% progress)

port-progress bot (Mar 06 2023 at 18:23):

mathlib port progress measure_theory.integral.bochner
Ported files: 722/1010 (71.5% of total)
Ported lines: 291989/460182 (63.5% of total)
Longest unported chain: 36/106 (66.0% progress)

port-progress bot (Mar 06 2023 at 18:27):

mathlib port progress data.complex.exponential
Ported files: 541/555 (97.5% of total)
Ported lines: 228775/235654 (97.1% of total)
Longest unported chain: 3/78 (96.2% progress)

port-progress bot (Mar 06 2023 at 18:31):

mathlib port progress linear_algebra.determinant
Ported files: 545/642 (84.9% of total)
Ported lines: 212336/263170 (80.7% of total)
Longest unported chain: 16/77 (79.2% progress)

port-progress bot (Mar 06 2023 at 18:35):

mathlib port progress ring_theory.polynomial.basic
Ported files: 508/564 (90.1% of total)
Ported lines: 197848/229823 (86.1% of total)
Longest unported chain: 11/70 (84.3% progress)

port-progress bot (Mar 06 2023 at 18:38):

mathlib port progress linear_algebra.basis
Ported files: 433/442 (98.0% of total)
Ported lines: 174312/177995 (97.9% of total)
Longest unported chain: 1/59 (98.3% progress)

port-progress bot (Mar 06 2023 at 18:42):

mathlib port progress topology.continuous_function.bounded
Ported files: 643/720 (89.3% of total)
Ported lines: 266320/310002 (85.9% of total)
Longest unported chain: 16/87 (81.6% progress)

port-progress bot (Mar 06 2023 at 18:45):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 691/894 (77.3% of total)
Ported lines: 283952/391597 (72.5% of total)
Longest unported chain: 24/93 (74.2% progress)

port-progress bot (Mar 06 2023 at 18:49):

mathlib port progress probability.independence
Ported files: 725/1025 (70.7% of total)
Ported lines: 292362/467887 (62.5% of total)
Longest unported chain: 41/111 (63.1% progress)

port-progress bot (Mar 06 2023 at 18:53):

mathlib port progress category_theory.abelian.basic
Ported files: 335/371 (90.3% of total)
Ported lines: 125664/142539 (88.2% of total)
Longest unported chain: 8/48 (83.3% progress)

port-progress bot (Mar 06 2023 at 18:57):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 340/398 (85.4% of total)
Ported lines: 128179/150311 (85.3% of total)
Longest unported chain: 14/54 (74.1% progress)

port-progress bot (Mar 06 2023 at 19:00):

mathlib port progress category_theory.monoidal.tor
Ported files: 600/751 (79.9% of total)
Ported lines: 223951/287962 (77.8% of total)
Longest unported chain: 23/82 (72.0% progress)

port-progress bot (Mar 06 2023 at 19:06):

mathlib port progress all
Ported files: 1166/2882 (40.5% of total)
Ported lines: 386990/1002774 (38.6% of total)
Longest unported chain: 56/126 (55.6% progress)

Johan Commelin (Mar 06 2023 at 19:16):

0.4%

Moritz Doll (Mar 07 2023 at 10:51):

fyi: RingTheory.Ideal.Operations seems to be portable, but not started yet, if anyone looks for a file to port.

port-progress bot (Mar 07 2023 at 18:03):

mathlib port progress data.polynomial.basic
Ported files: 387/398 (97.2% of total)
Ported lines: 155187/161318 (96.2% of total)
Longest unported chain: 1/58 (98.3% progress)

port-progress bot (Mar 07 2023 at 18:07):

mathlib port progress data.complex.basic
Ported files: 539/551 (97.8% of total)
Ported lines: 227996/232967 (97.9% of total)
Longest unported chain: 1/77 (98.7% progress)

port-progress bot (Mar 07 2023 at 18:11):

mathlib port progress data.complex.exponential
Ported files: 542/555 (97.7% of total)
Ported lines: 229012/235654 (97.2% of total)
Longest unported chain: 2/78 (97.4% progress)

port-progress bot (Mar 07 2023 at 18:15):

mathlib port progress category_theory.abelian.basic
Ported files: 345/371 (93.0% of total)
Ported lines: 130063/142539 (91.2% of total)
Longest unported chain: 7/48 (85.4% progress)

port-progress bot (Mar 07 2023 at 18:19):

mathlib port progress ring_theory.polynomial.basic
Ported files: 508/564 (90.1% of total)
Ported lines: 197848/229823 (86.1% of total)
Longest unported chain: 11/70 (84.3% progress)

port-progress bot (Mar 07 2023 at 18:22):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 353/398 (88.7% of total)
Ported lines: 134241/150311 (89.3% of total)
Longest unported chain: 13/54 (75.9% progress)

port-progress bot (Mar 07 2023 at 18:26):

mathlib port progress topology.continuous_function.bounded
Ported files: 635/703 (90.3% of total)
Ported lines: 264131/305116 (86.6% of total)
Longest unported chain: 13/87 (85.1% progress)

port-progress bot (Mar 07 2023 at 18:30):

mathlib port progress linear_algebra.determinant
Ported files: 545/642 (84.9% of total)
Ported lines: 212336/263170 (80.7% of total)
Longest unported chain: 16/77 (79.2% progress)

port-progress bot (Mar 07 2023 at 18:34):

mathlib port progress analysis.calculus.fderiv
Ported files: 629/703 (89.5% of total)
Ported lines: 262221/308774 (84.9% of total)
Longest unported chain: 15/89 (83.1% progress)

port-progress bot (Mar 07 2023 at 18:37):

mathlib port progress category_theory.monoidal.tor
Ported files: 615/751 (81.9% of total)
Ported lines: 229993/287962 (79.9% of total)
Longest unported chain: 23/82 (72.0% progress)

port-progress bot (Mar 07 2023 at 18:41):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 695/895 (77.7% of total)
Ported lines: 284698/391617 (72.7% of total)
Longest unported chain: 24/93 (74.2% progress)

port-progress bot (Mar 07 2023 at 18:45):

mathlib port progress combinatorics.additive.behrend
Ported files: 715/970 (73.7% of total)
Ported lines: 287701/427055 (67.4% of total)
Longest unported chain: 32/102 (68.6% progress)

port-progress bot (Mar 07 2023 at 18:49):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 722/1036 (69.7% of total)
Ported lines: 288236/439450 (65.6% of total)
Longest unported chain: 38/99 (61.6% progress)

port-progress bot (Mar 07 2023 at 18:54):

mathlib port progress measure_theory.integral.bochner
Ported files: 726/1011 (71.8% of total)
Ported lines: 292735/460203 (63.6% of total)
Longest unported chain: 36/106 (66.0% progress)

port-progress bot (Mar 07 2023 at 18:57):

mathlib port progress probability.independence
Ported files: 729/1026 (71.1% of total)
Ported lines: 293108/467908 (62.6% of total)
Longest unported chain: 41/111 (63.1% progress)

port-progress bot (Mar 07 2023 at 19:04):

mathlib port progress all
Ported files: 1191/2883 (41.3% of total)
Ported lines: 395178/1002796 (39.4% of total)
Longest unported chain: 56/126 (55.6% progress)

Johan Commelin (Mar 07 2023 at 19:05):

0.8%

Eric Wieser (Mar 07 2023 at 20:32):

Moritz Doll said:

fyi: RingTheory.Ideal.Operations seems to be portable, but not started yet, if anyone looks for a file to port.

port-status#ring_theory/ideal/operations

Yury G. Kudryashov (Mar 07 2023 at 22:41):

It would be nice if one of the meta programming people reviews !4#2419, then the path to normed groups will be clear.

Yury G. Kudryashov (Mar 07 2023 at 23:29):

(Should we add a taggable group @metahumans?)

Johan Commelin (Mar 08 2023 at 07:04):

Kudos to @Pol'tta / Kô Miyahara for porting algebra.monoid_algebra.basic. We can probably tick data.polynomial.basic off the list in the next 24 hrs.

Johan Commelin (Mar 08 2023 at 07:07):

Ooh! And the longest unported chain no longer leads to gelfand_duality... The new winner is analysis.normed_space.star.continuous_functional_calculus which imports gelfand_duality :rofl:

Moritz Doll (Mar 08 2023 at 12:33):

Jireh is using all the maths

port-progress bot (Mar 08 2023 at 18:03):

mathlib port progress data.polynomial.basic
Ported files: 389/398 (97.7% of total)
Ported lines: 157635/161318 (97.7% of total)
Longest unported chain: 1/58 (98.3% progress)

Johan Commelin (Mar 08 2023 at 18:03):

@Scott Morrison this one is done

port-progress bot (Mar 08 2023 at 18:07):

mathlib port progress data.complex.basic
Ported files: 540/551 (98.0% of total)
Ported lines: 228400/233003 (98.0% of total)
Longest unported chain: 1/77 (98.7% progress)

port-progress bot (Mar 08 2023 at 18:10):

mathlib port progress data.complex.exponential
Ported files: 543/555 (97.8% of total)
Ported lines: 229416/235690 (97.3% of total)
Longest unported chain: 1/78 (98.7% progress)

port-progress bot (Mar 08 2023 at 18:14):

mathlib port progress category_theory.abelian.basic
Ported files: 351/371 (94.6% of total)
Ported lines: 132901/142599 (93.2% of total)
Longest unported chain: 3/48 (93.8% progress)

port-progress bot (Mar 08 2023 at 18:18):

mathlib port progress ring_theory.polynomial.basic
Ported files: 518/564 (91.8% of total)
Ported lines: 203957/229829 (88.7% of total)
Longest unported chain: 9/70 (87.1% progress)

port-progress bot (Mar 08 2023 at 18:22):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 359/397 (90.4% of total)
Ported lines: 136456/150089 (90.9% of total)
Longest unported chain: 12/53 (77.4% progress)

port-progress bot (Mar 08 2023 at 18:26):

mathlib port progress topology.continuous_function.bounded
Ported files: 644/703 (91.6% of total)
Ported lines: 267392/305215 (87.6% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 08 2023 at 18:30):

mathlib port progress linear_algebra.determinant
Ported files: 555/642 (86.4% of total)
Ported lines: 218474/263205 (83.0% of total)
Longest unported chain: 16/77 (79.2% progress)

port-progress bot (Mar 08 2023 at 18:34):

mathlib port progress analysis.calculus.fderiv
Ported files: 638/703 (90.8% of total)
Ported lines: 265450/308841 (86.0% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 08 2023 at 18:38):

mathlib port progress category_theory.monoidal.tor
Ported files: 617/710 (86.9% of total)
Ported lines: 235188/275298 (85.4% of total)
Longest unported chain: 18/79 (77.2% progress)

port-progress bot (Mar 08 2023 at 18:42):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 714/895 (79.8% of total)
Ported lines: 294065/391719 (75.1% of total)
Longest unported chain: 24/92 (73.9% progress)

port-progress bot (Mar 08 2023 at 18:46):

mathlib port progress combinatorics.additive.behrend
Ported files: 735/970 (75.8% of total)
Ported lines: 297401/427157 (69.6% of total)
Longest unported chain: 32/101 (68.3% progress)

port-progress bot (Mar 08 2023 at 18:50):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 742/1036 (71.6% of total)
Ported lines: 297939/439555 (67.8% of total)
Longest unported chain: 38/99 (61.6% progress)

port-progress bot (Mar 08 2023 at 18:54):

mathlib port progress measure_theory.integral.bochner
Ported files: 746/1011 (73.8% of total)
Ported lines: 302438/460308 (65.7% of total)
Longest unported chain: 36/105 (65.7% progress)

port-progress bot (Mar 08 2023 at 18:58):

mathlib port progress probability.independence
Ported files: 749/1026 (73.0% of total)
Ported lines: 302811/468013 (64.7% of total)
Longest unported chain: 41/110 (62.7% progress)

port-progress bot (Mar 08 2023 at 19:04):

mathlib port progress all
Ported files: 1221/2887 (42.3% of total)
Ported lines: 409403/1003692 (40.8% of total)
Longest unported chain: 56/125 (55.2% progress)

Johan Commelin (Mar 08 2023 at 19:07):

1.4%

Kevin Buzzard (Mar 08 2023 at 20:16):

Many thanks to all the hard-working porters! It's great to see the rss feed racing along.

Johan Commelin (Mar 08 2023 at 20:32):

30 files were ported in the past 24hrs!

Jeremy Tan (Mar 09 2023 at 17:04):

https://github.com/leanprover-community/mathlib4/pull/2743 Just watching for the moment, but this specific PR I feel will enable a lot of other files to be ported, right?

Eric Wieser (Mar 09 2023 at 17:18):

I skimmed over it and added some comments

port-progress bot (Mar 09 2023 at 18:04):

mathlib port progress data.complex.basic
Ported files: 540/551 (98.0% of total)
Ported lines: 228400/233003 (98.0% of total)
Longest unported chain: 1/77 (98.7% progress)

port-progress bot (Mar 09 2023 at 18:08):

mathlib port progress data.complex.exponential
Ported files: 543/555 (97.8% of total)
Ported lines: 229416/235690 (97.3% of total)
Longest unported chain: 1/78 (98.7% progress)

port-progress bot (Mar 09 2023 at 18:12):

mathlib port progress category_theory.abelian.basic
Ported files: 359/371 (96.8% of total)
Ported lines: 136667/142599 (95.8% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 09 2023 at 18:16):

mathlib port progress ring_theory.polynomial.basic
Ported files: 527/564 (93.4% of total)
Ported lines: 209882/229829 (91.3% of total)
Longest unported chain: 8/70 (88.6% progress)

port-progress bot (Mar 09 2023 at 18:20):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 362/397 (91.2% of total)
Ported lines: 136950/150089 (91.2% of total)
Longest unported chain: 12/53 (77.4% progress)

port-progress bot (Mar 09 2023 at 18:24):

mathlib port progress topology.continuous_function.bounded
Ported files: 647/703 (92.0% of total)
Ported lines: 271769/305215 (89.0% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 09 2023 at 18:28):

mathlib port progress linear_algebra.determinant
Ported files: 564/642 (87.9% of total)
Ported lines: 224399/263209 (85.3% of total)
Longest unported chain: 15/77 (80.5% progress)

port-progress bot (Mar 09 2023 at 18:32):

mathlib port progress analysis.calculus.fderiv
Ported files: 642/703 (91.3% of total)
Ported lines: 270270/308841 (87.5% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 09 2023 at 18:36):

mathlib port progress category_theory.monoidal.tor
Ported files: 630/710 (88.7% of total)
Ported lines: 242058/275298 (87.9% of total)
Longest unported chain: 17/79 (78.5% progress)

port-progress bot (Mar 09 2023 at 18:40):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 725/895 (81.0% of total)
Ported lines: 302445/391723 (77.2% of total)
Longest unported chain: 23/92 (75.0% progress)

port-progress bot (Mar 09 2023 at 18:44):

mathlib port progress combinatorics.additive.behrend
Ported files: 746/970 (76.9% of total)
Ported lines: 305569/427161 (71.5% of total)
Longest unported chain: 31/101 (69.3% progress)

port-progress bot (Mar 09 2023 at 18:49):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 752/1036 (72.6% of total)
Ported lines: 305986/439559 (69.6% of total)
Longest unported chain: 37/99 (62.6% progress)

port-progress bot (Mar 09 2023 at 18:53):

mathlib port progress measure_theory.integral.bochner
Ported files: 758/1011 (75.0% of total)
Ported lines: 310787/460312 (67.5% of total)
Longest unported chain: 35/105 (66.7% progress)

port-progress bot (Mar 09 2023 at 18:57):

mathlib port progress probability.independence
Ported files: 763/1026 (74.4% of total)
Ported lines: 311400/468017 (66.5% of total)
Longest unported chain: 40/110 (63.6% progress)

port-progress bot (Mar 09 2023 at 19:03):

mathlib port progress all
Ported files: 1249/2887 (43.3% of total)
Ported lines: 420469/1003709 (41.9% of total)
Longest unported chain: 55/125 (56.0% progress)

Chris Hughes (Mar 09 2023 at 20:25):

1.1%

Kevin Buzzard (Mar 09 2023 at 21:39):

So over the last two days 1/40th of mathlib was ported :-)

Adam Topaz (Mar 09 2023 at 23:34):

So we'll be done in < 3 months?

Jireh Loreaux (Mar 09 2023 at 23:44):

well, at that breakneck pace we'd be done in 47 days. We ported 1/40th of the total in the past two days, not 1/40th of what's remaining. But I think that's a bit optimistic. Mid-June definitely seems feasible though.

Adam Topaz (Mar 09 2023 at 23:45):

I'm being a bit conservative with our speed in my estimate :)

Jeremy Tan (Mar 09 2023 at 23:57):

Adam Topaz said:

I'm being a bit conservative with our speed in my estimate :)

Well the port's not gonna be complete until we fix the data.matrix.basic blocker

Adam Topaz (Mar 10 2023 at 00:00):

what's the issue with data.matrix.basic?

Jeremy Tan (Mar 10 2023 at 00:05):

Adam Topaz said:

what's the issue with data.matrix.basic?

"Likely to be annoying without leanprover/lean4#2042". And nobody has bothered about this HUGE problem for two months despite it being high prio

Adam Topaz (Mar 10 2023 at 00:05):

is this really a huge problem?

Jeremy Tan (Mar 10 2023 at 00:06):

(at this moment I can't help with that either; I just picked up the language two days ago)

Jeremy Tan (Mar 10 2023 at 00:06):

It is a huge problem because it has many dependents

Jeremy Tan (Mar 10 2023 at 00:07):

In particular, suppose we managed to port enough of it to formalise the determinant. Then the Cassini's identity proof could be drastically simplified

Jeremy Tan (Mar 10 2023 at 00:07):

(that I sussed out in the new members stream)

Adam Topaz (Mar 10 2023 at 00:08):

I think tagging defs with simp is bad practice anyway (unless you want them to be unfolded by (d)simp). And I would have expected a def tagged with simp to indeed just unfold the definition regardless of whether it's a function or not (and whether it's applied or not)

Jeremy Tan (Mar 10 2023 at 00:10):

Wait, the mathlib3 data.matrix.basic does tagging defs with simp a lot?

Adam Topaz (Mar 10 2023 at 00:10):

no, but I suppose it does things like simp [transpose] (just guessing based on the comments in the lean4 issue)

Adam Topaz (Mar 10 2023 at 00:14):

IMO the current lean4 behavior is what I would expect to happen, while the lean3 behavior seems unexpected to me.

Adam Topaz (Mar 10 2023 at 00:27):

For example, I find it strange that in lean3 simp closes the second example but not the first:

@[simp]
def bar (x : ) :  := 2 * x

example : bar = λ x, 2 * x := begin
  simp,
  sorry
end

@[simp]
def bar' :    := λ x, 2 * x

example : bar' = λ x, 2 * x := begin
  simp,
end

Kevin Buzzard (Mar 10 2023 at 00:30):

Jeremy Tan said:

Adam Topaz said:

what's the issue with data.matrix.basic?

"Likely to be annoying without leanprover/lean4#2042". And nobody has bothered about this HUGE problem for two months despite it being high prio

This is an open source project run by a small overworked group at Microsoft and a collection of unpaid volunteers from around the world.

Kevin Buzzard (Mar 10 2023 at 00:31):

People sometimes have to wait.

Jeremy Tan (Mar 10 2023 at 00:45):

Right then, I'd like to try my hand at porting some files to mathlib4. I request access to the mathlib4 repo; my GitHub username is Parcly-Taxel

Jeremy Tan (Mar 10 2023 at 00:45):

data.nat.choose.vandermonde is what I want to start with

Scott Morrison (Mar 10 2023 at 01:59):

@Jeremy Tan, I have sent invites for both the mathlib and mathlib4 repos.

Eric Wieser (Mar 10 2023 at 07:32):

Adam Topaz said:

I think tagging defs with simp is bad practice anyway (unless you want them to be unfolded by (d)simp). And I would have expected a def tagged with simp to indeed just unfold the definition regardless of whether it's a function or not (and whether it's applied or not)

I think if we agree on that stance we should make the change in lean 3 first

Johan Commelin (Mar 10 2023 at 07:34):

How often does it happen?

Johan Commelin (Mar 10 2023 at 07:37):

My guesstimate is 350 occurences in ml3.

Eric Wieser (Mar 10 2023 at 07:37):

Adam Topaz said:

IMO the current lean4 behavior is what I would expect to happen, while the lean3 behavior seems unexpected to me.

I don't really agree with that; what's actually changed here is that lean 4 generates worse equation lemmas; before pattern matching against 0 and succ n would generate an equation lemma for each; now it generates a single equation lemmas that unfolds to a match statement

Mario Carneiro (Mar 10 2023 at 07:48):

note that it does generate equation lemmas for each match branch, but these are lemmas for the match splitter function, not for the function wrapping it

Chris Hughes (Mar 10 2023 at 08:08):

But you don't want to unfold stuff unless it's applied to a constructor. I don't want to see any matches in my goal ever.

Adam Topaz (Mar 10 2023 at 14:33):

Chris Hughes said:

But you don't want to unfold stuff unless it's applied to a constructor. I don't want to see any matches in my goal ever.

I agree with this completely. But my point is not that I want more lambdas and matches in goals, but rather that if you write simp [someFunc] then it's your fault that lean unfolded someFunc and not lean's fault. If we leave the current behavior in lean4 as is, we would have to write more boilerplate simp lemmas, or perhaps upgrade simps to generate the proper simp lemmas that we want. But there are times where I do dsimp [thing1, thing2, someFunc] where I want lean to unfold someFunc and in lean3 it was annoying to have to use unfold on a second line as well in some cases.

port-progress bot (Mar 10 2023 at 18:03):

mathlib port progress data.complex.basic
Ported files: 541/551 (98.2% of total)
Ported lines: 229179/233003 (98.4% of total)
Longest unported chain: 1/77 (98.7% progress)

port-progress bot (Mar 10 2023 at 18:07):

mathlib port progress data.complex.exponential
Ported files: 544/555 (98.0% of total)
Ported lines: 230195/235690 (97.7% of total)
Longest unported chain: 1/78 (98.7% progress)

port-progress bot (Mar 10 2023 at 18:11):

mathlib port progress category_theory.abelian.basic
Ported files: 360/371 (97.0% of total)
Ported lines: 137710/142599 (96.6% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 10 2023 at 18:15):

mathlib port progress ring_theory.polynomial.basic
Ported files: 528/564 (93.6% of total)
Ported lines: 211011/229829 (91.8% of total)
Longest unported chain: 8/70 (88.6% progress)

port-progress bot (Mar 10 2023 at 18:19):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 364/397 (91.7% of total)
Ported lines: 137377/150089 (91.5% of total)
Longest unported chain: 11/53 (79.2% progress)

port-progress bot (Mar 10 2023 at 18:23):

mathlib port progress topology.continuous_function.bounded
Ported files: 651/703 (92.6% of total)
Ported lines: 275425/305215 (90.2% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 10 2023 at 18:27):

mathlib port progress linear_algebra.determinant
Ported files: 565/642 (88.0% of total)
Ported lines: 225528/263209 (85.7% of total)
Longest unported chain: 15/77 (80.5% progress)

port-progress bot (Mar 10 2023 at 18:31):

mathlib port progress analysis.calculus.fderiv
Ported files: 646/703 (91.9% of total)
Ported lines: 273239/308849 (88.5% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 10 2023 at 18:35):

mathlib port progress category_theory.monoidal.tor
Ported files: 634/710 (89.3% of total)
Ported lines: 244789/275298 (88.9% of total)
Longest unported chain: 17/79 (78.5% progress)

port-progress bot (Mar 10 2023 at 18:39):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 733/895 (81.9% of total)
Ported lines: 307179/391723 (78.4% of total)
Longest unported chain: 23/92 (75.0% progress)

port-progress bot (Mar 10 2023 at 18:43):

mathlib port progress combinatorics.additive.behrend
Ported files: 755/970 (77.8% of total)
Ported lines: 310356/427169 (72.7% of total)
Longest unported chain: 31/101 (69.3% progress)

port-progress bot (Mar 10 2023 at 18:48):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 760/1036 (73.4% of total)
Ported lines: 310720/439559 (70.7% of total)
Longest unported chain: 37/99 (62.6% progress)

port-progress bot (Mar 10 2023 at 18:52):

mathlib port progress measure_theory.integral.bochner
Ported files: 767/1011 (75.9% of total)
Ported lines: 315434/460320 (68.5% of total)
Longest unported chain: 35/105 (66.7% progress)

port-progress bot (Mar 10 2023 at 18:56):

mathlib port progress probability.independence
Ported files: 770/1026 (75.0% of total)
Ported lines: 315807/468025 (67.5% of total)
Longest unported chain: 40/110 (63.6% progress)

port-progress bot (Mar 10 2023 at 19:02):

mathlib port progress all
Ported files: 1264/2889 (43.8% of total)
Ported lines: 427619/1004772 (42.6% of total)
Longest unported chain: 55/125 (56.0% progress)

Johan Commelin (Mar 10 2023 at 19:24):

0.7%

port-progress bot (Mar 11 2023 at 18:03):

mathlib port progress data.complex.basic
Ported files: 541/551 (98.2% of total)
Ported lines: 229179/233003 (98.4% of total)
Longest unported chain: 1/77 (98.7% progress)

Jeremy Tan (Mar 11 2023 at 18:04):

^ there's nothing left for this, we should replace it with some other goal file

Adam Topaz (Mar 11 2023 at 18:05):

Oh man, we’re moving FAST!

port-progress bot (Mar 11 2023 at 18:08):

mathlib port progress data.complex.exponential
Ported files: 544/555 (98.0% of total)
Ported lines: 230195/235690 (97.7% of total)
Longest unported chain: 1/78 (98.7% progress)

port-progress bot (Mar 11 2023 at 18:12):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138162/142599 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 11 2023 at 18:16):

mathlib port progress ring_theory.polynomial.basic
Ported files: 526/560 (93.9% of total)
Ported lines: 210393/228266 (92.2% of total)
Longest unported chain: 7/70 (90.0% progress)

port-progress bot (Mar 11 2023 at 18:21):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 367/397 (92.4% of total)
Ported lines: 138166/150089 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 11 2023 at 18:25):

mathlib port progress topology.continuous_function.bounded
Ported files: 652/703 (92.7% of total)
Ported lines: 275555/305215 (90.3% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 11 2023 at 18:29):

mathlib port progress linear_algebra.determinant
Ported files: 566/641 (88.3% of total)
Ported lines: 225658/262398 (86.0% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 11 2023 at 18:34):

mathlib port progress analysis.calculus.fderiv
Ported files: 647/703 (92.0% of total)
Ported lines: 273369/308849 (88.5% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 11 2023 at 18:38):

mathlib port progress category_theory.monoidal.tor
Ported files: 636/711 (89.5% of total)
Ported lines: 245168/275225 (89.1% of total)
Longest unported chain: 17/80 (78.8% progress)

port-progress bot (Mar 11 2023 at 18:43):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 734/894 (82.1% of total)
Ported lines: 307309/390912 (78.6% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 11 2023 at 18:47):

mathlib port progress combinatorics.additive.behrend
Ported files: 756/970 (77.9% of total)
Ported lines: 310486/426871 (72.7% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 11 2023 at 18:52):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 761/1039 (73.2% of total)
Ported lines: 310850/439583 (70.7% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 11 2023 at 18:57):

mathlib port progress measure_theory.integral.bochner
Ported files: 768/1011 (76.0% of total)
Ported lines: 315564/460022 (68.6% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 11 2023 at 19:02):

mathlib port progress probability.independence
Ported files: 771/1026 (75.1% of total)
Ported lines: 315937/467727 (67.5% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 11 2023 at 19:08):

mathlib port progress all
Ported files: 1281/2893 (44.3% of total)
Ported lines: 431700/1004913 (43.0% of total)
Longest unported chain: 54/125 (56.8% progress)

Johan Commelin (Mar 11 2023 at 19:13):

0.4%

port-progress bot (Mar 12 2023 at 18:04):

mathlib port progress data.complex.basic
Ported files: 542/551 (98.4% of total)
Ported lines: 229330/233013 (98.4% of total)
Longest unported chain: 1/77 (98.7% progress)

port-progress bot (Mar 12 2023 at 18:10):

mathlib port progress data.complex.exponential
Ported files: 545/555 (98.2% of total)
Ported lines: 230346/235700 (97.7% of total)
Longest unported chain: 1/78 (98.7% progress)

port-progress bot (Mar 12 2023 at 18:15):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138162/142599 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 12 2023 at 18:20):

mathlib port progress ring_theory.polynomial.basic
Ported files: 528/560 (94.3% of total)
Ported lines: 210913/228276 (92.4% of total)
Longest unported chain: 7/70 (90.0% progress)

port-progress bot (Mar 12 2023 at 18:25):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 367/397 (92.4% of total)
Ported lines: 138166/150089 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 12 2023 at 18:29):

mathlib port progress topology.continuous_function.bounded
Ported files: 654/703 (93.0% of total)
Ported lines: 276075/305225 (90.4% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 12 2023 at 18:34):

mathlib port progress linear_algebra.determinant
Ported files: 568/641 (88.6% of total)
Ported lines: 226178/262408 (86.2% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 12 2023 at 18:39):

mathlib port progress analysis.calculus.fderiv
Ported files: 649/703 (92.3% of total)
Ported lines: 273889/308859 (88.7% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 12 2023 at 18:43):

mathlib port progress category_theory.monoidal.tor
Ported files: 638/711 (89.7% of total)
Ported lines: 245688/275235 (89.3% of total)
Longest unported chain: 17/80 (78.8% progress)

port-progress bot (Mar 12 2023 at 18:48):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 736/894 (82.3% of total)
Ported lines: 307829/390922 (78.7% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 12 2023 at 18:53):

mathlib port progress combinatorics.additive.behrend
Ported files: 758/970 (78.1% of total)
Ported lines: 311006/426881 (72.9% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 12 2023 at 18:58):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 763/1039 (73.4% of total)
Ported lines: 311370/439593 (70.8% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 12 2023 at 19:03):

mathlib port progress measure_theory.integral.bochner
Ported files: 770/1011 (76.2% of total)
Ported lines: 316084/460032 (68.7% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 12 2023 at 19:08):

mathlib port progress probability.independence
Ported files: 773/1026 (75.3% of total)
Ported lines: 316457/467737 (67.7% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 12 2023 at 19:15):

mathlib port progress all
Ported files: 1284/2893 (44.4% of total)
Ported lines: 432264/1004923 (43.0% of total)
Longest unported chain: 54/125 (56.8% progress)

Kevin Buzzard (Mar 12 2023 at 23:57):

We are a week or two away from the half way stage

Johan Commelin (Mar 13 2023 at 04:58):

0.0%

Kevin Buzzard (Mar 13 2023 at 07:37):

Lol (I blame the weekend)

port-progress bot (Mar 13 2023 at 18:04):

mathlib port progress data.complex.exponential
Ported files: 545/555 (98.2% of total)
Ported lines: 230346/235700 (97.7% of total)
Longest unported chain: 1/78 (98.7% progress)

port-progress bot (Mar 13 2023 at 18:08):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138198/142635 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 13 2023 at 18:12):

mathlib port progress ring_theory.polynomial.basic
Ported files: 530/560 (94.6% of total)
Ported lines: 211623/228336 (92.7% of total)
Longest unported chain: 7/70 (90.0% progress)

port-progress bot (Mar 13 2023 at 18:15):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 368/397 (92.7% of total)
Ported lines: 138315/150122 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 13 2023 at 18:20):

mathlib port progress topology.continuous_function.bounded
Ported files: 656/703 (93.3% of total)
Ported lines: 277633/305290 (90.9% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 13 2023 at 18:23):

mathlib port progress linear_algebra.determinant
Ported files: 570/641 (88.9% of total)
Ported lines: 226908/262488 (86.4% of total)
Longest unported chain: 14/77 (81.8% progress)

Eric Wieser (Mar 13 2023 at 18:24):

Would port-status#analysis/inner_product_space/pi_L2` be a good target? docs#euclidean_space is regularly a thing needed by beginners wanting to talk about the distance between points

port-progress bot (Mar 13 2023 at 18:27):

mathlib port progress analysis.calculus.fderiv
Ported files: 650/703 (92.5% of total)
Ported lines: 274803/308907 (89.0% of total)
Longest unported chain: 14/88 (84.1% progress)

Jeremy Tan (Mar 13 2023 at 18:28):

Eric Wieser said:

Would port-status#analysis/inner_product_space/pi_L2` be a good target? docs#euclidean_space is regularly a thing needed by beginners wanting to talk about the distance between points

I say yes

port-progress bot (Mar 13 2023 at 18:31):

mathlib port progress category_theory.monoidal.tor
Ported files: 640/711 (90.0% of total)
Ported lines: 246440/275337 (89.5% of total)
Longest unported chain: 17/80 (78.8% progress)

port-progress bot (Mar 13 2023 at 18:35):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 740/894 (82.8% of total)
Ported lines: 310106/391056 (79.3% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 13 2023 at 18:40):

mathlib port progress combinatorics.additive.behrend
Ported files: 763/970 (78.7% of total)
Ported lines: 313554/427021 (73.4% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 13 2023 at 18:44):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 771/1039 (74.2% of total)
Ported lines: 314270/439727 (71.5% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 13 2023 at 18:48):

mathlib port progress measure_theory.integral.bochner
Ported files: 775/1011 (76.7% of total)
Ported lines: 318635/460175 (69.2% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 13 2023 at 18:52):

mathlib port progress probability.independence
Ported files: 778/1026 (75.8% of total)
Ported lines: 319008/467880 (68.2% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 13 2023 at 18:58):

mathlib port progress all
Ported files: 1311/2893 (45.3% of total)
Ported lines: 438929/1005222 (43.7% of total)
Longest unported chain: 54/125 (56.8% progress)

Johan Commelin (Mar 13 2023 at 19:04):

0.7%

port-progress bot (Mar 14 2023 at 18:04):

mathlib port progress data.complex.exponential
Ported files: 545/555 (98.2% of total)
Ported lines: 230346/235700 (97.7% of total)
Longest unported chain: 1/78 (98.7% progress)

port-progress bot (Mar 14 2023 at 18:08):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138198/142635 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 14 2023 at 18:12):

mathlib port progress ring_theory.polynomial.basic
Ported files: 532/562 (94.7% of total)
Ported lines: 212789/229167 (92.9% of total)
Longest unported chain: 7/70 (90.0% progress)

port-progress bot (Mar 14 2023 at 18:16):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 368/397 (92.7% of total)
Ported lines: 138315/150122 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 14 2023 at 18:20):

mathlib port progress topology.continuous_function.bounded
Ported files: 657/703 (93.5% of total)
Ported lines: 277842/305303 (91.0% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 14 2023 at 18:25):

mathlib port progress linear_algebra.determinant
Ported files: 572/643 (89.0% of total)
Ported lines: 228074/263319 (86.6% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 14 2023 at 18:29):

mathlib port progress analysis.calculus.fderiv
Ported files: 650/703 (92.5% of total)
Ported lines: 274809/308920 (89.0% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 14 2023 at 18:33):

mathlib port progress category_theory.monoidal.tor
Ported files: 642/713 (90.0% of total)
Ported lines: 247606/276168 (89.7% of total)
Longest unported chain: 17/80 (78.8% progress)

port-progress bot (Mar 14 2023 at 18:37):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 743/896 (82.9% of total)
Ported lines: 311343/391900 (79.4% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 14 2023 at 18:42):

mathlib port progress combinatorics.additive.behrend
Ported files: 768/972 (79.0% of total)
Ported lines: 315070/427875 (73.6% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 14 2023 at 18:46):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 778/1041 (74.7% of total)
Ported lines: 316418/440571 (71.8% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 14 2023 at 18:51):

mathlib port progress measure_theory.integral.bochner
Ported files: 783/1013 (77.3% of total)
Ported lines: 321736/461019 (69.8% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 14 2023 at 18:55):

mathlib port progress probability.independence
Ported files: 786/1028 (76.5% of total)
Ported lines: 322109/468724 (68.7% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 14 2023 at 19:01):

mathlib port progress all
Ported files: 1331/2893 (46.0% of total)
Ported lines: 444221/1005307 (44.2% of total)
Longest unported chain: 54/125 (56.8% progress)

Johan Commelin (Mar 14 2023 at 19:01):

0.5%

port-progress bot (Mar 15 2023 at 18:04):

mathlib port progress data.complex.exponential
Ported files: 546/555 (98.4% of total)
Ported lines: 232034/235717 (98.4% of total)
Longest unported chain: 1/78 (98.7% progress)

port-progress bot (Mar 15 2023 at 18:08):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138209/142646 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 15 2023 at 18:12):

mathlib port progress ring_theory.polynomial.basic
Ported files: 535/562 (95.2% of total)
Ported lines: 214446/229190 (93.6% of total)
Longest unported chain: 7/70 (90.0% progress)

port-progress bot (Mar 15 2023 at 18:16):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 368/397 (92.7% of total)
Ported lines: 138329/150136 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 15 2023 at 18:21):

mathlib port progress topology.continuous_function.bounded
Ported files: 657/703 (93.5% of total)
Ported lines: 277865/305326 (91.0% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 15 2023 at 18:25):

mathlib port progress linear_algebra.determinant
Ported files: 575/643 (89.4% of total)
Ported lines: 229762/263373 (87.2% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 15 2023 at 18:29):

mathlib port progress analysis.calculus.fderiv
Ported files: 650/703 (92.5% of total)
Ported lines: 274829/308940 (89.0% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 15 2023 at 18:33):

mathlib port progress category_theory.monoidal.tor
Ported files: 645/713 (90.5% of total)
Ported lines: 249263/276191 (90.3% of total)
Longest unported chain: 17/80 (78.8% progress)

port-progress bot (Mar 15 2023 at 18:37):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 747/896 (83.4% of total)
Ported lines: 314708/391965 (80.3% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 15 2023 at 18:42):

mathlib port progress combinatorics.additive.behrend
Ported files: 772/972 (79.4% of total)
Ported lines: 318444/427949 (74.4% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 15 2023 at 18:47):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 785/1041 (75.4% of total)
Ported lines: 320114/440660 (72.6% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 15 2023 at 18:51):

mathlib port progress measure_theory.integral.bochner
Ported files: 787/1013 (77.7% of total)
Ported lines: 325119/461102 (70.5% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 15 2023 at 18:56):

mathlib port progress probability.independence
Ported files: 790/1028 (76.8% of total)
Ported lines: 325492/468807 (69.4% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 15 2023 at 19:02):

mathlib port progress all
Ported files: 1343/2894 (46.4% of total)
Ported lines: 449015/1005647 (44.6% of total)
Longest unported chain: 54/125 (56.8% progress)

Johan Commelin (Mar 15 2023 at 19:02):

0.4%

port-progress bot (Mar 16 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138202/142639 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 16 2023 at 18:08):

mathlib port progress ring_theory.polynomial.basic
Ported files: 535/561 (95.4% of total)
Ported lines: 214439/228833 (93.7% of total)
Longest unported chain: 7/70 (90.0% progress)

port-progress bot (Mar 16 2023 at 18:12):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 368/397 (92.7% of total)
Ported lines: 138322/150129 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 16 2023 at 18:16):

mathlib port progress topology.continuous_function.bounded
Ported files: 657/704 (93.3% of total)
Ported lines: 277833/305346 (91.0% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 16 2023 at 18:20):

mathlib port progress linear_algebra.determinant
Ported files: 575/642 (89.6% of total)
Ported lines: 229755/263016 (87.4% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 16 2023 at 18:24):

mathlib port progress analysis.calculus.fderiv
Ported files: 650/704 (92.3% of total)
Ported lines: 274797/308960 (88.9% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 16 2023 at 18:28):

mathlib port progress category_theory.monoidal.tor
Ported files: 645/712 (90.6% of total)
Ported lines: 249256/275833 (90.4% of total)
Longest unported chain: 17/80 (78.8% progress)

port-progress bot (Mar 16 2023 at 18:32):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 747/896 (83.4% of total)
Ported lines: 314676/391635 (80.3% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 16 2023 at 18:37):

mathlib port progress combinatorics.additive.behrend
Ported files: 772/972 (79.4% of total)
Ported lines: 318412/427619 (74.5% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 16 2023 at 18:41):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 785/1041 (75.4% of total)
Ported lines: 320082/440329 (72.7% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 16 2023 at 18:45):

mathlib port progress measure_theory.integral.bochner
Ported files: 787/1013 (77.7% of total)
Ported lines: 325087/460775 (70.6% of total)
Longest unported chain: 34/105 (67.6% progress)

Eric Wieser (Mar 16 2023 at 18:48):

Eric Wieser said:

Would port-status#analysis/inner_product_space/pi_L2` be a good target? docs#euclidean_space is regularly a thing needed by beginners wanting to talk about the distance between points

:ping_pong: @Scott Morrison

port-progress bot (Mar 16 2023 at 18:50):

mathlib port progress probability.independence
Ported files: 790/1028 (76.8% of total)
Ported lines: 325460/468480 (69.5% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 16 2023 at 18:56):

mathlib port progress all
Ported files: 1348/2899 (46.5% of total)
Ported lines: 449617/1005926 (44.7% of total)
Longest unported chain: 54/125 (56.8% progress)

Johan Commelin (Mar 16 2023 at 20:27):

0.1%

Chris Hughes (Mar 17 2023 at 12:12):

I checked the mathlib port status yesterday. It was on 45.0%. Today it's 44.9%. It makes me a bit sad that we went backwards, even if just for one day.

Scott Morrison (Mar 17 2023 at 12:41):

Next time it happens, we'll close down mathlib3 for PRs. :-)

Yaël Dillies (Mar 17 2023 at 12:42):

Well, you know, we're not going backwards. The #queue keeps going down.

Yaël Dillies (Mar 17 2023 at 12:43):

Understand, the lines that mathlib3 is gaining are not new code, but instead code that was already written but not merged.

Eric Wieser (Mar 17 2023 at 12:44):

Scott Morrison said:

Next time it happens, we'll close down mathlib3 for PRs. :-)

I don't think it would be totally unreasonable to say "if the progress goes down from A to B, pause mathlib3 reviews and focus on mathlib4 reviews until it exceeds A again"

Eric Wieser (Mar 17 2023 at 12:45):

Of course this can be gamified by just PRing lorem ipsum text to logic/basic in mathlib3, to artificially inflate the port progress

Jeremy Tan (Mar 17 2023 at 16:34):

image.png wow, I'll be surprised if this 10-PR staging build goes in on the first try

Chris Hughes (Mar 17 2023 at 17:29):

It happens all the time. I would not be surprised at all if it goes through.

Jeremy Tan (Mar 17 2023 at 17:36):

It went through

port-progress bot (Mar 17 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138208/142645 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 17 2023 at 18:08):

mathlib port progress ring_theory.polynomial.basic
Ported files: 536/561 (95.5% of total)
Ported lines: 215189/228850 (94.0% of total)
Longest unported chain: 7/70 (90.0% progress)

port-progress bot (Mar 17 2023 at 18:12):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 368/397 (92.7% of total)
Ported lines: 138328/150135 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 17 2023 at 18:16):

mathlib port progress topology.continuous_function.bounded
Ported files: 658/704 (93.5% of total)
Ported lines: 277904/305365 (91.0% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 17 2023 at 18:21):

mathlib port progress linear_algebra.determinant
Ported files: 579/642 (90.2% of total)
Ported lines: 232841/263038 (88.5% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 17 2023 at 18:25):

mathlib port progress analysis.calculus.fderiv
Ported files: 651/704 (92.5% of total)
Ported lines: 274863/308974 (89.0% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 17 2023 at 18:29):

mathlib port progress category_theory.monoidal.tor
Ported files: 648/712 (91.0% of total)
Ported lines: 250169/275850 (90.7% of total)
Longest unported chain: 17/80 (78.8% progress)

port-progress bot (Mar 17 2023 at 18:33):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 752/896 (83.9% of total)
Ported lines: 317814/391673 (81.1% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 17 2023 at 18:38):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 775/967 (80.1% of total)
Ported lines: 320719/425772 (75.3% of total)
Longest unported chain: 29/100 (71.0% progress)

port-progress bot (Mar 17 2023 at 18:42):

mathlib port progress combinatorics.additive.behrend
Ported files: 777/972 (79.9% of total)
Ported lines: 321550/427683 (75.2% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 17 2023 at 18:47):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 790/1041 (75.9% of total)
Ported lines: 323220/440350 (73.4% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 17 2023 at 18:52):

mathlib port progress measure_theory.integral.bochner
Ported files: 792/1013 (78.2% of total)
Ported lines: 328225/460797 (71.2% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 17 2023 at 18:56):

mathlib port progress probability.independence
Ported files: 795/1028 (77.3% of total)
Ported lines: 328598/468502 (70.1% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 17 2023 at 19:02):

mathlib port progress all
Ported files: 1365/2902 (47.0% of total)
Ported lines: 454913/1006398 (45.2% of total)
Longest unported chain: 54/125 (56.8% progress)

Chris Hughes (Mar 17 2023 at 19:05):

0.5%

port-progress bot (Mar 18 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138243/142680 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

Jeremy Tan (Mar 18 2023 at 18:05):

Are !4#2692 and !4#2880 ready to merge? (The latter was invalidated from other merges, and has been fixed as far as the CI is concerned)

port-progress bot (Mar 18 2023 at 18:08):

mathlib port progress ring_theory.polynomial.basic
Ported files: 540/561 (96.3% of total)
Ported lines: 217390/228904 (95.0% of total)
Longest unported chain: 6/70 (91.4% progress)

port-progress bot (Mar 18 2023 at 18:12):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 368/397 (92.7% of total)
Ported lines: 138363/150170 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 18 2023 at 18:16):

mathlib port progress topology.continuous_function.bounded
Ported files: 655/699 (93.7% of total)
Ported lines: 276929/304031 (91.1% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 18 2023 at 18:20):

mathlib port progress linear_algebra.determinant
Ported files: 583/642 (90.8% of total)
Ported lines: 235051/263101 (89.3% of total)
Longest unported chain: 13/77 (83.1% progress)

port-progress bot (Mar 18 2023 at 18:24):

mathlib port progress analysis.calculus.fderiv
Ported files: 648/699 (92.7% of total)
Ported lines: 273888/307640 (89.0% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 18 2023 at 18:28):

mathlib port progress category_theory.monoidal.tor
Ported files: 652/712 (91.6% of total)
Ported lines: 252376/275910 (91.5% of total)
Longest unported chain: 16/80 (80.0% progress)

port-progress bot (Mar 18 2023 at 18:32):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 756/897 (84.3% of total)
Ported lines: 320027/391760 (81.7% of total)
Longest unported chain: 21/92 (77.2% progress)

port-progress bot (Mar 18 2023 at 18:36):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 780/968 (80.6% of total)
Ported lines: 323976/425859 (76.1% of total)
Longest unported chain: 28/100 (72.0% progress)

Henrik Böving (Mar 18 2023 at 18:40):

Why is the L2 part not properly linked O_o

port-progress bot (Mar 18 2023 at 18:40):

mathlib port progress combinatorics.additive.behrend
Ported files: 782/973 (80.4% of total)
Ported lines: 324807/427770 (75.9% of total)
Longest unported chain: 29/101 (71.3% progress)

Eric Wieser (Mar 18 2023 at 18:41):

Because this bot is using a regex to generate a markdown table out of plaintext output

Eric Wieser (Mar 18 2023 at 18:41):

A copy of the script is at https://github.com/leanprover-community/mathlib-port-status/blob/main/scripts/port-progress-bot.sh, but I have no idea whether it's the version being run by @Scott Morrison

Eric Wieser (Mar 18 2023 at 18:43):

The cause is the capital L not being matched by [0-9a-z_\.]

port-progress bot (Mar 18 2023 at 18:45):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 795/1039 (76.5% of total)
Ported lines: 325761/439439 (74.1% of total)
Longest unported chain: 35/99 (64.6% progress)

port-progress bot (Mar 18 2023 at 18:49):

mathlib port progress measure_theory.integral.bochner
Ported files: 797/1014 (78.6% of total)
Ported lines: 331482/460884 (71.9% of total)
Longest unported chain: 33/105 (68.6% progress)

port-progress bot (Mar 18 2023 at 18:53):

mathlib port progress probability.independence
Ported files: 800/1029 (77.7% of total)
Ported lines: 331855/468589 (70.8% of total)
Longest unported chain: 38/110 (65.5% progress)

port-progress bot (Mar 18 2023 at 18:59):

mathlib port progress all
Ported files: 1377/2904 (47.4% of total)
Ported lines: 458994/1006814 (45.6% of total)
Longest unported chain: 53/125 (57.6% progress)

Johan Commelin (Mar 18 2023 at 19:06):

0.4%

Jeremy Tan (Mar 18 2023 at 19:15):

Jeremy Tan said:

Are !4#2692 and !4#2880 ready to merge?

Right, both should be ready now

Ayush Agrawal (Mar 19 2023 at 17:49):

Kevin Buzzard said:

If I type

leanproject import-graph --to group_theory.monoid_localization --exclude-tactics --reduce --port-status --exclude-ported --show-unused group_theory.monoid_localization.pdf

into my home PC I get a graph. If I type it into my laptop I get

The node group_theory.monoid_localization is not in the digraph.

Is this something to do with not having enough graph library installed?

I also bumped into the same problem. Can somebody explain what is causing this?

port-progress bot (Mar 19 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138278/142715 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 19 2023 at 18:08):

mathlib port progress ring_theory.polynomial.basic
Ported files: 542/561 (96.6% of total)
Ported lines: 218250/228951 (95.3% of total)
Longest unported chain: 6/70 (91.4% progress)

port-progress bot (Mar 19 2023 at 18:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 368/397 (92.7% of total)
Ported lines: 138398/150205 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 19 2023 at 18:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 655/699 (93.7% of total)
Ported lines: 276964/304064 (91.1% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 19 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 585/643 (91.0% of total)
Ported lines: 235911/263188 (89.6% of total)
Longest unported chain: 14/78 (82.1% progress)

port-progress bot (Mar 19 2023 at 18:24):

mathlib port progress analysis.calculus.fderiv
Ported files: 648/699 (92.7% of total)
Ported lines: 273923/307673 (89.0% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 19 2023 at 18:27):

mathlib port progress category_theory.monoidal.tor
Ported files: 654/712 (91.9% of total)
Ported lines: 253236/275957 (91.8% of total)
Longest unported chain: 16/80 (80.0% progress)

port-progress bot (Mar 19 2023 at 18:31):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 758/898 (84.4% of total)
Ported lines: 320887/391849 (81.9% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 19 2023 at 18:36):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 783/969 (80.8% of total)
Ported lines: 325065/425951 (76.3% of total)
Longest unported chain: 29/100 (71.0% progress)

port-progress bot (Mar 19 2023 at 18:40):

mathlib port progress combinatorics.additive.behrend
Ported files: 785/974 (80.6% of total)
Ported lines: 325896/427862 (76.2% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 19 2023 at 18:44):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 799/1039 (76.9% of total)
Ported lines: 326894/439494 (74.4% of total)
Longest unported chain: 36/100 (64.0% progress)

port-progress bot (Mar 19 2023 at 18:49):

mathlib port progress measure_theory.integral.bochner
Ported files: 800/1015 (78.8% of total)
Ported lines: 332571/460976 (72.1% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 19 2023 at 18:53):

mathlib port progress probability.independence
Ported files: 803/1030 (78.0% of total)
Ported lines: 332944/468681 (71.0% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 19 2023 at 18:58):

mathlib port progress all
Ported files: 1386/2904 (47.7% of total)
Ported lines: 460648/1006896 (45.7% of total)
Longest unported chain: 54/125 (56.8% progress)

Jireh Loreaux (Mar 19 2023 at 19:27):

0.1%

Scott Morrison (Mar 19 2023 at 20:40):

Ayush Agrawal said:

Kevin Buzzard said:

If I type

leanproject import-graph --to group_theory.monoid_localization --exclude-tactics --reduce --port-status --exclude-ported --show-unused group_theory.monoid_localization.pdf

into my home PC I get a graph. If I type it into my laptop I get

The node group_theory.monoid_localization is not in the digraph.

Is this something to do with not having enough graph library installed?

I also bumped into the same problem. Can somebody explain what is causing this?

For some people, the import-graph command only seems to work when run from inside the src folder.

Ayush Agrawal (Mar 20 2023 at 06:12):

Scott Morrison said:

Ayush Agrawal said:

Kevin Buzzard said:

If I type

leanproject import-graph --to group_theory.monoid_localization --exclude-tactics --reduce --port-status --exclude-ported --show-unused group_theory.monoid_localization.pdf

into my home PC I get a graph. If I type it into my laptop I get

The node group_theory.monoid_localization is not in the digraph.

Is this something to do with not having enough graph library installed?

I also bumped into the same problem. Can somebody explain what is causing this?

For some people, the import-graph command only seems to work when run from inside the src folder.

I am running that inside src folder only. This happens for some files only.

Jon Eugster (Mar 20 2023 at 09:08):

Which files do not work? already ported files would raise this error, for example.

Scott Morrison (Mar 20 2023 at 09:17):

Oh yeah! As Jon is implicitly indicating, you've used the flag --exclude-ported, and group_theory.monoid_localization has already been ported to mathlib4, so it's not in the digraph, as expected!

Jon Eugster (Mar 20 2023 at 09:31):

( I did change that for myself a few months ago: mathlib-tools#162. So instead of failing, the script would output a file with a single green node. But never bothered to ping any devs to review and merge it)

port-progress bot (Mar 20 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138278/142715 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 20 2023 at 18:07):

mathlib port progress ring_theory.polynomial.basic
Ported files: 542/561 (96.6% of total)
Ported lines: 218256/228957 (95.3% of total)
Longest unported chain: 6/70 (91.4% progress)

port-progress bot (Mar 20 2023 at 18:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 368/397 (92.7% of total)
Ported lines: 138398/150205 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 20 2023 at 18:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 655/699 (93.7% of total)
Ported lines: 276982/304082 (91.1% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 20 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 586/643 (91.1% of total)
Ported lines: 235975/263208 (89.7% of total)
Longest unported chain: 14/78 (82.1% progress)

port-progress bot (Mar 20 2023 at 18:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 648/699 (92.7% of total)
Ported lines: 273930/307680 (89.0% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 20 2023 at 18:27):

mathlib port progress category_theory.monoidal.tor
Ported files: 654/712 (91.9% of total)
Ported lines: 253242/275963 (91.8% of total)
Longest unported chain: 16/80 (80.0% progress)

port-progress bot (Mar 20 2023 at 18:31):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 759/898 (84.5% of total)
Ported lines: 320955/391873 (81.9% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 20 2023 at 18:35):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 784/969 (80.9% of total)
Ported lines: 325136/425978 (76.3% of total)
Longest unported chain: 29/100 (71.0% progress)

port-progress bot (Mar 20 2023 at 18:39):

mathlib port progress combinatorics.additive.behrend
Ported files: 786/974 (80.7% of total)
Ported lines: 325967/427889 (76.2% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 20 2023 at 18:44):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 801/1039 (77.1% of total)
Ported lines: 327384/439524 (74.5% of total)
Longest unported chain: 36/100 (64.0% progress)

port-progress bot (Mar 20 2023 at 18:48):

mathlib port progress measure_theory.integral.bochner
Ported files: 801/1015 (78.9% of total)
Ported lines: 332642/461003 (72.2% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 20 2023 at 18:52):

mathlib port progress probability.independence
Ported files: 804/1030 (78.1% of total)
Ported lines: 333015/468708 (71.0% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 20 2023 at 18:57):

mathlib port progress all
Ported files: 1388/2904 (47.8% of total)
Ported lines: 461150/1007247 (45.8% of total)
Longest unported chain: 54/125 (56.8% progress)

Johan Commelin (Mar 20 2023 at 19:00):

0.1%

port-progress bot (Mar 21 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138278/142715 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 21 2023 at 18:07):

mathlib port progress ring_theory.polynomial.basic
Ported files: 546/561 (97.3% of total)
Ported lines: 221327/228957 (96.7% of total)
Longest unported chain: 4/70 (94.3% progress)

port-progress bot (Mar 21 2023 at 18:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 368/397 (92.7% of total)
Ported lines: 138398/150205 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 21 2023 at 18:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 655/699 (93.7% of total)
Ported lines: 276982/304101 (91.1% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 21 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 591/643 (91.9% of total)
Ported lines: 239428/263208 (91.0% of total)
Longest unported chain: 14/78 (82.1% progress)

port-progress bot (Mar 21 2023 at 18:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 648/699 (92.7% of total)
Ported lines: 273930/307924 (89.0% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 21 2023 at 18:26):

mathlib port progress category_theory.monoidal.tor
Ported files: 659/712 (92.6% of total)
Ported lines: 256541/275963 (93.0% of total)
Longest unported chain: 15/80 (81.2% progress)

port-progress bot (Mar 21 2023 at 18:30):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 764/898 (85.1% of total)
Ported lines: 324408/392001 (82.8% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 21 2023 at 18:34):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 789/969 (81.4% of total)
Ported lines: 328589/426408 (77.1% of total)
Longest unported chain: 29/100 (71.0% progress)

port-progress bot (Mar 21 2023 at 18:39):

mathlib port progress combinatorics.additive.behrend
Ported files: 791/974 (81.2% of total)
Ported lines: 329420/428319 (76.9% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 21 2023 at 18:43):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 807/1039 (77.7% of total)
Ported lines: 331277/439652 (75.3% of total)
Longest unported chain: 36/100 (64.0% progress)

port-progress bot (Mar 21 2023 at 18:47):

mathlib port progress measure_theory.integral.bochner
Ported files: 806/1015 (79.4% of total)
Ported lines: 336095/461433 (72.8% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 21 2023 at 18:51):

mathlib port progress probability.independence
Ported files: 809/1030 (78.5% of total)
Ported lines: 336468/469138 (71.7% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 21 2023 at 18:56):

mathlib port progress all
Ported files: 1397/2904 (48.1% of total)
Ported lines: 465615/1007677 (46.2% of total)
Longest unported chain: 54/125 (56.8% progress)

Johan Commelin (Mar 21 2023 at 21:25):

0.4%

Jeremy Tan (Mar 22 2023 at 17:08):

As of now the number of unported files (excluding in-progress ones) is less than the number of ported files

Jeremy Tan (Mar 22 2023 at 17:08):

So in a sense we have reached halfway

port-progress bot (Mar 22 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138278/142715 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 22 2023 at 18:08):

mathlib port progress ring_theory.polynomial.basic
Ported files: 547/562 (97.3% of total)
Ported lines: 221705/229185 (96.7% of total)
Longest unported chain: 3/70 (95.7% progress)

port-progress bot (Mar 22 2023 at 18:12):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 368/397 (92.7% of total)
Ported lines: 138398/150205 (92.1% of total)
Longest unported chain: 10/53 (81.1% progress)

port-progress bot (Mar 22 2023 at 18:16):

mathlib port progress topology.continuous_function.bounded
Ported files: 655/699 (93.7% of total)
Ported lines: 276982/304101 (91.1% of total)
Longest unported chain: 12/86 (86.0% progress)

port-progress bot (Mar 22 2023 at 18:20):

mathlib port progress linear_algebra.determinant
Ported files: 593/644 (92.1% of total)
Ported lines: 240093/263445 (91.1% of total)
Longest unported chain: 14/78 (82.1% progress)

port-progress bot (Mar 22 2023 at 18:24):

mathlib port progress analysis.calculus.fderiv
Ported files: 648/699 (92.7% of total)
Ported lines: 273930/307924 (89.0% of total)
Longest unported chain: 14/88 (84.1% progress)

port-progress bot (Mar 22 2023 at 18:28):

mathlib port progress category_theory.monoidal.tor
Ported files: 661/713 (92.7% of total)
Ported lines: 257141/276194 (93.1% of total)
Longest unported chain: 15/80 (81.2% progress)

port-progress bot (Mar 22 2023 at 18:32):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 768/899 (85.4% of total)
Ported lines: 326093/392238 (83.1% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 22 2023 at 18:36):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 794/971 (81.8% of total)
Ported lines: 330775/426682 (77.5% of total)
Longest unported chain: 29/100 (71.0% progress)

port-progress bot (Mar 22 2023 at 18:40):

mathlib port progress combinatorics.additive.behrend
Ported files: 796/976 (81.6% of total)
Ported lines: 331606/428593 (77.4% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 22 2023 at 18:45):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 813/1040 (78.2% of total)
Ported lines: 333726/439898 (75.9% of total)
Longest unported chain: 36/100 (64.0% progress)

port-progress bot (Mar 22 2023 at 18:49):

mathlib port progress measure_theory.integral.bochner
Ported files: 811/1017 (79.7% of total)
Ported lines: 338281/461707 (73.3% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 22 2023 at 18:53):

mathlib port progress probability.independence
Ported files: 814/1032 (78.9% of total)
Ported lines: 338654/469412 (72.1% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 22 2023 at 18:58):

mathlib port progress all
Ported files: 1411/2907 (48.5% of total)
Ported lines: 470349/1008132 (46.7% of total)
Longest unported chain: 54/125 (56.8% progress)

Johan Commelin (Mar 22 2023 at 19:40):

0.5%

port-progress bot (Mar 23 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138278/142715 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 23 2023 at 18:07):

mathlib port progress ring_theory.polynomial.basic
Ported files: 548/562 (97.5% of total)
Ported lines: 222812/229188 (97.2% of total)
Longest unported chain: 2/70 (97.1% progress)

port-progress bot (Mar 23 2023 at 18:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 369/397 (92.9% of total)
Ported lines: 139152/150205 (92.6% of total)
Longest unported chain: 9/53 (83.0% progress)

port-progress bot (Mar 23 2023 at 18:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 657/699 (94.0% of total)
Ported lines: 278525/304101 (91.6% of total)
Longest unported chain: 11/86 (87.2% progress)

port-progress bot (Mar 23 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 594/644 (92.2% of total)
Ported lines: 241200/263448 (91.6% of total)
Longest unported chain: 14/78 (82.1% progress)

port-progress bot (Mar 23 2023 at 18:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 650/699 (93.0% of total)
Ported lines: 275473/307924 (89.5% of total)
Longest unported chain: 13/88 (85.2% progress)

port-progress bot (Mar 23 2023 at 18:26):

mathlib port progress category_theory.monoidal.tor
Ported files: 662/713 (92.8% of total)
Ported lines: 258251/276200 (93.5% of total)
Longest unported chain: 15/80 (81.2% progress)

port-progress bot (Mar 23 2023 at 18:30):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 771/899 (85.8% of total)
Ported lines: 328749/392247 (83.8% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 23 2023 at 18:34):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 797/971 (82.1% of total)
Ported lines: 333434/426694 (78.1% of total)
Longest unported chain: 29/100 (71.0% progress)

port-progress bot (Mar 23 2023 at 18:38):

mathlib port progress combinatorics.additive.behrend
Ported files: 799/976 (81.9% of total)
Ported lines: 334265/428605 (78.0% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 23 2023 at 18:43):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 818/1040 (78.7% of total)
Ported lines: 336628/439910 (76.5% of total)
Longest unported chain: 36/100 (64.0% progress)

port-progress bot (Mar 23 2023 at 18:47):

mathlib port progress measure_theory.integral.bochner
Ported files: 814/1017 (80.0% of total)
Ported lines: 340940/461719 (73.8% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 23 2023 at 18:51):

mathlib port progress probability.independence
Ported files: 817/1032 (79.2% of total)
Ported lines: 341313/469424 (72.7% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 23 2023 at 18:56):

mathlib port progress all
Ported files: 1427/2907 (49.1% of total)
Ported lines: 476660/1008146 (47.3% of total)
Longest unported chain: 54/125 (56.8% progress)

Chris Hughes (Mar 23 2023 at 19:16):

1.1%

Scott Morrison (Mar 23 2023 at 21:55):

Err, not to rain on the parade, but I think it is only 0.6% = 47.3% - 46.7%.

port-progress bot (Mar 24 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138314/142751 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 24 2023 at 18:07):

mathlib port progress ring_theory.polynomial.basic
Ported files: 548/562 (97.5% of total)
Ported lines: 222867/229254 (97.2% of total)
Longest unported chain: 2/70 (97.1% progress)

port-progress bot (Mar 24 2023 at 18:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 369/397 (92.9% of total)
Ported lines: 139191/150244 (92.6% of total)
Longest unported chain: 9/53 (83.0% progress)

port-progress bot (Mar 24 2023 at 18:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 657/699 (94.0% of total)
Ported lines: 278602/304178 (91.6% of total)
Longest unported chain: 11/86 (87.2% progress)

port-progress bot (Mar 24 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 594/644 (92.2% of total)
Ported lines: 241255/263514 (91.6% of total)
Longest unported chain: 14/78 (82.1% progress)

port-progress bot (Mar 24 2023 at 18:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 650/699 (93.0% of total)
Ported lines: 275550/308001 (89.5% of total)
Longest unported chain: 13/88 (85.2% progress)

port-progress bot (Mar 24 2023 at 18:26):

mathlib port progress category_theory.monoidal.tor
Ported files: 665/713 (93.3% of total)
Ported lines: 259530/276268 (93.9% of total)
Longest unported chain: 15/80 (81.2% progress)

port-progress bot (Mar 24 2023 at 18:30):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 777/899 (86.4% of total)
Ported lines: 332723/392338 (84.8% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 24 2023 at 18:34):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 803/971 (82.7% of total)
Ported lines: 337408/426785 (79.1% of total)
Longest unported chain: 29/100 (71.0% progress)

port-progress bot (Mar 24 2023 at 18:39):

mathlib port progress combinatorics.additive.behrend
Ported files: 805/976 (82.5% of total)
Ported lines: 338239/428696 (78.9% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 24 2023 at 18:43):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 824/1040 (79.2% of total)
Ported lines: 340608/440007 (77.4% of total)
Longest unported chain: 36/100 (64.0% progress)

port-progress bot (Mar 24 2023 at 18:47):

mathlib port progress measure_theory.integral.bochner
Ported files: 820/1017 (80.6% of total)
Ported lines: 344914/461810 (74.7% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 24 2023 at 18:51):

mathlib port progress probability.independence
Ported files: 823/1032 (79.7% of total)
Ported lines: 345287/469515 (73.5% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 24 2023 at 18:56):

mathlib port progress all
Ported files: 1445/2909 (49.7% of total)
Ported lines: 485237/1008667 (48.1% of total)
Longest unported chain: 54/125 (56.8% progress)

Johan Commelin (Mar 24 2023 at 18:58):

0.8%

Jeremy Tan (Mar 25 2023 at 12:51):

And with the merging of Algebra.MonoidAlgebra.Division we are now officially over 50% done in terms of file count

Jeremy Tan (Mar 25 2023 at 12:53):

Our next target will be 75% in terms of file count

Kevin Buzzard (Mar 25 2023 at 14:26):

That will be your next target. My next target will be 60%.

port-progress bot (Mar 25 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138327/142764 (96.9% of total)
Longest unported chain: 1/48 (97.9% progress)

port-progress bot (Mar 25 2023 at 18:08):

mathlib port progress ring_theory.polynomial.basic
Ported files: 552/562 (98.2% of total)
Ported lines: 224647/229423 (97.9% of total)
Longest unported chain: 1/70 (98.6% progress)

port-progress bot (Mar 25 2023 at 18:12):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 373/397 (94.0% of total)
Ported lines: 140679/150269 (93.6% of total)
Longest unported chain: 8/53 (84.9% progress)

port-progress bot (Mar 25 2023 at 18:16):

mathlib port progress topology.continuous_function.bounded
Ported files: 662/700 (94.6% of total)
Ported lines: 281845/304514 (92.6% of total)
Longest unported chain: 8/86 (90.7% progress)

port-progress bot (Mar 25 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 598/644 (92.9% of total)
Ported lines: 243035/263683 (92.2% of total)
Longest unported chain: 14/78 (82.1% progress)

port-progress bot (Mar 25 2023 at 18:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 655/700 (93.6% of total)
Ported lines: 278793/308337 (90.4% of total)
Longest unported chain: 10/88 (88.6% progress)

port-progress bot (Mar 25 2023 at 18:27):

mathlib port progress category_theory.monoidal.tor
Ported files: 668/713 (93.7% of total)
Ported lines: 260609/276443 (94.3% of total)
Longest unported chain: 15/80 (81.2% progress)

port-progress bot (Mar 25 2023 at 18:31):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 781/899 (86.9% of total)
Ported lines: 333733/392585 (85.0% of total)
Longest unported chain: 22/92 (76.1% progress)

port-progress bot (Mar 25 2023 at 18:35):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 807/971 (83.1% of total)
Ported lines: 338418/427034 (79.2% of total)
Longest unported chain: 29/100 (71.0% progress)

port-progress bot (Mar 25 2023 at 18:39):

mathlib port progress combinatorics.additive.behrend
Ported files: 809/976 (82.9% of total)
Ported lines: 339249/428945 (79.1% of total)
Longest unported chain: 30/101 (70.3% progress)

port-progress bot (Mar 25 2023 at 18:43):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 828/1040 (79.6% of total)
Ported lines: 341618/440241 (77.6% of total)
Longest unported chain: 36/100 (64.0% progress)

port-progress bot (Mar 25 2023 at 18:48):

mathlib port progress measure_theory.integral.bochner
Ported files: 825/1017 (81.1% of total)
Ported lines: 346218/462046 (74.9% of total)
Longest unported chain: 34/105 (67.6% progress)

port-progress bot (Mar 25 2023 at 18:52):

mathlib port progress probability.independence
Ported files: 828/1032 (80.2% of total)
Ported lines: 346591/469757 (73.8% of total)
Longest unported chain: 39/110 (64.5% progress)

port-progress bot (Mar 25 2023 at 18:57):

mathlib port progress all
Ported files: 1455/2908 (50.0% of total)
Ported lines: 489088/1009002 (48.5% of total)
Longest unported chain: 54/125 (56.8% progress)

Johan Commelin (Mar 25 2023 at 19:02):

0.4%

port-progress bot (Mar 26 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 360/371 (97.0% of total)
Ported lines: 137892/142680 (96.6% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Mar 26 2023 at 18:07):

mathlib port progress ring_theory.polynomial.basic
Ported files: 551/563 (97.9% of total)
Ported lines: 224216/229466 (97.7% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Mar 26 2023 at 18:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 373/397 (94.0% of total)
Ported lines: 140465/150185 (93.5% of total)
Longest unported chain: 7/52 (86.5% progress)

port-progress bot (Mar 26 2023 at 18:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 661/701 (94.3% of total)
Ported lines: 281423/304566 (92.4% of total)
Longest unported chain: 8/85 (90.6% progress)

port-progress bot (Mar 26 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 597/645 (92.6% of total)
Ported lines: 242604/263726 (92.0% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 26 2023 at 18:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 654/701 (93.3% of total)
Ported lines: 278371/308389 (90.3% of total)
Longest unported chain: 10/87 (88.5% progress)

port-progress bot (Mar 26 2023 at 18:26):

mathlib port progress category_theory.monoidal.tor
Ported files: 667/714 (93.4% of total)
Ported lines: 260178/276486 (94.1% of total)
Longest unported chain: 15/79 (81.0% progress)

port-progress bot (Mar 26 2023 at 18:30):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 780/900 (86.7% of total)
Ported lines: 333311/392637 (84.9% of total)
Longest unported chain: 22/91 (75.8% progress)

port-progress bot (Mar 26 2023 at 18:35):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 806/972 (82.9% of total)
Ported lines: 337996/427086 (79.1% of total)
Longest unported chain: 29/99 (70.7% progress)

port-progress bot (Mar 26 2023 at 18:39):

mathlib port progress combinatorics.additive.behrend
Ported files: 808/977 (82.7% of total)
Ported lines: 338827/428997 (79.0% of total)
Longest unported chain: 30/100 (70.0% progress)

port-progress bot (Mar 26 2023 at 18:43):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 827/1041 (79.4% of total)
Ported lines: 341196/440293 (77.5% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 26 2023 at 18:47):

mathlib port progress measure_theory.integral.bochner
Ported files: 824/1018 (80.9% of total)
Ported lines: 345796/462098 (74.8% of total)
Longest unported chain: 34/104 (67.3% progress)

port-progress bot (Mar 26 2023 at 18:51):

mathlib port progress probability.independence
Ported files: 827/1033 (80.1% of total)
Ported lines: 346169/469809 (73.7% of total)
Longest unported chain: 39/109 (64.2% progress)

port-progress bot (Mar 26 2023 at 18:56):

mathlib port progress all
Ported files: 1458/2909 (50.1% of total)
Ported lines: 489188/1009057 (48.5% of total)
Longest unported chain: 54/124 (56.5% progress)

Jeremy Tan (Mar 26 2023 at 18:56):

-0.1%

Jeremy Tan (Mar 26 2023 at 18:57):

We've got some ready PRs but nobody approved them

James Gallicchio (Mar 26 2023 at 20:18):

Hey, number of ported files still went up :joy:

Scott Morrison (Mar 26 2023 at 22:12):

@Jeremy Tan, the number you posted just seems to be wrong. Johan has been posting the difference for the number of ported lines. It was 48.5% yesterday, and 48.5% today.

Scott Morrison (Mar 26 2023 at 22:18):

Jeremy Tan said:

We've got some ready PRs but nobody approved them

Moreover, I would ask (repeating early requests others have made) that you be patient, and understand that many people are involved, and they are working as hard as they can on this porting effort.

Saying "but nobody approved them" is not helpful at the moment. Please remember that everyone is working within their time constraints. Also, given that there are many open files for porting at the moment, approving PRs is not actually the bottleneck right now.

Similarly above saying "our next target will be 75%" is inappropriate. We certainly appreciate the considerable effort you've been putting into porting recently, but please use caution in telling others what their priorities should be.

Patrick Stevens (Mar 26 2023 at 22:20):

(indeed, fraction of ported lines has increased by over 0.007% since yesterday - still positive, even if it rounds to 0 to one decimal place!)

Jeremy Tan (Mar 27 2023 at 02:58):

@Scott Morrison I live in Singapore, on the other side of the world from where most of you are. I can stare for hours in my afternoon at the recently changed PRs, when you're all sleeping, not knowing what to do with those PRs

Jeremy Tan (Mar 27 2023 at 02:59):

Constantly pressing F5, and seeing that nothing changed

Scott Morrison (Mar 27 2023 at 03:00):

Don't press F5? Work on files that don't yet have a PR open for them? It seems unproductive to wait on other people unnecessarily? I fear, though, that you're not understanding the point I'm making about social interactions.

Jeremy Tan (Mar 27 2023 at 03:03):

My brain is too small for most of the standard mathlib ports. Where can I get a list of forward ports from mathlib3 that need to be done?

Jeremy Tan (Mar 27 2023 at 03:13):

Scott Morrison said:

Work on files that don't yet have a PR open for them?

Where are those files???

James Gallicchio (Mar 27 2023 at 03:17):

(I think scott is suggesting to focus on opening new PRs for files that haven't been started yet, since there are dozens of files that are ready to port but haven't been started yet)

Jeremy Tan (Mar 27 2023 at 03:20):

@James Gallicchio I was asking for where I can find those files that haven't been started. I have no reply so far

Jeremy Tan (Mar 27 2023 at 03:20):

Not just the files without a mathlib4 equiv yet

Jeremy Tan (Mar 27 2023 at 03:21):

I'm talking about the forwardports that need to be done

James Gallicchio (Mar 27 2023 at 03:22):

As far as I'm aware, forward ports are a bit trickier to orchestrate (see https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/forward.20porting ). So it would probably be a better use of your time to focus on unported files.

Jeremy Tan (Mar 27 2023 at 03:23):

Right then

Moritz Doll (Mar 27 2023 at 04:16):

James Gallicchio I was asking for where I can find those files that haven't been started. I have no reply so far

#port-dashboard

Jeremy Tan (Mar 27 2023 at 05:40):

Right now #port-dashboard is mangled because of the Data.Set.Pairwise.Basic file that will be introduced by !4#3117

Jeremy Tan (Mar 27 2023 at 05:41):

I'll have to wait until that is merged

Eric Wieser (Mar 27 2023 at 07:52):

Contributions to #port-dashboard itself to fix that behavior would also be welcome!

Chris Hughes (Mar 27 2023 at 12:35):

Jeremy Tan said:

Scott Morrison said:

Work on files that don't yet have a PR open for them?

Where are those files???

There's a list of files that aren't ported yet here. There should be quite a few on the "Maybe ready to port" list that you could work on. Right now there are a few polynomial related files there, and those are fairly straightforward in my experience.

port-progress bot (Mar 27 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 360/371 (97.0% of total)
Ported lines: 137905/142693 (96.6% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Mar 27 2023 at 18:07):

mathlib port progress ring_theory.polynomial.basic
Ported files: 551/563 (97.9% of total)
Ported lines: 224273/229523 (97.7% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Mar 27 2023 at 18:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 373/397 (94.0% of total)
Ported lines: 140478/150198 (93.5% of total)
Longest unported chain: 7/52 (86.5% progress)

port-progress bot (Mar 27 2023 at 18:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 655/688 (95.2% of total)
Ported lines: 279402/298721 (93.5% of total)
Longest unported chain: 8/85 (90.6% progress)

port-progress bot (Mar 27 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 597/645 (92.6% of total)
Ported lines: 242687/263809 (92.0% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 27 2023 at 18:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 654/700 (93.4% of total)
Ported lines: 278406/308208 (90.3% of total)
Longest unported chain: 10/87 (88.5% progress)

port-progress bot (Mar 27 2023 at 18:26):

mathlib port progress category_theory.monoidal.tor
Ported files: 668/714 (93.6% of total)
Ported lines: 260319/276565 (94.1% of total)
Longest unported chain: 15/79 (81.0% progress)

port-progress bot (Mar 27 2023 at 18:30):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 780/899 (86.8% of total)
Ported lines: 333394/392504 (84.9% of total)
Longest unported chain: 22/91 (75.8% progress)

port-progress bot (Mar 27 2023 at 18:34):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 807/971 (83.1% of total)
Ported lines: 338529/426981 (79.3% of total)
Longest unported chain: 29/99 (70.7% progress)

port-progress bot (Mar 27 2023 at 18:39):

mathlib port progress combinatorics.additive.behrend
Ported files: 809/976 (82.9% of total)
Ported lines: 339360/428892 (79.1% of total)
Longest unported chain: 30/100 (70.0% progress)

port-progress bot (Mar 27 2023 at 18:43):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 828/1040 (79.6% of total)
Ported lines: 341729/440206 (77.6% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 27 2023 at 18:47):

mathlib port progress measure_theory.integral.bochner
Ported files: 825/1017 (81.1% of total)
Ported lines: 346329/461993 (75.0% of total)
Longest unported chain: 34/104 (67.3% progress)

port-progress bot (Mar 27 2023 at 18:51):

mathlib port progress probability.independence
Ported files: 828/1032 (80.2% of total)
Ported lines: 346702/469704 (73.8% of total)
Longest unported chain: 39/109 (64.2% progress)

port-progress bot (Mar 27 2023 at 18:57):

mathlib port progress all
Ported files: 1468/2911 (50.4% of total)
Ported lines: 491237/1009595 (48.7% of total)
Longest unported chain: 54/124 (56.5% progress)

Scott Morrison (Mar 27 2023 at 19:00):

0.2%

Chris Hughes (Mar 28 2023 at 12:23):

The "Maybe ready to port" section on https://leanprover-community.github.io/mathlib-port-status/old has suddenly got far fewer files on it than it did yesterday. Is there a reason for this. It's the tool I've been using to figure the next file to have a go at.

Eric Wieser (Mar 28 2023 at 15:47):

That section tracked files which had an unported dependency somewhere that wasn't a direct dependency

Eric Wieser (Mar 28 2023 at 15:47):

port-status#data/set/pairwise/basic was added in a mathlib3 refactor and so caused most of the files to end up in that section

port-progress bot (Mar 28 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138274/142711 (96.9% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Mar 28 2023 at 18:07):

mathlib port progress ring_theory.polynomial.basic
Ported files: 553/563 (98.2% of total)
Ported lines: 224765/229541 (97.9% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Mar 28 2023 at 18:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 374/397 (94.2% of total)
Ported lines: 140847/150218 (93.8% of total)
Longest unported chain: 7/52 (86.5% progress)

port-progress bot (Mar 28 2023 at 18:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 659/688 (95.8% of total)
Ported lines: 280642/298739 (93.9% of total)
Longest unported chain: 8/85 (90.6% progress)

port-progress bot (Mar 28 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 599/645 (92.9% of total)
Ported lines: 243179/263827 (92.2% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 28 2023 at 18:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 659/700 (94.1% of total)
Ported lines: 280031/308226 (90.9% of total)
Longest unported chain: 10/87 (88.5% progress)

port-progress bot (Mar 28 2023 at 18:27):

mathlib port progress category_theory.monoidal.tor
Ported files: 670/714 (93.8% of total)
Ported lines: 260811/276585 (94.3% of total)
Longest unported chain: 15/79 (81.0% progress)

port-progress bot (Mar 28 2023 at 18:30):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 785/899 (87.3% of total)
Ported lines: 335019/392522 (85.4% of total)
Longest unported chain: 22/91 (75.8% progress)

port-progress bot (Mar 28 2023 at 18:35):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 813/971 (83.7% of total)
Ported lines: 341011/426999 (79.9% of total)
Longest unported chain: 29/99 (70.7% progress)

port-progress bot (Mar 28 2023 at 18:39):

mathlib port progress combinatorics.additive.behrend
Ported files: 815/976 (83.5% of total)
Ported lines: 341842/428910 (79.7% of total)
Longest unported chain: 30/100 (70.0% progress)

port-progress bot (Mar 28 2023 at 18:43):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 834/1040 (80.2% of total)
Ported lines: 344211/440224 (78.2% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 28 2023 at 18:47):

mathlib port progress measure_theory.integral.bochner
Ported files: 831/1017 (81.7% of total)
Ported lines: 348811/462011 (75.5% of total)
Longest unported chain: 34/104 (67.3% progress)

port-progress bot (Mar 28 2023 at 18:51):

mathlib port progress probability.independence
Ported files: 834/1032 (80.8% of total)
Ported lines: 349184/469722 (74.3% of total)
Longest unported chain: 39/109 (64.2% progress)

port-progress bot (Mar 28 2023 at 18:56):

mathlib port progress all
Ported files: 1476/2911 (50.7% of total)
Ported lines: 494271/1009606 (49.0% of total)
Longest unported chain: 54/124 (56.5% progress)

Johan Commelin (Mar 28 2023 at 19:13):

0.3%

port-progress bot (Mar 29 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138278/142715 (96.9% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Mar 29 2023 at 18:08):

mathlib port progress ring_theory.polynomial.basic
Ported files: 553/563 (98.2% of total)
Ported lines: 224796/229572 (97.9% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Mar 29 2023 at 18:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 375/397 (94.5% of total)
Ported lines: 141121/150222 (93.9% of total)
Longest unported chain: 7/52 (86.5% progress)

port-progress bot (Mar 29 2023 at 18:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 659/688 (95.8% of total)
Ported lines: 280673/298770 (93.9% of total)
Longest unported chain: 8/85 (90.6% progress)

port-progress bot (Mar 29 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 599/645 (92.9% of total)
Ported lines: 243210/263858 (92.2% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 29 2023 at 18:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 659/700 (94.1% of total)
Ported lines: 280062/308262 (90.9% of total)
Longest unported chain: 10/87 (88.5% progress)

port-progress bot (Mar 29 2023 at 18:27):

mathlib port progress category_theory.monoidal.tor
Ported files: 672/714 (94.1% of total)
Ported lines: 261137/276955 (94.3% of total)
Longest unported chain: 14/79 (82.3% progress)

port-progress bot (Mar 29 2023 at 18:31):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 785/899 (87.3% of total)
Ported lines: 335050/392558 (85.4% of total)
Longest unported chain: 22/91 (75.8% progress)

port-progress bot (Mar 29 2023 at 18:35):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 816/971 (84.0% of total)
Ported lines: 341794/427039 (80.0% of total)
Longest unported chain: 29/99 (70.7% progress)

port-progress bot (Mar 29 2023 at 18:39):

mathlib port progress combinatorics.additive.behrend
Ported files: 818/976 (83.8% of total)
Ported lines: 342625/428950 (79.9% of total)
Longest unported chain: 30/100 (70.0% progress)

port-progress bot (Mar 29 2023 at 18:44):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 839/1040 (80.7% of total)
Ported lines: 345301/440264 (78.4% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 29 2023 at 18:48):

mathlib port progress measure_theory.integral.bochner
Ported files: 834/1017 (82.0% of total)
Ported lines: 349594/462051 (75.7% of total)
Longest unported chain: 34/104 (67.3% progress)

port-progress bot (Mar 29 2023 at 18:52):

mathlib port progress probability.independence
Ported files: 837/1032 (81.1% of total)
Ported lines: 349967/469762 (74.5% of total)
Longest unported chain: 39/109 (64.2% progress)

port-progress bot (Mar 29 2023 at 18:57):

mathlib port progress all
Ported files: 1492/2913 (51.2% of total)
Ported lines: 497268/1010096 (49.2% of total)
Longest unported chain: 54/124 (56.5% progress)

Johan Commelin (Mar 29 2023 at 19:31):

0.2%

port-progress bot (Mar 30 2023 at 18:04):

mathlib port progress category_theory.abelian.basic
Ported files: 361/371 (97.3% of total)
Ported lines: 138412/142709 (97.0% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Mar 30 2023 at 18:07):

mathlib port progress ring_theory.polynomial.basic
Ported files: 554/563 (98.4% of total)
Ported lines: 226114/229657 (98.5% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Mar 30 2023 at 18:10):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 375/397 (94.5% of total)
Ported lines: 141255/150216 (94.0% of total)
Longest unported chain: 7/52 (86.5% progress)

port-progress bot (Mar 30 2023 at 18:14):

mathlib port progress topology.continuous_function.bounded
Ported files: 659/688 (95.8% of total)
Ported lines: 280898/298858 (94.0% of total)
Longest unported chain: 8/85 (90.6% progress)

port-progress bot (Mar 30 2023 at 18:18):

mathlib port progress linear_algebra.determinant
Ported files: 600/645 (93.0% of total)
Ported lines: 244528/263943 (92.6% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 30 2023 at 18:22):

mathlib port progress analysis.calculus.fderiv
Ported files: 659/700 (94.1% of total)
Ported lines: 280287/308350 (90.9% of total)
Longest unported chain: 10/87 (88.5% progress)

port-progress bot (Mar 30 2023 at 18:26):

mathlib port progress category_theory.monoidal.tor
Ported files: 673/714 (94.3% of total)
Ported lines: 262455/277040 (94.7% of total)
Longest unported chain: 14/79 (82.3% progress)

port-progress bot (Mar 30 2023 at 18:30):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 786/899 (87.4% of total)
Ported lines: 336368/392646 (85.7% of total)
Longest unported chain: 22/91 (75.8% progress)

port-progress bot (Mar 30 2023 at 18:34):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 817/971 (84.1% of total)
Ported lines: 343112/427465 (80.3% of total)
Longest unported chain: 29/99 (70.7% progress)

port-progress bot (Mar 30 2023 at 18:38):

mathlib port progress combinatorics.additive.behrend
Ported files: 819/976 (83.9% of total)
Ported lines: 343943/429376 (80.1% of total)
Longest unported chain: 30/100 (70.0% progress)

port-progress bot (Mar 30 2023 at 18:42):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 840/1040 (80.8% of total)
Ported lines: 346619/440352 (78.7% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 30 2023 at 18:47):

mathlib port progress measure_theory.integral.bochner
Ported files: 835/1017 (82.1% of total)
Ported lines: 350912/462477 (75.9% of total)
Longest unported chain: 34/104 (67.3% progress)

port-progress bot (Mar 30 2023 at 18:51):

mathlib port progress probability.independence
Ported files: 838/1032 (81.2% of total)
Ported lines: 351285/470188 (74.7% of total)
Longest unported chain: 39/109 (64.2% progress)

port-progress bot (Mar 30 2023 at 18:56):

mathlib port progress all
Ported files: 1498/2915 (51.4% of total)
Ported lines: 499634/1011276 (49.4% of total)
Longest unported chain: 54/124 (56.5% progress)

Scott Morrison (Mar 30 2023 at 21:32):

0.2%

port-progress bot (Mar 31 2023 at 18:05):

mathlib port progress category_theory.abelian.basic
Ported files: 362/371 (97.6% of total)
Ported lines: 138519/142747 (97.0% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Mar 31 2023 at 18:07):

mathlib port progress ring_theory.polynomial.basic
Ported files: 555/563 (98.6% of total)
Ported lines: 226265/229739 (98.5% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Mar 31 2023 at 18:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 377/397 (95.0% of total)
Ported lines: 141620/150268 (94.2% of total)
Longest unported chain: 7/52 (86.5% progress)

port-progress bot (Mar 31 2023 at 18:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 660/688 (95.9% of total)
Ported lines: 281055/298946 (94.0% of total)
Longest unported chain: 8/85 (90.6% progress)

port-progress bot (Mar 31 2023 at 18:19):

mathlib port progress linear_algebra.determinant
Ported files: 602/645 (93.3% of total)
Ported lines: 244792/264145 (92.7% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Mar 31 2023 at 18:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 660/700 (94.3% of total)
Ported lines: 280444/308497 (90.9% of total)
Longest unported chain: 10/87 (88.5% progress)

port-progress bot (Mar 31 2023 at 18:27):

mathlib port progress category_theory.monoidal.tor
Ported files: 366/395 (92.7% of total)
Ported lines: 139196/150683 (92.4% of total)
Longest unported chain: 14/56 (75.0% progress)

port-progress bot (Mar 31 2023 at 18:31):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 788/900 (87.6% of total)
Ported lines: 336638/392883 (85.7% of total)
Longest unported chain: 22/91 (75.8% progress)

port-progress bot (Mar 31 2023 at 18:35):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 819/972 (84.3% of total)
Ported lines: 343382/427702 (80.3% of total)
Longest unported chain: 29/99 (70.7% progress)

port-progress bot (Mar 31 2023 at 18:39):

mathlib port progress combinatorics.additive.behrend
Ported files: 821/977 (84.0% of total)
Ported lines: 344213/429613 (80.1% of total)
Longest unported chain: 30/100 (70.0% progress)

port-progress bot (Mar 31 2023 at 18:44):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 843/1041 (81.0% of total)
Ported lines: 347070/440815 (78.7% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Mar 31 2023 at 18:48):

mathlib port progress measure_theory.integral.bochner
Ported files: 837/1017 (82.3% of total)
Ported lines: 351182/462511 (75.9% of total)
Longest unported chain: 34/104 (67.3% progress)

port-progress bot (Mar 31 2023 at 18:52):

mathlib port progress probability.independence
Ported files: 840/1032 (81.4% of total)
Ported lines: 351555/470222 (74.8% of total)
Longest unported chain: 39/109 (64.2% progress)

port-progress bot (Mar 31 2023 at 18:57):

mathlib port progress all
Ported files: 1503/2918 (51.5% of total)
Ported lines: 500767/1011593 (49.5% of total)
Longest unported chain: 54/124 (56.5% progress)

Johan Commelin (Mar 31 2023 at 20:24):

0.1%

Matthew Ballard (Mar 31 2023 at 20:25):

And half a milly

port-progress bot (Apr 01 2023 at 19:05):

mathlib port progress category_theory.abelian.basic
Ported files: 362/371 (97.6% of total)
Ported lines: 138513/142741 (97.0% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Apr 01 2023 at 19:07):

mathlib port progress ring_theory.polynomial.basic
Ported files: 555/563 (98.6% of total)
Ported lines: 226378/229852 (98.5% of total)
Longest unported chain: 1/69 (98.6% progress)

port-progress bot (Apr 01 2023 at 19:11):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 377/397 (95.0% of total)
Ported lines: 141614/150262 (94.2% of total)
Longest unported chain: 7/52 (86.5% progress)

port-progress bot (Apr 01 2023 at 19:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 660/688 (95.9% of total)
Ported lines: 281119/299010 (94.0% of total)
Longest unported chain: 8/85 (90.6% progress)

port-progress bot (Apr 01 2023 at 19:19):

mathlib port progress linear_algebra.determinant
Ported files: 602/645 (93.3% of total)
Ported lines: 244905/264258 (92.7% of total)
Longest unported chain: 14/77 (81.8% progress)

port-progress bot (Apr 01 2023 at 19:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 660/700 (94.3% of total)
Ported lines: 280559/308612 (90.9% of total)
Longest unported chain: 10/87 (88.5% progress)

port-progress bot (Apr 01 2023 at 19:27):

mathlib port progress category_theory.monoidal.tor
Ported files: 366/395 (92.7% of total)
Ported lines: 139190/150677 (92.4% of total)
Longest unported chain: 14/56 (75.0% progress)

port-progress bot (Apr 01 2023 at 19:31):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 788/900 (87.6% of total)
Ported lines: 336751/392996 (85.7% of total)
Longest unported chain: 22/91 (75.8% progress)

port-progress bot (Apr 01 2023 at 19:36):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 819/972 (84.3% of total)
Ported lines: 343495/427815 (80.3% of total)
Longest unported chain: 29/99 (70.7% progress)

port-progress bot (Apr 01 2023 at 19:40):

mathlib port progress combinatorics.additive.behrend
Ported files: 821/977 (84.0% of total)
Ported lines: 344326/429726 (80.1% of total)
Longest unported chain: 30/100 (70.0% progress)

Ruben Van de Velde (Apr 01 2023 at 19:41):

port-progress bot said:

mathlib port progress ring_theory.polynomial.basic
Ported files: 555/563 (98.6% of total)
Ported lines: 226378/229852 (98.5% of total)
Longest unported chain: 1/69 (98.6% progress)

This one's done

port-progress bot (Apr 01 2023 at 19:44):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 843/1041 (81.0% of total)
Ported lines: 347183/440927 (78.7% of total)
Longest unported chain: 36/99 (63.6% progress)

port-progress bot (Apr 01 2023 at 19:49):

mathlib port progress measure_theory.integral.bochner
Ported files: 837/1017 (82.3% of total)
Ported lines: 351250/462583 (75.9% of total)
Longest unported chain: 34/104 (67.3% progress)

port-progress bot (Apr 01 2023 at 19:53):

mathlib port progress probability.independence
Ported files: 840/1032 (81.4% of total)
Ported lines: 351623/470294 (74.8% of total)
Longest unported chain: 39/109 (64.2% progress)

port-progress bot (Apr 01 2023 at 19:58):

mathlib port progress all
Ported files: 1503/2920 (51.5% of total)
Ported lines: 500835/1011927 (49.5% of total)
Longest unported chain: 54/124 (56.5% progress)

Scott Morrison (Apr 01 2023 at 20:22):

0.0%

Kevin Buzzard (Apr 01 2023 at 20:28):

Is this "clearly progress has been made but it's 0.0%" related to the fact that we finally have under 500 mathlib3 PRs for the first time in ages?

Kevin Buzzard (Apr 01 2023 at 20:28):

(deleted)

Scott Morrison (Apr 01 2023 at 20:43):

I think actually it is that the #queue4 has quite a lot of ready-to-merge material, just that no one got to yesterday.

Jireh Loreaux (Apr 01 2023 at 22:07):

If you ever want to know how much (and what) has been ported recently, you can go to #port-status and sort the ported files by date ported.

port-progress bot (Apr 02 2023 at 19:05):

mathlib port progress category_theory.abelian.basic
Ported files: 362/371 (97.6% of total)
Ported lines: 138513/142741 (97.0% of total)
Longest unported chain: 1/47 (97.9% progress)

Eric Wieser (Apr 02 2023 at 19:08):

Jireh Loreaux said:

If you ever want to know how much (and what) has been ported recently, you can go to #port-status and sort the ported files by date ported.

(you mean #port-dashboard)

port-progress bot (Apr 02 2023 at 19:08):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 377/397 (95.0% of total)
Ported lines: 141614/150262 (94.2% of total)
Longest unported chain: 7/52 (86.5% progress)

port-progress bot (Apr 02 2023 at 19:12):

mathlib port progress topology.continuous_function.bounded
Ported files: 660/688 (95.9% of total)
Ported lines: 281124/299015 (94.0% of total)
Longest unported chain: 8/85 (90.6% progress)

port-progress bot (Apr 02 2023 at 19:17):

mathlib port progress linear_algebra.determinant
Ported files: 604/645 (93.6% of total)
Ported lines: 247102/264290 (93.5% of total)
Longest unported chain: 13/77 (83.1% progress)

port-progress bot (Apr 02 2023 at 19:21):

mathlib port progress analysis.calculus.fderiv
Ported files: 660/700 (94.3% of total)
Ported lines: 280564/308617 (90.9% of total)
Longest unported chain: 10/87 (88.5% progress)

port-progress bot (Apr 02 2023 at 19:25):

mathlib port progress category_theory.monoidal.tor
Ported files: 366/395 (92.7% of total)
Ported lines: 139190/150677 (92.4% of total)
Longest unported chain: 14/56 (75.0% progress)

port-progress bot (Apr 02 2023 at 19:29):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 790/900 (87.8% of total)
Ported lines: 338948/393028 (86.2% of total)
Longest unported chain: 21/91 (76.9% progress)

port-progress bot (Apr 02 2023 at 19:33):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 821/972 (84.5% of total)
Ported lines: 345692/427847 (80.8% of total)
Longest unported chain: 28/99 (71.7% progress)

port-progress bot (Apr 02 2023 at 19:37):

mathlib port progress combinatorics.additive.behrend
Ported files: 823/977 (84.2% of total)
Ported lines: 346523/429758 (80.6% of total)
Longest unported chain: 29/100 (71.0% progress)

port-progress bot (Apr 02 2023 at 19:42):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 846/1041 (81.3% of total)
Ported lines: 349524/440959 (79.3% of total)
Longest unported chain: 35/99 (64.6% progress)

port-progress bot (Apr 02 2023 at 19:46):

mathlib port progress measure_theory.integral.bochner
Ported files: 839/1017 (82.5% of total)
Ported lines: 353447/462615 (76.4% of total)
Longest unported chain: 33/104 (68.3% progress)

port-progress bot (Apr 02 2023 at 19:50):

mathlib port progress probability.independence
Ported files: 842/1032 (81.6% of total)
Ported lines: 353820/470326 (75.2% of total)
Longest unported chain: 38/109 (65.1% progress)

port-progress bot (Apr 02 2023 at 19:55):

mathlib port progress all
Ported files: 1507/2920 (51.6% of total)
Ported lines: 503335/1011968 (49.7% of total)
Longest unported chain: 53/124 (57.3% progress)

Mauricio Collares (Apr 02 2023 at 19:56):

#port-dashboard says 50% ported lines

Scott Morrison (Apr 02 2023 at 20:38):

0.2%

port-progress bot (Apr 03 2023 at 19:05):

mathlib port progress category_theory.abelian.basic
Ported files: 362/371 (97.6% of total)
Ported lines: 138530/142758 (97.0% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Apr 03 2023 at 19:09):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 378/397 (95.2% of total)
Ported lines: 142685/150288 (94.9% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Apr 03 2023 at 19:14):

mathlib port progress topology.continuous_function.bounded
Ported files: 661/689 (95.9% of total)
Ported lines: 281509/299400 (94.0% of total)
Longest unported chain: 8/85 (90.6% progress)

port-progress bot (Apr 03 2023 at 19:18):

mathlib port progress linear_algebra.determinant
Ported files: 607/646 (94.0% of total)
Ported lines: 248406/264678 (93.9% of total)
Longest unported chain: 12/74 (83.8% progress)

port-progress bot (Apr 03 2023 at 19:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 661/701 (94.3% of total)
Ported lines: 280952/309005 (90.9% of total)
Longest unported chain: 10/87 (88.5% progress)

port-progress bot (Apr 03 2023 at 19:27):

mathlib port progress category_theory.monoidal.tor
Ported files: 367/395 (92.9% of total)
Ported lines: 139946/150700 (92.9% of total)
Longest unported chain: 14/56 (75.0% progress)

port-progress bot (Apr 03 2023 at 19:32):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 793/901 (88.0% of total)
Ported lines: 340264/393428 (86.5% of total)
Longest unported chain: 20/91 (78.0% progress)

port-progress bot (Apr 03 2023 at 19:37):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 824/973 (84.7% of total)
Ported lines: 347023/428262 (81.0% of total)
Longest unported chain: 27/99 (72.7% progress)

port-progress bot (Apr 03 2023 at 19:42):

mathlib port progress combinatorics.additive.behrend
Ported files: 826/978 (84.5% of total)
Ported lines: 347854/430173 (80.9% of total)
Longest unported chain: 28/100 (72.0% progress)

port-progress bot (Apr 03 2023 at 19:47):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 849/1042 (81.5% of total)
Ported lines: 350878/441397 (79.5% of total)
Longest unported chain: 34/96 (64.6% progress)

port-progress bot (Apr 03 2023 at 19:52):

mathlib port progress measure_theory.integral.bochner
Ported files: 842/1018 (82.7% of total)
Ported lines: 354781/463033 (76.6% of total)
Longest unported chain: 32/104 (69.2% progress)

port-progress bot (Apr 03 2023 at 19:57):

mathlib port progress probability.independence
Ported files: 845/1033 (81.8% of total)
Ported lines: 355154/470744 (75.4% of total)
Longest unported chain: 37/109 (66.1% progress)

port-progress bot (Apr 03 2023 at 20:03):

mathlib port progress all
Ported files: 1521/2923 (52.0% of total)
Ported lines: 507872/1012627 (50.2% of total)
Longest unported chain: 52/124 (58.1% progress)

Scott Morrison (Apr 03 2023 at 20:03):

Over 50%!

Scott Morrison (Apr 03 2023 at 20:03):

0.5%

port-progress bot (Apr 04 2023 at 19:04):

mathlib port progress category_theory.abelian.basic
Ported files: 362/371 (97.6% of total)
Ported lines: 138564/142792 (97.0% of total)
Longest unported chain: 1/47 (97.9% progress)

port-progress bot (Apr 04 2023 at 19:07):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 378/397 (95.2% of total)
Ported lines: 142719/150322 (94.9% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Apr 04 2023 at 19:11):

mathlib port progress topology.continuous_function.bounded
Ported files: 662/689 (96.1% of total)
Ported lines: 283665/299449 (94.7% of total)
Longest unported chain: 7/85 (91.8% progress)

port-progress bot (Apr 04 2023 at 19:15):

mathlib port progress linear_algebra.determinant
Ported files: 609/646 (94.3% of total)
Ported lines: 248775/264721 (94.0% of total)
Longest unported chain: 11/74 (85.1% progress)

port-progress bot (Apr 04 2023 at 19:19):

mathlib port progress analysis.calculus.fderiv
Ported files: 662/701 (94.4% of total)
Ported lines: 283108/309054 (91.6% of total)
Longest unported chain: 9/87 (89.7% progress)

port-progress bot (Apr 04 2023 at 19:23):

mathlib port progress category_theory.monoidal.tor
Ported files: 367/395 (92.9% of total)
Ported lines: 139980/150734 (92.9% of total)
Longest unported chain: 14/56 (75.0% progress)

port-progress bot (Apr 04 2023 at 19:27):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 796/901 (88.3% of total)
Ported lines: 342740/393648 (87.1% of total)
Longest unported chain: 19/91 (79.1% progress)

port-progress bot (Apr 04 2023 at 19:31):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 827/973 (85.0% of total)
Ported lines: 349499/428482 (81.6% of total)
Longest unported chain: 26/99 (73.7% progress)

port-progress bot (Apr 04 2023 at 19:35):

mathlib port progress combinatorics.additive.behrend
Ported files: 829/978 (84.8% of total)
Ported lines: 350330/430393 (81.4% of total)
Longest unported chain: 27/100 (73.0% progress)

port-progress bot (Apr 04 2023 at 19:39):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 853/1042 (81.9% of total)
Ported lines: 353997/441442 (80.2% of total)
Longest unported chain: 33/96 (65.6% progress)

port-progress bot (Apr 04 2023 at 19:44):

mathlib port progress measure_theory.integral.bochner
Ported files: 845/1018 (83.0% of total)
Ported lines: 357257/463077 (77.1% of total)
Longest unported chain: 31/104 (70.2% progress)

port-progress bot (Apr 04 2023 at 19:47):

mathlib port progress probability.independence
Ported files: 848/1033 (82.1% of total)
Ported lines: 357630/470971 (75.9% of total)
Longest unported chain: 36/109 (67.0% progress)

port-progress bot (Apr 04 2023 at 19:52):

mathlib port progress all
Ported files: 1533/2923 (52.4% of total)
Ported lines: 511828/1013033 (50.5% of total)
Longest unported chain: 51/124 (58.9% progress)

Johan Commelin (Apr 04 2023 at 19:56):

0.3%

port-progress bot (Apr 05 2023 at 19:05):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 379/397 (95.5% of total)
Ported lines: 143362/150355 (95.3% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Apr 05 2023 at 19:09):

mathlib port progress topology.continuous_function.bounded
Ported files: 663/689 (96.2% of total)
Ported lines: 283888/299497 (94.8% of total)
Longest unported chain: 7/85 (91.8% progress)

port-progress bot (Apr 05 2023 at 19:14):

mathlib port progress linear_algebra.determinant
Ported files: 610/646 (94.4% of total)
Ported lines: 249494/264768 (94.2% of total)
Longest unported chain: 11/74 (85.1% progress)

port-progress bot (Apr 05 2023 at 19:19):

mathlib port progress analysis.calculus.fderiv
Ported files: 663/701 (94.6% of total)
Ported lines: 283331/309102 (91.7% of total)
Longest unported chain: 9/87 (89.7% progress)

port-progress bot (Apr 05 2023 at 19:23):

mathlib port progress category_theory.monoidal.tor
Ported files: 367/395 (92.9% of total)
Ported lines: 140013/150767 (92.9% of total)
Longest unported chain: 14/56 (75.0% progress)

port-progress bot (Apr 05 2023 at 19:28):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 800/901 (88.8% of total)
Ported lines: 343794/393713 (87.3% of total)
Longest unported chain: 19/91 (79.1% progress)

port-progress bot (Apr 05 2023 at 19:32):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 832/973 (85.5% of total)
Ported lines: 351070/428547 (81.9% of total)
Longest unported chain: 26/99 (73.7% progress)

port-progress bot (Apr 05 2023 at 19:37):

mathlib port progress combinatorics.additive.behrend
Ported files: 834/978 (85.3% of total)
Ported lines: 351901/430458 (81.8% of total)
Longest unported chain: 27/100 (73.0% progress)

port-progress bot (Apr 05 2023 at 19:42):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 859/1042 (82.4% of total)
Ported lines: 355649/441530 (80.5% of total)
Longest unported chain: 34/97 (64.9% progress)

port-progress bot (Apr 05 2023 at 19:47):

mathlib port progress measure_theory.integral.bochner
Ported files: 850/1018 (83.5% of total)
Ported lines: 358828/463142 (77.5% of total)
Longest unported chain: 31/104 (70.2% progress)

port-progress bot (Apr 05 2023 at 19:52):

mathlib port progress probability.independence
Ported files: 853/1033 (82.6% of total)
Ported lines: 359201/471036 (76.3% of total)
Longest unported chain: 36/109 (67.0% progress)

port-progress bot (Apr 05 2023 at 19:57):

mathlib port progress all
Ported files: 1552/2924 (53.1% of total)
Ported lines: 516635/1013332 (51.0% of total)
Longest unported chain: 51/124 (58.9% progress)

Scott Morrison (Apr 05 2023 at 22:00):

0.5%

Ruben Van de Velde (Apr 06 2023 at 13:55):

Whoa, Data.Vector3 (!4#633 !4#1204) is on the queue!

Eric Wieser (Apr 06 2023 at 14:12):

I'm inclined to say we should take it off the queue and check that the latest mathport output is still reasonable

Eric Wieser (Apr 06 2023 at 14:30):

Yep, this PR had some misnamed lemmas that new mathport fixed automatically

Eric Wieser (Apr 06 2023 at 14:31):

I think we should be wary of stale PRs, and prefer to run start_port.sh again and merge the output when reviving them

Matthew Ballard (Apr 07 2023 at 00:23):

Where is the bot?

Jeremy Tan (Apr 07 2023 at 01:34):

@Scott Morrison your bot is probably down

Scott Morrison (Apr 07 2023 at 03:20):

Sorry, that server is not available at the moment. Johan says he is likely to be able to provide a substitute.

Johan Commelin (Apr 07 2023 at 07:24):

Yes, I'll run it now!

Johan Commelin (Apr 07 2023 at 07:28):

Ooh, I should first get an up to date list of targets.

port progress bot (jmc) (Apr 07 2023 at 08:38):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 379/397 (95.5% of total)
Ported lines: 143365/150358 (95.3% of total)
Longest unported chain: 6/52 (88.5% progress)

port progress bot (jmc) (Apr 07 2023 at 08:41):

mathlib port progress topology.continuous_function.bounded
Ported files: 664/689 (96.4% of total)
Ported lines: 284316/299506 (94.9% of total)
Longest unported chain: 7/85 (91.8% progress)

port progress bot (jmc) (Apr 07 2023 at 08:44):

mathlib port progress linear_algebra.determinant
Ported files: 611/646 (94.6% of total)
Ported lines: 249785/264800 (94.3% of total)
Longest unported chain: 10/74 (86.5% progress)

port progress bot (jmc) (Apr 07 2023 at 08:46):

mathlib port progress analysis.calculus.fderiv
Ported files: 665/701 (94.9% of total)
Ported lines: 284353/309111 (92.0% of total)
Longest unported chain: 9/87 (89.7% progress)

port progress bot (jmc) (Apr 07 2023 at 08:48):

mathlib port progress category_theory.monoidal.tor
Ported files: 367/395 (92.9% of total)
Ported lines: 140013/150767 (92.9% of total)
Longest unported chain: 14/56 (75.0% progress)

port progress bot (jmc) (Apr 07 2023 at 08:51):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 805/901 (89.3% of total)
Ported lines: 345340/393754 (87.7% of total)
Longest unported chain: 18/91 (80.2% progress)

port progress bot (jmc) (Apr 07 2023 at 08:54):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 837/973 (86.0% of total)
Ported lines: 352619/428591 (82.3% of total)
Longest unported chain: 25/99 (74.7% progress)

port progress bot (jmc) (Apr 07 2023 at 08:57):

mathlib port progress combinatorics.additive.behrend
Ported files: 839/978 (85.8% of total)
Ported lines: 353450/430502 (82.1% of total)
Longest unported chain: 26/100 (74.0% progress)

port progress bot (jmc) (Apr 07 2023 at 09:00):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 865/1042 (83.0% of total)
Ported lines: 357188/441580 (80.9% of total)
Longest unported chain: 33/97 (66.0% progress)

port progress bot (jmc) (Apr 07 2023 at 09:03):

mathlib port progress measure_theory.integral.bochner
Ported files: 855/1018 (84.0% of total)
Ported lines: 360377/463186 (77.8% of total)
Longest unported chain: 30/104 (71.2% progress)

port progress bot (jmc) (Apr 07 2023 at 09:05):

mathlib port progress probability.independence
Ported files: 858/1033 (83.1% of total)
Ported lines: 360750/471080 (76.6% of total)
Longest unported chain: 35/109 (67.9% progress)

port progress bot (jmc) (Apr 07 2023 at 10:19):

mathlib port progress all
Ported files: 1571/2925 (53.7% of total)
Ported lines: 521885/1013608 (51.5% of total)
Longest unported chain: 50/124 (59.7% progress)

Johan Commelin (Apr 07 2023 at 10:36):

0.5%

Notification Bot (Apr 07 2023 at 12:06):

Eric Rodriguez has marked this topic as resolved.

Notification Bot (Apr 07 2023 at 12:07):

Jeremy Tan has marked this topic as unresolved.

Jeremy Tan (Apr 07 2023 at 15:40):

@Johan Commelin at what time is your version of the port progress bot running?

Johan Commelin (Apr 07 2023 at 17:08):

The rest of the week it should run at 05:00 UTC, if everything goes as planned.

Jeremy Tan (Apr 08 2023 at 09:16):

@Johan Commelin it didn't run

Jeremy Tan (Apr 08 2023 at 09:17):

(well, it generated the files but didn't post here)

Jeremy Tan (Apr 08 2023 at 09:17):

https://math.commelin.net/files/mathlib4/2023-04-08/probability.independence.pdf

Johan Commelin (Apr 08 2023 at 09:46):

Hmm, I'm not sure what happened. I just started the script manually, so hopefully the stats will appear in a few minutes.

port progress bot (jmc) (Apr 08 2023 at 09:48):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 379/397 (95.5% of total)
Ported lines: 143368/150361 (95.3% of total)
Longest unported chain: 6/52 (88.5% progress)

port progress bot (jmc) (Apr 08 2023 at 09:51):

mathlib port progress topology.continuous_function.bounded
Ported files: 665/689 (96.5% of total)
Ported lines: 284542/299523 (95.0% of total)
Longest unported chain: 7/85 (91.8% progress)

port progress bot (jmc) (Apr 08 2023 at 09:54):

mathlib port progress linear_algebra.determinant
Ported files: 619/646 (95.8% of total)
Ported lines: 252160/264817 (95.2% of total)
Longest unported chain: 7/74 (90.5% progress)

port progress bot (jmc) (Apr 08 2023 at 09:56):

mathlib port progress analysis.calculus.fderiv
Ported files: 667/701 (95.1% of total)
Ported lines: 286944/309128 (92.8% of total)
Longest unported chain: 9/87 (89.7% progress)

port progress bot (jmc) (Apr 08 2023 at 09:59):

mathlib port progress category_theory.monoidal.tor
Ported files: 367/395 (92.9% of total)
Ported lines: 140016/150770 (92.9% of total)
Longest unported chain: 14/56 (75.0% progress)

port progress bot (jmc) (Apr 08 2023 at 10:01):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 817/901 (90.7% of total)
Ported lines: 350739/393771 (89.1% of total)
Longest unported chain: 15/91 (83.5% progress)

port progress bot (jmc) (Apr 08 2023 at 10:04):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 849/973 (87.3% of total)
Ported lines: 358018/428608 (83.5% of total)
Longest unported chain: 22/99 (77.8% progress)

port progress bot (jmc) (Apr 08 2023 at 10:07):

mathlib port progress combinatorics.additive.behrend
Ported files: 851/978 (87.0% of total)
Ported lines: 358849/430519 (83.4% of total)
Longest unported chain: 23/100 (77.0% progress)

port progress bot (jmc) (Apr 08 2023 at 10:10):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 877/1042 (84.2% of total)
Ported lines: 362587/441597 (82.1% of total)
Longest unported chain: 30/97 (69.1% progress)

port progress bot (jmc) (Apr 08 2023 at 10:13):

mathlib port progress measure_theory.integral.bochner
Ported files: 867/1018 (85.2% of total)
Ported lines: 365776/463203 (79.0% of total)
Longest unported chain: 27/104 (74.0% progress)

port progress bot (jmc) (Apr 08 2023 at 10:15):

mathlib port progress probability.independence
Ported files: 870/1033 (84.2% of total)
Ported lines: 366149/471097 (77.7% of total)
Longest unported chain: 32/109 (70.6% progress)

port progress bot (jmc) (Apr 08 2023 at 10:18):

mathlib port progress all
Ported files: 1588/2925 (54.3% of total)
Ported lines: 528077/1013777 (52.1% of total)
Longest unported chain: 47/124 (62.1% progress)

Johan Commelin (Apr 08 2023 at 10:47):

0.6%

port progress bot (jmc) (Apr 09 2023 at 07:27):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 379/397 (95.5% of total)
Ported lines: 143374/150367 (95.3% of total)
Longest unported chain: 6/52 (88.5% progress)

port progress bot (jmc) (Apr 09 2023 at 07:30):

mathlib port progress topology.continuous_function.bounded
Ported files: 665/689 (96.5% of total)
Ported lines: 284548/299529 (95.0% of total)
Longest unported chain: 7/85 (91.8% progress)

port progress bot (jmc) (Apr 09 2023 at 07:33):

mathlib port progress linear_algebra.determinant
Ported files: 619/646 (95.8% of total)
Ported lines: 252187/264866 (95.2% of total)
Longest unported chain: 7/74 (90.5% progress)

port progress bot (jmc) (Apr 09 2023 at 07:35):

mathlib port progress analysis.calculus.fderiv
Ported files: 667/701 (95.1% of total)
Ported lines: 286956/309146 (92.8% of total)
Longest unported chain: 9/87 (89.7% progress)

port progress bot (jmc) (Apr 09 2023 at 07:38):

mathlib port progress category_theory.monoidal.tor
Ported files: 367/395 (92.9% of total)
Ported lines: 140022/150776 (92.9% of total)
Longest unported chain: 14/56 (75.0% progress)

port progress bot (jmc) (Apr 09 2023 at 07:40):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 817/901 (90.7% of total)
Ported lines: 350790/393884 (89.1% of total)
Longest unported chain: 15/91 (83.5% progress)

port progress bot (jmc) (Apr 09 2023 at 07:43):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 849/973 (87.3% of total)
Ported lines: 358069/428722 (83.5% of total)
Longest unported chain: 22/99 (77.8% progress)

port progress bot (jmc) (Apr 09 2023 at 07:46):

mathlib port progress combinatorics.additive.behrend
Ported files: 851/978 (87.0% of total)
Ported lines: 358900/430633 (83.3% of total)
Longest unported chain: 23/100 (77.0% progress)

port progress bot (jmc) (Apr 09 2023 at 07:49):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 877/1042 (84.2% of total)
Ported lines: 362638/441676 (82.1% of total)
Longest unported chain: 30/97 (69.1% progress)

port progress bot (jmc) (Apr 09 2023 at 07:51):

mathlib port progress measure_theory.integral.bochner
Ported files: 867/1018 (85.2% of total)
Ported lines: 365827/463283 (79.0% of total)
Longest unported chain: 27/104 (74.0% progress)

port progress bot (jmc) (Apr 09 2023 at 07:54):

mathlib port progress probability.independence
Ported files: 870/1033 (84.2% of total)
Ported lines: 366200/471177 (77.7% of total)
Longest unported chain: 32/109 (70.6% progress)

port progress bot (jmc) (Apr 09 2023 at 07:57):

mathlib port progress all
Ported files: 1591/2925 (54.4% of total)
Ported lines: 528798/1013961 (52.2% of total)
Longest unported chain: 47/124 (62.1% progress)

Scott Morrison (Apr 09 2023 at 08:10):

0.1%

port progress bot (jmc) (Apr 10 2023 at 07:02):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 379/397 (95.5% of total)
Ported lines: 143374/150367 (95.3% of total)
Longest unported chain: 6/52 (88.5% progress)

port progress bot (jmc) (Apr 10 2023 at 07:04):

mathlib port progress topology.continuous_function.bounded
Ported files: 665/689 (96.5% of total)
Ported lines: 284548/299529 (95.0% of total)
Longest unported chain: 7/85 (91.8% progress)

port progress bot (jmc) (Apr 10 2023 at 07:07):

mathlib port progress linear_algebra.determinant
Ported files: 619/645 (96.0% of total)
Ported lines: 252187/264762 (95.3% of total)
Longest unported chain: 6/74 (91.9% progress)

port progress bot (jmc) (Apr 10 2023 at 07:09):

mathlib port progress analysis.calculus.fderiv
Ported files: 667/701 (95.1% of total)
Ported lines: 286956/309146 (92.8% of total)
Longest unported chain: 9/87 (89.7% progress)

port progress bot (jmc) (Apr 10 2023 at 07:12):

mathlib port progress category_theory.monoidal.tor
Ported files: 367/395 (92.9% of total)
Ported lines: 140022/150776 (92.9% of total)
Longest unported chain: 14/56 (75.0% progress)

port progress bot (jmc) (Apr 10 2023 at 07:14):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 817/902 (90.6% of total)
Ported lines: 350790/393931 (89.0% of total)
Longest unported chain: 14/91 (84.6% progress)

port progress bot (jmc) (Apr 10 2023 at 07:17):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 849/974 (87.2% of total)
Ported lines: 358069/428769 (83.5% of total)
Longest unported chain: 21/99 (78.8% progress)

port progress bot (jmc) (Apr 10 2023 at 07:20):

mathlib port progress combinatorics.additive.behrend
Ported files: 851/979 (86.9% of total)
Ported lines: 358900/430680 (83.3% of total)
Longest unported chain: 22/100 (78.0% progress)

port progress bot (jmc) (Apr 10 2023 at 07:23):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 877/1043 (84.1% of total)
Ported lines: 362638/441724 (82.1% of total)
Longest unported chain: 30/97 (69.1% progress)

port progress bot (jmc) (Apr 10 2023 at 07:25):

mathlib port progress measure_theory.integral.bochner
Ported files: 867/1019 (85.1% of total)
Ported lines: 365827/463330 (79.0% of total)
Longest unported chain: 26/104 (75.0% progress)

port progress bot (jmc) (Apr 10 2023 at 07:28):

mathlib port progress probability.independence
Ported files: 870/1034 (84.1% of total)
Ported lines: 366200/471224 (77.7% of total)
Longest unported chain: 31/109 (71.6% progress)

port progress bot (jmc) (Apr 10 2023 at 07:31):

mathlib port progress all
Ported files: 1591/2925 (54.4% of total)
Ported lines: 528798/1013914 (52.2% of total)
Longest unported chain: 46/124 (62.9% progress)

Johan Commelin (Apr 10 2023 at 07:33):

0.0%

Jeremy Tan (Apr 11 2023 at 06:40):

Where is the bot again?

Johan Commelin (Apr 11 2023 at 13:57):

Sorry, I was travelling. I don't know why the cronjob on my server is failing. I'll login to give it a kick.

Johan Commelin (Apr 11 2023 at 13:58):

It's running again. It should start posting stats in ~15 mins.

port progress bot (jmc) (Apr 11 2023 at 14:29):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 380/397 (95.7% of total)
Ported lines: 143722/150362 (95.6% of total)
Longest unported chain: 6/52 (88.5% progress)

port progress bot (jmc) (Apr 11 2023 at 14:32):

mathlib port progress topology.continuous_function.bounded
Ported files: 666/689 (96.7% of total)
Ported lines: 285507/299524 (95.3% of total)
Longest unported chain: 7/85 (91.8% progress)

port progress bot (jmc) (Apr 11 2023 at 14:34):

mathlib port progress linear_algebra.determinant
Ported files: 623/645 (96.6% of total)
Ported lines: 254833/264766 (96.2% of total)
Longest unported chain: 6/74 (91.9% progress)

port progress bot (jmc) (Apr 11 2023 at 14:37):

mathlib port progress analysis.calculus.fderiv
Ported files: 668/701 (95.3% of total)
Ported lines: 287915/309141 (93.1% of total)
Longest unported chain: 9/87 (89.7% progress)

port progress bot (jmc) (Apr 11 2023 at 14:39):

mathlib port progress category_theory.monoidal.tor
Ported files: 368/395 (93.2% of total)
Ported lines: 140215/150768 (93.0% of total)
Longest unported chain: 14/56 (75.0% progress)

port progress bot (jmc) (Apr 11 2023 at 14:42):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 822/902 (91.1% of total)
Ported lines: 354403/393938 (90.0% of total)
Longest unported chain: 14/91 (84.6% progress)

port progress bot (jmc) (Apr 11 2023 at 14:45):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 856/974 (87.9% of total)
Ported lines: 362727/428805 (84.6% of total)
Longest unported chain: 21/99 (78.8% progress)

port progress bot (jmc) (Apr 11 2023 at 14:48):

mathlib port progress combinatorics.additive.behrend
Ported files: 858/979 (87.6% of total)
Ported lines: 363558/430716 (84.4% of total)
Longest unported chain: 22/100 (78.0% progress)

port progress bot (jmc) (Apr 11 2023 at 14:50):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 883/1043 (84.7% of total)
Ported lines: 367060/441731 (83.1% of total)
Longest unported chain: 29/97 (70.1% progress)

port progress bot (jmc) (Apr 11 2023 at 14:53):

mathlib port progress measure_theory.integral.bochner
Ported files: 874/1019 (85.8% of total)
Ported lines: 370485/463467 (79.9% of total)
Longest unported chain: 26/104 (75.0% progress)

port progress bot (jmc) (Apr 11 2023 at 14:56):

mathlib port progress probability.independence
Ported files: 877/1034 (84.8% of total)
Ported lines: 370858/471361 (78.7% of total)
Longest unported chain: 31/109 (71.6% progress)

port progress bot (jmc) (Apr 11 2023 at 14:59):

mathlib port progress all
Ported files: 1626/2925 (55.6% of total)
Ported lines: 542795/1014354 (53.5% of total)
Longest unported chain: 46/124 (62.9% progress)

Johan Commelin (Apr 11 2023 at 15:59):

1.3%

Ruben Van de Velde (Apr 11 2023 at 16:02):

Thanks to the tireless reviewers!

Jeremy Tan (Apr 12 2023 at 14:47):

The bot didn't run again – or has it shifted to the original 2am UTC+8 time it ran when Scott ran the bot?

port progress bot (jmc) (Apr 12 2023 at 18:43):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 380/397 (95.7% of total)
Ported lines: 143722/150362 (95.6% of total)
Longest unported chain: 6/52 (88.5% progress)

port progress bot (jmc) (Apr 12 2023 at 18:45):

mathlib port progress topology.continuous_function.bounded
Ported files: 668/689 (97.0% of total)
Ported lines: 286405/299538 (95.6% of total)
Longest unported chain: 6/85 (92.9% progress)

port progress bot (jmc) (Apr 12 2023 at 18:48):

mathlib port progress linear_algebra.determinant
Ported files: 623/645 (96.6% of total)
Ported lines: 254854/264796 (96.2% of total)
Longest unported chain: 6/74 (91.9% progress)

port progress bot (jmc) (Apr 12 2023 at 18:50):

mathlib port progress analysis.calculus.fderiv
Ported files: 673/701 (96.0% of total)
Ported lines: 291008/309158 (94.1% of total)
Longest unported chain: 8/87 (90.8% progress)

port progress bot (jmc) (Apr 12 2023 at 18:53):

mathlib port progress category_theory.monoidal.tor
Ported files: 368/395 (93.2% of total)
Ported lines: 140218/150771 (93.0% of total)
Longest unported chain: 14/56 (75.0% progress)

port progress bot (jmc) (Apr 12 2023 at 18:55):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 829/902 (91.9% of total)
Ported lines: 357726/393974 (90.8% of total)
Longest unported chain: 14/91 (84.6% progress)

port progress bot (jmc) (Apr 12 2023 at 18:58):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 863/974 (88.6% of total)
Ported lines: 366056/428847 (85.4% of total)
Longest unported chain: 21/99 (78.8% progress)

port progress bot (jmc) (Apr 12 2023 at 19:01):

mathlib port progress combinatorics.additive.behrend
Ported files: 865/979 (88.4% of total)
Ported lines: 366887/430758 (85.2% of total)
Longest unported chain: 22/100 (78.0% progress)

port progress bot (jmc) (Apr 12 2023 at 19:04):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 890/1043 (85.3% of total)
Ported lines: 370513/441773 (83.9% of total)
Longest unported chain: 29/97 (70.1% progress)

port progress bot (jmc) (Apr 12 2023 at 19:06):

mathlib port progress measure_theory.integral.bochner
Ported files: 881/1019 (86.5% of total)
Ported lines: 373814/463509 (80.6% of total)
Longest unported chain: 26/104 (75.0% progress)

port progress bot (jmc) (Apr 12 2023 at 19:09):

mathlib port progress probability.independence
Ported files: 884/1034 (85.5% of total)
Ported lines: 374187/471403 (79.4% of total)
Longest unported chain: 31/109 (71.6% progress)

port progress bot (jmc) (Apr 12 2023 at 19:12):

mathlib port progress all
Ported files: 1638/2925 (56.0% of total)
Ported lines: 547020/1014460 (53.9% of total)
Longest unported chain: 46/124 (62.9% progress)

Jireh Loreaux (Apr 12 2023 at 19:31):

0.4%

port progress bot (jmc) (Apr 13 2023 at 21:10):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 381/397 (96.0% of total)
Ported lines: 144380/150362 (96.0% of total)
Longest unported chain: 6/52 (88.5% progress)

port progress bot (jmc) (Apr 13 2023 at 21:13):

mathlib port progress topology.continuous_function.bounded
Ported files: 671/689 (97.4% of total)
Ported lines: 288767/299547 (96.4% of total)
Longest unported chain: 6/85 (92.9% progress)

port progress bot (jmc) (Apr 13 2023 at 21:15):

mathlib port progress linear_algebra.determinant
Ported files: 624/645 (96.7% of total)
Ported lines: 255405/264846 (96.4% of total)
Longest unported chain: 6/74 (91.9% progress)

port progress bot (jmc) (Apr 13 2023 at 21:18):

mathlib port progress analysis.calculus.fderiv
Ported files: 674/701 (96.1% of total)
Ported lines: 291272/309167 (94.2% of total)
Longest unported chain: 8/87 (90.8% progress)

port progress bot (jmc) (Apr 13 2023 at 21:20):

mathlib port progress category_theory.monoidal.tor
Ported files: 368/395 (93.2% of total)
Ported lines: 140218/150771 (93.0% of total)
Longest unported chain: 14/56 (75.0% progress)

port progress bot (jmc) (Apr 13 2023 at 21:22):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 831/902 (92.1% of total)
Ported lines: 358547/394039 (91.0% of total)
Longest unported chain: 14/91 (84.6% progress)

port progress bot (jmc) (Apr 13 2023 at 21:25):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 866/974 (88.9% of total)
Ported lines: 367071/428912 (85.6% of total)
Longest unported chain: 21/99 (78.8% progress)

port progress bot (jmc) (Apr 13 2023 at 21:28):

mathlib port progress combinatorics.additive.behrend
Ported files: 868/979 (88.7% of total)
Ported lines: 367902/430823 (85.4% of total)
Longest unported chain: 22/100 (78.0% progress)

port progress bot (jmc) (Apr 13 2023 at 21:31):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 893/1043 (85.6% of total)
Ported lines: 371525/441835 (84.1% of total)
Longest unported chain: 29/97 (70.1% progress)

port progress bot (jmc) (Apr 13 2023 at 21:34):

mathlib port progress measure_theory.integral.bochner
Ported files: 884/1019 (86.8% of total)
Ported lines: 374829/463574 (80.9% of total)
Longest unported chain: 26/104 (75.0% progress)

port progress bot (jmc) (Apr 13 2023 at 21:36):

mathlib port progress probability.independence
Ported files: 887/1034 (85.8% of total)
Ported lines: 375202/471468 (79.6% of total)
Longest unported chain: 31/109 (71.6% progress)

port progress bot (jmc) (Apr 13 2023 at 21:39):

mathlib port progress all
Ported files: 1647/2925 (56.3% of total)
Ported lines: 549858/1014563 (54.2% of total)
Longest unported chain: 46/124 (62.9% progress)

Moritz Doll (Apr 14 2023 at 00:10):

0.3%

port progress bot (jmc) (Apr 14 2023 at 05:39):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 381/397 (96.0% of total)
Ported lines: 144380/150362 (96.0% of total)
Longest unported chain: 6/52 (88.5% progress)

port progress bot (jmc) (Apr 14 2023 at 05:42):

mathlib port progress topology.continuous_function.bounded
Ported files: 671/689 (97.4% of total)
Ported lines: 288767/299550 (96.4% of total)
Longest unported chain: 6/85 (92.9% progress)

port progress bot (jmc) (Apr 14 2023 at 05:44):

mathlib port progress linear_algebra.determinant
Ported files: 624/645 (96.7% of total)
Ported lines: 255405/264846 (96.4% of total)
Longest unported chain: 6/74 (91.9% progress)

port progress bot (jmc) (Apr 14 2023 at 05:47):

mathlib port progress analysis.calculus.fderiv
Ported files: 674/701 (96.1% of total)
Ported lines: 291272/309170 (94.2% of total)
Longest unported chain: 8/87 (90.8% progress)

port progress bot (jmc) (Apr 14 2023 at 05:49):

mathlib port progress category_theory.monoidal.tor
Ported files: 368/395 (93.2% of total)
Ported lines: 140218/150771 (93.0% of total)
Longest unported chain: 14/56 (75.0% progress)

port progress bot (jmc) (Apr 14 2023 at 05:52):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 831/902 (92.1% of total)
Ported lines: 358547/394042 (91.0% of total)
Longest unported chain: 14/91 (84.6% progress)

port progress bot (jmc) (Apr 14 2023 at 05:54):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 866/974 (88.9% of total)
Ported lines: 367071/428915 (85.6% of total)
Longest unported chain: 21/99 (78.8% progress)

port progress bot (jmc) (Apr 14 2023 at 05:57):

mathlib port progress combinatorics.additive.behrend
Ported files: 868/979 (88.7% of total)
Ported lines: 367902/430826 (85.4% of total)
Longest unported chain: 22/100 (78.0% progress)

port progress bot (jmc) (Apr 14 2023 at 06:00):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 893/1043 (85.6% of total)
Ported lines: 371525/441838 (84.1% of total)
Longest unported chain: 29/97 (70.1% progress)

port progress bot (jmc) (Apr 14 2023 at 06:03):

mathlib port progress measure_theory.integral.bochner
Ported files: 884/1019 (86.8% of total)
Ported lines: 374829/463577 (80.9% of total)
Longest unported chain: 26/104 (75.0% progress)

port progress bot (jmc) (Apr 14 2023 at 06:05):

mathlib port progress probability.independence
Ported files: 887/1034 (85.8% of total)
Ported lines: 375202/471471 (79.6% of total)
Longest unported chain: 31/109 (71.6% progress)

port progress bot (jmc) (Apr 14 2023 at 06:09):

mathlib port progress all
Ported files: 1647/2925 (56.3% of total)
Ported lines: 549858/1014621 (54.2% of total)
Longest unported chain: 46/124 (62.9% progress)

Scott Morrison (Apr 14 2023 at 08:11):

Not sure if I should say 0.0%, since that was the second run today?

Johan Commelin (Apr 14 2023 at 08:21):

Yeah the one yesterday night was really late. Running in the morning is somehow what should have happened.

port progress bot (jmc) (Apr 15 2023 at 17:00):

mathlib port progress topology.continuous_function.bounded
Ported files: 671/689 (97.4% of total)
Ported lines: 288770/299553 (96.4% of total)
Longest unported chain: 6/85 (92.9% progress)

port progress bot (jmc) (Apr 15 2023 at 17:03):

mathlib port progress linear_algebra.determinant
Ported files: 625/645 (96.9% of total)
Ported lines: 255590/264970 (96.5% of total)
Longest unported chain: 6/74 (91.9% progress)

port progress bot (jmc) (Apr 15 2023 at 17:05):

mathlib port progress analysis.calculus.fderiv
Ported files: 674/701 (96.1% of total)
Ported lines: 291275/309173 (94.2% of total)
Longest unported chain: 8/87 (90.8% progress)

port progress bot (jmc) (Apr 15 2023 at 17:08):

mathlib port progress category_theory.monoidal.tor
Ported files: 370/395 (93.7% of total)
Ported lines: 140771/150774 (93.4% of total)
Longest unported chain: 13/56 (76.8% progress)

port progress bot (jmc) (Apr 15 2023 at 17:10):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 832/902 (92.2% of total)
Ported lines: 358735/394169 (91.0% of total)
Longest unported chain: 14/91 (84.6% progress)

port progress bot (jmc) (Apr 15 2023 at 17:13):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 867/974 (89.0% of total)
Ported lines: 367262/429067 (85.6% of total)
Longest unported chain: 21/99 (78.8% progress)

port progress bot (jmc) (Apr 15 2023 at 17:16):

mathlib port progress combinatorics.additive.behrend
Ported files: 869/979 (88.8% of total)
Ported lines: 368093/430978 (85.4% of total)
Longest unported chain: 22/100 (78.0% progress)

port progress bot (jmc) (Apr 15 2023 at 17:18):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 894/1043 (85.7% of total)
Ported lines: 371716/441968 (84.1% of total)
Longest unported chain: 28/97 (71.1% progress)

port progress bot (jmc) (Apr 15 2023 at 17:21):

mathlib port progress measure_theory.integral.bochner
Ported files: 885/1019 (86.8% of total)
Ported lines: 375020/463729 (80.9% of total)
Longest unported chain: 26/104 (75.0% progress)

port progress bot (jmc) (Apr 15 2023 at 17:24):

mathlib port progress probability.independence
Ported files: 888/1034 (85.9% of total)
Ported lines: 375393/471623 (79.6% of total)
Longest unported chain: 31/109 (71.6% progress)

port progress bot (jmc) (Apr 15 2023 at 17:27):

mathlib port progress all
Ported files: 1657/2925 (56.6% of total)
Ported lines: 553285/1014824 (54.5% of total)
Longest unported chain: 46/124 (62.9% progress)

Johan Commelin (Apr 15 2023 at 17:29):

0.3%

port progress bot (jmc) (Apr 16 2023 at 16:03):

mathlib port progress topology.continuous_function.bounded
Ported files: 671/689 (97.4% of total)
Ported lines: 288770/299553 (96.4% of total)
Longest unported chain: 6/85 (92.9% progress)

port progress bot (jmc) (Apr 16 2023 at 16:05):

mathlib port progress linear_algebra.determinant
Ported files: 626/645 (97.1% of total)
Ported lines: 255786/264970 (96.5% of total)
Longest unported chain: 6/74 (91.9% progress)

port progress bot (jmc) (Apr 16 2023 at 16:08):

mathlib port progress analysis.calculus.fderiv
Ported files: 674/701 (96.1% of total)
Ported lines: 291275/309173 (94.2% of total)
Longest unported chain: 8/87 (90.8% progress)

port progress bot (jmc) (Apr 16 2023 at 16:10):

mathlib port progress category_theory.monoidal.tor
Ported files: 370/395 (93.7% of total)
Ported lines: 140771/150774 (93.4% of total)
Longest unported chain: 13/56 (76.8% progress)

port progress bot (jmc) (Apr 16 2023 at 16:12):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 833/902 (92.4% of total)
Ported lines: 358931/394169 (91.1% of total)
Longest unported chain: 14/91 (84.6% progress)

port progress bot (jmc) (Apr 16 2023 at 16:15):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 868/974 (89.1% of total)
Ported lines: 367458/429067 (85.6% of total)
Longest unported chain: 21/99 (78.8% progress)

port progress bot (jmc) (Apr 16 2023 at 16:18):

mathlib port progress combinatorics.additive.behrend
Ported files: 870/979 (88.9% of total)
Ported lines: 368289/430978 (85.5% of total)
Longest unported chain: 22/100 (78.0% progress)

port progress bot (jmc) (Apr 16 2023 at 16:21):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 895/1043 (85.8% of total)
Ported lines: 371912/441968 (84.1% of total)
Longest unported chain: 27/97 (72.2% progress)

port progress bot (jmc) (Apr 16 2023 at 16:23):

mathlib port progress measure_theory.integral.bochner
Ported files: 886/1019 (86.9% of total)
Ported lines: 375216/463729 (80.9% of total)
Longest unported chain: 26/104 (75.0% progress)

port progress bot (jmc) (Apr 16 2023 at 16:26):

mathlib port progress probability.independence
Ported files: 889/1034 (86.0% of total)
Ported lines: 375589/471623 (79.6% of total)
Longest unported chain: 31/109 (71.6% progress)

port progress bot (jmc) (Apr 16 2023 at 16:29):

mathlib port progress all
Ported files: 1658/2925 (56.7% of total)
Ported lines: 553481/1014824 (54.5% of total)
Longest unported chain: 46/124 (62.9% progress)

Yaël Dillies (Apr 16 2023 at 16:48):

port progress bot (jmc) said:

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 868/974 (89.1% of total)
Ported lines: 367458/429067 (85.6% of total)
Longest unported chain: 21/99 (78.8% progress)

The linkifier is broken on this one.

Eric Wieser (Apr 16 2023 at 16:50):

This has been raised before

Henrik Böving said:

Why is the L2 part not properly linked O_o

Eric Wieser (Apr 16 2023 at 16:51):

Eric Wieser said:

A copy of the script is at https://github.com/leanprover-community/mathlib-port-status/blob/main/scripts/port-progress-bot.sh, but I have no idea whether it's the version being run by Scott Morrison

Eric Wieser said:

The cause is the capital L not being matched by [0-9a-z_\.]

cc @Scott Morrison / @Johan Commelin, as I believe you have divergent copies of the script on your hard drives

Eric Wieser (Apr 16 2023 at 16:52):

Feel free to push the version you're actually running to the link above

port progress bot (jmc) (Apr 17 2023 at 05:54):

mathlib port progress topology.continuous_function.bounded
Ported files: 671/689 (97.4% of total)
Ported lines: 288770/299553 (96.4% of total)
Longest unported chain: 6/85 (92.9% progress)

Jeremy Tan (Apr 17 2023 at 05:55):

:question:

port progress bot (jmc) (Apr 17 2023 at 05:56):

mathlib port progress linear_algebra.determinant
Ported files: 626/645 (97.1% of total)
Ported lines: 255786/264970 (96.5% of total)
Longest unported chain: 6/74 (91.9% progress)

port progress bot (jmc) (Apr 17 2023 at 05:59):

mathlib port progress analysis.calculus.fderiv
Ported files: 674/701 (96.1% of total)
Ported lines: 291275/309173 (94.2% of total)
Longest unported chain: 8/87 (90.8% progress)

port progress bot (jmc) (Apr 17 2023 at 06:01):

mathlib port progress category_theory.monoidal.tor
Ported files: 370/395 (93.7% of total)
Ported lines: 140771/150774 (93.4% of total)
Longest unported chain: 13/56 (76.8% progress)

port progress bot (jmc) (Apr 17 2023 at 06:04):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 833/902 (92.4% of total)
Ported lines: 358931/394169 (91.1% of total)
Longest unported chain: 14/91 (84.6% progress)

port progress bot (jmc) (Apr 17 2023 at 06:06):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 868/974 (89.1% of total)
Ported lines: 367458/429067 (85.6% of total)
Longest unported chain: 21/99 (78.8% progress)

port progress bot (jmc) (Apr 17 2023 at 06:09):

mathlib port progress combinatorics.additive.behrend
Ported files: 870/979 (88.9% of total)
Ported lines: 368289/430978 (85.5% of total)
Longest unported chain: 22/100 (78.0% progress)

port progress bot (jmc) (Apr 17 2023 at 06:12):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 895/1043 (85.8% of total)
Ported lines: 371912/441968 (84.1% of total)
Longest unported chain: 27/97 (72.2% progress)

port progress bot (jmc) (Apr 17 2023 at 06:15):

mathlib port progress measure_theory.integral.bochner
Ported files: 886/1019 (86.9% of total)
Ported lines: 375216/463729 (80.9% of total)
Longest unported chain: 26/104 (75.0% progress)

port progress bot (jmc) (Apr 17 2023 at 06:17):

mathlib port progress probability.independence
Ported files: 889/1034 (86.0% of total)
Ported lines: 375589/471623 (79.6% of total)
Longest unported chain: 31/109 (71.6% progress)

port progress bot (jmc) (Apr 17 2023 at 06:21):

mathlib port progress all
Ported files: 1659/2925 (56.7% of total)
Ported lines: 553643/1014824 (54.6% of total)
Longest unported chain: 46/124 (62.9% progress)

Scott Morrison (Apr 17 2023 at 06:28):

0.1%

Jeremy Tan (Apr 17 2023 at 06:29):

port progress bot (jmc) said:

mathlib port progress topology.continuous_function.bounded
Ported files: 671/689 (97.4% of total)
Ported lines: 288770/299553 (96.4% of total)
Longest unported chain: 6/85 (92.9% progress)

I starred this one, because !4#3063 seems ready to merge

Jeremy Tan (Apr 17 2023 at 06:43):

Well we always seem to get a backlog of ready PRs on Monday

Scott Morrison (Apr 17 2023 at 06:44):

Hopefully I'll get through some in the next few hours, we'll see. :-)

Jeremy Tan (Apr 18 2023 at 05:37):

image.png This (the open PR count) is the lowest it's been in a long time

Mario Carneiro (Apr 18 2023 at 05:41):

:tada: , but also... that's not a small number :sad:

Sebastian Ullrich (Apr 18 2023 at 12:51):

PR merges are now outpacing the speed center for I believe the first time http://speedcenter.informatik.kit.edu/mathlib4/queue

Jeremy Tan (Apr 18 2023 at 12:58):

And #port-dashboard is probably broken, it needs to be restarted

Eric Wieser (Apr 18 2023 at 13:06):

What makes you say that? #port-dashboard shouldn't need restarting ever, its a static page that's generated every half hour from #port-wiki

Jeremy Tan (Apr 18 2023 at 13:07):

It hasn't updated in a whole hour, I believe

Eric Wieser (Apr 18 2023 at 13:10):

#port-wiki looks stale

Scott Morrison (Apr 18 2023 at 13:49):

(The port progress bot will be resuming its usual schedule; the delay is expected.)

Eric Wieser (Apr 18 2023 at 14:02):

@Scott Morrison, @Jeremy Tan is referring to the script that updates the port wiki which is a different thing entirely; https://github.com/leanprover-community/mathlib-port-status#architecture shows the architecture, and Johan's machine is the weak link

Scott Morrison (Apr 18 2023 at 14:03):

Sorry, yes, I understood. I even put it in parentheses to indicate it was an aside to the main conversation. :-)

Eric Wieser (Apr 18 2023 at 14:04):

Would you mind reviewing https://github.com/leanprover-community/mathlib-port-status/pull/8/files#r1102872715 and writing a better description for the port progress bot you run on your machine?

Johan Commelin (Apr 18 2023 at 14:27):

Eric Wieser said:

Scott Morrison, Jeremy Tan is referring to the script that updates the port wiki which is a different thing entirely; https://github.com/leanprover-community/mathlib-port-status#architecture shows the architecture, and Johan's machine is the weak link

My machine has been having troubles last week. And I didn't have any time to look into it. I might give it a hard reboot soonish. Hopefully that fixes the issues. Otherwise, it will have to wait till Saturday.

Johan Commelin (Apr 18 2023 at 14:28):

Atm, math.commelin.net is down. Which is not good.

yannis monbru (Apr 18 2023 at 15:15):

Hi, i don't know what to do with this information but the file https://leanprover-community.github.io/mathlib-port-status/file/topology/algebra/valuation is marked as unported and i have a ported version of it on my copy of mathlib4
(and that one too: https://leanprover-community.github.io/mathlib-port-status/file/topology/metric_space/cantor_scheme)

Yaël Dillies (Apr 18 2023 at 15:19):

file#topology/metric_space/cantor_scheme was just added to mathlib, so just wait for @Felix Weilacher to port it. I don't know what's up with the other one.

Johan Commelin (Apr 18 2023 at 15:21):

Was topology.algebra.valuation ported recently? If so, it's explained by my server being down.

Johan Commelin (Apr 18 2023 at 15:21):

I'm on my way home. Expect a reboot in ~ 30 mins. So hopefully everything is back on track in ~ 1hr. But if my server misbehaves, it might take longer.

yannis monbru (Apr 18 2023 at 15:23):

oh yes 4 ours ago then everything is ok

Johan Commelin (Apr 18 2023 at 17:04):

my server seems to be running again

Johan Commelin (Apr 18 2023 at 17:04):

hopefully things are back to normal

port-progress bot (Apr 18 2023 at 19:03):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 381/397 (96.0% of total)
Ported lines: 144391/150373 (96.0% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Apr 18 2023 at 19:07):

mathlib port progress topology.continuous_function.bounded
Ported files: 672/689 (97.5% of total)
Ported lines: 289054/299596 (96.5% of total)
Longest unported chain: 5/85 (94.1% progress)

port-progress bot (Apr 18 2023 at 19:11):

mathlib port progress linear_algebra.determinant
Ported files: 626/645 (97.1% of total)
Ported lines: 255829/265012 (96.5% of total)
Longest unported chain: 5/73 (93.2% progress)

port-progress bot (Apr 18 2023 at 19:15):

mathlib port progress analysis.calculus.fderiv
Ported files: 676/701 (96.4% of total)
Ported lines: 291882/309219 (94.4% of total)
Longest unported chain: 7/87 (92.0% progress)

port-progress bot (Apr 18 2023 at 19:18):

mathlib port progress category_theory.monoidal.tor
Ported files: 380/395 (96.2% of total)
Ported lines: 145123/150806 (96.2% of total)
Longest unported chain: 5/56 (91.1% progress)

port-progress bot (Apr 18 2023 at 19:22):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 838/901 (93.0% of total)
Ported lines: 360454/393826 (91.5% of total)
Longest unported chain: 12/91 (86.8% progress)

port-progress bot (Apr 18 2023 at 19:26):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 873/973 (89.7% of total)
Ported lines: 368981/428724 (86.1% of total)
Longest unported chain: 19/99 (80.8% progress)

port-progress bot (Apr 18 2023 at 19:30):

mathlib port progress combinatorics.additive.behrend
Ported files: 875/978 (89.5% of total)
Ported lines: 369812/430635 (85.9% of total)
Longest unported chain: 20/100 (80.0% progress)

port-progress bot (Apr 18 2023 at 19:35):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 899/1042 (86.3% of total)
Ported lines: 372950/441619 (84.5% of total)
Longest unported chain: 27/97 (72.2% progress)

port-progress bot (Apr 18 2023 at 19:39):

mathlib port progress measure_theory.integral.bochner
Ported files: 892/1018 (87.6% of total)
Ported lines: 377034/463499 (81.3% of total)
Longest unported chain: 24/104 (76.9% progress)

port-progress bot (Apr 18 2023 at 19:42):

mathlib port progress probability.independence
Ported files: 895/1033 (86.6% of total)
Ported lines: 377407/471393 (80.1% of total)
Longest unported chain: 29/109 (73.4% progress)

port-progress bot (Apr 18 2023 at 19:47):

mathlib port progress all
Ported files: 1703/2927 (58.2% of total)
Ported lines: 568295/1015462 (56.0% of total)
Longest unported chain: 44/124 (64.5% progress)

Johan Commelin (Apr 18 2023 at 19:55):

1.4%

port-progress bot (Apr 19 2023 at 19:03):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 381/397 (96.0% of total)
Ported lines: 144391/150373 (96.0% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Apr 19 2023 at 19:07):

mathlib port progress topology.continuous_function.bounded
Ported files: 672/689 (97.5% of total)
Ported lines: 289054/299596 (96.5% of total)
Longest unported chain: 5/85 (94.1% progress)

port-progress bot (Apr 19 2023 at 19:11):

mathlib port progress linear_algebra.determinant
Ported files: 626/645 (97.1% of total)
Ported lines: 255829/265012 (96.5% of total)
Longest unported chain: 5/73 (93.2% progress)

port-progress bot (Apr 19 2023 at 19:15):

mathlib port progress analysis.calculus.fderiv
Ported files: 676/701 (96.4% of total)
Ported lines: 291882/309219 (94.4% of total)
Longest unported chain: 7/87 (92.0% progress)

port-progress bot (Apr 19 2023 at 19:19):

mathlib port progress category_theory.monoidal.tor
Ported files: 380/395 (96.2% of total)
Ported lines: 145132/150815 (96.2% of total)
Longest unported chain: 5/56 (91.1% progress)

port-progress bot (Apr 19 2023 at 19:23):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 838/901 (93.0% of total)
Ported lines: 360454/393826 (91.5% of total)
Longest unported chain: 12/91 (86.8% progress)

port-progress bot (Apr 19 2023 at 19:27):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 873/973 (89.7% of total)
Ported lines: 368981/428724 (86.1% of total)
Longest unported chain: 19/99 (80.8% progress)

port-progress bot (Apr 19 2023 at 19:31):

mathlib port progress combinatorics.additive.behrend
Ported files: 875/978 (89.5% of total)
Ported lines: 369812/430635 (85.9% of total)
Longest unported chain: 20/100 (80.0% progress)

port-progress bot (Apr 19 2023 at 19:35):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 899/1042 (86.3% of total)
Ported lines: 372953/441622 (84.5% of total)
Longest unported chain: 27/97 (72.2% progress)

port-progress bot (Apr 19 2023 at 19:39):

mathlib port progress measure_theory.integral.bochner
Ported files: 892/1018 (87.6% of total)
Ported lines: 377037/463502 (81.3% of total)
Longest unported chain: 24/104 (76.9% progress)

port-progress bot (Apr 19 2023 at 19:43):

mathlib port progress probability.independence
Ported files: 895/1033 (86.6% of total)
Ported lines: 377410/471396 (80.1% of total)
Longest unported chain: 29/109 (73.4% progress)

port-progress bot (Apr 19 2023 at 19:48):

mathlib port progress all
Ported files: 1703/2928 (58.2% of total)
Ported lines: 568343/1015676 (56.0% of total)
Longest unported chain: 44/124 (64.5% progress)

Johan Commelin (Apr 19 2023 at 19:48):

0.0%

Yaël Dillies (Apr 19 2023 at 19:50):

Le calme avant la tempête...

Adam Topaz (Apr 19 2023 at 19:52):

Johan Commelin said:

1.4%

avant ou après?

Scott Morrison (Apr 19 2023 at 20:40):

Something seems wrong with these numbers. Just looking at the PRs merged during the last 24 hours, starting at https://leanprover.zulipchat.com/#narrow/stream/116290-rss/topic/Recent.20Commits.20to.20mathlib4.3Amaster/near/350988933, I count many thousands of lines of code, but the bot claims only about 50.

Scott Morrison (Apr 19 2023 at 20:50):

Who/what is responsible for updating https://raw.githubusercontent.com/wiki/leanprover-community/mathlib/mathlib4-port-status.md?

Scott Morrison (Apr 19 2023 at 20:51):

It is out-of-date, and that is what the port-progress-bot is relying on.

Scott Morrison (Apr 19 2023 at 20:53):

@Johan Commelin, I guess this is your server?

Eric Wieser (Apr 19 2023 at 23:56):

Sometimes github decides to serve a stale copy of the raw version. You can look at #port-wiki to see whether it's been updated by Johan's server

Scott Morrison (Apr 20 2023 at 00:22):

I was going off the history page at https://github.com/leanprover-community/mathlib/wiki/mathlib4-port-status/_history.

Johan Commelin (Apr 20 2023 at 05:42):

I have no clue what is wrong with my server. But we seem to be having unreliable internet problems...

Johan Commelin (Apr 20 2023 at 05:43):

Since the internet problems are unreliable, there are many heisenbugs lurking everywhere :sad:

Johan Commelin (Apr 20 2023 at 05:47):

Traceback (most recent call last):
File "/home/jmc/data/math/mathlib4_bot/./scripts/make_port_status.py", line 135, in <module>
import_, repo, commit = get_mathlib4_module_commit_info(f.stdout.decode())
UnicodeDecodeError: 'utf-8' codec can't decode byte 0x80 in position 3131: invalid start byte

Johan Commelin (Apr 20 2023 at 05:51):

I just removed a ' in the middle of a sentence in the yaml input file. Let's see if that helps.

Johan Commelin (Apr 20 2023 at 05:54):

Nope, didn't help

Scott Morrison (Apr 20 2023 at 05:55):

Does https://stackoverflow.com/questions/38518023/unicodedecodeerror-utf8-codec-cant-decode-byte-0x80-in-position-3131-invali help? It's the same byte and position!

Johan Commelin (Apr 20 2023 at 05:58):

I need to catch a train now... this is getting mysterious.

Johan Commelin (Apr 20 2023 at 05:58):

Can we scan the various git/wiki repos involved for .DS_store files?

Scott Morrison (Apr 20 2023 at 05:58):

I don't think it's about that file.

Scott Morrison (Apr 20 2023 at 05:59):

Just some bad character.

Jeremy Tan (Apr 20 2023 at 06:13):

Johan Commelin said:

Can we scan the various git/wiki repos involved for .DS_store files?

!4#3511 has .DS_Store files

Johan Commelin (Apr 20 2023 at 06:15):

@Jeremy Tan Thanks for finding them! Can you see since when?

Jeremy Tan (Apr 20 2023 at 06:16):

The commit that introduced them is https://github.com/leanprover-community/mathlib4/pull/3511/commits/394572f30b56d07a9401690701f928c1e74dbcda,

Johan Commelin (Apr 20 2023 at 06:17):

so recently... it might explain the problems

Johan Commelin (Apr 20 2023 at 06:20):

I'm running the script with more debug output. Let's see what it says

Scott Morrison (Apr 20 2023 at 06:21):

It seems strange those files could have affected your script... I've nuked them in any case.

Johan Commelin (Apr 20 2023 at 06:22):

The script indeed crashes on 3511

Johan Commelin (Apr 20 2023 at 06:26):

For every PR, the script parses all the new files in the PR, and scans them for mathlib3 hashes. It probably gets stuck trying to parse these .DS_store files.

Johan Commelin (Apr 20 2023 at 06:27):

  1. I think we should have CI that checks specifically against these files. It's not the first time they ended up in a PR.
  2. I can tweak the script, so that it doesn't parse files that do not end in .lean.

Scott Morrison (Apr 20 2023 at 06:28):

How about we just add .DS_Store to the .gitignore? Really people should have it in their own .gitignore if they use a mac, but obviously not everyone does.

Johan Commelin (Apr 20 2023 at 06:29):

That's also fine with me. But stuff in .gitignore can still be added (although much less likely).

Kevin Buzzard (Apr 20 2023 at 06:30):

Presumably it's being added by people who just have that "when I click commit, add everything you can" option switched on in VS Code.

Scott Morrison (Apr 20 2023 at 06:31):

https://github.com/leanprover-community/mathlib4/pull/3538

Johan Commelin (Apr 20 2023 at 06:31):

Scott Morrison said:

It seems strange those files could have affected your script... I've nuked them in any case.

And the script just finished without errors!

Kevin Buzzard (Apr 20 2023 at 06:32):

So what was the actual port progress? :-)

Johan Commelin (Apr 20 2023 at 06:32):

I just triggered the other bot that generates the dashboard

Johan Commelin (Apr 20 2023 at 06:33):

We'll know in ~ 10 mins

Scott Morrison (Apr 20 2023 at 06:33):

Should I re-run the one that posts here?

Jeremy Tan (Apr 20 2023 at 06:35):

Yes, Scott

Johan Commelin (Apr 20 2023 at 06:50):

#port-dashboard has updated

port-progress bot (Apr 20 2023 at 07:14):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 382/397 (96.2% of total)
Ported lines: 144697/150456 (96.2% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Apr 20 2023 at 07:18):

mathlib port progress topology.continuous_function.bounded
Ported files: 672/689 (97.5% of total)
Ported lines: 289137/299679 (96.5% of total)
Longest unported chain: 5/85 (94.1% progress)

port-progress bot (Apr 20 2023 at 07:23):

mathlib port progress linear_algebra.determinant
Ported files: 627/645 (97.2% of total)
Ported lines: 256448/265222 (96.7% of total)
Longest unported chain: 4/73 (94.5% progress)

port-progress bot (Apr 20 2023 at 07:27):

mathlib port progress analysis.calculus.fderiv
Ported files: 676/701 (96.4% of total)
Ported lines: 291965/309302 (94.4% of total)
Longest unported chain: 7/87 (92.0% progress)

port-progress bot (Apr 20 2023 at 07:31):

mathlib port progress category_theory.monoidal.tor
Ported files: 382/395 (96.7% of total)
Ported lines: 146369/150898 (97.0% of total)
Longest unported chain: 3/56 (94.6% progress)

port-progress bot (Apr 20 2023 at 07:35):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 839/901 (93.1% of total)
Ported lines: 361073/394036 (91.6% of total)
Longest unported chain: 11/91 (87.9% progress)

port-progress bot (Apr 20 2023 at 07:39):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 874/973 (89.8% of total)
Ported lines: 369600/428934 (86.2% of total)
Longest unported chain: 19/99 (80.8% progress)

port-progress bot (Apr 20 2023 at 07:43):

mathlib port progress combinatorics.additive.behrend
Ported files: 876/978 (89.6% of total)
Ported lines: 370431/430845 (86.0% of total)
Longest unported chain: 20/100 (80.0% progress)

port-progress bot (Apr 20 2023 at 07:48):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 901/1042 (86.5% of total)
Ported lines: 373982/441832 (84.6% of total)
Longest unported chain: 27/97 (72.2% progress)

port-progress bot (Apr 20 2023 at 07:52):

mathlib port progress measure_theory.integral.bochner
Ported files: 893/1018 (87.7% of total)
Ported lines: 377656/463712 (81.4% of total)
Longest unported chain: 24/104 (76.9% progress)

port-progress bot (Apr 20 2023 at 07:58):

mathlib port progress probability.independence
Ported files: 896/1033 (86.7% of total)
Ported lines: 378029/471606 (80.2% of total)
Longest unported chain: 29/109 (73.4% progress)

Scott Morrison (Apr 20 2023 at 08:02):

I think it is open season on

These are both marked help-wanted, and have massive downstream dependencies.

Scott Morrison (Apr 20 2023 at 08:04):

To a lesser degree

  • !4#3292 RingTheory.Polynomial.Quotient
  • !4#3341 LinearAlgebra.AffineSpace.Independent

port-progress bot (Apr 20 2023 at 08:05):

mathlib port progress all
Ported files: 1721/2928 (58.8% of total)
Ported lines: 573477/1015886 (56.5% of total)
Longest unported chain: 44/124 (64.5% progress)

Johan Commelin (Apr 20 2023 at 08:06):

0.5%

Eric Wieser (Apr 20 2023 at 08:11):

!4#3466 had some meta code issues that I've flagged in other threads; while we can certainly work around them, it might be more valuable for the people who have meta experience to fix apply_fun and by_cases instead

Eric Rodriguez (Apr 20 2023 at 08:51):

(and cases and cases')

Jeremy Tan (Apr 20 2023 at 15:51):

image.png
Our open PR count is now sitting at a shockingly low 137

port-progress bot (Apr 20 2023 at 19:03):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 382/397 (96.2% of total)
Ported lines: 144811/150570 (96.2% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Apr 20 2023 at 19:07):

mathlib port progress topology.continuous_function.bounded
Ported files: 672/689 (97.5% of total)
Ported lines: 289270/299812 (96.5% of total)
Longest unported chain: 5/85 (94.1% progress)

port-progress bot (Apr 20 2023 at 19:11):

mathlib port progress linear_algebra.determinant
Ported files: 631/645 (97.8% of total)
Ported lines: 257657/265424 (97.1% of total)
Longest unported chain: 2/73 (97.3% progress)

port-progress bot (Apr 20 2023 at 19:15):

mathlib port progress analysis.calculus.fderiv
Ported files: 676/701 (96.4% of total)
Ported lines: 292098/309435 (94.4% of total)
Longest unported chain: 7/87 (92.0% progress)

port-progress bot (Apr 20 2023 at 19:19):

mathlib port progress category_theory.monoidal.tor
Ported files: 382/395 (96.7% of total)
Ported lines: 146483/151012 (97.0% of total)
Longest unported chain: 3/56 (94.6% progress)

port-progress bot (Apr 20 2023 at 19:23):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 843/901 (93.6% of total)
Ported lines: 362291/394247 (91.9% of total)
Longest unported chain: 11/91 (87.9% progress)

port-progress bot (Apr 20 2023 at 19:27):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 878/973 (90.2% of total)
Ported lines: 370818/429145 (86.4% of total)
Longest unported chain: 19/99 (80.8% progress)

port-progress bot (Apr 20 2023 at 19:31):

mathlib port progress combinatorics.additive.behrend
Ported files: 880/978 (90.0% of total)
Ported lines: 371649/431056 (86.2% of total)
Longest unported chain: 20/100 (80.0% progress)

port-progress bot (Apr 20 2023 at 19:35):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 906/1042 (86.9% of total)
Ported lines: 375820/442043 (85.0% of total)
Longest unported chain: 27/97 (72.2% progress)

port-progress bot (Apr 20 2023 at 19:39):

mathlib port progress measure_theory.integral.bochner
Ported files: 897/1018 (88.1% of total)
Ported lines: 378874/463923 (81.7% of total)
Longest unported chain: 24/104 (76.9% progress)

port-progress bot (Apr 20 2023 at 19:43):

mathlib port progress probability.independence
Ported files: 900/1033 (87.1% of total)
Ported lines: 379247/471817 (80.4% of total)
Longest unported chain: 29/109 (73.4% progress)

port-progress bot (Apr 20 2023 at 19:48):

mathlib port progress all
Ported files: 1739/2929 (59.4% of total)
Ported lines: 579253/1016207 (57.0% of total)
Longest unported chain: 44/124 (64.5% progress)

Johan Commelin (Apr 20 2023 at 20:20):

0.5%

Tobias Grosser (Apr 21 2023 at 06:04):

Nice!

port-progress bot (Apr 21 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 382/397 (96.2% of total)
Ported lines: 144853/150612 (96.2% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Apr 21 2023 at 19:08):

mathlib port progress topology.continuous_function.bounded
Ported files: 672/689 (97.5% of total)
Ported lines: 289349/299891 (96.5% of total)
Longest unported chain: 5/85 (94.1% progress)

port-progress bot (Apr 21 2023 at 19:12):

mathlib port progress linear_algebra.determinant
Ported files: 632/645 (98.0% of total)
Ported lines: 258287/265579 (97.3% of total)
Longest unported chain: 2/73 (97.3% progress)

port-progress bot (Apr 21 2023 at 19:16):

mathlib port progress analysis.calculus.fderiv
Ported files: 677/701 (96.6% of total)
Ported lines: 293116/309514 (94.7% of total)
Longest unported chain: 7/87 (92.0% progress)

port-progress bot (Apr 21 2023 at 19:19):

mathlib port progress category_theory.monoidal.tor
Ported files: 382/395 (96.7% of total)
Ported lines: 146528/151057 (97.0% of total)
Longest unported chain: 3/56 (94.6% progress)

port-progress bot (Apr 21 2023 at 19:23):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 845/901 (93.8% of total)
Ported lines: 363860/394402 (92.3% of total)
Longest unported chain: 11/91 (87.9% progress)

port-progress bot (Apr 21 2023 at 19:27):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 880/973 (90.4% of total)
Ported lines: 372387/429300 (86.7% of total)
Longest unported chain: 19/99 (80.8% progress)

port-progress bot (Apr 21 2023 at 19:31):

mathlib port progress combinatorics.additive.behrend
Ported files: 882/978 (90.2% of total)
Ported lines: 373218/431211 (86.6% of total)
Longest unported chain: 20/100 (80.0% progress)

port-progress bot (Apr 21 2023 at 19:36):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 909/1042 (87.2% of total)
Ported lines: 377463/442204 (85.4% of total)
Longest unported chain: 27/97 (72.2% progress)

port-progress bot (Apr 21 2023 at 19:40):

mathlib port progress measure_theory.integral.bochner
Ported files: 899/1018 (88.3% of total)
Ported lines: 380443/464078 (82.0% of total)
Longest unported chain: 24/104 (76.9% progress)

port-progress bot (Apr 21 2023 at 19:43):

mathlib port progress probability.independence
Ported files: 902/1033 (87.3% of total)
Ported lines: 380816/471972 (80.7% of total)
Longest unported chain: 29/109 (73.4% progress)

port-progress bot (Apr 21 2023 at 19:48):

mathlib port progress all
Ported files: 1751/2929 (59.8% of total)
Ported lines: 582648/1016446 (57.3% of total)
Longest unported chain: 44/124 (64.5% progress)

Scott Morrison (Apr 21 2023 at 22:47):

0.3%

port-progress bot (Apr 22 2023 at 19:03):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 382/397 (96.2% of total)
Ported lines: 144853/150612 (96.2% of total)
Longest unported chain: 6/52 (88.5% progress)

port-progress bot (Apr 22 2023 at 19:07):

mathlib port progress topology.continuous_function.bounded
Ported files: 673/690 (97.5% of total)
Ported lines: 289578/300120 (96.5% of total)
Longest unported chain: 5/85 (94.1% progress)

port-progress bot (Apr 22 2023 at 19:11):

mathlib port progress linear_algebra.determinant
Ported files: 632/645 (98.0% of total)
Ported lines: 258290/265582 (97.3% of total)
Longest unported chain: 2/73 (97.3% progress)

port-progress bot (Apr 22 2023 at 19:15):

mathlib port progress analysis.calculus.fderiv
Ported files: 679/702 (96.7% of total)
Ported lines: 293622/309746 (94.8% of total)
Longest unported chain: 7/87 (92.0% progress)

port-progress bot (Apr 22 2023 at 19:18):

mathlib port progress category_theory.monoidal.tor
Ported files: 382/395 (96.7% of total)
Ported lines: 146528/151057 (97.0% of total)
Longest unported chain: 3/56 (94.6% progress)

port-progress bot (Apr 22 2023 at 19:22):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 846/901 (93.9% of total)
Ported lines: 364178/394446 (92.3% of total)
Longest unported chain: 11/91 (87.9% progress)

port-progress bot (Apr 22 2023 at 19:26):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 881/973 (90.5% of total)
Ported lines: 372705/429415 (86.8% of total)
Longest unported chain: 19/99 (80.8% progress)

port-progress bot (Apr 22 2023 at 19:30):

mathlib port progress combinatorics.additive.behrend
Ported files: 883/978 (90.3% of total)
Ported lines: 373536/431326 (86.6% of total)
Longest unported chain: 20/100 (80.0% progress)

port-progress bot (Apr 22 2023 at 19:35):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 911/1043 (87.3% of total)
Ported lines: 377975/442442 (85.4% of total)
Longest unported chain: 27/97 (72.2% progress)

port-progress bot (Apr 22 2023 at 19:39):

mathlib port progress measure_theory.integral.bochner
Ported files: 900/1018 (88.4% of total)
Ported lines: 380735/464196 (82.0% of total)
Longest unported chain: 24/104 (76.9% progress)

port-progress bot (Apr 22 2023 at 19:42):

mathlib port progress probability.independence
Ported files: 903/1033 (87.4% of total)
Ported lines: 381108/472090 (80.7% of total)
Longest unported chain: 29/109 (73.4% progress)

port-progress bot (Apr 22 2023 at 19:47):

mathlib port progress all
Ported files: 1754/2930 (59.9% of total)
Ported lines: 583478/1016927 (57.4% of total)
Longest unported chain: 44/124 (64.5% progress)

Scott Morrison (Apr 22 2023 at 23:20):

0.1%

port-progress bot (Apr 23 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 383/397 (96.5% of total)
Ported lines: 145254/150612 (96.4% of total)
Longest unported chain: 5/52 (90.4% progress)

Eric Wieser (Apr 23 2023 at 19:05):

@Johan Commelin said:

I have no clue what is wrong with my server. But we seem to be having unreliable internet problems...

It looks like #port-wiki is stale again, it's not reflecting the most-recently-merged PRs

port-progress bot (Apr 23 2023 at 19:08):

mathlib port progress topology.continuous_function.bounded
Ported files: 673/690 (97.5% of total)
Ported lines: 289578/300120 (96.5% of total)
Longest unported chain: 5/85 (94.1% progress)

port-progress bot (Apr 23 2023 at 19:12):

mathlib port progress linear_algebra.determinant
Ported files: 632/645 (98.0% of total)
Ported lines: 258290/265582 (97.3% of total)
Longest unported chain: 2/73 (97.3% progress)

port-progress bot (Apr 23 2023 at 19:16):

mathlib port progress analysis.calculus.fderiv
Ported files: 679/702 (96.7% of total)
Ported lines: 293622/309746 (94.8% of total)
Longest unported chain: 7/87 (92.0% progress)

port-progress bot (Apr 23 2023 at 19:20):

mathlib port progress category_theory.monoidal.tor
Ported files: 382/395 (96.7% of total)
Ported lines: 146528/151057 (97.0% of total)
Longest unported chain: 3/56 (94.6% progress)

port-progress bot (Apr 23 2023 at 19:24):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 846/901 (93.9% of total)
Ported lines: 364178/394446 (92.3% of total)
Longest unported chain: 11/91 (87.9% progress)

port-progress bot (Apr 23 2023 at 19:28):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 881/973 (90.5% of total)
Ported lines: 372705/429415 (86.8% of total)
Longest unported chain: 19/99 (80.8% progress)

port-progress bot (Apr 23 2023 at 19:32):

mathlib port progress combinatorics.additive.behrend
Ported files: 883/978 (90.3% of total)
Ported lines: 373536/431326 (86.6% of total)
Longest unported chain: 20/100 (80.0% progress)

port-progress bot (Apr 23 2023 at 19:37):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 911/1043 (87.3% of total)
Ported lines: 377975/442442 (85.4% of total)
Longest unported chain: 27/97 (72.2% progress)

port-progress bot (Apr 23 2023 at 19:41):

mathlib port progress measure_theory.integral.bochner
Ported files: 900/1018 (88.4% of total)
Ported lines: 380735/464196 (82.0% of total)
Longest unported chain: 24/104 (76.9% progress)

port-progress bot (Apr 23 2023 at 19:45):

mathlib port progress probability.independence
Ported files: 903/1033 (87.4% of total)
Ported lines: 381108/472090 (80.7% of total)
Longest unported chain: 29/109 (73.4% progress)

port-progress bot (Apr 23 2023 at 19:50):

mathlib port progress all
Ported files: 1756/2930 (59.9% of total)
Ported lines: 584130/1016927 (57.4% of total)
Longest unported chain: 44/124 (64.5% progress)

Scott Morrison (Apr 23 2023 at 21:25):

0.0%, but see Eric's message above about the data pipeline being down.

Eric Wieser (Apr 24 2023 at 00:02):

I think @Bulhwi Cha accidentally took down the pipeline with https://github.com/leanprover-community/mathlib4/wiki/port-comments/_compare/9b53e9e3a0ec6ff357ba7fab293d2d5bb459eb51...97ee0be8e9e0ed932d30edc097ce86a3b07045df which introduces invalid yaml syntax to the port comments file

Eric Wieser (Apr 24 2023 at 00:03):

It's unfortunate that the CI that checks this file runs only on Johan's server where no one else can see it

Eric Wieser (Apr 24 2023 at 00:09):

In their defense, YAML is horribly hard to write correctly

Scott Morrison (Apr 24 2023 at 00:09):

Maybe editing the port comments file needs a human intermediary. (Or, I guess, we write a bot that asks GPT to make it into correct yaml... :-)

Eric Wieser (Apr 24 2023 at 00:11):

Putting it in a real git repo rather than a wiki would mean that people who pushed bad yaml would get an email telling them CI failed, which is probably better than having to ask Johan each time why things went silent

Eric Wieser (Apr 24 2023 at 00:12):

Teaching Johan's bot to post to zulip if it crashes would probably also do the trick

Eric Wieser (Apr 24 2023 at 00:13):

I can confirm #port-wiki is live again

Bulhwi Cha (Apr 24 2023 at 00:58):

Eric Wieser said:

I think Bulhwi Cha accidentally took down the pipeline with https://github.com/leanprover-community/mathlib4/wiki/port-comments/_compare/9b53e9e3a0ec6ff357ba7fab293d2d5bb459eb51...97ee0be8e9e0ed932d30edc097ce86a3b07045df which introduces invalid yaml syntax to the port comments file

Oh, I'm so sorry. I'll be careful of it.

port-progress bot (Apr 24 2023 at 02:32):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 384/397 (96.7% of total)
Ported lines: 145363/150612 (96.5% of total)
Longest unported chain: 4/52 (92.3% progress)

port-progress bot (Apr 24 2023 at 02:36):

mathlib port progress topology.continuous_function.bounded
Ported files: 673/690 (97.5% of total)
Ported lines: 289578/300120 (96.5% of total)
Longest unported chain: 5/85 (94.1% progress)

port-progress bot (Apr 24 2023 at 02:41):

mathlib port progress linear_algebra.determinant
Ported files: 632/645 (98.0% of total)
Ported lines: 258290/265582 (97.3% of total)
Longest unported chain: 2/73 (97.3% progress)

port-progress bot (Apr 24 2023 at 02:46):

mathlib port progress analysis.calculus.fderiv
Ported files: 679/702 (96.7% of total)
Ported lines: 293622/309746 (94.8% of total)
Longest unported chain: 7/87 (92.0% progress)

port-progress bot (Apr 24 2023 at 02:50):

mathlib port progress category_theory.monoidal.tor
Ported files: 382/395 (96.7% of total)
Ported lines: 146528/151057 (97.0% of total)
Longest unported chain: 3/56 (94.6% progress)

port-progress bot (Apr 24 2023 at 02:54):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 846/901 (93.9% of total)
Ported lines: 364178/394446 (92.3% of total)
Longest unported chain: 11/91 (87.9% progress)

port-progress bot (Apr 24 2023 at 02:59):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 880/972 (90.5% of total)
Ported lines: 372663/429373 (86.8% of total)
Longest unported chain: 19/99 (80.8% progress)

port-progress bot (Apr 24 2023 at 03:35):

mathlib port progress combinatorics.additive.behrend
Ported files: 882/977 (90.3% of total)
Ported lines: 373494/431284 (86.6% of total)
Longest unported chain: 20/100 (80.0% progress)

port-progress bot (Apr 24 2023 at 03:40):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 911/1043 (87.3% of total)
Ported lines: 377975/442442 (85.4% of total)
Longest unported chain: 27/97 (72.2% progress)

port-progress bot (Apr 24 2023 at 03:46):

mathlib port progress measure_theory.integral.bochner
Ported files: 899/1017 (88.4% of total)
Ported lines: 380693/464154 (82.0% of total)
Longest unported chain: 24/104 (76.9% progress)

port-progress bot (Apr 24 2023 at 03:51):

mathlib port progress probability.independence
Ported files: 902/1032 (87.4% of total)
Ported lines: 381066/472048 (80.7% of total)
Longest unported chain: 29/109 (73.4% progress)

port-progress bot (Apr 24 2023 at 03:57):

mathlib port progress all
Ported files: 1760/2930 (60.1% of total)
Ported lines: 584435/1016927 (57.5% of total)
Longest unported chain: 44/124 (64.5% progress)

Johan Commelin (Apr 24 2023 at 05:46):

0.1%

Jeremy Tan (Apr 24 2023 at 15:55):

We are now at over 60% ported files

port-progress bot (Apr 24 2023 at 19:06):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 385/397 (97.0% of total)
Ported lines: 145425/150616 (96.6% of total)
Longest unported chain: 4/52 (92.3% progress)

port-progress bot (Apr 24 2023 at 19:14):

mathlib port progress topology.continuous_function.bounded
Ported files: 674/690 (97.7% of total)
Ported lines: 289632/300116 (96.5% of total)
Longest unported chain: 5/85 (94.1% progress)

port-progress bot (Apr 24 2023 at 19:19):

mathlib port progress linear_algebra.determinant
Ported files: 633/645 (98.1% of total)
Ported lines: 258360/265505 (97.3% of total)
Longest unported chain: 2/73 (97.3% progress)

port-progress bot (Apr 24 2023 at 19:24):

mathlib port progress analysis.calculus.fderiv
Ported files: 681/702 (97.0% of total)
Ported lines: 294159/309742 (95.0% of total)
Longest unported chain: 7/87 (92.0% progress)

port-progress bot (Apr 24 2023 at 19:29):

mathlib port progress category_theory.monoidal.tor
Ported files: 384/395 (97.2% of total)
Ported lines: 146793/151061 (97.2% of total)
Longest unported chain: 3/56 (94.6% progress)

port-progress bot (Apr 24 2023 at 19:33):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 848/901 (94.1% of total)
Ported lines: 364731/394369 (92.5% of total)
Longest unported chain: 11/91 (87.9% progress)

port-progress bot (Apr 24 2023 at 19:38):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 882/972 (90.7% of total)
Ported lines: 373216/429296 (86.9% of total)
Longest unported chain: 19/99 (80.8% progress)

port-progress bot (Apr 24 2023 at 19:42):

mathlib port progress combinatorics.additive.behrend
Ported files: 884/977 (90.5% of total)
Ported lines: 374047/431207 (86.7% of total)
Longest unported chain: 20/100 (80.0% progress)

port-progress bot (Apr 24 2023 at 19:47):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 914/1043 (87.6% of total)
Ported lines: 378681/442365 (85.6% of total)
Longest unported chain: 27/97 (72.2% progress)

port-progress bot (Apr 24 2023 at 19:52):

mathlib port progress measure_theory.integral.bochner
Ported files: 901/1017 (88.6% of total)
Ported lines: 381246/464077 (82.2% of total)
Longest unported chain: 24/104 (76.9% progress)

port-progress bot (Apr 24 2023 at 19:56):

mathlib port progress probability.independence
Ported files: 904/1032 (87.6% of total)
Ported lines: 381619/471971 (80.9% of total)
Longest unported chain: 29/109 (73.4% progress)

port-progress bot (Apr 24 2023 at 20:02):

mathlib port progress all
Ported files: 1772/2930 (60.5% of total)
Ported lines: 586518/1016944 (57.7% of total)
Longest unported chain: 44/124 (64.5% progress)

Scott Morrison (Apr 24 2023 at 21:29):

0.2%

Kevin Buzzard (Apr 24 2023 at 21:30):

We officially made it to 60% of files though :-)

port-progress bot (Apr 25 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 385/397 (97.0% of total)
Ported lines: 145425/150616 (96.6% of total)
Longest unported chain: 4/52 (92.3% progress)

port-progress bot (Apr 25 2023 at 19:08):

mathlib port progress topology.continuous_function.bounded
Ported files: 675/690 (97.8% of total)
Ported lines: 290463/300116 (96.8% of total)
Longest unported chain: 5/85 (94.1% progress)

port-progress bot (Apr 25 2023 at 19:12):

mathlib port progress linear_algebra.determinant
Ported files: 635/645 (98.4% of total)
Ported lines: 260415/265505 (98.1% of total)
Longest unported chain: 2/73 (97.3% progress)

port-progress bot (Apr 25 2023 at 19:16):

mathlib port progress analysis.calculus.fderiv
Ported files: 683/702 (97.3% of total)
Ported lines: 295337/309742 (95.3% of total)
Longest unported chain: 7/87 (92.0% progress)

port-progress bot (Apr 25 2023 at 19:19):

mathlib port progress category_theory.monoidal.tor
Ported files: 384/395 (97.2% of total)
Ported lines: 146793/151061 (97.2% of total)
Longest unported chain: 3/56 (94.6% progress)

port-progress bot (Apr 25 2023 at 19:23):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 854/901 (94.8% of total)
Ported lines: 368243/394369 (93.4% of total)
Longest unported chain: 11/91 (87.9% progress)

port-progress bot (Apr 25 2023 at 19:27):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 892/975 (91.5% of total)
Ported lines: 377144/429823 (87.7% of total)
Longest unported chain: 19/99 (80.8% progress)

port-progress bot (Apr 25 2023 at 19:31):

mathlib port progress combinatorics.additive.behrend
Ported files: 894/980 (91.2% of total)
Ported lines: 377975/431734 (87.5% of total)
Longest unported chain: 20/100 (80.0% progress)

port-progress bot (Apr 25 2023 at 19:36):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 920/1043 (88.2% of total)
Ported lines: 382193/442365 (86.4% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (Apr 25 2023 at 19:40):

mathlib port progress measure_theory.integral.bochner
Ported files: 911/1020 (89.3% of total)
Ported lines: 385174/464604 (82.9% of total)
Longest unported chain: 24/104 (76.9% progress)

port-progress bot (Apr 25 2023 at 19:44):

mathlib port progress probability.independence
Ported files: 914/1035 (88.3% of total)
Ported lines: 385547/472498 (81.6% of total)
Longest unported chain: 29/109 (73.4% progress)

port-progress bot (Apr 25 2023 at 19:48):

mathlib port progress all
Ported files: 1791/2930 (61.1% of total)
Ported lines: 593504/1017308 (58.3% of total)
Longest unported chain: 44/124 (64.5% progress)

Scott Morrison (Apr 25 2023 at 21:52):

0.6%

port-progress bot (Apr 25 2023 at 21:56):

mathlib port progress topology.category.CompHaus.projective
Ported files: 782/793 (98.6% of total)
Ported lines: 319258/324312 (98.4% of total)
Longest unported chain: 2/82 (97.6% progress)

port-progress bot (Apr 25 2023 at 22:00):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 768/779 (98.6% of total)
Ported lines: 313829/318931 (98.4% of total)
Longest unported chain: 3/83 (96.4% progress)

port-progress bot (Apr 26 2023 at 19:05):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 385/397 (97.0% of total)
Ported lines: 145425/150616 (96.6% of total)
Longest unported chain: 4/52 (92.3% progress)

port-progress bot (Apr 26 2023 at 19:09):

mathlib port progress topology.category.CompHaus.projective
Ported files: 779/790 (98.6% of total)
Ported lines: 319242/323409 (98.7% of total)
Longest unported chain: 2/82 (97.6% progress)

port-progress bot (Apr 26 2023 at 19:14):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 765/776 (98.6% of total)
Ported lines: 313813/318028 (98.7% of total)
Longest unported chain: 3/83 (96.4% progress)

port-progress bot (Apr 26 2023 at 19:18):

mathlib port progress topology.continuous_function.bounded
Ported files: 677/690 (98.1% of total)
Ported lines: 291896/300214 (97.2% of total)
Longest unported chain: 4/85 (95.3% progress)

port-progress bot (Apr 26 2023 at 19:23):

mathlib port progress linear_algebra.determinant
Ported files: 635/645 (98.4% of total)
Ported lines: 260523/265613 (98.1% of total)
Longest unported chain: 2/73 (97.3% progress)

port-progress bot (Apr 26 2023 at 19:27):

mathlib port progress analysis.calculus.fderiv
Ported files: 684/702 (97.4% of total)
Ported lines: 296499/309840 (95.7% of total)
Longest unported chain: 6/87 (93.1% progress)

port-progress bot (Apr 26 2023 at 19:31):

mathlib port progress category_theory.monoidal.tor
Ported files: 384/395 (97.2% of total)
Ported lines: 146793/151061 (97.2% of total)
Longest unported chain: 3/56 (94.6% progress)

port-progress bot (Apr 26 2023 at 19:36):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 857/901 (95.1% of total)
Ported lines: 370134/394496 (93.8% of total)
Longest unported chain: 10/91 (89.0% progress)

port-progress bot (Apr 26 2023 at 19:40):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 895/975 (91.8% of total)
Ported lines: 379035/429950 (88.2% of total)
Longest unported chain: 18/99 (81.8% progress)

port-progress bot (Apr 26 2023 at 19:45):

mathlib port progress combinatorics.additive.behrend
Ported files: 897/980 (91.5% of total)
Ported lines: 379866/431861 (88.0% of total)
Longest unported chain: 19/100 (81.0% progress)

port-progress bot (Apr 26 2023 at 19:50):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 922/1043 (88.4% of total)
Ported lines: 383655/442492 (86.7% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (Apr 26 2023 at 19:55):

mathlib port progress measure_theory.integral.bochner
Ported files: 914/1020 (89.6% of total)
Ported lines: 387065/464731 (83.3% of total)
Longest unported chain: 23/104 (77.9% progress)

port-progress bot (Apr 26 2023 at 19:59):

mathlib port progress probability.independence
Ported files: 917/1035 (88.6% of total)
Ported lines: 387438/472625 (82.0% of total)
Longest unported chain: 28/109 (74.3% progress)

port-progress bot (Apr 26 2023 at 20:04):

mathlib port progress all
Ported files: 1797/2934 (61.2% of total)
Ported lines: 596588/1017558 (58.6% of total)
Longest unported chain: 43/124 (65.3% progress)

Johan Commelin (Apr 26 2023 at 20:06):

0.3%

port-progress bot (Apr 27 2023 at 19:03):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 385/397 (97.0% of total)
Ported lines: 145434/150625 (96.6% of total)
Longest unported chain: 4/52 (92.3% progress)

port-progress bot (Apr 27 2023 at 19:07):

mathlib port progress topology.category.CompHaus.projective
Ported files: 780/790 (98.7% of total)
Ported lines: 319604/323609 (98.8% of total)
Longest unported chain: 1/82 (98.8% progress)

port-progress bot (Apr 27 2023 at 19:11):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 766/776 (98.7% of total)
Ported lines: 314175/318228 (98.7% of total)
Longest unported chain: 2/83 (97.6% progress)

port-progress bot (Apr 27 2023 at 19:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 679/690 (98.4% of total)
Ported lines: 292672/300426 (97.4% of total)
Longest unported chain: 2/85 (97.6% progress)

port-progress bot (Apr 27 2023 at 19:19):

mathlib port progress linear_algebra.determinant
Ported files: 635/645 (98.4% of total)
Ported lines: 260730/265820 (98.1% of total)
Longest unported chain: 2/73 (97.3% progress)

port-progress bot (Apr 27 2023 at 19:22):

mathlib port progress analysis.calculus.fderiv
Ported files: 686/702 (97.7% of total)
Ported lines: 297281/310058 (95.9% of total)
Longest unported chain: 4/87 (95.4% progress)

port-progress bot (Apr 27 2023 at 19:26):

mathlib port progress category_theory.monoidal.tor
Ported files: 384/395 (97.2% of total)
Ported lines: 146799/151067 (97.2% of total)
Longest unported chain: 3/56 (94.6% progress)

port-progress bot (Apr 27 2023 at 19:30):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 859/901 (95.3% of total)
Ported lines: 370935/394732 (94.0% of total)
Longest unported chain: 10/91 (89.0% progress)

port-progress bot (Apr 27 2023 at 19:34):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 897/975 (92.0% of total)
Ported lines: 379839/430189 (88.3% of total)
Longest unported chain: 17/99 (82.8% progress)

port-progress bot (Apr 27 2023 at 19:38):

mathlib port progress combinatorics.additive.behrend
Ported files: 899/980 (91.7% of total)
Ported lines: 380670/432100 (88.1% of total)
Longest unported chain: 18/100 (82.0% progress)

port-progress bot (Apr 27 2023 at 19:43):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 924/1043 (88.6% of total)
Ported lines: 384456/442730 (86.8% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (Apr 27 2023 at 19:47):

mathlib port progress measure_theory.integral.bochner
Ported files: 916/1020 (89.8% of total)
Ported lines: 387933/465044 (83.4% of total)
Longest unported chain: 22/104 (78.8% progress)

port-progress bot (Apr 27 2023 at 19:50):

mathlib port progress probability.independence
Ported files: 919/1035 (88.8% of total)
Ported lines: 388306/472938 (82.1% of total)
Longest unported chain: 27/109 (75.2% progress)

port-progress bot (Apr 27 2023 at 19:55):

mathlib port progress all
Ported files: 1804/2934 (61.5% of total)
Ported lines: 598772/1018052 (58.8% of total)
Longest unported chain: 42/124 (66.1% progress)

Scott Morrison (Apr 27 2023 at 22:35):

0.2%

port-progress bot (Apr 28 2023 at 19:03):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 386/397 (97.2% of total)
Ported lines: 145837/150640 (96.8% of total)
Longest unported chain: 3/52 (94.2% progress)

port-progress bot (Apr 28 2023 at 19:07):

mathlib port progress topology.category.CompHaus.projective
Ported files: 782/790 (99.0% of total)
Ported lines: 320148/323628 (98.9% of total)
Longest unported chain: 1/82 (98.8% progress)

port-progress bot (Apr 28 2023 at 19:11):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 767/776 (98.8% of total)
Ported lines: 314419/318224 (98.8% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (Apr 28 2023 at 19:15):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 292894/300407 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (Apr 28 2023 at 19:19):

mathlib port progress linear_algebra.determinant
Ported files: 637/645 (98.8% of total)
Ported lines: 261805/265836 (98.5% of total)
Longest unported chain: 1/73 (98.6% progress)

port-progress bot (Apr 28 2023 at 19:23):

mathlib port progress analysis.calculus.fderiv
Ported files: 688/702 (98.0% of total)
Ported lines: 298008/310054 (96.1% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (Apr 28 2023 at 19:26):

mathlib port progress category_theory.monoidal.tor
Ported files: 385/395 (97.5% of total)
Ported lines: 147093/151084 (97.4% of total)
Longest unported chain: 2/56 (96.4% progress)

port-progress bot (Apr 28 2023 at 19:30):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 864/900 (96.0% of total)
Ported lines: 372844/394713 (94.5% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (Apr 28 2023 at 19:34):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 902/974 (92.6% of total)
Ported lines: 381748/430170 (88.7% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (Apr 28 2023 at 19:38):

mathlib port progress combinatorics.additive.behrend
Ported files: 904/979 (92.3% of total)
Ported lines: 382579/432081 (88.5% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (Apr 28 2023 at 19:42):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 929/1042 (89.2% of total)
Ported lines: 386365/442711 (87.3% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (Apr 28 2023 at 19:46):

mathlib port progress measure_theory.integral.bochner
Ported files: 921/1019 (90.4% of total)
Ported lines: 389842/465038 (83.8% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (Apr 28 2023 at 19:50):

mathlib port progress probability.independence
Ported files: 924/1034 (89.4% of total)
Ported lines: 390215/472932 (82.5% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (Apr 28 2023 at 19:55):

mathlib port progress all
Ported files: 1822/2935 (62.1% of total)
Ported lines: 603370/1018316 (59.3% of total)
Longest unported chain: 40/124 (67.7% progress)

Johan Commelin (Apr 28 2023 at 19:58):

0.6%

Scott Morrison (Apr 28 2023 at 22:04):

topology.category.CompHaus.projective is complete, and I will remove it from the bot!

Jeremy Tan (Apr 29 2023 at 02:08):

Data.MvPolynomial.Polynomial is already in mathlib4. Why does #port-dashboard show it as unported?

Kevin Buzzard (Apr 29 2023 at 11:30):

port-progress bot said:

mathlib port progress category_theory.sites.dense_subsite
Ported files: 386/397 (97.2% of total)
Ported lines: 145837/150640 (96.8% of total)
Longest unported chain: 3/52 (94.2% progress)

Why this does say 386/397 ported files, when the pdf indicates that the answer should be x-4 / x for some x?

Eric Wieser (Apr 29 2023 at 11:31):

What doe port-status#category_theory/sites/dense_subsite say?

Eric Wieser (Apr 29 2023 at 11:32):

Heh, 344/347 which is different again

Kevin Buzzard (Apr 29 2023 at 11:33):

But maybe that's OK, I could have made an off by one error. Is a file which has all prerequisites ported x/x or x-1/x?

Eric Wieser (Apr 29 2023 at 11:34):

For port-status (which doesn't actually show the /x bit) it's x/x

Eric Wieser (Apr 29 2023 at 11:34):

I assume this is down to different handling of tactic files

Kevin Buzzard (Apr 29 2023 at 11:35):

Yes, I assume so. And from your other response it looks like I did make an off by one error, so the port-status page is perhaps the one to trust.

Eric Wieser (Apr 29 2023 at 11:35):

Hey, at least the graphs agree!

port-progress bot (Apr 29 2023 at 19:03):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 386/397 (97.2% of total)
Ported lines: 145843/150646 (96.8% of total)
Longest unported chain: 3/52 (94.2% progress)

port-progress bot (Apr 29 2023 at 19:07):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 767/776 (98.8% of total)
Ported lines: 314428/318233 (98.8% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (Apr 29 2023 at 19:11):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 292903/300416 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (Apr 29 2023 at 19:15):

mathlib port progress linear_algebra.determinant
Ported files: 637/645 (98.8% of total)
Ported lines: 261814/265845 (98.5% of total)
Longest unported chain: 1/73 (98.6% progress)

port-progress bot (Apr 29 2023 at 19:19):

mathlib port progress analysis.calculus.fderiv
Ported files: 688/702 (98.0% of total)
Ported lines: 298020/310066 (96.1% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (Apr 29 2023 at 19:22):

mathlib port progress category_theory.monoidal.tor
Ported files: 385/395 (97.5% of total)
Ported lines: 147099/151090 (97.4% of total)
Longest unported chain: 2/56 (96.4% progress)

port-progress bot (Apr 29 2023 at 19:26):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 864/900 (96.0% of total)
Ported lines: 372865/394734 (94.5% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (Apr 29 2023 at 19:30):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 902/974 (92.6% of total)
Ported lines: 381769/430191 (88.7% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (Apr 29 2023 at 19:34):

mathlib port progress combinatorics.additive.behrend
Ported files: 904/979 (92.3% of total)
Ported lines: 382600/432102 (88.5% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (Apr 29 2023 at 19:39):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 929/1042 (89.2% of total)
Ported lines: 386386/442732 (87.3% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (Apr 29 2023 at 19:43):

mathlib port progress measure_theory.integral.bochner
Ported files: 921/1019 (90.4% of total)
Ported lines: 389863/465059 (83.8% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (Apr 29 2023 at 19:47):

mathlib port progress probability.independence
Ported files: 924/1034 (89.4% of total)
Ported lines: 390236/472953 (82.5% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (Apr 29 2023 at 19:51):

mathlib port progress all
Ported files: 1828/2935 (62.3% of total)
Ported lines: 604333/1018308 (59.3% of total)
Longest unported chain: 40/124 (67.7% progress)

Scott Morrison (Apr 29 2023 at 22:24):

0.0%

Scott Morrison (Apr 29 2023 at 23:28):

@porters, I would like to make a small attempt at channeling available effort towards porting. It's great that people are porting available files, but I'm concerned about the number of high priority files that are marked help-wanted, and want to just draw attention to these. I think everyone (who feels competent to do so!) who wants to work on the port should consider starting by looking through this list for places they can contribute.

I've made this list by going through the priority porting targets above, and looking at the highest files. These are the files that begin the longest chains towards the targets:

  • Analysis.NormedSpace.OperatorNorm !4#3708
  • Analysis.SpecificLimits.Normed !4#3419
  • CategoryTheory.Functor.Flat !4#3703
  • RingTheory.TensorProduct !4#3649
  • RingTheory.Polynomial.Quotient !4#3292
  • Topology.ContinuousFunction.Algebra !4#3332

There is also open for porting:

  • category_theory.preadditive.projective_resolution

And a PR not marked as help-wanted, but for which I will nevertheless ping the author here, to check if they would in fact like help!

  • LinearAlgebra.Determinant !4#3694 (@Pol'tta / Miyahara Kō)

The files on the first list are all marked help-wanted, so it's fine for anyone to jump in. (A polite convention we often follow is to post a comment on the PR saying you are "locking" and "unlocking" the PR while you're actively working on it, to avoid duplicating work; but I wouldn't say doing so is compulsory.)

I will hopefully try to update this list regularly if it proves useful.

Moritz Doll (Apr 29 2023 at 23:47):

fyi: in the case of Analysis.NormedSpace.OperatorNorm it is probably good to ask Anatole first whether he has any uncommited work. The help-wanted label was added by someone else (on the same day as the initial commit).

Jeremy Tan (Apr 30 2023 at 01:29):

I had asked Dedecker here and he said there was no uncommitted work

Jeremy Tan (Apr 30 2023 at 01:33):

OperatorNorm is effectively mine now

Scott Morrison (Apr 30 2023 at 03:31):

Jeremy Tan said:

OperatorNorm is effectively mine now

What do you mean by this?

Jeremy Tan (Apr 30 2023 at 04:12):

Dedecker did nothing but run the script and create the PR; I was the first one to actually push some fixes

Scott Morrison (Apr 30 2023 at 04:15):

Yes, what I meant was --- do you not want other people working on it? That seemed the obvious interpretation of your comment.

Jeremy Tan (Apr 30 2023 at 04:21):

I sure want others to work on it

Kevin Buzzard (Apr 30 2023 at 10:10):

CategoryTheory.Functor.Flat is on route to one of the Copenhagen targets and I've been slowly but surely working on it since Scott made the PR. I don't mind it being tagged "help wanted" -- it's Scott's PR after all -- but I'll remark that if I'd opened that PR instead (and Scott beat me by 45 minutes) then I would not have tagged it "help wanted" and I would just be working on it when I had time. I've just spent some time documenting what I know about the remaining issues in the file (6 or so sorries) and I'm now going to spend about 7 hours marking, so others can feel free to take over.

Matthew Ballard (Apr 30 2023 at 13:15):

All remaining files have now have < 400 dependents. 10 more and it’s < 300

Pol'tta / Miyahara Kō (Apr 30 2023 at 13:33):

I had to finish my part-time job so I was late to finish !4#3694. Now I have finished, but I'm welcome to help.

port-progress bot (Apr 30 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 386/397 (97.2% of total)
Ported lines: 145851/150654 (96.8% of total)
Longest unported chain: 3/52 (94.2% progress)

port-progress bot (Apr 30 2023 at 19:07):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 767/776 (98.8% of total)
Ported lines: 314597/318402 (98.8% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (Apr 30 2023 at 19:11):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 293072/300585 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (Apr 30 2023 at 19:15):

mathlib port progress linear_algebra.determinant
Ported files: 637/645 (98.8% of total)
Ported lines: 261822/265853 (98.5% of total)
Longest unported chain: 1/73 (98.6% progress)

port-progress bot (Apr 30 2023 at 19:19):

mathlib port progress analysis.calculus.fderiv
Ported files: 688/702 (98.0% of total)
Ported lines: 298189/310235 (96.1% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (Apr 30 2023 at 19:22):

mathlib port progress category_theory.monoidal.tor
Ported files: 385/395 (97.5% of total)
Ported lines: 147107/151098 (97.4% of total)
Longest unported chain: 2/56 (96.4% progress)

port-progress bot (Apr 30 2023 at 19:26):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 865/900 (96.1% of total)
Ported lines: 373198/394903 (94.5% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (Apr 30 2023 at 19:30):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 903/974 (92.7% of total)
Ported lines: 382262/430520 (88.8% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (Apr 30 2023 at 19:34):

mathlib port progress combinatorics.additive.behrend
Ported files: 905/979 (92.4% of total)
Ported lines: 383093/432431 (88.6% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (Apr 30 2023 at 19:39):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 930/1042 (89.3% of total)
Ported lines: 386879/443061 (87.3% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (Apr 30 2023 at 19:43):

mathlib port progress measure_theory.integral.bochner
Ported files: 922/1019 (90.5% of total)
Ported lines: 390356/465388 (83.9% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (Apr 30 2023 at 19:47):

mathlib port progress probability.independence
Ported files: 925/1034 (89.5% of total)
Ported lines: 390729/473282 (82.6% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (Apr 30 2023 at 19:51):

mathlib port progress all
Ported files: 1832/2936 (62.4% of total)
Ported lines: 605383/1018669 (59.4% of total)
Longest unported chain: 41/125 (67.2% progress)

Scott Morrison (Apr 30 2023 at 23:19):

0.1%

Joël Riou (May 01 2023 at 10:04):

The target category_theory.monoidal.tor may soon be removed from the bot: !4#3740 !4#3751 !4#3754

port-progress bot (May 01 2023 at 19:03):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 388/399 (97.2% of total)
Ported lines: 147359/152162 (96.8% of total)
Longest unported chain: 3/52 (94.2% progress)

port-progress bot (May 01 2023 at 19:07):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 768/776 (99.0% of total)
Ported lines: 314888/318395 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 01 2023 at 19:11):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 293065/300578 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 01 2023 at 19:15):

mathlib port progress linear_algebra.determinant
Ported files: 637/645 (98.8% of total)
Ported lines: 261815/265846 (98.5% of total)
Longest unported chain: 1/73 (98.6% progress)

port-progress bot (May 01 2023 at 19:19):

mathlib port progress analysis.calculus.fderiv
Ported files: 688/702 (98.0% of total)
Ported lines: 298182/310228 (96.1% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 01 2023 at 19:22):

mathlib port progress category_theory.monoidal.tor
Ported files: 387/397 (97.5% of total)
Ported lines: 148615/152606 (97.4% of total)
Longest unported chain: 2/56 (96.4% progress)

port-progress bot (May 01 2023 at 19:26):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 865/900 (96.1% of total)
Ported lines: 373191/394903 (94.5% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 01 2023 at 19:30):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 903/974 (92.7% of total)
Ported lines: 382255/430520 (88.8% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 01 2023 at 19:34):

mathlib port progress combinatorics.additive.behrend
Ported files: 905/979 (92.4% of total)
Ported lines: 383086/432431 (88.6% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 01 2023 at 19:39):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 930/1044 (89.1% of total)
Ported lines: 386872/443609 (87.2% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 01 2023 at 19:43):

mathlib port progress measure_theory.integral.bochner
Ported files: 922/1020 (90.4% of total)
Ported lines: 390349/465414 (83.9% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 01 2023 at 19:47):

mathlib port progress probability.independence
Ported files: 925/1035 (89.4% of total)
Ported lines: 390722/473452 (82.5% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (May 01 2023 at 19:51):

mathlib port progress all
Ported files: 1835/2937 (62.5% of total)
Ported lines: 606904/1018942 (59.6% of total)
Longest unported chain: 41/125 (67.2% progress)

Johan Commelin (May 01 2023 at 19:57):

0.2%

Scott Morrison (May 01 2023 at 19:57):

0.2%

Scott Morrison (May 02 2023 at 11:49):

We've just had two of the porting goals LinearAlgebra.Determinant and CategoryTheory.Monoidal.Tor hit master! Thanks for everyone who contributed to these.

Scott Morrison (May 02 2023 at 11:49):

I'll remove them from port-progress-bot now.

Scott Morrison (May 02 2023 at 11:59):

Our list of "high priority and help wanted files" remains more or less the same:

Kevin is working on CategoryTheory.Functor.Flat !4#3703, and it looks like it is getting very close now.

LinearAlgebra.Determinant was just merged.

Please, if you have time to help with the port, prioritize working on these ones! :-)

Ruben Van de Velde (May 02 2023 at 12:04):

I started looking at a few, but had no clue how to make progress on the timeouts :(

Scott Morrison (May 02 2023 at 12:07):

Even just doing what I did in RingTheory.Polynomial.Quotient !4#3292 just now is helpful:

  • if it's a term mode proof that is making heavy use of unification, ungolf it and write out the steps with type annotations, to help identify which step is timing out
  • turn on set_option profiler true in and set_option set_option trace.Meta.isDefEq true in, then click through the trace logs (always following whichever branch is slowest), and then copy and paste the section of the log that is timing out into a comment in the file, so others looking at it can quickly see what is going on.

Sebastian Ullrich (May 02 2023 at 12:10):

Use set_option trace.profiler true in instead to be shown only the slow branches!

Ruben Van de Velde (May 02 2023 at 12:15):

I learned something today, thanks :)

I'm guessing I don't want to see "[46.190159s] try rfl "

port-progress bot (May 02 2023 at 19:05):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 388/399 (97.2% of total)
Ported lines: 147359/152162 (96.8% of total)
Longest unported chain: 3/52 (94.2% progress)

port-progress bot (May 02 2023 at 19:09):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 768/776 (99.0% of total)
Ported lines: 314896/318403 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 02 2023 at 19:13):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 293070/300583 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 02 2023 at 19:17):

mathlib port progress analysis.calculus.fderiv
Ported files: 688/702 (98.0% of total)
Ported lines: 298187/310232 (96.1% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 02 2023 at 19:21):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 868/900 (96.4% of total)
Ported lines: 374242/394911 (94.8% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 02 2023 at 19:26):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 904/973 (92.9% of total)
Ported lines: 382260/430129 (88.9% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 02 2023 at 19:30):

mathlib port progress combinatorics.additive.behrend
Ported files: 906/978 (92.6% of total)
Ported lines: 383091/432040 (88.7% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 02 2023 at 19:35):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 931/1044 (89.2% of total)
Ported lines: 387080/443505 (87.3% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 02 2023 at 19:39):

mathlib port progress measure_theory.integral.bochner
Ported files: 923/1019 (90.6% of total)
Ported lines: 390354/465023 (83.9% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 02 2023 at 19:43):

mathlib port progress probability.independence
Ported files: 926/1034 (89.6% of total)
Ported lines: 390727/473061 (82.6% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (May 02 2023 at 19:48):

mathlib port progress all
Ported files: 1842/2937 (62.7% of total)
Ported lines: 608481/1018939 (59.7% of total)
Longest unported chain: 41/125 (67.2% progress)

Johan Commelin (May 02 2023 at 20:15):

0.1%

James Gallicchio (May 03 2023 at 05:10):

It's been a month since we hit 50% ported lines. 10% progress since then!

port-progress bot (May 03 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 388/399 (97.2% of total)
Ported lines: 147403/152206 (96.8% of total)
Longest unported chain: 3/52 (94.2% progress)

port-progress bot (May 03 2023 at 19:08):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 768/776 (99.0% of total)
Ported lines: 314998/318505 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 03 2023 at 19:12):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 293172/300685 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 03 2023 at 19:16):

mathlib port progress analysis.calculus.fderiv
Ported files: 688/702 (98.0% of total)
Ported lines: 298289/310334 (96.1% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 03 2023 at 19:20):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 868/900 (96.4% of total)
Ported lines: 374358/395027 (94.8% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 03 2023 at 19:24):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 904/973 (92.9% of total)
Ported lines: 382376/430251 (88.9% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 03 2023 at 19:28):

mathlib port progress combinatorics.additive.behrend
Ported files: 906/978 (92.6% of total)
Ported lines: 383207/432162 (88.7% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 03 2023 at 19:33):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 931/1044 (89.2% of total)
Ported lines: 387196/443627 (87.3% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 03 2023 at 19:37):

mathlib port progress measure_theory.integral.bochner
Ported files: 924/1019 (90.7% of total)
Ported lines: 391920/465145 (84.3% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 03 2023 at 19:41):

mathlib port progress probability.independence
Ported files: 927/1034 (89.7% of total)
Ported lines: 392293/473183 (82.9% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (May 03 2023 at 19:45):

mathlib port progress all
Ported files: 1854/2939 (63.1% of total)
Ported lines: 612297/1019399 (60.1% of total)
Longest unported chain: 41/125 (67.2% progress)

Johan Commelin (May 03 2023 at 19:52):

0.4%

port-progress bot (May 04 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 383/394 (97.2% of total)
Ported lines: 145806/150609 (96.8% of total)
Longest unported chain: 3/50 (94.0% progress)

port-progress bot (May 04 2023 at 19:08):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 768/776 (99.0% of total)
Ported lines: 314998/318505 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 04 2023 at 19:12):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 293172/300685 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 04 2023 at 19:16):

mathlib port progress analysis.calculus.fderiv
Ported files: 688/702 (98.0% of total)
Ported lines: 298320/310365 (96.1% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 04 2023 at 19:21):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 868/900 (96.4% of total)
Ported lines: 374448/394902 (94.8% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 04 2023 at 19:25):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 904/973 (92.9% of total)
Ported lines: 382466/430122 (88.9% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 04 2023 at 19:30):

mathlib port progress combinatorics.additive.behrend
Ported files: 906/978 (92.6% of total)
Ported lines: 383297/432033 (88.7% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 04 2023 at 19:34):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 930/1043 (89.2% of total)
Ported lines: 387241/443452 (87.3% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 04 2023 at 19:39):

mathlib port progress measure_theory.integral.bochner
Ported files: 925/1019 (90.8% of total)
Ported lines: 392598/465026 (84.4% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 04 2023 at 19:43):

mathlib port progress probability.independence
Ported files: 928/1034 (89.7% of total)
Ported lines: 392971/473103 (83.1% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (May 04 2023 at 19:48):

mathlib port progress all
Ported files: 1860/2941 (63.2% of total)
Ported lines: 613899/1019572 (60.2% of total)
Longest unported chain: 40/124 (67.7% progress)

Scott Morrison (May 04 2023 at 23:28):

0.1%

port-progress bot (May 05 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 383/394 (97.2% of total)
Ported lines: 145811/150614 (96.8% of total)
Longest unported chain: 3/50 (94.0% progress)

port-progress bot (May 05 2023 at 19:07):

mathlib port progress topology.category.CompHaus.projective
Ported files: 783/790 (99.1% of total)
Ported lines: 320504/323920 (98.9% of total)
Longest unported chain: 1/82 (98.8% progress)

port-progress bot (May 05 2023 at 19:10):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 768/776 (99.0% of total)
Ported lines: 315006/318513 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 05 2023 at 19:14):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 293180/300693 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 05 2023 at 19:17):

mathlib port progress linear_algebra.determinant
Ported files: 638/645 (98.9% of total)
Ported lines: 262643/266059 (98.7% of total)
Longest unported chain: 1/73 (98.6% progress)

port-progress bot (May 05 2023 at 19:21):

mathlib port progress analysis.calculus.fderiv
Ported files: 688/702 (98.0% of total)
Ported lines: 298328/310373 (96.1% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 05 2023 at 19:24):

mathlib port progress category_theory.monoidal.tor
Ported files: 390/397 (98.2% of total)
Ported lines: 149248/152664 (97.8% of total)
Longest unported chain: 1/56 (98.2% progress)

port-progress bot (May 05 2023 at 19:28):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 868/900 (96.4% of total)
Ported lines: 374456/394903 (94.8% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 05 2023 at 19:33):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 904/973 (92.9% of total)
Ported lines: 382474/430123 (88.9% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 05 2023 at 19:37):

mathlib port progress combinatorics.additive.behrend
Ported files: 906/978 (92.6% of total)
Ported lines: 383305/432034 (88.7% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 05 2023 at 19:41):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 930/1043 (89.2% of total)
Ported lines: 387249/443474 (87.3% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 05 2023 at 19:46):

mathlib port progress measure_theory.integral.bochner
Ported files: 926/1019 (90.9% of total)
Ported lines: 392755/465027 (84.5% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 05 2023 at 19:50):

mathlib port progress probability.independence
Ported files: 929/1034 (89.8% of total)
Ported lines: 393128/473104 (83.1% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (May 05 2023 at 19:55):

mathlib port progress all
Ported files: 1861/2942 (63.3% of total)
Ported lines: 614054/1019680 (60.2% of total)
Longest unported chain: 40/124 (67.7% progress)

Johan Commelin (May 05 2023 at 19:57):

0.0%

Ruben Van de Velde (May 05 2023 at 20:00):

topology.category.CompHaus.projective, linear_algebra.determinant, and category_theory.monoidal.tor are done

Scott Morrison (May 05 2023 at 22:31):

I had a bad git accident at home, and accidentally reverted the changes to the script which had dropped these targets...

Jireh Loreaux (May 06 2023 at 02:24):

There's always reflog for git accidents

Eric Wieser (May 06 2023 at 04:12):

That only helps if the accident was in the history and not in uncommitted changes in the working tree...

Pol'tta / Miyahara Kō (May 06 2023 at 10:03):

MeasureTheory.Measure.MeasureSpace is now ready to merge except some dependent PRs.
This is the second longest file in Mathlib. (BTW the first longest one is Data.List.Basic)
@MonadMaverick and I ported this, so it was a hard job.

Johan Commelin (May 06 2023 at 10:42):

Thanks a lot for all your efforts!

port-progress bot (May 06 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 383/394 (97.2% of total)
Ported lines: 145811/150614 (96.8% of total)
Longest unported chain: 3/50 (94.0% progress)

port-progress bot (May 06 2023 at 19:08):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 768/776 (99.0% of total)
Ported lines: 315006/318513 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 06 2023 at 19:12):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 293174/300687 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 06 2023 at 19:16):

mathlib port progress analysis.calculus.fderiv
Ported files: 688/702 (98.0% of total)
Ported lines: 298328/310373 (96.1% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 06 2023 at 19:20):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 868/900 (96.4% of total)
Ported lines: 374456/394903 (94.8% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 06 2023 at 19:24):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 904/973 (92.9% of total)
Ported lines: 382474/430230 (88.9% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 06 2023 at 19:29):

mathlib port progress combinatorics.additive.behrend
Ported files: 906/978 (92.6% of total)
Ported lines: 383305/432141 (88.7% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 06 2023 at 19:33):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 930/1043 (89.2% of total)
Ported lines: 387249/443581 (87.3% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 06 2023 at 19:38):

mathlib port progress measure_theory.integral.bochner
Ported files: 928/1019 (91.1% of total)
Ported lines: 393304/465128 (84.6% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 06 2023 at 19:42):

mathlib port progress probability.independence
Ported files: 931/1034 (90.0% of total)
Ported lines: 393677/473205 (83.2% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (May 06 2023 at 19:47):

mathlib port progress all
Ported files: 1865/2942 (63.4% of total)
Ported lines: 615346/1019794 (60.3% of total)
Longest unported chain: 40/124 (67.7% progress)

Scott Morrison (May 07 2023 at 00:48):

0.1%

port-progress bot (May 07 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 383/394 (97.2% of total)
Ported lines: 145993/150796 (96.8% of total)
Longest unported chain: 3/50 (94.0% progress)

port-progress bot (May 07 2023 at 19:07):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 768/776 (99.0% of total)
Ported lines: 315188/318695 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 07 2023 at 19:11):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 293356/300869 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 07 2023 at 19:15):

mathlib port progress analysis.calculus.fderiv
Ported files: 688/702 (98.0% of total)
Ported lines: 298510/310555 (96.1% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 07 2023 at 19:19):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 868/900 (96.4% of total)
Ported lines: 374638/395085 (94.8% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 07 2023 at 19:23):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 904/973 (92.9% of total)
Ported lines: 382656/430414 (88.9% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 07 2023 at 19:27):

mathlib port progress combinatorics.additive.behrend
Ported files: 906/978 (92.6% of total)
Ported lines: 383487/432325 (88.7% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 07 2023 at 19:32):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 930/1043 (89.2% of total)
Ported lines: 387431/443765 (87.3% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 07 2023 at 19:36):

mathlib port progress measure_theory.integral.bochner
Ported files: 928/1019 (91.1% of total)
Ported lines: 393498/465324 (84.6% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 07 2023 at 19:40):

mathlib port progress probability.independence
Ported files: 931/1034 (90.0% of total)
Ported lines: 393871/473401 (83.2% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (May 07 2023 at 19:45):

mathlib port progress all
Ported files: 1866/2944 (63.4% of total)
Ported lines: 615908/1020112 (60.4% of total)
Longest unported chain: 40/124 (67.7% progress)

Mauricio Collares (May 07 2023 at 19:45):

Milestone: Fewer than 1000 unported files on #port-dashboard (probably happened yesterday but I missed it)

Scott Morrison (May 07 2023 at 23:59):

0.1%

Scott Morrison (May 08 2023 at 13:04):

An update on high priority files:

Our list of "high priority and help wanted files" is only moving slowly:

Almost there:

  • Topology.ContinuousFunction.Algebra !4#3332 (see thread. Did some more work on this today, looks like just some linting to go, if someone would like to take that!)
  • CategoryTheory.Functor.Flat !4#3703 (@Kevin Buzzard?)

Recently merged:

  • Analysis.SpecificLimits.Normed !4#3419

Scott Morrison (May 08 2023 at 13:11):

As previously, if you have something you can contribute to one of these files, that's probably the most helpful thing to do in terms of mathlib4!

Ruben Van de Velde (May 08 2023 at 13:21):

I'll do Topology.ContinuousFunction.Algebra now

Ruben Van de Velde (May 08 2023 at 14:13):

Ruben Van de Velde said:

I'll do Topology.ContinuousFunction.Algebra now

!4#3332 up for review

Kevin Buzzard (May 08 2023 at 14:17):

For CategoryTheory.Functor.Flat I was slowly trying to work out whether unification hints could help with the forget (Type u) issue but nobody has got them working. I think the other issues can just be ignored; so I think that what is needed is that I move the forget issues to a more appropriate place (which I'll do at some point within the next 8 hours) and then I'd be happy to merge.

port-progress bot (May 08 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 383/394 (97.2% of total)
Ported lines: 146005/150808 (96.8% of total)
Longest unported chain: 3/50 (94.0% progress)

port-progress bot (May 08 2023 at 19:08):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 768/776 (99.0% of total)
Ported lines: 315200/318707 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

Eric Wieser (May 08 2023 at 19:09):

Kevin Buzzard said:

For CategoryTheory.Functor.Flat I was slowly trying to work out whether unification hints could help with the forget (Type u) issue.

Wasn't this easily solved with @[reducible]?

Kevin Buzzard (May 08 2023 at 19:10):

Not as far as I know (neither Adam nor I could solve it). See the thread linked in the PR

port-progress bot (May 08 2023 at 19:12):

mathlib port progress topology.continuous_function.bounded
Ported files: 680/690 (98.6% of total)
Ported lines: 293368/300881 (97.5% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 08 2023 at 19:16):

mathlib port progress analysis.calculus.fderiv
Ported files: 689/702 (98.1% of total)
Ported lines: 299169/310567 (96.3% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 08 2023 at 19:20):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 869/900 (96.6% of total)
Ported lines: 375297/394968 (95.0% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 08 2023 at 19:24):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 906/973 (93.1% of total)
Ported lines: 383958/430347 (89.2% of total)
Longest unported chain: 15/99 (84.8% progress)

Eric Wieser (May 08 2023 at 19:25):

Kevin Buzzard said:

Not as far as I know (neither Adam nor I could solve it). See the thread linked in the PR

See my comment on that thread from hours ago

Eric Wieser (May 08 2023 at 19:27):

Eric Wieser said:

Adam Topaz said:

Adding reducible to literally everything in this file doesn't seem to work. So I guess the answer is no, it's not possible?

attribute [reducible] ConcreteCategory.Forget ConcreteCategory.types works

port-progress bot (May 08 2023 at 19:28):

mathlib port progress combinatorics.additive.behrend
Ported files: 908/978 (92.8% of total)
Ported lines: 384789/432258 (89.0% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 08 2023 at 19:32):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 932/1043 (89.4% of total)
Ported lines: 388733/443667 (87.6% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 08 2023 at 19:36):

mathlib port progress measure_theory.integral.bochner
Ported files: 931/1019 (91.4% of total)
Ported lines: 394981/465339 (84.9% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 08 2023 at 19:40):

mathlib port progress probability.independence
Ported files: 934/1034 (90.3% of total)
Ported lines: 395354/473416 (83.5% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (May 08 2023 at 19:45):

mathlib port progress all
Ported files: 1875/2945 (63.7% of total)
Ported lines: 619147/1020618 (60.7% of total)
Longest unported chain: 40/124 (67.7% progress)

Kevin Buzzard (May 08 2023 at 20:42):

Eric Wieser said:

Kevin Buzzard said:

Not as far as I know (neither Adam nor I could solve it). See the thread linked in the PR

See my comment on that thread from hours ago

Oh I missed that comment (even though I'd read the thread!) Thanks!

Scott Morrison (May 08 2023 at 21:27):

0.3%

Kevin Buzzard (May 08 2023 at 22:12):

Scott merged master (and hence Sebastien's refactoring of the algebra hierarchy) into the RingTheory.TensorProduct PR, and this solves several problems in RingTheory.TensorProduct; I tried solving a few more. I couldn't get the Semiring (A ⊗[R] B) instance working so I sorried some proofs; there's now a panic in the file :-/

Kevin Buzzard (May 08 2023 at 23:12):

Re CategoryTheory.Functor.Flat !4#3703 : the only remaining issue is whether we merge it with the rw [Comma.eqToHom_right] hacks or wait for several days for #18973 and its corresponding forward-port to make its way through the system first.

Kevin Buzzard (May 09 2023 at 16:51):

#18973 isn't passing CI. Should we merge !4#3703 first, or wait? !4#3703 is on the critical path to category_theory.sites.dense_subsite, which we need for Copenhagen.

Kevin Buzzard (May 09 2023 at 16:52):

Related: should I start porting the next file on the critical path or should I wait until !4#3703 is merged?

Eric Wieser (May 09 2023 at 17:11):

(I have no strong opinions here: though I'm a bit worried that the mathlib3 change didn't go through as trivially as I expected)

Kevin Buzzard (May 09 2023 at 18:55):

When I made the change in mathlib4 to check it would fix the issue, I had to edit two other files (comma and something else).

port-progress bot (May 09 2023 at 19:03):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 383/394 (97.2% of total)
Ported lines: 146005/150808 (96.8% of total)
Longest unported chain: 3/50 (94.0% progress)

port-progress bot (May 09 2023 at 19:07):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 768/776 (99.0% of total)
Ported lines: 315252/318759 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 09 2023 at 19:11):

mathlib port progress topology.continuous_function.bounded
Ported files: 681/690 (98.7% of total)
Ported lines: 294380/300936 (97.8% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 09 2023 at 19:15):

mathlib port progress analysis.calculus.fderiv
Ported files: 689/702 (98.1% of total)
Ported lines: 299235/310633 (96.3% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 09 2023 at 19:19):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 869/900 (96.6% of total)
Ported lines: 375370/395041 (95.0% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 09 2023 at 19:23):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 906/973 (93.1% of total)
Ported lines: 384034/430423 (89.2% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 09 2023 at 19:27):

mathlib port progress combinatorics.additive.behrend
Ported files: 908/978 (92.8% of total)
Ported lines: 384865/432334 (89.0% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 09 2023 at 19:31):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 932/1043 (89.4% of total)
Ported lines: 388809/443780 (87.6% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 09 2023 at 19:35):

mathlib port progress measure_theory.integral.bochner
Ported files: 933/1019 (91.6% of total)
Ported lines: 400210/465421 (86.0% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 09 2023 at 19:39):

mathlib port progress probability.independence
Ported files: 936/1034 (90.5% of total)
Ported lines: 400583/473498 (84.6% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (May 09 2023 at 19:44):

mathlib port progress all
Ported files: 1883/2945 (63.9% of total)
Ported lines: 625971/1020755 (61.3% of total)
Longest unported chain: 40/124 (67.7% progress)

Scott Morrison (May 09 2023 at 23:07):

@Kevin Buzzard, I've merged !4#3703, using Copenhagen as an excuse to keep things moving!

Scott Morrison (May 09 2023 at 23:07):

0.6%

port-progress bot (May 10 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 384/394 (97.5% of total)
Ported lines: 146410/150821 (97.1% of total)
Longest unported chain: 2/50 (96.0% progress)

port-progress bot (May 10 2023 at 19:06):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 769/776 (99.1% of total)
Ported lines: 315348/318764 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 10 2023 at 19:10):

mathlib port progress topology.continuous_function.bounded
Ported files: 681/690 (98.7% of total)
Ported lines: 294385/300941 (97.8% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 10 2023 at 19:14):

mathlib port progress analysis.calculus.fderiv
Ported files: 689/702 (98.1% of total)
Ported lines: 299240/310638 (96.3% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 10 2023 at 19:18):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 869/900 (96.6% of total)
Ported lines: 375375/395046 (95.0% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 10 2023 at 19:23):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 906/974 (93.0% of total)
Ported lines: 384039/430626 (89.2% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 10 2023 at 19:27):

mathlib port progress combinatorics.additive.behrend
Ported files: 908/979 (92.7% of total)
Ported lines: 384870/432537 (89.0% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 10 2023 at 19:31):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 932/1044 (89.3% of total)
Ported lines: 388814/443983 (87.6% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 10 2023 at 19:36):

mathlib port progress measure_theory.integral.bochner
Ported files: 939/1020 (92.1% of total)
Ported lines: 402057/465630 (86.3% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 10 2023 at 19:40):

mathlib port progress probability.independence
Ported files: 942/1035 (91.0% of total)
Ported lines: 402430/473707 (85.0% of total)
Longest unported chain: 25/109 (77.1% progress)

port-progress bot (May 10 2023 at 19:44):

mathlib port progress all
Ported files: 1908/2946 (64.8% of total)
Ported lines: 632953/1021620 (62.0% of total)
Longest unported chain: 40/124 (67.7% progress)

Scott Morrison (May 10 2023 at 21:25):

0.7%

port-progress bot (May 11 2023 at 19:05):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 387/396 (97.7% of total)
Ported lines: 146947/151137 (97.2% of total)
Longest unported chain: 1/50 (98.0% progress)

port-progress bot (May 11 2023 at 19:07):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 769/776 (99.1% of total)
Ported lines: 315434/318850 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 11 2023 at 19:11):

mathlib port progress topology.continuous_function.bounded
Ported files: 681/690 (98.7% of total)
Ported lines: 294511/301067 (97.8% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 11 2023 at 19:16):

mathlib port progress analysis.calculus.fderiv
Ported files: 689/702 (98.1% of total)
Ported lines: 299323/310721 (96.3% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 11 2023 at 19:20):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 869/900 (96.6% of total)
Ported lines: 375458/395129 (95.0% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 11 2023 at 19:24):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 907/975 (93.0% of total)
Ported lines: 384531/431323 (89.2% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 11 2023 at 19:28):

mathlib port progress combinatorics.additive.behrend
Ported files: 909/980 (92.8% of total)
Ported lines: 385362/433234 (89.0% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 11 2023 at 19:33):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 933/1045 (89.3% of total)
Ported lines: 389306/444680 (87.5% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 11 2023 at 19:37):

mathlib port progress measure_theory.integral.bochner
Ported files: 940/1021 (92.1% of total)
Ported lines: 402617/466395 (86.3% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 11 2023 at 19:44):

mathlib port progress all
Ported files: 1920/2947 (65.2% of total)
Ported lines: 636917/1022203 (62.3% of total)
Longest unported chain: 40/124 (67.7% progress)

Johan Commelin (May 11 2023 at 20:23):

0.3%

Mario Carneiro (May 12 2023 at 17:15):

Can I add a suggestion for a metric for the bot to display? As we get closer to the end of the port, more files will get all their reverse dependencies ported. These files are important because they are essentially "done" as far as porting is concerned: you can make modifications to them without any porting hazards as long as you fix the mathlib4 side of things.

So how about tracking the number of files that have no unported dependent files? It is probably quite low right now, maybe in the 10-20% range, but it will start to jump up toward the end.

Eric Wieser (May 12 2023 at 17:27):

Modifications to them can still create hazards with forward-ports; though hopefully the only things touching these files in mathlib3 are propagation of some trivial rename, which should be easy to apply from scratch in the forward-port

Eric Wieser (May 12 2023 at 17:29):

I could add this to the progress bar on #port-dashboard as a dark green section

port-progress bot (May 12 2023 at 19:05):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 388/396 (98.0% of total)
Ported lines: 147240/151144 (97.4% of total)
Longest unported chain: 1/50 (98.0% progress)

port-progress bot (May 12 2023 at 19:08):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 769/776 (99.1% of total)
Ported lines: 315438/318854 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 12 2023 at 19:13):

mathlib port progress topology.continuous_function.bounded
Ported files: 681/690 (98.7% of total)
Ported lines: 294515/301071 (97.8% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 12 2023 at 19:17):

mathlib port progress analysis.calculus.fderiv
Ported files: 690/702 (98.3% of total)
Ported lines: 299653/310725 (96.4% of total)
Longest unported chain: 3/87 (96.6% progress)

port-progress bot (May 12 2023 at 19:22):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 871/900 (96.8% of total)
Ported lines: 376499/395177 (95.3% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 12 2023 at 19:26):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 910/975 (93.3% of total)
Ported lines: 385791/431395 (89.4% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 12 2023 at 19:31):

mathlib port progress combinatorics.additive.behrend
Ported files: 912/980 (93.1% of total)
Ported lines: 386622/433306 (89.2% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 12 2023 at 19:36):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 936/1045 (89.6% of total)
Ported lines: 390522/444684 (87.8% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 12 2023 at 19:40):

mathlib port progress measure_theory.integral.bochner
Ported files: 943/1021 (92.4% of total)
Ported lines: 403908/466498 (86.6% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 12 2023 at 19:49):

mathlib port progress all
Ported files: 1935/2949 (65.6% of total)
Ported lines: 642439/1022749 (62.8% of total)
Longest unported chain: 40/124 (67.7% progress)

Pol'tta / Miyahara Kō (May 12 2023 at 19:51):

0.5%

port-progress bot (May 13 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 388/396 (98.0% of total)
Ported lines: 147240/151155 (97.4% of total)
Longest unported chain: 1/50 (98.0% progress)

port-progress bot (May 13 2023 at 19:07):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 769/776 (99.1% of total)
Ported lines: 315438/318854 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 13 2023 at 19:12):

mathlib port progress topology.continuous_function.bounded
Ported files: 681/690 (98.7% of total)
Ported lines: 294515/301071 (97.8% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 13 2023 at 19:19):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 871/900 (96.8% of total)
Ported lines: 376505/395183 (95.3% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 13 2023 at 19:24):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 911/975 (93.4% of total)
Ported lines: 386755/431404 (89.7% of total)
Longest unported chain: 15/99 (84.8% progress)

port-progress bot (May 13 2023 at 19:28):

mathlib port progress combinatorics.additive.behrend
Ported files: 913/980 (93.2% of total)
Ported lines: 387586/433315 (89.4% of total)
Longest unported chain: 16/100 (84.0% progress)

port-progress bot (May 13 2023 at 19:33):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 937/1045 (89.7% of total)
Ported lines: 391486/444693 (88.0% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 13 2023 at 19:38):

mathlib port progress measure_theory.integral.bochner
Ported files: 944/1021 (92.5% of total)
Ported lines: 404872/466507 (86.8% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 13 2023 at 19:46):

mathlib port progress all
Ported files: 1947/2949 (66.0% of total)
Ported lines: 646177/1022974 (63.2% of total)
Longest unported chain: 40/124 (67.7% progress)

Johan Commelin (May 13 2023 at 19:51):

0.4%

Kevin Buzzard (May 13 2023 at 20:00):

Good for a weekend :-)

port-progress bot (May 14 2023 at 19:04):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 388/396 (98.0% of total)
Ported lines: 147240/151155 (97.4% of total)
Longest unported chain: 1/50 (98.0% progress)

port-progress bot (May 14 2023 at 19:06):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 769/776 (99.1% of total)
Ported lines: 315438/318854 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 14 2023 at 19:10):

mathlib port progress topology.continuous_function.bounded
Ported files: 681/690 (98.7% of total)
Ported lines: 294515/301071 (97.8% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 14 2023 at 19:17):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 871/900 (96.8% of total)
Ported lines: 376505/395183 (95.3% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 14 2023 at 19:22):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 911/983 (92.7% of total)
Ported lines: 386755/431720 (89.6% of total)
Longest unported chain: 19/103 (81.6% progress)

port-progress bot (May 14 2023 at 19:26):

mathlib port progress combinatorics.additive.behrend
Ported files: 913/988 (92.4% of total)
Ported lines: 387586/433631 (89.4% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 14 2023 at 19:30):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 937/1045 (89.7% of total)
Ported lines: 391486/444693 (88.0% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 14 2023 at 19:34):

mathlib port progress measure_theory.integral.bochner
Ported files: 944/1029 (91.7% of total)
Ported lines: 404872/466823 (86.7% of total)
Longest unported chain: 24/108 (77.8% progress)

port-progress bot (May 14 2023 at 19:42):

mathlib port progress all
Ported files: 1952/2959 (66.0% of total)
Ported lines: 646855/1023338 (63.2% of total)
Longest unported chain: 44/128 (65.6% progress)

Pol'tta / Miyahara Kō (May 14 2023 at 22:59):

0.0%

Kevin Buzzard (May 15 2023 at 14:49):

We can now remove category_theory.sites.dense_subsite from this list, as !4#3985 is merged. Looks like the second file on the list, topology.category.Profinite.as_limit, is also done.

Matthew Ballard (May 15 2023 at 14:51):

How about group cohomology as a target?

Kevin Buzzard (May 15 2023 at 14:53):

This is the file representation_theory.group_cohomology.basic.

Matthew Ballard (May 15 2023 at 14:59):

Lots of stuck things on that path that need attention

Kevin Buzzard (May 15 2023 at 15:10):

The next four files in the list are all blocked on Analysis.NormedSpace.OperatorNorm, whose PR is not compiling !4#3708 with Lean 4 master but which works fine !4#3903 with what I believe is the Lean 4 PR lean4#2210 . The fifth file on the list is quadratic reciprocity, which is blocked on ring_theory.polynomial.quotient, which is stuck in PR !4#3292 but which is working fine with lean4#2210 in !4#3932 (or at least I think it is, it compiles locally on my machine and I just fixed what I believe are the last few linting issues). The final file (Bochner integral) is also blocked on the OperatorNorm PR. So we are slowly grinding to a halt now, waiting for a decision on Gabriel's Lean 4 PR.

Matthew Ballard (May 15 2023 at 15:13):

The things along the path representation_theory.group_cohomology.basic have the possibility of becoming unstuck without changes to core

Matthew Ballard (May 15 2023 at 15:16):

Bonus points if it can be done by Monday :wink:

Kevin Buzzard (May 15 2023 at 15:18):

There's ring_theory.tensor_product along the path to group cohomology, which is another port in a similar situation: it's stuck at !4#3649 but as far as I know nobody yet attempted to get it working with the modification to core Lean. Maybe I'll give it a go?

Ruben Van de Velde (May 15 2023 at 15:24):

Is lean4#2210 likely to land soon?

Ruben Van de Velde (May 15 2023 at 15:36):

And congrats @Eric Wieser on !4#4000!

Matthew Ballard (May 15 2023 at 15:49):

What we should focus on in the current state might be a good topic for discussion later today

Matthew Ballard (May 15 2023 at 16:06):

Ruben Van de Velde said:

Is lean4#2210 likely to land soon?

:rocket:

Kevin Buzzard (May 15 2023 at 16:22):

!4#4004 is RingTheory.TensorProduct with reenableeta, just because I kind of don't know what else to work on right now.

Matthew Ballard (May 15 2023 at 16:35):

I guess it is open season on bumping heartbeats to merge (after checking against reenableeta) until we get the toolchain updated

Mauricio Collares (May 15 2023 at 16:36):

Isn't it better to just merge !4#3414 now (with the toolchain currently used there) and then move back to a nightly tomorrow?

Matthew Ballard (May 15 2023 at 16:38):

I'll see if it is simple to update reenableeta to master.

Matthew Ballard (May 15 2023 at 18:11):

It was wasn't simple for me despite there only being two broken files (including one I just ported) :/

Mauricio Collares (May 15 2023 at 18:30):

In both cases there is one extra goal being created and then the rest of the proof is trying to close the wrong goal

Matthew Ballard (May 15 2023 at 18:31):

I pushed sorried versions to the reeanableeta_20230515 branch in case any one else wants to play along

Matthew Ballard (May 15 2023 at 18:48):

Ok I guess we are down to 1 sorry now.

Mauricio Collares (May 15 2023 at 18:51):

(deleted)

Mauricio Collares (May 15 2023 at 18:53):

The remaining sorry is easy to fill but I don't get why we need to fill it. In particular, I don't get why some local state is reverted.

Matthew Ballard (May 15 2023 at 18:53):

Yeah. I used your trick of library_search lol

port-progress bot (May 15 2023 at 19:03):

mathlib port progress category_theory.sites.dense_subsite
Ported files: 389/396 (98.2% of total)
Ported lines: 147739/151155 (97.7% of total)
Longest unported chain: 1/50 (98.0% progress)

port-progress bot (May 15 2023 at 19:06):

mathlib port progress topology.category.Profinite.as_limit
Ported files: 769/776 (99.1% of total)
Ported lines: 315438/318854 (98.9% of total)
Longest unported chain: 1/83 (98.8% progress)

port-progress bot (May 15 2023 at 19:10):

mathlib port progress topology.continuous_function.bounded
Ported files: 681/690 (98.7% of total)
Ported lines: 294515/301071 (97.8% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 15 2023 at 19:16):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 871/900 (96.8% of total)
Ported lines: 376558/395236 (95.3% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 15 2023 at 19:21):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 912/983 (92.8% of total)
Ported lines: 387248/431780 (89.7% of total)
Longest unported chain: 19/103 (81.6% progress)

port-progress bot (May 15 2023 at 19:25):

mathlib port progress combinatorics.additive.behrend
Ported files: 914/988 (92.5% of total)
Ported lines: 388079/433691 (89.5% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 15 2023 at 19:29):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 937/1045 (89.7% of total)
Ported lines: 391539/444811 (88.0% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 15 2023 at 19:33):

mathlib port progress measure_theory.integral.bochner
Ported files: 939/1018 (92.2% of total)
Ported lines: 403489/459496 (87.8% of total)
Longest unported chain: 24/108 (77.8% progress)

port-progress bot (May 15 2023 at 19:41):

mathlib port progress all
Ported files: 1959/2963 (66.1% of total)
Ported lines: 649285/1023635 (63.4% of total)
Longest unported chain: 44/128 (65.6% progress)

Kevin Buzzard (May 15 2023 at 23:11):

!4#4004 has just one sorry but I need to sleep now. simp was closing it in Lean 3 it seems.

Eric Rodriguez (May 15 2023 at 23:33):

fixed; it seems LinearEquiv.coe_symm_mk isn't firing within simp; moving it to rw fixed things.

Eric Rodriguez (May 15 2023 at 23:36):

is this expected? I see a porting note says this:

-- Porting note: below needed to be rewritten due to changed `simp` behaviour for `coe`

Johan Commelin (May 16 2023 at 04:59):

0.2%

Kevin Buzzard (May 16 2023 at 08:50):

There were several instances in the part of the file I ported where simp was not working but rw worked instead; I can remember at least three proofs in that file where lean 3 simp only [A, B, C, D, E] had to turn into lean 4 simp only [A,B], rw [C,D], simp only [E]. Probably worth investigating.

Ruben Van de Velde (May 16 2023 at 08:52):

Can that be an issue with the discrimination tree?

Kevin Buzzard (May 16 2023 at 08:52):

I'll try to minimise at some point today

Ruben Van de Velde (May 16 2023 at 08:54):

It's somewhat common - https://github.com/leanprover-community/mathlib4/commit/017781e6ac3c66813822930e4007baa0d518250f#diff-26ed6932a1d4a0b23b3b4a7d27e1bdd1ab6145d69e4aee002374792c1bca30f2R169 is another example I just noticed

port-progress bot (May 16 2023 at 19:04):

mathlib port progress topology.continuous_function.bounded
Ported files: 681/690 (98.7% of total)
Ported lines: 294515/301071 (97.8% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 16 2023 at 19:11):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 872/900 (96.9% of total)
Ported lines: 377021/395236 (95.4% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 16 2023 at 19:15):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 917/987 (92.9% of total)
Ported lines: 389234/431972 (90.1% of total)
Longest unported chain: 19/103 (81.6% progress)

port-progress bot (May 16 2023 at 19:19):

mathlib port progress combinatorics.additive.behrend
Ported files: 919/992 (92.6% of total)
Ported lines: 390065/433883 (89.9% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 16 2023 at 19:24):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 942/1045 (90.1% of total)
Ported lines: 393525/444811 (88.5% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 16 2023 at 19:28):

mathlib port progress measure_theory.integral.bochner
Ported files: 944/1022 (92.4% of total)
Ported lines: 405475/459688 (88.2% of total)
Longest unported chain: 24/108 (77.8% progress)

port-progress bot (May 16 2023 at 19:35):

mathlib port progress representation_theory.group_cohomology.basic
Ported files: 918/964 (95.2% of total)
Ported lines: 363946/380035 (95.8% of total)
Longest unported chain: 11/79 (86.1% progress)

port-progress bot (May 16 2023 at 19:39):

mathlib port progress all
Ported files: 1972/2967 (66.5% of total)
Ported lines: 654204/1023759 (63.9% of total)
Longest unported chain: 44/128 (65.6% progress)

Johan Commelin (May 16 2023 at 19:52):

0.5%

Daniel Fabian (May 16 2023 at 20:13):

I've been out of the loop for quite a while. @Johan Commelin, @Kevin Buzzard or @Mario Carneiro would you mind explaining to me roughly where we stand w.r.t. being able to rely on lean 4 for mathlib?

Johan Commelin (May 16 2023 at 20:13):

Roughly at 63.9%, I would say :rofl:

Daniel Fabian (May 16 2023 at 20:14):

lol. Is the current plan to get everything to 100% first, or are new contributions already sometimes made mathlib 4?

Johan Commelin (May 16 2023 at 20:14):

More seriously: for basic topology and algebra, you're good to go. For stuff like manifolds, advanced analysis, and stuff like that, we'll need another 3 months maybe?

Johan Commelin (May 16 2023 at 20:15):

New contributions are fine, if they are orthogonal to stuff that is in mathlib3

Ruben Van de Velde (May 16 2023 at 20:15):

There's been at least one new file added to mathlib 4 :)

Daniel Fabian (May 16 2023 at 20:15):

that's really neat. Great to hear the progress :)

Johan Commelin (May 16 2023 at 20:15):

In other words, if the new contribution will not cause a headache down the road, when we try to port something.

Heather Macbeth (May 17 2023 at 02:26):

What's the incantation to generate a port-progress graph locally?

Yakov Pechersky (May 17 2023 at 02:38):

My (albeit old, maybe outdated) command history says:

leanproject --debug import-graph --to algebra.order.field.defs algebra.order.ring.pdf --port-status --mathlib4 ~/math/mathlib4 --reduce

Heather Macbeth (May 17 2023 at 02:51):

Thanks! That works but doesn't do the new thing of hiding the green nodes. I'll try to read the manual ...

Heather Macbeth (May 17 2023 at 03:04):

Hmm, my local leanproject doesn't have the --really-exclude-ported flag added on Jan 27, and when I tried updating leanproject nothing changed. Is that because the latest release is from Dec 15? cc @Patrick Massot

Yakov Pechersky (May 17 2023 at 03:37):

You can always do a pip install git+https://github.com/leanprover-community/mathlib-tools.git -U

Pol'tta / Miyahara Kō (May 17 2023 at 09:48):

I've finished porting MeasureTheory.Function.SimpleFunc; MeasureTheory.Integral.Lebesgue is ready to port.
I'm going to sleep.

port-progress bot (May 17 2023 at 19:04):

mathlib port progress topology.continuous_function.bounded
Ported files: 681/690 (98.7% of total)
Ported lines: 294530/301086 (97.8% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 17 2023 at 19:12):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 872/900 (96.9% of total)
Ported lines: 377039/395254 (95.4% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 17 2023 at 19:17):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 920/987 (93.2% of total)
Ported lines: 391359/432087 (90.6% of total)
Longest unported chain: 19/103 (81.6% progress)

port-progress bot (May 17 2023 at 19:21):

mathlib port progress combinatorics.additive.behrend
Ported files: 922/992 (92.9% of total)
Ported lines: 392190/433998 (90.4% of total)
Longest unported chain: 20/104 (80.8% progress)

port-progress bot (May 17 2023 at 19:26):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 945/1045 (90.4% of total)
Ported lines: 395880/444841 (89.0% of total)
Longest unported chain: 26/97 (73.2% progress)

port-progress bot (May 17 2023 at 19:31):

mathlib port progress measure_theory.integral.bochner
Ported files: 947/1022 (92.7% of total)
Ported lines: 407600/459738 (88.7% of total)
Longest unported chain: 24/108 (77.8% progress)

port-progress bot (May 17 2023 at 19:39):

mathlib port progress representation_theory.group_cohomology.basic
Ported files: 921/964 (95.5% of total)
Ported lines: 364762/380035 (96.0% of total)
Longest unported chain: 11/79 (86.1% progress)

port-progress bot (May 17 2023 at 19:44):

mathlib port progress all
Ported files: 1986/2968 (66.9% of total)
Ported lines: 658960/1025166 (64.3% of total)
Longest unported chain: 44/128 (65.6% progress)

Kevin Buzzard (May 17 2023 at 19:47):

We now have our first claim to be 2/3 of the way through!

Johan Commelin (May 17 2023 at 19:55):

0.4%

Pol'tta / Miyahara Kō (May 18 2023 at 03:30):

Haha! I've finished porting MeasureTheory.Integral.Lebesgue!
Whoever expected that integrals comes to Lean 4 earlier than derivatives?

Rémy Degenne (May 18 2023 at 06:32):

It looks like probability.independence got removed from the port-progress bot output. I guess it is because its name changed to probability.independence.basic recently. Can someone with access to the bot fix the name in the script it is running?

Eric Wieser (May 18 2023 at 06:34):

(deleted)

Johan Commelin (May 18 2023 at 07:06):

cc @Scott Morrison

Scott Morrison (May 18 2023 at 11:46):

A quick high-priority/help-wanted post, if anyone is looking for something to work on:

  • Analysis.NormedSpace.Multilinear !4#4057 <--- especially this one!
  • Analysis.NormedSpace.AffineIsometry !4#3651
  • LinearAlgebra.Dual !4#3659
  • Algebra.Category.Mon.Limits !4#3073
  • CategoryTheory.Bicategory.Coherence !4#4062

Jeremy Tan (May 18 2023 at 13:15):

Scott Morrison said:

A quick high-priority/help-wanted post, if anyone is looking for something to work on:

  • Analysis.NormedSpace.Multilinear !4#4057 <--- especially this one!
  • Analysis.NormedSpace.AffineIsometry !4#3651
  • LinearAlgebra.Dual !4#3659
  • Algebra.Category.Mon.Limits !4#3073
  • CategoryTheory.Bicategory.Coherence !4#4062

I'd like to add to this list

Floris van Doorn (May 18 2023 at 18:48):

!4#4057 is ready for review!

port-progress bot (May 18 2023 at 19:04):

mathlib port progress topology.continuous_function.bounded
Ported files: 682/690 (98.8% of total)
Ported lines: 296301/301089 (98.4% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 18 2023 at 19:12):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 876/900 (97.3% of total)
Ported lines: 379478/395259 (96.0% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 18 2023 at 19:17):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 911/938 (97.1% of total)
Ported lines: 392558/411395 (95.4% of total)
Longest unported chain: 6/92 (93.5% progress)

port-progress bot (May 18 2023 at 19:21):

mathlib port progress combinatorics.additive.behrend
Ported files: 929/983 (94.5% of total)
Ported lines: 396184/431139 (91.9% of total)
Longest unported chain: 15/100 (85.0% progress)

port-progress bot (May 18 2023 at 19:26):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 955/1045 (91.4% of total)
Ported lines: 401477/444876 (90.2% of total)
Longest unported chain: 25/97 (74.2% progress)

port-progress bot (May 18 2023 at 19:31):

mathlib port progress measure_theory.integral.bochner
Ported files: 926/965 (96.0% of total)
Ported lines: 405349/436324 (92.9% of total)
Longest unported chain: 10/97 (89.7% progress)

port-progress bot (May 18 2023 at 19:35):

mathlib port progress probability.independence.basic
Ported files: 930/980 (94.9% of total)
Ported lines: 405902/444211 (91.4% of total)
Longest unported chain: 15/102 (85.3% progress)

port-progress bot (May 18 2023 at 19:40):

mathlib port progress representation_theory.group_cohomology.basic
Ported files: 923/964 (95.7% of total)
Ported lines: 366036/380047 (96.3% of total)
Longest unported chain: 10/79 (87.3% progress)

port-progress bot (May 18 2023 at 19:45):

mathlib port progress all
Ported files: 2020/2971 (68.0% of total)
Ported lines: 669637/1026030 (65.3% of total)
Longest unported chain: 30/117 (74.4% progress)

Johan Commelin (May 18 2023 at 19:56):

1.0%

Johan Commelin (May 18 2023 at 19:57):

Shout out to Heather, who conquered 10% of the longest unported chain single-handedly :octopus:

Heather Macbeth (May 18 2023 at 20:00):

Hold your hats, more to come :)

Scott Morrison (May 18 2023 at 20:25):

I've just sent Algebra.Category.Mon.Limits !4#3073 to bors. Hopefully GroupCat.Limits and ModuleCat.Limits are easier if you follow the template of defining and using GroupCatMax and ModuleCatMax.

Heather Macbeth (May 18 2023 at 20:47):

Another day, another split. Actually two today:

#19040 removes the dependence of measure_theory/function/special_functions/basic (which is on the way to the Bochner integral) on normed_space/finite_dimension.

#19039 is a big split and a measure theory specialist might want to look at it. It removes the dependence of the construction of the Lebesgue measure on the Bochner integral.

Heather Macbeth (May 18 2023 at 20:48):

After #19039, the length of the longest chain in mathlib decreases again (to 114) and, even better, the longest unported chain is now in algebra rather than analysis :)

- ring_theory.matrix_algebra
- ring_theory.polynomial_algebra
- linear_algebra.matrix.charpoly.basic
- linear_algebra.matrix.charpoly.coeff
- linear_algebra.matrix.charpoly.linear_map
- ring_theory.integral_closure
- field_theory.minpoly.basic
- field_theory.minpoly.field
- ring_theory.power_basis
- ring_theory.adjoin_root
  ring_theory.localization.away
  algebra.category.Ring.instances
  algebra.category.Ring.constructions
  topology.sheaves.sheaf_condition.pairwise_intersections
  topology.sheaves.sheaf_condition.equalizer_products
  topology.sheaves.forget
  topology.sheaves.sheaf_condition.unique_gluing
  topology.sheaves.stalks
  algebraic_geometry.ringed_space
  algebraic_geometry.locally_ringed_space
  algebraic_geometry.Spec
  algebraic_geometry.Scheme
  algebraic_geometry.open_immersion
  algebraic_geometry.locally_ringed_space.has_colimits
  algebraic_geometry.presheafed_space.gluing
  algebraic_geometry.gluing
  algebraic_geometry.pullbacks
  algebraic_geometry.morphisms.basic
  algebraic_geometry.morphisms.quasi_compact
  algebraic_geometry.morphisms.quasi_separated

Ruben Van de Velde (May 18 2023 at 21:01):

Time for the algebraists to get to work, huh :)

Scott Morrison (May 18 2023 at 21:04):

That long initial sequence of lines beginning with - was irresistible: #19041.

Heather Macbeth (May 18 2023 at 21:06):

Darn! :)

Kevin Buzzard (May 19 2023 at 07:21):

Perhaps schemes should now be considered a new target for the port, now that it is apparently on the naughty chair (i.e. part of the longest chain).

Just trying to get a feeling as to where we are with respect to the targets that are already being tracked, I realise that the percentages in "ported files" are now becoming quite misleading. The fact that in some sense we are "95.7 percent of the way to group cohomology" sounds great but also gives no real indication of how much work is left. "37 files to go!" would be more helpful at this point. Conversely, with the "all" category the percentage is very much unmisleading.

Indeed out of our 8 currently chosen target files, they're all over 90% done and most are over 95% done, so someone giving a cursory glance might conclude that there's no point joining in because probably they'll all be done next week. A perhaps more useful representation of the amount of work left to do for the target files at this point would simply be the number of files left in the pdf, which cannot be computed by the data being presented because the difference between the numerator and denominator of the displayed fraction is always more than this for some reason I've never really understood (someone once explained it to me as "tactic files", but if they're not on the pdf I'm not interested: for example in group cohomology the difference is 41).

port-progress bot (May 19 2023 at 12:26):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Ported files: 923/985 (93.7% of total)
Ported lines: 374367/400636 (93.4% of total)
Longest unported chain: 28/101 (72.3% progress)

port-progress bot (May 19 2023 at 12:30):

mathlib port progress algebra.category.Module.abelian
Ported files: 662/674 (98.2% of total)
Ported lines: 253213/257971 (98.2% of total)
Longest unported chain: 2/71 (97.2% progress)

port-progress bot (May 19 2023 at 12:35):

mathlib port progress algebra.category.Module.adjunctions
Ported files: 568/579 (98.1% of total)
Ported lines: 217872/222253 (98.0% of total)
Longest unported chain: 2/63 (96.8% progress)

port-progress bot (May 19 2023 at 19:04):

mathlib port progress topology.continuous_function.bounded
Ported files: 682/691 (98.7% of total)
Ported lines: 296307/301164 (98.4% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 19 2023 at 19:12):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 842/854 (98.6% of total)
Ported lines: 365739/370852 (98.6% of total)
Longest unported chain: 2/87 (97.7% progress)

port-progress bot (May 19 2023 at 19:16):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 913/939 (97.2% of total)
Ported lines: 394835/411470 (96.0% of total)
Longest unported chain: 5/92 (94.6% progress)

port-progress bot (May 19 2023 at 19:21):

mathlib port progress combinatorics.additive.behrend
Ported files: 931/984 (94.6% of total)
Ported lines: 398461/431214 (92.4% of total)
Longest unported chain: 14/100 (86.0% progress)

port-progress bot (May 19 2023 at 19:26):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 961/1046 (91.9% of total)
Ported lines: 404878/444973 (91.0% of total)
Longest unported chain: 24/97 (75.3% progress)

port-progress bot (May 19 2023 at 19:31):

mathlib port progress measure_theory.integral.bochner
Ported files: 928/965 (96.2% of total)
Ported lines: 407626/436250 (93.4% of total)
Longest unported chain: 10/97 (89.7% progress)

port-progress bot (May 19 2023 at 19:35):

mathlib port progress probability.independence.basic
Ported files: 660/677 (97.5% of total)
Ported lines: 288619/301256 (95.8% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 19 2023 at 19:40):

mathlib port progress representation_theory.group_cohomology.basic
Ported files: 926/968 (95.7% of total)
Ported lines: 366889/380130 (96.5% of total)
Longest unported chain: 10/79 (87.3% progress)

port-progress bot (May 19 2023 at 19:44):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Ported files: 920/977 (94.2% of total)
Ported lines: 374189/398194 (94.0% of total)
Longest unported chain: 19/92 (79.3% progress)

port-progress bot (May 19 2023 at 19:48):

mathlib port progress algebra.category.Module.abelian
Ported files: 662/674 (98.2% of total)
Ported lines: 253213/257971 (98.2% of total)
Longest unported chain: 2/71 (97.2% progress)

port-progress bot (May 19 2023 at 19:53):

mathlib port progress algebra.category.Module.adjunctions
Ported files: 569/579 (98.3% of total)
Ported lines: 218206/222253 (98.2% of total)
Longest unported chain: 1/63 (98.4% progress)

port-progress bot (May 19 2023 at 19:58):

mathlib port progress all
Ported files: 2035/2983 (68.2% of total)
Ported lines: 675794/1026465 (65.8% of total)
Longest unported chain: 28/114 (75.4% progress)

Kevin Buzzard (May 19 2023 at 19:59):

Earlier people were posting lists of files with -s in and someone asked what the - sign means. Can I ask how to see the - signs? I'm wondering how many - signs there are for (random file I'm interested in seeing ported).

Heather Macbeth (May 19 2023 at 20:06):

@Kevin Buzzard in a terminal at cd the top level of mathlib3, with the oleans downloaded, type leanproject port-progress --to measure_theory.integral.bochner and wait about a minute

Heather Macbeth (May 19 2023 at 20:07):

(a summary table comes quickly, you wait, and then the full list comes)

Eric Wieser (May 19 2023 at 20:11):

Can I ask how to see the - signs?

click on the words "longest unported chain"

Kevin Buzzard (May 19 2023 at 20:12):

buzzard@buster:~/lean-projects/mathlib$ leanproject port-progress --to algebraic_geometry.morphisms.quasi_separated
division by zero
buzzard@buster:~/lean-projects/mathlib$

I was hoping for subtractions, not divisions :-)

Kalle Kytölä (May 19 2023 at 21:13):

That looks like a bug: an undefined division by zero instead of a junk value?!? :wink:

Heather Macbeth (May 19 2023 at 21:18):

Possibly try deleting src/all, building again (should only take a second), and then retry?

Jeremy Tan (May 20 2023 at 16:44):

Only three unported files now have over 200 dependents, and none of them have over 250:

  • LinearAlgebra.Dual
  • LinearAlgebra.BilinearForm
  • Analysis.SpecialFunctions.Pow.NNReal

And !4#3659 is awaiting review

port-progress bot (May 20 2023 at 19:04):

mathlib port progress topology.continuous_function.bounded
Ported files: 683/691 (98.8% of total)
Ported lines: 296445/301233 (98.4% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 20 2023 at 19:12):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 845/854 (98.9% of total)
Ported lines: 366635/370921 (98.8% of total)
Longest unported chain: 1/87 (98.9% progress)

port-progress bot (May 20 2023 at 19:16):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 921/939 (98.1% of total)
Ported lines: 397915/411538 (96.7% of total)
Longest unported chain: 5/92 (94.6% progress)

port-progress bot (May 20 2023 at 19:21):

mathlib port progress combinatorics.additive.behrend
Ported files: 940/984 (95.5% of total)
Ported lines: 402003/431282 (93.2% of total)
Longest unported chain: 13/100 (87.0% progress)

port-progress bot (May 20 2023 at 19:26):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 965/1046 (92.3% of total)
Ported lines: 406007/445042 (91.2% of total)
Longest unported chain: 24/97 (75.3% progress)

port-progress bot (May 20 2023 at 19:31):

mathlib port progress measure_theory.integral.bochner
Ported files: 932/965 (96.6% of total)
Ported lines: 409743/436371 (93.9% of total)
Longest unported chain: 10/97 (89.7% progress)

port-progress bot (May 20 2023 at 19:35):

mathlib port progress probability.independence.basic
Ported files: 660/677 (97.5% of total)
Ported lines: 288710/301347 (95.8% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (May 20 2023 at 19:39):

mathlib port progress representation_theory.group_cohomology.basic
Ported files: 928/968 (95.9% of total)
Ported lines: 367002/380130 (96.5% of total)
Longest unported chain: 10/79 (87.3% progress)

port-progress bot (May 20 2023 at 19:44):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Ported files: 920/977 (94.2% of total)
Ported lines: 374189/398194 (94.0% of total)
Longest unported chain: 19/92 (79.3% progress)

port-progress bot (May 20 2023 at 19:48):

mathlib port progress algebra.category.Module.abelian
Ported files: 662/674 (98.2% of total)
Ported lines: 253213/257971 (98.2% of total)
Longest unported chain: 2/71 (97.2% progress)

port-progress bot (May 20 2023 at 19:53):

mathlib port progress algebra.category.Module.adjunctions
Ported files: 570/579 (98.4% of total)
Ported lines: 218260/222253 (98.2% of total)
Longest unported chain: 1/63 (98.4% progress)

port-progress bot (May 20 2023 at 19:57):

mathlib port progress all
Ported files: 2055/2985 (68.8% of total)
Ported lines: 681294/1027335 (66.3% of total)
Longest unported chain: 27/114 (76.3% progress)

Scott Morrison (May 20 2023 at 22:03):

0.5%

Kevin Buzzard (May 21 2023 at 08:31):

I love how the rate was "usually >= 0.5%" but a few weeks ago dropped to "usually <= 0.3%", but after lean4#2210 it has now come back up to "usually >= 0.5%".

Chris Hughes (May 21 2023 at 18:52):

Today's gonna be a big day

port-progress bot (May 21 2023 at 19:04):

mathlib port progress topology.continuous_function.bounded
Ported files: 683/691 (98.8% of total)
Ported lines: 296448/301236 (98.4% of total)
Longest unported chain: 1/85 (98.8% progress)

port-progress bot (May 21 2023 at 19:12):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 845/854 (98.9% of total)
Ported lines: 366650/370936 (98.8% of total)
Longest unported chain: 1/87 (98.9% progress)

port-progress bot (May 21 2023 at 19:17):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 922/939 (98.2% of total)
Ported lines: 398742/411583 (96.9% of total)
Longest unported chain: 5/92 (94.6% progress)

port-progress bot (May 21 2023 at 19:21):

mathlib port progress combinatorics.additive.behrend
Ported files: 941/984 (95.6% of total)
Ported lines: 402833/431330 (93.4% of total)
Longest unported chain: 13/100 (87.0% progress)

port-progress bot (May 21 2023 at 19:26):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 968/1046 (92.5% of total)
Ported lines: 406704/445090 (91.4% of total)
Longest unported chain: 21/97 (78.4% progress)

port-progress bot (May 21 2023 at 19:31):

mathlib port progress measure_theory.integral.bochner
Ported files: 939/965 (97.3% of total)
Ported lines: 416053/436398 (95.3% of total)
Longest unported chain: 10/97 (89.7% progress)

port-progress bot (May 21 2023 at 19:35):

mathlib port progress probability.independence.basic
Ported files: 664/677 (98.1% of total)
Ported lines: 294372/301347 (97.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (May 21 2023 at 19:40):

mathlib port progress representation_theory.group_cohomology.basic
Ported files: 930/968 (96.1% of total)
Ported lines: 367444/380148 (96.7% of total)
Longest unported chain: 10/79 (87.3% progress)

port-progress bot (May 21 2023 at 19:44):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Ported files: 927/977 (94.9% of total)
Ported lines: 376138/398227 (94.5% of total)
Longest unported chain: 19/92 (79.3% progress)

port-progress bot (May 21 2023 at 19:48):

mathlib port progress algebra.category.Module.abelian
Ported files: 664/674 (98.5% of total)
Ported lines: 253640/257974 (98.3% of total)
Longest unported chain: 2/71 (97.2% progress)

port-progress bot (May 21 2023 at 19:53):

mathlib port progress algebra.category.Module.adjunctions
Ported files: 570/579 (98.4% of total)
Ported lines: 218266/222259 (98.2% of total)
Longest unported chain: 1/63 (98.4% progress)

port-progress bot (May 21 2023 at 19:58):

mathlib port progress all
Ported files: 2086/2985 (69.9% of total)
Ported lines: 694826/1027524 (67.6% of total)
Longest unported chain: 27/114 (76.3% progress)

Chris Hughes (May 21 2023 at 19:58):

1.3%

Tobias Grosser (May 22 2023 at 05:58):

Congratulations!

Patrick Massot (May 22 2023 at 16:49):

@Scott Morrison topology.continuous_function.bounded can be removed from this list.

port-progress bot (May 22 2023 at 19:07):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 845/854 (98.9% of total)
Ported lines: 366660/370946 (98.8% of total)
Longest unported chain: 1/87 (98.9% progress)

port-progress bot (May 22 2023 at 19:12):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 924/939 (98.4% of total)
Ported lines: 401464/411595 (97.5% of total)
Longest unported chain: 3/92 (96.7% progress)

port-progress bot (May 22 2023 at 19:16):

mathlib port progress combinatorics.additive.behrend
Ported files: 949/984 (96.4% of total)
Ported lines: 408012/431368 (94.6% of total)
Longest unported chain: 10/100 (90.0% progress)

port-progress bot (May 22 2023 at 19:20):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 975/1046 (93.2% of total)
Ported lines: 413308/445298 (92.8% of total)
Longest unported chain: 19/97 (80.4% progress)

port-progress bot (May 22 2023 at 19:25):

mathlib port progress measure_theory.integral.bochner
Ported files: 943/965 (97.7% of total)
Ported lines: 418025/436435 (95.8% of total)
Longest unported chain: 8/97 (91.8% progress)

port-progress bot (May 22 2023 at 19:29):

mathlib port progress probability.independence.basic
Ported files: 665/677 (98.2% of total)
Ported lines: 294612/301395 (97.7% of total)
Longest unported chain: 3/91 (96.7% progress)

port-progress bot (May 22 2023 at 19:33):

mathlib port progress representation_theory.group_cohomology.basic
Ported files: 932/968 (96.3% of total)
Ported lines: 369094/380164 (97.1% of total)
Longest unported chain: 10/79 (87.3% progress)

port-progress bot (May 22 2023 at 19:37):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Ported files: 932/977 (95.4% of total)
Ported lines: 378516/398261 (95.0% of total)
Longest unported chain: 18/92 (80.4% progress)

port-progress bot (May 22 2023 at 19:41):

mathlib port progress algebra.category.Module.abelian
Ported files: 664/674 (98.5% of total)
Ported lines: 253653/257987 (98.3% of total)
Longest unported chain: 2/71 (97.2% progress)

port-progress bot (May 22 2023 at 19:45):

mathlib port progress algebra.category.Module.adjunctions
Ported files: 570/579 (98.4% of total)
Ported lines: 218273/222266 (98.2% of total)
Longest unported chain: 1/63 (98.4% progress)

port-progress bot (May 22 2023 at 19:49):

mathlib port progress all
Ported files: 2141/2987 (71.7% of total)
Ported lines: 717672/1028472 (69.8% of total)
Longest unported chain: 24/113 (78.8% progress)

Johan Commelin (May 22 2023 at 19:51):

2.2%

Chris Hughes (May 22 2023 at 19:57):

55 files

port-progress bot (May 23 2023 at 19:07):

mathlib port progress analysis.normed_space.hahn_banach.extension
Ported files: 846/854 (99.1% of total)
Ported lines: 367390/370962 (99.0% of total)
Longest unported chain: 1/87 (98.9% progress)

port-progress bot (May 23 2023 at 19:11):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 924/939 (98.4% of total)
Ported lines: 401486/411617 (97.5% of total)
Longest unported chain: 3/92 (96.7% progress)

port-progress bot (May 23 2023 at 19:15):

mathlib port progress combinatorics.additive.behrend
Ported files: 952/985 (96.6% of total)
Ported lines: 409185/431535 (94.8% of total)
Longest unported chain: 10/100 (90.0% progress)

port-progress bot (May 23 2023 at 19:20):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 990/1046 (94.6% of total)
Ported lines: 419401/445340 (94.2% of total)
Longest unported chain: 16/97 (83.5% progress)

port-progress bot (May 23 2023 at 19:24):

mathlib port progress measure_theory.integral.bochner
Ported files: 944/965 (97.8% of total)
Ported lines: 419991/436457 (96.2% of total)
Longest unported chain: 8/97 (91.8% progress)

port-progress bot (May 23 2023 at 19:28):

mathlib port progress probability.independence.basic
Ported files: 665/677 (98.2% of total)
Ported lines: 294615/301398 (97.7% of total)
Longest unported chain: 3/91 (96.7% progress)

port-progress bot (May 23 2023 at 19:32):

mathlib port progress representation_theory.group_cohomology.basic
Ported files: 933/968 (96.4% of total)
Ported lines: 369497/380170 (97.2% of total)
Longest unported chain: 10/79 (87.3% progress)

port-progress bot (May 23 2023 at 19:36):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Ported files: 937/977 (95.9% of total)
Ported lines: 380066/398276 (95.4% of total)
Longest unported chain: 18/92 (80.4% progress)

port-progress bot (May 23 2023 at 19:40):

mathlib port progress algebra.category.Module.abelian
Ported files: 664/674 (98.5% of total)
Ported lines: 253653/257987 (98.3% of total)
Longest unported chain: 2/71 (97.2% progress)

port-progress bot (May 23 2023 at 19:44):

mathlib port progress algebra.category.Module.adjunctions
Ported files: 570/579 (98.4% of total)
Ported lines: 218273/222266 (98.2% of total)
Longest unported chain: 1/63 (98.4% progress)

port-progress bot (May 23 2023 at 19:49):

mathlib port progress all
Ported files: 2171/2989 (72.6% of total)
Ported lines: 731351/1029369 (71.0% of total)
Longest unported chain: 24/113 (78.8% progress)

Chris Hughes (May 23 2023 at 20:00):

1.2%

port-progress bot (May 24 2023 at 03:36):

459 files completely ported, out of 2992.

Tobias Grosser (May 24 2023 at 11:13):

Wow, things are moving super fast now. That's impressive.

port-progress bot (May 24 2023 at 14:53):

465/2992 files completely ported (15.00%).

Scott Morrison (May 24 2023 at 15:50):

@Eric Wieser, do you know what is going on with analysis.calculus.deriv on the port dashboard? It says that it is in progress via !4#4254 , but that is an unrelated PR adding new material.

Eric Wieser (May 24 2023 at 15:50):

The port dashboard (port-status#analysis/calculus/deriv) is just regurgitating what #port-wiki says

Eric Wieser (May 24 2023 at 15:52):

Though I think it's somewhat moot because @Yury G. Kudryashov indicated they were going to split the file in mathlib3 first

Eric Wieser (May 24 2023 at 15:52):

#port-wiki in turn is generated from https://github.com/leanprover-community/mathlib4/blob/master/scripts/make_port_status.py, and evidently this script uses the wrong heuristics to identify PRs

Eric Wieser (May 24 2023 at 15:53):

But if you modify that script you have to ask Johan Commelin nicely to update the version that is actually being run

Patrick Massot (May 24 2023 at 15:53):

Does anyone knows why the port-progress bot posts mysterious outdated statistics such as 465/2992 files completely ported (15.00%).?

Yury G. Kudryashov (May 24 2023 at 15:53):

I ported it, then my PR that drops some unneeded assumptions was merged.

Eric Wieser (May 24 2023 at 15:53):

(obligatory diagram link)

Yury G. Kudryashov (May 24 2023 at 15:55):

I will split deriv today, wait for mathport, then mirror changes in mathlib4. I know how to rewrite git history so that it will be easy to review.

Chris Hughes (May 24 2023 at 15:59):

Patrick Massot said:

Does anyone knows why the port-progress bot posts mysterious outdated statistics such as 465/2992 files completely ported (15.00%).?

I think completely ported means everything that depends on it is ported. This could be made clearer.

Scott Morrison (May 24 2023 at 16:10):

Chris Hughes said:

Patrick Massot said:

Does anyone knows why the port-progress bot posts mysterious outdated statistics such as 465/2992 files completely ported (15.00%).?

I think completely ported means everything that depends on it is ported. This could be made clearer.

Updated.

Scott Morrison (May 24 2023 at 16:13):

I have removed analysis.normed_space.hahn_banach.extension from the port-progress-bot, as it is done! :tada:

I've added four new targets Heather suggested, which the bot will post on shortly.

Patrick Massot (May 24 2023 at 16:15):

Oooh! Thanks a lot Chris, I was very far from guessing that.

port-progress bot (May 24 2023 at 16:20):

mathlib port progress analysis.complex.cauchy_integral
Ported files: 1031/1101 (93.6% of total)
Ported lines: 445740/495748 (89.9% of total)
Longest unported chain: 14/104 (86.5% progress)

port-progress bot (May 24 2023 at 16:26):

mathlib port progress analysis.fourier.add_circle
Ported files: 1028/1103 (93.2% of total)
Ported lines: 445308/497469 (89.5% of total)
Longest unported chain: 13/103 (87.4% progress)

port-progress bot (May 24 2023 at 16:31):

mathlib port progress geometry.manifold.whitney_embedding
Ported files: 1033/1115 (92.6% of total)
Ported lines: 448302/504838 (88.8% of total)
Longest unported chain: 18/109 (83.5% progress)

port-progress bot (May 24 2023 at 16:35):

mathlib port progress measure_theory.function.jacobian
Ported files: 1027/1088 (94.4% of total)
Ported lines: 446634/495115 (90.2% of total)
Longest unported chain: 16/106 (84.9% progress)

port-progress bot (May 24 2023 at 16:37):

465/2994 files completely ported (15.00%), in the sense that also all downstream dependencies are ported.

Patrick Massot (May 24 2023 at 16:39):

Do we have any file that is less than 90% ported?

Heather Macbeth (May 24 2023 at 16:40):

Yes, a few, you can order by dependencies on the #port-status page.

Heather Macbeth (May 24 2023 at 16:41):

For example, number_theory.modular_forms.jacobi_theta has 118 + 18 unported dependencies and 1063 ported dependencies, which I make to be 88.6% ported.

Heather Macbeth (May 24 2023 at 16:43):

That's files rather than lines -- actually I see that several of the newly-added analysis targets are also less than 90% ported on files.

Eric Wieser (May 24 2023 at 16:44):

There's a (lines) column you can now sort on too

port-progress bot (May 24 2023 at 19:07):

mathlib port progress analysis.inner_product_space.pi_L2
Ported files: 925/940 (98.4% of total)
Ported lines: 401617/411748 (97.5% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (May 24 2023 at 19:11):

mathlib port progress combinatorics.additive.behrend
Ported files: 955/986 (96.9% of total)
Ported lines: 409723/431706 (94.9% of total)
Longest unported chain: 10/101 (90.1% progress)

Kevin Buzzard (May 24 2023 at 19:13):

Patrick Massot said:

Do we have any file that is less than 90% ported?

Yes I made this point recently, the percentages are very misleading now. A better figure is simply the number of files in the pdf, which you can't work out from the 1033/1115 fraction because this includes random tactic files which are not going to be ported. Example: analysis.inner_product_space.pi_L2 is 98.4% ported (meaningless), 925/940 (still kind of meaningless), and 8 nodes in the pdf (concrete information about how much work is actually left).

port-progress bot (May 24 2023 at 19:16):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Ported files: 997/1049 (95.0% of total)
Ported lines: 421774/445577 (94.7% of total)
Longest unported chain: 15/97 (84.5% progress)

Kevin Buzzard (May 24 2023 at 19:19):

45 files to go for that one

port-progress bot (May 24 2023 at 19:20):

mathlib port progress measure_theory.integral.bochner
Ported files: 946/966 (97.9% of total)
Ported lines: 420828/436539 (96.4% of total)
Longest unported chain: 8/98 (91.8% progress)

Kevin Buzzard (May 24 2023 at 19:21):

13 for that. Aah, is it always D-N-7 or so, if the ratio is N/D?

port-progress bot (May 24 2023 at 19:24):

mathlib port progress probability.independence.basic
Ported files: 665/677 (98.2% of total)
Ported lines: 294633/301416 (97.7% of total)
Longest unported chain: 3/91 (96.7% progress)

Ruben Van de Velde (May 24 2023 at 19:25):

Kevin Buzzard said:

13 for that. Aah, is it always D-N-7 or so, if the ratio is N/D?

I see we've got a number theorist in the room :)

Kevin Buzzard (May 24 2023 at 19:27):

yeah, that last one 665/677 so D-N=12 and there are 5 files in the pdf

port-progress bot (May 24 2023 at 19:28):

mathlib port progress representation_theory.group_cohomology.basic
Ported files: 934/968 (96.5% of total)
Ported lines: 370101/380176 (97.3% of total)
Longest unported chain: 10/79 (87.3% progress)

port-progress bot (May 24 2023 at 19:32):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Ported files: 939/977 (96.1% of total)
Ported lines: 381163/398283 (95.7% of total)
Longest unported chain: 18/92 (80.4% progress)

Kevin Buzzard (May 24 2023 at 19:33):

Conjecture holding up

port-progress bot (May 24 2023 at 19:36):

mathlib port progress algebra.category.Module.abelian
Ported files: 665/674 (98.7% of total)
Ported lines: 254251/257987 (98.6% of total)
Longest unported chain: 1/71 (98.6% progress)

Kevin Buzzard (May 24 2023 at 19:39):

Just 2 to go for that one

port-progress bot (May 24 2023 at 19:40):

mathlib port progress algebra.category.Module.adjunctions
Ported files: 570/579 (98.4% of total)
Ported lines: 218273/222266 (98.2% of total)
Longest unported chain: 1/63 (98.4% progress)

Eric Wieser (May 24 2023 at 19:40):

If you just want the number of unported files just read the #port-dashboard page?

Eric Wieser (May 24 2023 at 19:40):

Can we have the bot include links to that too?

Kevin Buzzard (May 24 2023 at 19:42):

The number of actually unported lines would also be a useful measure now we're at this stage, it's no longer helpful to know that we've ported 254251 lines towards abelian categories

Kevin Buzzard (May 24 2023 at 19:43):

Probably there is some other constant analogous to 7 where you do D-N-constant and see the actual number of lines left to go, but right now this involves subtracting 6 digit numbers from other 6 digit numbers

port-progress bot (May 24 2023 at 19:45):

mathlib port progress analysis.complex.cauchy_integral
Ported files: 1031/1101 (93.6% of total)
Ported lines: 445740/495748 (89.9% of total)
Longest unported chain: 14/104 (86.5% progress)

port-progress bot (May 24 2023 at 19:49):

mathlib port progress analysis.fourier.add_circle
Ported files: 1028/1103 (93.2% of total)
Ported lines: 445308/497469 (89.5% of total)
Longest unported chain: 13/103 (87.4% progress)

port-progress bot (May 24 2023 at 19:54):

mathlib port progress geometry.manifold.whitney_embedding
Ported files: 1033/1115 (92.6% of total)
Ported lines: 448302/504838 (88.8% of total)
Longest unported chain: 18/109 (83.5% progress)

port-progress bot (May 24 2023 at 19:58):

mathlib port progress measure_theory.function.jacobian
Ported files: 1027/1088 (94.4% of total)
Ported lines: 446634/495115 (90.2% of total)
Longest unported chain: 16/106 (84.9% progress)

port-progress bot (May 24 2023 at 20:03):

mathlib port progress all
Ported files: 2191/2993 (73.2% of total)
Ported lines: 737896/1030031 (71.6% of total)
Longest unported chain: 24/114 (78.9% progress)

port-progress bot (May 24 2023 at 20:04):

465/2994 files completely ported (15.00%), in the sense that also all downstream dependencies are ported.

Kevin Buzzard (May 24 2023 at 20:05):

If the D-N-7 conjecture is correct then there are under 800 files to go (the 7 saves us). Recall that we did over 50 in a day the other day.

Eric Wieser (May 24 2023 at 20:07):

Kevin Buzzard said:

The number of actually unported lines would also be a useful measure now we're at this stage, it's no longer helpful to know that we've ported 254251 lines towards abelian categories

Hovering over the progress bar at port-status#algebra/category/Module/abelian tells you the number of unported lines and files

Eric Wieser (May 24 2023 at 20:08):

Thought admittedly there are only 3 pixels or so of hover target!

Yaël Dillies (May 24 2023 at 20:14):

Kevin Buzzard said:

Conjecture holding up

Could it be backed up by a million pounds cash prize?

Kevin Buzzard (May 24 2023 at 20:33):

Eric Wieser said:

Thought admittedly there are only 3 pixels or so of hover target!

Oh lol it's the little yellow lines? Ha ha that's not something people are going to notice easily! Thanks! I still can't get the "number of lines" one working, I need to get my glasses I think.

Eric Wieser (May 24 2023 at 20:34):

No, the yellow line is the in progress ones. Depending on whether you're viewing the dashboard in dark/light mode, it's the even smaller black/white sections

Eric Wieser (May 24 2023 at 20:35):

(dark light mode matches whatever choice you made on the mathlib3 docs)

Kevin Buzzard (May 24 2023 at 20:36):

success2.png

Eric Wieser (May 24 2023 at 20:39):

Ah, in this case there are no unported lines, they're all in progress!

Kevin Buzzard (May 24 2023 at 20:42):

So in summary, obviously the tooling is fabulous and now after this investigation I realise that it's easy to work out the data which is meaningful to me from the data being offered to us. I guess one simple suggestion would be simply to change reporting "ported files" and "ported lines" to "unported files" and "unported lines" now we are well over half way through, as these numbers are easier to understand.

Ruben Van de Velde (May 24 2023 at 20:50):

If we're doing suggestions, can the page for unported files contain the lean-4-ified path that I need to pass to start_port.sh?

Eric Wieser (May 24 2023 at 21:03):

PRs welcome at https://github.com/leanprover-community/mathlib-port-status! It's unfortunately a pile of hacks, but you can open it gitpod and build (~10 minutes) the changes to see if things work

Eric Wieser (May 24 2023 at 21:03):

file.j2 is what renders each page

Scott Morrison (May 25 2023 at 00:39):

Okay, re-running the port progress bot reporting D-N-7. If someone feels like computing the magic constant for the number of lines I can include that too.

port-progress bot (May 25 2023 at 00:43):

mathlib port progress all
Unported files: 799/2993 (73.3% of total)
Unported lines: 291747/1030045 (71.7% of total)
Longest unported chain: 24/114 (78.9% progress)

port-progress bot (May 25 2023 at 00:45):

466/2994 files completely ported (15.00%), in the sense that also all downstream dependencies are ported.

Anne Baanen (May 25 2023 at 01:27):

0.7%

Scott Morrison (May 25 2023 at 02:29):

Oh, maybe we shouldn't count this one. It was an "extra" to test the new statistics (unported rather than ported).

Scott Morrison (May 25 2023 at 02:30):

Ah, I see, that's that difference since yesterday in any case, as no one did the difference earlier today. Sorry for the noise. :-)

Anne Baanen (May 25 2023 at 02:32):

Porting 0.7% in 4 hours is slightly too high of an expectation, even given the records we set in the past few days :)

Yury G. Kudryashov (May 25 2023 at 06:18):

!4#4327 brings the "out-of-date" list back below 20.

Yury G. Kudryashov (May 25 2023 at 06:25):

Forward-porting #18990 which is responsible for another 6 files on the list.

Yury G. Kudryashov (May 25 2023 at 07:09):

Done in !4#4328

Eric Wieser (May 25 2023 at 07:11):

Thanks, I was going to do that one myself in 4 hours or so; I'll review in 3 hours from now if no one else gets there first

Yury G. Kudryashov (May 25 2023 at 07:53):

See also !4#4330 (depends on !4#4327)

Eric Wieser (May 25 2023 at 15:05):

@Johan Commelin, you missed step 3 of the forward-porting review instructions, which suggests you didn't do step 4 either!

Eric Wieser (May 25 2023 at 15:05):

(And @Yury G. Kudryashov, you missed step 8 of the forward-proting PR instructions on the same page)

Eric Wieser (May 25 2023 at 15:06):

(meanwhile, I missed my target time by 5 hours...)

Johan Commelin (May 25 2023 at 15:06):

Ooh, sorry! I didn't know about this page! I just had the two PRs open side-by-side and compared them basically line-by-line

Eric Wieser (May 25 2023 at 15:07):

Ah, sounds like you just did the hard-mode version of what you were supposed to do!

Eric Wieser (May 25 2023 at 15:07):

I didn't know about this page!

It's linked from #outofsync now :)

Yury G. Kudryashov (May 25 2023 at 15:33):

!4#4342

Yury G. Kudryashov (May 25 2023 at 15:37):

Also updates !4#4330

port-progress bot (May 25 2023 at 19:08):

mathlib port progress analysis.inner_product_space.pi_L2
Unported files: 13/940 (98.6% of total)
Unported lines: 9074/411758 (97.8% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (May 25 2023 at 19:12):

mathlib port progress combinatorics.additive.behrend
Unported files: 25/986 (97.5% of total)
Unported lines: 20108/431725 (95.3% of total)
Longest unported chain: 8/101 (92.1% progress)

port-progress bot (May 25 2023 at 19:17):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 48/1049 (95.4% of total)
Unported lines: 22539/445605 (94.9% of total)
Longest unported chain: 14/97 (85.6% progress)

port-progress bot (May 25 2023 at 19:21):

mathlib port progress measure_theory.integral.bochner
Unported files: 13/966 (98.7% of total)
Unported lines: 12716/436653 (97.1% of total)
Longest unported chain: 5/98 (94.9% progress)

Mauricio Collares (May 25 2023 at 19:22):

I think this run missed the newest batch of commits that just landed a minute ago

Damiano Testa (May 25 2023 at 19:24):

Tomorrow will be a better day...

Mauricio Collares (May 25 2023 at 19:25):

Hopefully true! But today is looking good too

port-progress bot (May 25 2023 at 19:25):

mathlib port progress probability.independence.basic
Unported files: 12/677 (98.2% of total)
Unported lines: 6776/301423 (97.7% of total)
Longest unported chain: 3/91 (96.7% progress)

port-progress bot (May 25 2023 at 19:29):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 31/968 (96.8% of total)
Unported lines: 9697/380189 (97.4% of total)
Longest unported chain: 10/79 (87.3% progress)

port-progress bot (May 25 2023 at 19:33):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 35/977 (96.4% of total)
Unported lines: 15934/398296 (96.0% of total)
Longest unported chain: 17/92 (81.5% progress)

port-progress bot (May 25 2023 at 19:36):

mathlib port progress algebra.category.Module.abelian
Unported files: 7/674 (99.0% of total)
Unported lines: 3409/258000 (98.7% of total)
Longest unported chain: 1/71 (98.6% progress)

port-progress bot (May 25 2023 at 19:40):

mathlib port progress algebra.category.Module.adjunctions
Unported files: 9/579 (98.4% of total)
Unported lines: 3986/222273 (98.2% of total)
Longest unported chain: 1/63 (98.4% progress)

port-progress bot (May 25 2023 at 19:45):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 55/1101 (95.0% of total)
Unported lines: 43202/495874 (91.3% of total)
Longest unported chain: 11/104 (89.4% progress)

port-progress bot (May 25 2023 at 19:49):

mathlib port progress analysis.fourier.add_circle
Unported files: 61/1103 (94.5% of total)
Unported lines: 45867/497595 (90.8% of total)
Longest unported chain: 10/103 (90.3% progress)

port-progress bot (May 25 2023 at 19:54):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 69/1115 (93.8% of total)
Unported lines: 50487/504961 (90.0% of total)
Longest unported chain: 16/109 (85.3% progress)

port-progress bot (May 25 2023 at 19:59):

mathlib port progress measure_theory.function.jacobian
Unported files: 49/1088 (95.5% of total)
Unported lines: 42449/495235 (91.4% of total)
Longest unported chain: 13/106 (87.7% progress)

port-progress bot (May 25 2023 at 20:03):

mathlib port progress all
Unported files: 753/2993 (74.8% of total)
Unported lines: 275712/1030208 (73.2% of total)
Longest unported chain: 21/114 (81.6% progress)

port-progress bot (May 25 2023 at 20:04):

489/2994 files completely ported (16.00%), in the sense that also all downstream dependencies are ported.

Reid Barton (May 25 2023 at 20:08):

GHCi, version 8.6.5: http://www.haskell.org/ghc/  :? for help
Prelude> 489/2994
0.16332665330661322

Johan Commelin (May 25 2023 at 20:09):

1.5%

Anne Baanen (May 25 2023 at 20:09):

1.5%

Scott Morrison (May 25 2023 at 20:31):

Okay, bcs rounding behaviour is weird. More decimals places will be available in future runs. :-)

Sebastian Ullrich (May 25 2023 at 21:05):

I believe bc is one of those cursed Unix utils that is not actually meant to ever be used

Henrik Böving (May 25 2023 at 21:16):

https://xkcd.com/1172/ holds here. The day our internal IT at work decided to remove bc two people complained that their scripts stopped working.

port-progress bot (May 26 2023 at 19:07):

mathlib port progress analysis.inner_product_space.pi_L2
Unported files: 9/941 (99.0% of total)
Unported lines: 5114/412142 (98.8% of total)
Longest unported chain: 1/93 (98.9% progress)

port-progress bot (May 26 2023 at 19:11):

mathlib port progress combinatorics.additive.behrend
Unported files: 20/987 (98.0% of total)
Unported lines: 16009/432109 (96.3% of total)
Longest unported chain: 8/101 (92.1% progress)

port-progress bot (May 26 2023 at 19:16):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 42/1049 (96.0% of total)
Unported lines: 17609/445725 (96.0% of total)
Longest unported chain: 14/97 (85.6% progress)

port-progress bot (May 26 2023 at 19:20):

mathlib port progress measure_theory.integral.bochner
Unported files: 13/966 (98.7% of total)
Unported lines: 12835/436892 (97.1% of total)
Longest unported chain: 5/98 (94.9% progress)

port-progress bot (May 26 2023 at 19:24):

mathlib port progress probability.independence.basic
Unported files: 12/677 (98.2% of total)
Unported lines: 6776/301543 (97.8% of total)
Longest unported chain: 3/91 (96.7% progress)

port-progress bot (May 26 2023 at 19:28):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 30/968 (96.9% of total)
Unported lines: 9624/380301 (97.5% of total)
Longest unported chain: 10/79 (87.3% progress)

port-progress bot (May 26 2023 at 19:32):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 32/977 (96.7% of total)
Unported lines: 15210/398397 (96.2% of total)
Longest unported chain: 15/92 (83.7% progress)

port-progress bot (May 26 2023 at 19:35):

mathlib port progress algebra.category.Module.abelian
Unported files: 7/674 (99.0% of total)
Unported lines: 3409/258019 (98.7% of total)
Longest unported chain: 1/71 (98.6% progress)

port-progress bot (May 26 2023 at 19:39):

mathlib port progress algebra.category.Module.adjunctions
Unported files: 9/579 (98.4% of total)
Unported lines: 3986/222292 (98.2% of total)
Longest unported chain: 1/63 (98.4% progress)

port-progress bot (May 26 2023 at 19:44):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 52/1102 (95.3% of total)
Unported lines: 41458/496377 (91.6% of total)
Longest unported chain: 11/104 (89.4% progress)

port-progress bot (May 26 2023 at 19:48):

mathlib port progress analysis.fourier.add_circle
Unported files: 57/1104 (94.8% of total)
Unported lines: 44123/498148 (91.1% of total)
Longest unported chain: 10/103 (90.3% progress)

port-progress bot (May 26 2023 at 19:53):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 66/1116 (94.1% of total)
Unported lines: 48756/505477 (90.4% of total)
Longest unported chain: 16/109 (85.3% progress)

port-progress bot (May 26 2023 at 19:57):

mathlib port progress measure_theory.function.jacobian
Unported files: 46/1089 (95.8% of total)
Unported lines: 40705/495738 (91.8% of total)
Longest unported chain: 13/106 (87.7% progress)

port-progress bot (May 26 2023 at 20:02):

mathlib port progress all
Unported files: 721/2994 (75.9% of total)
Unported lines: 266996/1030994 (74.1% of total)
Longest unported chain: 21/114 (81.6% progress)

Anne Baanen (May 26 2023 at 20:03):

0.9%

port-progress bot (May 26 2023 at 20:03):

498/2995 files completely ported (16.62%), in the sense that also all downstream dependencies are ported.

Jeremy Tan (May 26 2023 at 20:56):

port-progress bot said:

mathlib port progress all
Unported files: 721/2994 (75.9% of total)
Unported lines: 266996/1030994 (74.1% of total)
Longest unported chain: 21/114 (81.6% progress)

The PDF for this is not being generated

Scott Morrison (May 27 2023 at 17:57):

port-progress bot said:

498/2995 files completely ported (16.62%), in the sense that also all downstream dependencies are ported.

Just a note that this percentage is expected to lag far behind the other numbers, and to move "discontinuously". It can only increase when leaf files are ported, and a single leaf file being ported can result in arbitrarily many files becoming "completely ported". In particular if the import graph were linear this would increase from 0% to 100% when the unique leaf was ported.

Scott Morrison (May 27 2023 at 18:34):

We did 8.3% over the last week. The last week was unusual, as many people active in porting were together in the same place (Banff), so presumably we won't continue at quite this pace. If we were to, however, then it would only be ~3 weeks until the end!

port-progress bot (May 27 2023 at 19:07):

mathlib port progress analysis.inner_product_space.pi_L2
Unported files: 8/941 (99.1% of total)
Unported lines: 4291/412213 (99.0% of total)
Longest unported chain: 1/93 (98.9% progress)

Ruben Van de Velde (May 27 2023 at 19:11):

port-progress bot said:

mathlib port progress analysis.inner_product_space.pi_L2
Unported files: 8/941 (99.1% of total)
Unported lines: 4291/412213 (99.0% of total)
Longest unported chain: 1/93 (98.9% progress)

This is !4#4420

port-progress bot (May 27 2023 at 19:11):

mathlib port progress combinatorics.additive.behrend
Unported files: 19/987 (98.1% of total)
Unported lines: 15186/432192 (96.5% of total)
Longest unported chain: 8/101 (92.1% progress)

port-progress bot (May 27 2023 at 19:16):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 41/1049 (96.1% of total)
Unported lines: 17085/445808 (96.2% of total)
Longest unported chain: 14/97 (85.6% progress)

Scott Morrison (May 27 2023 at 19:18):

Ruben Van de Velde said:

This is !4#4420

I fixed a few errors. This one is very close.

Scott Morrison (May 27 2023 at 19:19):

port-progress bot said:

combinatorics.additive.behrend

This is waiting on the refactor of deriv to land, which should be soon.

Scott Morrison (May 27 2023 at 19:20):

port-progress bot said:

number_theory.legendre_symbol.quadratic_reciprocity

is stuck on SplittingField.

port-progress bot (May 27 2023 at 19:20):

mathlib port progress measure_theory.integral.bochner
Unported files: 14/967 (98.6% of total)
Unported lines: 12871/436999 (97.1% of total)
Longest unported chain: 6/99 (93.9% progress)

port-progress bot (May 27 2023 at 19:25):

mathlib port progress probability.independence.basic
Unported files: 12/677 (98.2% of total)
Unported lines: 6776/301543 (97.8% of total)
Longest unported chain: 3/91 (96.7% progress)

port-progress bot (May 27 2023 at 19:33):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 29/968 (97.0% of total)
Unported lines: 9508/380313 (97.5% of total)
Longest unported chain: 10/79 (87.3% progress)

Scott Morrison (May 27 2023 at 19:44):

port-progress bot said:

measure_theory.integral.bochner

This unfortunately got snagged by mathlib3 PRs, and a bunch of work by @Pol'tta / Miyahara Kō had to be discarded (see !4#4341 and the chain of dependent PRs from there). I think the current status is that we are waiting for the next mathport run to restart this. As far as I can see #19083 was a mathlib3 PR that could have waited to happen in mathlib4, and consequently held up the port.

Scott Morrison (May 27 2023 at 19:50):

port-progress bot said:

representation_theory.group_cohomology.basic

is waiting on !4#4357 which @Kyle Miller is currently reviewing / refactoring.

port-progress bot (May 27 2023 at 19:55):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 28/977 (97.1% of total)
Unported lines: 14048/398471 (96.5% of total)
Longest unported chain: 12/92 (87.0% progress)

Eric Wieser (May 27 2023 at 19:55):

Scott Morrison said:

port-progress bot said:

measure_theory.integral.bochner

a bunch of work by Pol'tta / Miyahara Kō had to be discarded (see !4#4341 and the chain of dependent PRs from there).

The work in the dependent PRs should be salvageable; it was just the one file that needs to be discarded.

Eric Wieser (May 27 2023 at 19:55):

The porting dashboard was clear that there was a mathlib3 PR that modified the file, and that it should not be ported without waiting. I'm sad for @Pol'tta / Miyahara Kō that their work was wasted, but they made the choice to ignore the warning without starting a discussion about it.

Ruben Van de Velde (May 27 2023 at 19:56):

Scott Morrison said:

Ruben Van de Velde said:

This is !4#4420

I fixed a few errors. This one is very close.

Thanks. It's up for review now

Scott Morrison (May 27 2023 at 19:56):

port-progress bot said:

algebraic_geometry.morphisms.quasi_separated

This one is wide open, and needs someone to start porting files! Both topology.sheaves.sheaf_of_functions and topology.sheaves.stalks look like they are ready to go.

port-progress bot (May 27 2023 at 19:58):

mathlib port progress algebra.category.Module.abelian
Unported files: 7/674 (99.0% of total)
Unported lines: 3409/258022 (98.7% of total)
Longest unported chain: 1/71 (98.6% progress)

Scott Morrison (May 27 2023 at 20:01):

port-progress bot said:

algebra.category.Module.abelian

Oops, done, I need to remove this from the bot.

port-progress bot (May 27 2023 at 20:02):

mathlib port progress algebra.category.Module.adjunctions
Unported files: 9/579 (98.4% of total)
Unported lines: 3986/222292 (98.2% of total)
Longest unported chain: 1/63 (98.4% progress)

port-progress bot (May 27 2023 at 20:06):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 52/1103 (95.3% of total)
Unported lines: 40671/496517 (91.8% of total)
Longest unported chain: 12/105 (88.6% progress)

Scott Morrison (May 27 2023 at 20:09):

port-progress bot said:

algebra.category.Module.adjunctions

is waiting on !4#4368, which was marked on WIP but I think, @Matthew Ballard, is okay to mark as awaiting-review?

port-progress bot (May 27 2023 at 20:11):

mathlib port progress analysis.fourier.add_circle
Unported files: 57/1105 (94.8% of total)
Unported lines: 43336/498288 (91.3% of total)
Longest unported chain: 11/104 (89.4% progress)

Matthew Ballard (May 27 2023 at 20:12):

In !4#4368, there is a grotesque set_option maxHeartbeats 0 in because of a convert proof. I haven't had time to try to improve it yet but it should not be too hard.

Matthew Ballard (May 27 2023 at 20:13):

Please feel free to take a look. My hands are full for a bit.

port-progress bot (May 27 2023 at 20:16):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 66/1117 (94.1% of total)
Unported lines: 48044/505686 (90.5% of total)
Longest unported chain: 16/109 (85.3% progress)

port-progress bot (May 27 2023 at 20:20):

mathlib port progress measure_theory.function.jacobian
Unported files: 46/1090 (95.8% of total)
Unported lines: 39933/495884 (91.9% of total)
Longest unported chain: 14/107 (86.9% progress)

port-progress bot (May 27 2023 at 20:25):

mathlib port progress all
Unported files: 702/2995 (76.6% of total)
Unported lines: 261216/1031509 (74.7% of total)
Longest unported chain: 22/115 (80.9% progress)

port-progress bot (May 27 2023 at 20:25):

0/2996 files completely ported (0%), in the sense that also all downstream dependencies are ported.

Scott Morrison (May 27 2023 at 20:25):

port-progress bot said:

0/2996 files completely ported (0%), in the sense that also all downstream dependencies are ported.

Ooops, something went wrong there!

Scott Morrison (May 27 2023 at 20:42):

Hmm, runs okay locally. I've told the bot to try again?

port-progress bot (May 27 2023 at 20:43):

507/2996 files completely ported (16.92%), in the sense that also all downstream dependencies are ported.

Kyle Miller (May 27 2023 at 20:46):

@Matthew Ballard I'm guessing convert is having to unfold a whole lot of stuff. set_option trace.congr! true is a way to see what steps it actually ends up taking, and you can see that the main congruence step is just "show the left-hand sides and right-hand sides of these equalities are equal", and then it manages to prove the following goals using one of its methods to dispatch goals it generates; it doesn't report which one it uses, but I imagine it probably refl here. There probably should be an option for turning this off, or at least having it do only obvious refls.

Here are the goals. If you prove them as local hypotheses, then convert will pick them up using assumption.

R: Type u
inst: CommRing R
W: ModuleCat R
X: ModuleCat R
Y: ModuleCat R
Z: ModuleCat R
 ModuleCat.MonoidalCategory.tensorHom (ModuleCat.MonoidalCategory.associator W X Y).hom (𝟙 Z) 
    (ModuleCat.MonoidalCategory.associator W (ModuleCat.MonoidalCategory.tensorObj X Y) Z).hom 
      ModuleCat.MonoidalCategory.tensorHom (𝟙 W) (ModuleCat.MonoidalCategory.associator X Y Z).hom =
  LinearMap.comp
    (LinearMap.comp (TensorProduct.map 1 (TensorProduct.assoc R X Y Z))
      (TensorProduct.assoc R (W) (X [R] Y) Z))
    (TensorProduct.map ((TensorProduct.assoc R W X Y)) 1)
R: Type u
inst: CommRing R
W: ModuleCat R
X: ModuleCat R
Y: ModuleCat R
Z: ModuleCat R
 (ModuleCat.MonoidalCategory.associator (ModuleCat.MonoidalCategory.tensorObj W X) Y Z).hom 
    (ModuleCat.MonoidalCategory.associator W X (ModuleCat.MonoidalCategory.tensorObj Y Z)).hom =
  LinearMap.comp (TensorProduct.assoc R (W) (X) (Y [R] Z)) (TensorProduct.assoc R (W [R] X) Y Z)

Kyle Miller (May 27 2023 at 21:01):

Hmm, even just applying the congruence is really slow:

private lemma congr_eq (h : x = y) (hx : x = x') (hy' : y = y') : x' = y' := by subst_vars; rfl

set_option profiler true
set_option trace.profiler true
set_option maxHeartbeats 0 in
theorem pentagon (W X Y Z : ModuleCat R) :
    tensorHom (associator W X Y).hom (𝟙 Z) 
        (associator W (tensorObj X Y) Z).hom  tensorHom (𝟙 W) (associator X Y Z).hom =
      (associator (tensorObj W X) Y Z).hom  (associator W X (tensorObj Y Z)).hom := by
  refine congr_eq (pentagon_aux R W X Y Z) ?_ ?_ -- 35 seconds
  sorry -- rfl works, 32 seconds
  sorry -- rfl works, 7 seconds

Jeremy Tan (May 28 2023 at 02:06):

Still no PDF for the all target

Jon Eugster (May 28 2023 at 10:39):

Jeremy Tan said:

Still no PDF for the all target

I tracked this down to a misshaped comment: @Vierkantor: work in progress on `norm_num-bigop` branch\n apparently they cannot contain : unless wrapped in quotes. For now I just edited #port-comments removing that colon, so tonight it should work again. Here's my locally generated all.pdf

port-progress bot (May 28 2023 at 19:01):

507/3009 files completely ported (16.84%), in the sense that also all downstream dependencies are ported.

Scott Morrison (May 28 2023 at 20:33):

Jon Eugster said:

I tracked this down to a misshaped comment: @Vierkantor: work in progress on `norm_num-bigop` branch\n

Thanks. I thought this was going to be the problem, but apparently failed to notice that colon even though I was specifically looking for colons!

Eric Wieser (May 28 2023 at 21:55):

Mis-shaped according to which parser?

Eric Wieser (May 28 2023 at 21:57):

It looks like #port-wiki was unaffected, so presumably the yaml parsing of #port-comments itself is working just fine

Jon Eugster (May 29 2023 at 05:51):

pydot has a problem that node attributes cannot contain colons unless quoted in additional ""

Jon Eugster (May 29 2023 at 05:53):

and for some reason the nodes in the graph contain the porting-comment even though it seems like they wouldnt be needed for the creation of these graphs.

I guess one could also fix this in mathlib-tools by dropping the attribute comment for all nodes before passing the graph to pydot.

port-progress bot (May 29 2023 at 19:01):

512/3010 files completely ported (17.00%), in the sense that also all downstream dependencies are ported.

Patrick Stevens (May 29 2023 at 19:06):

A lovely round numerator and a lovely near-integer percentage!

Mario Carneiro (May 29 2023 at 19:17):

hopefully not another bc bug

Mario Carneiro (May 29 2023 at 19:18):

well, other than some questionable rounding it seems to be correct

Jireh Loreaux (May 29 2023 at 22:06):

It seems the port progress is not posting the other progress targets... @Scott Morrison I guess this is because you were in Banff?

Scott Morrison (May 30 2023 at 01:11):

Fixed, should run shortly.

port-progress bot (May 30 2023 at 01:17):

mathlib port progress analysis.inner_product_space.pi_L2
Unported files: 7/941 (99.3% of total)
Unported lines: 3409/412343 (99.2% of total)
Longest unported chain: 1/93 (98.9% progress)

port-progress bot (May 30 2023 at 01:27):

mathlib port progress combinatorics.additive.behrend
Unported files: 17/995 (98.3% of total)
Unported lines: 11790/432330 (97.3% of total)
Longest unported chain: 6/103 (94.2% progress)

port-progress bot (May 30 2023 at 01:32):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 41/1049 (96.1% of total)
Unported lines: 17085/445954 (96.2% of total)
Longest unported chain: 14/97 (85.6% progress)

port-progress bot (May 30 2023 at 01:36):

mathlib port progress measure_theory.integral.bochner
Unported files: 11/967 (98.9% of total)
Unported lines: 9453/437137 (97.8% of total)
Longest unported chain: 3/99 (97.0% progress)

port-progress bot (May 30 2023 at 01:41):

mathlib port progress probability.independence.basic
Unported files: 11/677 (98.4% of total)
Unported lines: 6009/301551 (98.0% of total)
Longest unported chain: 3/91 (96.7% progress)

port-progress bot (May 30 2023 at 01:45):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 26/968 (97.3% of total)
Unported lines: 8964/380321 (97.6% of total)
Longest unported chain: 6/79 (92.4% progress)

port-progress bot (May 30 2023 at 01:50):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 27/977 (97.2% of total)
Unported lines: 13938/398491 (96.5% of total)
Longest unported chain: 12/92 (87.0% progress)

port-progress bot (May 30 2023 at 01:54):

mathlib port progress algebra.category.Module.adjunctions
Unported files: 8/579 (98.6% of total)
Unported lines: 3752/222292 (98.3% of total)
Longest unported chain: 1/63 (98.4% progress)

port-progress bot (May 30 2023 at 01:59):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 46/1112 (95.9% of total)
Unported lines: 32452/496818 (93.5% of total)
Longest unported chain: 10/105 (90.5% progress)

port-progress bot (May 30 2023 at 02:04):

mathlib port progress analysis.fourier.add_circle
Unported files: 49/1112 (95.6% of total)
Unported lines: 34746/498218 (93.0% of total)
Longest unported chain: 9/104 (91.3% progress)

port-progress bot (May 30 2023 at 02:09):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 60/1125 (94.7% of total)
Unported lines: 40464/505836 (92.0% of total)
Longest unported chain: 14/111 (87.4% progress)

port-progress bot (May 30 2023 at 02:14):

mathlib port progress measure_theory.function.jacobian
Unported files: 37/1096 (96.6% of total)
Unported lines: 30634/495726 (93.8% of total)
Longest unported chain: 11/107 (89.7% progress)

port-progress bot (May 30 2023 at 02:19):

mathlib port progress all
Unported files: 684/3009 (77.3% of total)
Unported lines: 249065/1032875 (75.9% of total)
Longest unported chain: 20/116 (82.8% progress)

port-progress bot (May 30 2023 at 02:20):

512/3010 files completely ported (17.00%), in the sense that also all downstream dependencies are ported.

Anne Baanen (May 30 2023 at 09:42):

port-progress bot said:

mathlib port progress all
Unported files: 702/2995 (76.6% of total)
Unported lines: 261216/1031509 (74.7% of total)
Longest unported chain: 22/115 (80.9% progress)

0.6%

Anne Baanen (May 30 2023 at 09:43):

port-progress bot said:

mathlib port progress all
Unported files: 684/3009 (77.3% of total)
Unported lines: 249065/1032875 (75.9% of total)
Longest unported chain: 20/116 (82.8% progress)

1.2%

Kevin Buzzard (May 30 2023 at 10:01):

Thanks for bringing us up to speed :-) 22 percent to go, things are looking in great shape. There was only one question at the porting meeting yesterday.

port-progress bot (May 30 2023 at 19:08):

mathlib port progress combinatorics.additive.behrend
Unported files: 16/995 (98.4% of total)
Unported lines: 11572/432365 (97.3% of total)
Longest unported chain: 6/103 (94.2% progress)

port-progress bot (May 30 2023 at 19:13):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 40/1049 (96.2% of total)
Unported lines: 16125/445956 (96.4% of total)
Longest unported chain: 14/97 (85.6% progress)

port-progress bot (May 30 2023 at 19:18):

mathlib port progress measure_theory.integral.bochner
Unported files: 11/967 (98.9% of total)
Unported lines: 9453/437148 (97.8% of total)
Longest unported chain: 3/99 (97.0% progress)

port-progress bot (May 30 2023 at 19:22):

mathlib port progress probability.independence.basic
Unported files: 9/677 (98.7% of total)
Unported lines: 5045/301554 (98.3% of total)
Longest unported chain: 1/91 (98.9% progress)

port-progress bot (May 30 2023 at 19:26):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 24/968 (97.5% of total)
Unported lines: 8547/380330 (97.8% of total)
Longest unported chain: 6/79 (92.4% progress)

port-progress bot (May 30 2023 at 19:31):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 26/977 (97.3% of total)
Unported lines: 13346/398502 (96.6% of total)
Longest unported chain: 11/92 (88.0% progress)

port-progress bot (May 30 2023 at 19:34):

mathlib port progress algebra.category.Module.adjunctions
Unported files: 7/579 (98.8% of total)
Unported lines: 3409/222295 (98.5% of total)
Longest unported chain: 1/63 (98.4% progress)

port-progress bot (May 30 2023 at 19:39):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 41/1112 (96.3% of total)
Unported lines: 30996/496868 (93.8% of total)
Longest unported chain: 9/105 (91.4% progress)

port-progress bot (May 30 2023 at 19:44):

mathlib port progress analysis.fourier.add_circle
Unported files: 47/1112 (95.8% of total)
Unported lines: 33782/498268 (93.2% of total)
Longest unported chain: 9/104 (91.3% progress)

port-progress bot (May 30 2023 at 19:49):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 57/1125 (94.9% of total)
Unported lines: 39282/505883 (92.2% of total)
Longest unported chain: 14/111 (87.4% progress)

port-progress bot (May 30 2023 at 19:54):

mathlib port progress measure_theory.function.jacobian
Unported files: 34/1096 (96.9% of total)
Unported lines: 29201/495776 (94.1% of total)
Longest unported chain: 11/107 (89.7% progress)

port-progress bot (May 30 2023 at 19:59):

mathlib port progress all
Unported files: 664/3010 (77.9% of total)
Unported lines: 243778/1033873 (76.4% of total)
Longest unported chain: 20/116 (82.8% progress)

port-progress bot (May 30 2023 at 20:00):

524/3011 files completely ported (17.40%), in the sense that also all downstream dependencies are ported.

Scott Morrison (May 30 2023 at 23:15):

0.5%

port-progress bot (May 31 2023 at 19:07):

mathlib port progress combinatorics.additive.behrend
Unported files: 16/995 (98.4% of total)
Unported lines: 11572/432406 (97.3% of total)
Longest unported chain: 6/103 (94.2% progress)

port-progress bot (May 31 2023 at 19:12):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 40/1049 (96.2% of total)
Unported lines: 16123/445995 (96.4% of total)
Longest unported chain: 14/97 (85.6% progress)

port-progress bot (May 31 2023 at 19:17):

mathlib port progress measure_theory.integral.bochner
Unported files: 10/967 (99.0% of total)
Unported lines: 8152/437186 (98.1% of total)
Longest unported chain: 2/99 (98.0% progress)

port-progress bot (May 31 2023 at 19:21):

mathlib port progress probability.independence.basic
Unported files: 9/677 (98.7% of total)
Unported lines: 5045/301590 (98.3% of total)
Longest unported chain: 1/91 (98.9% progress)

port-progress bot (May 31 2023 at 19:26):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 24/968 (97.5% of total)
Unported lines: 8547/380348 (97.8% of total)
Longest unported chain: 6/79 (92.4% progress)

port-progress bot (May 31 2023 at 19:31):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 25/977 (97.4% of total)
Unported lines: 13040/398543 (96.7% of total)
Longest unported chain: 11/92 (88.0% progress)

port-progress bot (May 31 2023 at 19:36):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 37/1112 (96.7% of total)
Unported lines: 27799/496951 (94.4% of total)
Longest unported chain: 8/105 (92.4% progress)

port-progress bot (May 31 2023 at 19:41):

mathlib port progress analysis.fourier.add_circle
Unported files: 43/1112 (96.1% of total)
Unported lines: 30585/498342 (93.9% of total)
Longest unported chain: 9/104 (91.3% progress)

port-progress bot (May 31 2023 at 19:47):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 53/1125 (95.3% of total)
Unported lines: 36085/505960 (92.9% of total)
Longest unported chain: 14/111 (87.4% progress)

port-progress bot (May 31 2023 at 19:52):

mathlib port progress measure_theory.function.jacobian
Unported files: 29/1096 (97.4% of total)
Unported lines: 25445/495856 (94.9% of total)
Longest unported chain: 10/107 (90.7% progress)

port-progress bot (May 31 2023 at 19:57):

mathlib port progress all
Unported files: 656/3013 (78.2% of total)
Unported lines: 238481/1034777 (77.0% of total)
Longest unported chain: 19/116 (83.6% progress)

port-progress bot (May 31 2023 at 19:59):

528/3014 files completely ported (17.51%), in the sense that also all downstream dependencies are ported.

Jireh Loreaux (May 31 2023 at 20:02):

0.6%

Anne Baanen (Jun 01 2023 at 09:02):

port-progress bot said:

mathlib port progress all
Unported files: 656/3013 (78.2% of total)
Unported lines: 238481/1034777 (77.0% of total)
Longest unported chain: 19/116 (83.6% progress)

I can now actually read all.pdf on maximum zoom!

port-progress bot (Jun 01 2023 at 19:07):

mathlib port progress combinatorics.additive.behrend
Unported files: 15/995 (98.5% of total)
Unported lines: 9891/432407 (97.7% of total)
Longest unported chain: 6/103 (94.2% progress)

port-progress bot (Jun 01 2023 at 19:12):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 40/1049 (96.2% of total)
Unported lines: 16127/446008 (96.4% of total)
Longest unported chain: 14/97 (85.6% progress)

port-progress bot (Jun 01 2023 at 19:17):

mathlib port progress measure_theory.integral.bochner
Unported files: 10/967 (99.0% of total)
Unported lines: 8152/437189 (98.1% of total)
Longest unported chain: 2/99 (98.0% progress)

port-progress bot (Jun 01 2023 at 19:21):

mathlib port progress probability.independence.basic
Unported files: 8/677 (98.8% of total)
Unported lines: 4306/301590 (98.6% of total)
Longest unported chain: 1/91 (98.9% progress)

port-progress bot (Jun 01 2023 at 19:26):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 24/968 (97.5% of total)
Unported lines: 8547/380348 (97.8% of total)
Longest unported chain: 6/79 (92.4% progress)

port-progress bot (Jun 01 2023 at 19:30):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 23/977 (97.6% of total)
Unported lines: 11757/398546 (97.0% of total)
Longest unported chain: 11/92 (88.0% progress)

port-progress bot (Jun 01 2023 at 19:35):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 31/1112 (97.2% of total)
Unported lines: 23171/496967 (95.3% of total)
Longest unported chain: 8/105 (92.4% progress)

port-progress bot (Jun 01 2023 at 19:40):

mathlib port progress analysis.fourier.add_circle
Unported files: 37/1112 (96.7% of total)
Unported lines: 24838/498355 (95.0% of total)
Longest unported chain: 9/104 (91.3% progress)

port-progress bot (Jun 01 2023 at 19:45):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 47/1125 (95.8% of total)
Unported lines: 31184/505973 (93.8% of total)
Longest unported chain: 13/111 (88.3% progress)

port-progress bot (Jun 01 2023 at 19:52):

mathlib port progress measure_theory.function.jacobian
Unported files: 24/1096 (97.8% of total)
Unported lines: 20842/495869 (95.8% of total)
Longest unported chain: 10/107 (90.7% progress)

port-progress bot (Jun 01 2023 at 19:57):

mathlib port progress all
Unported files: 637/3013 (78.9% of total)
Unported lines: 227688/1035031 (78.0% of total)
Longest unported chain: 19/116 (83.6% progress)

port-progress bot (Jun 01 2023 at 19:59):

535/3014 files completely ported (17.75%), in the sense that also all downstream dependencies are ported.

Scott Morrison (Jun 01 2023 at 20:02):

1.0%

Kevin Buzzard (Jun 01 2023 at 20:36):

Oh it's now reporting number of unported files! Thank you to whoever changed this -- it's now a much better measure of progress for most of our goals :-)

Michael Stoll (Jun 01 2023 at 20:40):

But the percentages still refer to ported files/lines/files in the original(?) longest chain, which I find slightly confusing.

Johan Commelin (Jun 02 2023 at 05:25):

Only 5 more files with > 100 dependents!

port-progress bot (Jun 02 2023 at 19:07):

mathlib port progress combinatorics.additive.behrend
Unported files: 13/994 (98.7% of total)
Unported lines: 7671/431623 (98.2% of total)
Longest unported chain: 5/103 (95.1% progress)

port-progress bot (Jun 02 2023 at 19:12):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 37/1050 (96.5% of total)
Unported lines: 15293/446033 (96.6% of total)
Longest unported chain: 14/97 (85.6% progress)

port-progress bot (Jun 02 2023 at 19:17):

mathlib port progress measure_theory.integral.bochner
Unported files: 8/967 (99.2% of total)
Unported lines: 5245/437189 (98.8% of total)
Longest unported chain: 1/99 (99.0% progress)

port-progress bot (Jun 02 2023 at 19:20):

mathlib port progress probability.independence.basic
Unported files: 7/677 (99.0% of total)
Unported lines: 3409/301593 (98.9% of total)
Longest unported chain: 1/91 (98.9% progress)

port-progress bot (Jun 02 2023 at 19:24):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 22/968 (97.7% of total)
Unported lines: 7133/380347 (98.1% of total)
Longest unported chain: 5/79 (93.7% progress)

port-progress bot (Jun 02 2023 at 19:28):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 21/977 (97.9% of total)
Unported lines: 11299/398551 (97.2% of total)
Longest unported chain: 9/92 (90.2% progress)

port-progress bot (Jun 02 2023 at 19:33):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 25/1111 (97.7% of total)
Unported lines: 17418/496195 (96.5% of total)
Longest unported chain: 6/105 (94.3% progress)

port-progress bot (Jun 02 2023 at 19:38):

mathlib port progress analysis.fourier.add_circle
Unported files: 29/1107 (97.4% of total)
Unported lines: 18223/494829 (96.3% of total)
Longest unported chain: 6/104 (94.2% progress)

port-progress bot (Jun 02 2023 at 19:43):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 41/1124 (96.4% of total)
Unported lines: 26074/505201 (94.8% of total)
Longest unported chain: 13/111 (88.3% progress)

port-progress bot (Jun 02 2023 at 19:48):

mathlib port progress measure_theory.function.jacobian
Unported files: 20/1096 (98.2% of total)
Unported lines: 17280/495884 (96.5% of total)
Longest unported chain: 8/107 (92.5% progress)

port-progress bot (Jun 02 2023 at 19:53):

mathlib port progress all
Unported files: 602/3016 (80.0% of total)
Unported lines: 211561/1035518 (79.6% of total)
Longest unported chain: 17/116 (85.3% progress)

port-progress bot (Jun 02 2023 at 19:54):

548/3017 files completely ported (18.16%), in the sense that also all downstream dependencies are ported.

Johan Commelin (Jun 02 2023 at 20:13):

1.6%

Michael Stoll (Jun 02 2023 at 20:39):

port-progress bot said:

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 37/1050 (96.5% of total)
Unported lines: 15293/446033 (96.6% of total)
Longest unported chain: 14/97 (85.6% progress)

If I click on the link, I get a graph that shows 30 nodes. Is the difference the magic number 7 that @Kevin Buzzard recently discovered? I thought that this was being corrected for...

Eric Wieser (Jun 02 2023 at 22:05):

Those 7 files are the ones in core that appear on #port-dashboard I think

port-progress bot (Jun 03 2023 at 19:07):

mathlib port progress combinatorics.additive.behrend
Unported files: 13/994 (98.7% of total)
Unported lines: 7671/431623 (98.2% of total)
Longest unported chain: 5/103 (95.1% progress)

port-progress bot (Jun 03 2023 at 19:12):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 36/1050 (96.6% of total)
Unported lines: 15174/446045 (96.6% of total)
Longest unported chain: 14/97 (85.6% progress)

port-progress bot (Jun 03 2023 at 19:16):

mathlib port progress measure_theory.integral.bochner
Unported files: 8/967 (99.2% of total)
Unported lines: 5245/437195 (98.8% of total)
Longest unported chain: 1/99 (99.0% progress)

port-progress bot (Jun 03 2023 at 19:19):

mathlib port progress probability.independence.basic
Unported files: 7/677 (99.0% of total)
Unported lines: 3409/301596 (98.9% of total)
Longest unported chain: 1/91 (98.9% progress)

port-progress bot (Jun 03 2023 at 19:24):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 22/968 (97.7% of total)
Unported lines: 7133/380353 (98.1% of total)
Longest unported chain: 5/79 (93.7% progress)

port-progress bot (Jun 03 2023 at 19:28):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 21/977 (97.9% of total)
Unported lines: 11299/398557 (97.2% of total)
Longest unported chain: 9/92 (90.2% progress)

port-progress bot (Jun 03 2023 at 19:33):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 25/1111 (97.7% of total)
Unported lines: 17418/496207 (96.5% of total)
Longest unported chain: 6/105 (94.3% progress)

port-progress bot (Jun 03 2023 at 19:37):

mathlib port progress analysis.fourier.add_circle
Unported files: 27/1107 (97.6% of total)
Unported lines: 17973/494847 (96.4% of total)
Longest unported chain: 5/104 (95.2% progress)

port-progress bot (Jun 03 2023 at 19:42):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 41/1124 (96.4% of total)
Unported lines: 26074/505216 (94.8% of total)
Longest unported chain: 13/111 (88.3% progress)

port-progress bot (Jun 03 2023 at 19:47):

mathlib port progress measure_theory.function.jacobian
Unported files: 20/1096 (98.2% of total)
Unported lines: 17280/495896 (96.5% of total)
Longest unported chain: 8/107 (92.5% progress)

port-progress bot (Jun 03 2023 at 19:52):

mathlib port progress all
Unported files: 582/3016 (80.7% of total)
Unported lines: 207152/1035635 (80.0% of total)
Longest unported chain: 17/116 (85.3% progress)

port-progress bot (Jun 03 2023 at 19:53):

558/3017 files completely ported (18.49%), in the sense that also all downstream dependencies are ported.

Johan Commelin (Jun 03 2023 at 19:53):

0.4%

port-progress bot (Jun 04 2023 at 19:07):

mathlib port progress combinatorics.additive.behrend
Unported files: 11/994 (98.9% of total)
Unported lines: 4610/431623 (98.9% of total)
Longest unported chain: 3/103 (97.1% progress)

port-progress bot (Jun 04 2023 at 19:12):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 36/1050 (96.6% of total)
Unported lines: 15174/446048 (96.6% of total)
Longest unported chain: 14/97 (85.6% progress)

port-progress bot (Jun 04 2023 at 19:17):

mathlib port progress measure_theory.integral.bochner
Unported files: 8/967 (99.2% of total)
Unported lines: 5245/437195 (98.8% of total)
Longest unported chain: 1/99 (99.0% progress)

port-progress bot (Jun 04 2023 at 19:21):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 21/968 (97.8% of total)
Unported lines: 6972/380368 (98.2% of total)
Longest unported chain: 5/79 (93.7% progress)

port-progress bot (Jun 04 2023 at 19:25):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 21/977 (97.9% of total)
Unported lines: 11299/398585 (97.2% of total)
Longest unported chain: 9/92 (90.2% progress)

port-progress bot (Jun 04 2023 at 19:30):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 23/1111 (97.9% of total)
Unported lines: 14357/496207 (97.1% of total)
Longest unported chain: 6/105 (94.3% progress)

port-progress bot (Jun 04 2023 at 19:35):

mathlib port progress analysis.fourier.add_circle
Unported files: 25/1107 (97.7% of total)
Unported lines: 14912/494850 (97.0% of total)
Longest unported chain: 5/104 (95.2% progress)

port-progress bot (Jun 04 2023 at 19:40):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 39/1124 (96.5% of total)
Unported lines: 23013/505216 (95.4% of total)
Longest unported chain: 12/111 (89.2% progress)

port-progress bot (Jun 04 2023 at 19:45):

mathlib port progress measure_theory.function.jacobian
Unported files: 18/1096 (98.4% of total)
Unported lines: 13606/495896 (97.3% of total)
Longest unported chain: 8/107 (92.5% progress)

port-progress bot (Jun 04 2023 at 19:50):

mathlib port progress all
Unported files: 575/3016 (80.9% of total)
Unported lines: 202439/1035720 (80.5% of total)
Longest unported chain: 17/116 (85.3% progress)

Jireh Loreaux (Jun 04 2023 at 19:51):

0.5%

port-progress bot (Jun 04 2023 at 19:51):

560/3017 files completely ported (18.56%), in the sense that also all downstream dependencies are ported.

Kevin Buzzard (Jun 04 2023 at 22:43):

geometry.manifold.whitney_embedding is a counterexample to the "off-by-seven" conjecture: the difference between the number of unported files claimed by the bot and the number of files listed on the pdf is 8.

Kevin Buzzard (Jun 04 2023 at 22:44):

huh -- for group cohomology the difference is 9.

Eric Wieser (Jun 04 2023 at 22:59):

What does #port-dashboard say in those cases?

Kevin Buzzard (Jun 04 2023 at 23:21):

It says this about group cohomology https://leanprover-community.github.io/mathlib-port-status/file/representation_theory/group_cohomology/basic . I must be honest, I don't really understand much of what is on those websites other than the bits I need to understand. It says 6+7+925. It says there are 14 files to go in the sense that there are 14 bullet points. There are 12 nodes on the graph and experience suggests that we'll be finished when we port those 12 files. Those 12 files on the pdf are what I actually need to know in practice.

Eric Wieser (Jun 05 2023 at 00:05):

Hovering over the 6 and 7 tell you what they each mean. The 14 is 6 + 7 + 1 (the file itself)

Eric Wieser (Jun 05 2023 at 00:05):

The graph has 14 nodes but two of them aren't connected!

Joël Riou (Jun 05 2023 at 08:16):

The discrepancy is because the dependency to bicategory.coherence_tactic was removed (at least temporarily) when monoidal.coherence was ported.

Kevin Buzzard (Jun 05 2023 at 10:46):

wooah it now says 5+3+930 :-)

Johan Commelin (Jun 05 2023 at 10:47):

Is that good or bad news?

Kevin Buzzard (Jun 05 2023 at 10:47):

Definitely good :-) (while I was sleeping 5 files got merged)

Johan Commelin (Jun 05 2023 at 10:48):

If only 15 files got ported while you slept...

Kevin Buzzard (Jun 05 2023 at 10:48):

I'll go back to bed.

Johan Commelin (Jun 05 2023 at 10:49):

Exactly!

Kevin Buzzard (Jun 05 2023 at 10:49):

It's not 5 files in total, it's 5 files on the route to group cohomology!

Johan Commelin (Jun 05 2023 at 10:49):

They always say that sleeping is good for you... turns out it's actually true :rofl:

Kevin Buzzard (Jun 05 2023 at 10:55):

When I was trying to make sense of this area 5.5 years ago, working out what was easy or hard, I quickly got the impression that generating a ton of category theory in a theorem prover looked very easy, whereas doing things I regarded as far more basic such as proving quadratic reciprocity seemed to be far rarer and perhaps even far harder. Then you and I started experimenting with Lean 3 and we realised that actually making basic group theory, ring theory, topological ring theory etc was not hard at all, it's just that nobody was doing it because nobody in the community particularly cared about it. Category theory on the other hand was struggling a bit, with Scott having universe problems and having to include category instances etc etc, and also with it being connected to nothing else in the library at the time. However with the port to mathlib4 I feel like currently things are a little bit returning to the old days: I have ported some category theory files and on the whole they sail through (modulo perhaps some issues with simp not behaving), whereas the algebraists are complaining about splitting fields and the analysts are complaining about differentiation. This might just be random noise though; if we have got to 80% (which, as Oliver pointed out to me on Friday, is really more like 95% given all the work that people like Mario and Gabriel and others have put in in order for us to even start the porting procedure) then one has to be optimistic that all the noise we're running into now is nothing more than noise.

Kevin Buzzard (Jun 05 2023 at 11:16):

I mention this because much of what is left on the road to group cohomology is category theory :-) (no splitting fields required! Although when we get to Galois cohomology...)

Johan Commelin (Jun 05 2023 at 15:30):

We need to port less than 10 files, and after that every unported file will have < 50 dependents.

Eric Wieser (Jun 05 2023 at 15:37):

port-status#number_theory/zeta_function claims to have 71 files that aren't yet ported in mathlib4 master

Eric Wieser (Jun 05 2023 at 15:38):

Are you considering the 9 in-progress ones as "ported"?

port-progress bot (Jun 05 2023 at 19:07):

mathlib port progress combinatorics.additive.behrend
Unported files: 8/994 (99.2% of total)
Unported lines: 3948/431641 (99.1% of total)
Longest unported chain: 1/103 (99.0% progress)

Ruben Van de Velde (Jun 05 2023 at 19:09):

port-progress bot said:

mathlib port progress combinatorics.additive.behrend
Unported files: 8/994 (99.2% of total)
Unported lines: 3948/431641 (99.1% of total)
Longest unported chain: 1/103 (99.0% progress)

This one's up for grabs!

port-progress bot (Jun 05 2023 at 19:11):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 37/1051 (96.5% of total)
Unported lines: 15221/446104 (96.6% of total)
Longest unported chain: 14/97 (85.6% progress)

port-progress bot (Jun 05 2023 at 19:14):

mathlib port progress measure_theory.integral.bochner
Unported files: 7/967 (99.3% of total)
Unported lines: 3409/437204 (99.2% of total)
Longest unported chain: 1/99 (99.0% progress)

Johan Commelin (Jun 05 2023 at 19:14):

Done

port-progress bot (Jun 05 2023 at 19:18):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 16/968 (98.3% of total)
Unported lines: 6602/380380 (98.3% of total)
Longest unported chain: 3/79 (96.2% progress)

port-progress bot (Jun 05 2023 at 19:22):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 22/978 (97.8% of total)
Unported lines: 11326/398621 (97.2% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 05 2023 at 19:26):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 18/1111 (98.4% of total)
Unported lines: 11278/496225 (97.7% of total)
Longest unported chain: 5/105 (95.2% progress)

port-progress bot (Jun 05 2023 at 19:31):

mathlib port progress analysis.fourier.add_circle
Unported files: 18/1107 (98.4% of total)
Unported lines: 10545/494868 (97.9% of total)
Longest unported chain: 4/104 (96.2% progress)

port-progress bot (Jun 05 2023 at 19:35):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 30/1124 (97.3% of total)
Unported lines: 17580/505237 (96.5% of total)
Longest unported chain: 11/111 (90.1% progress)

port-progress bot (Jun 05 2023 at 19:40):

mathlib port progress measure_theory.function.jacobian
Unported files: 16/1096 (98.5% of total)
Unported lines: 10903/495911 (97.8% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 05 2023 at 19:44):

mathlib port progress all
Unported files: 529/3018 (82.5% of total)
Unported lines: 187085/1036326 (81.9% of total)
Longest unported chain: 17/117 (85.5% progress)

port-progress bot (Jun 05 2023 at 19:45):

581/3019 files completely ported (19.24%), in the sense that also all downstream dependencies are ported.

Chris Hughes (Jun 05 2023 at 19:50):

1.4%

Joël Riou (Jun 05 2023 at 19:55):

After I struggled with RepresentationTheory.Action !4#4700 there are only three remaining files to port on the way to GroupCohomology.Basic.

Johan Commelin (Jun 05 2023 at 20:04):

About 46 files today, I think!

Pol'tta / Miyahara Kō (Jun 06 2023 at 00:21):

MeasureTheory.Integral.SetIntegral is ready to review, the last file which has >100 dependents.

Scott Morrison (Jun 06 2023 at 01:38):

Kevin Buzzard said:

However with the port to mathlib4 I feel like currently things are a little bit returning to the old days: I have ported some category theory files and on the whole they sail through (modulo perhaps some issues with simp not behaving), whereas the algebraists are complaining about splitting fields and the analysts are complaining about differentiation.

I don't think this is particularly accurate. I think a lot of the variation in ease-of-porting we're seeing comes down to how much defeq abuse (abuse is maybe overstating it) the mathlib3 library was using; many things have changed in Lean4 that then cause problems. I think in the "trivial" parts of the category theory library, it was smooth sailing, mostly because we were pretty good at avoiding defeq abuse (some old horrors like opposite notwithstanding). Now that we're porting algebraic geometry we're seeing some of the same issues: there are worryingly many appearances of erw in setting up Spec and Scheme and so forth, and sure enough this is now causing troubling during porting.

Tobias Grosser (Jun 06 2023 at 04:24):

Chris Hughes said:

1.4%

Wow!

Scott Morrison (Jun 06 2023 at 05:51):

Anyone wanting to work on algebraic geometry porting could:

  • give further review to !4#4693
  • help continue Topology.Gluing !4#3987
  • begin porting algebraic_geometry.open_immersion.basic

Damiano Testa (Jun 06 2023 at 05:52):

I'll give open_immersion a shot!

Jireh Loreaux (Jun 06 2023 at 21:13):

@Scott Morrison I think the port progress bot may have died again.

Scott Morrison (Jun 06 2023 at 22:34):

Flaky internet here. I'll re-run now.

port-progress bot (Jun 06 2023 at 22:40):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 36/1051 (96.6% of total)
Unported lines: 15073/446104 (96.6% of total)
Longest unported chain: 13/97 (86.6% progress)

port-progress bot (Jun 06 2023 at 22:42):

mathlib port progress combinatorics.additive.behrend
Unported files: 7/994 (99.3% of total)
Unported lines: 3409/431647 (99.2% of total)
Longest unported chain: 1/103 (99.0% progress)

port-progress bot (Jun 06 2023 at 22:44):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 12/968 (98.8% of total)
Unported lines: 5260/380395 (98.6% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 06 2023 at 22:49):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 22/978 (97.8% of total)
Unported lines: 11326/398621 (97.2% of total)
Longest unported chain: 7/90 (92.2% progress)

Scott Morrison (Jun 06 2023 at 22:51):

Maybe group_cohomology can be finished today! Just three files, in a linear chain, and representation_theory.Rep is currently open for porting.

Scott Morrison (Jun 06 2023 at 22:54):

(err, apparently the previous run of the bot was just delayed by flaky internet, not aborted, and we now have two interleaved runs happening. I'll clean up as we go, I guess.)

port-progress bot (Jun 06 2023 at 22:54):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 13/1111 (98.8% of total)
Unported lines: 8107/496237 (98.4% of total)
Longest unported chain: 4/105 (96.2% progress)

port-progress bot (Jun 06 2023 at 22:59):

mathlib port progress analysis.fourier.add_circle
Unported files: 15/1107 (98.6% of total)
Unported lines: 8170/494889 (98.3% of total)
Longest unported chain: 2/104 (98.1% progress)

port-progress bot (Jun 06 2023 at 23:04):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 26/1124 (97.7% of total)
Unported lines: 15351/505261 (97.0% of total)
Longest unported chain: 11/111 (90.1% progress)

Scott Morrison (Jun 06 2023 at 23:04):

The following dependencies of analysis.fourier.add_circle are labelled help-wanted:

  • MeasureTheory.Integral.IntervalIntegral !4#4710 (see discussion here)
  • MeasureTheory.Group.Integration !4#4694

Scott Morrison (Jun 06 2023 at 23:07):

geometry.manifold.whitney_embedding also has help-wanted on

  • MeasureTheory.Group.Integration !4#4694

port-progress bot (Jun 06 2023 at 23:09):

mathlib port progress measure_theory.function.jacobian
Unported files: 12/1096 (98.9% of total)
Unported lines: 8600/495917 (98.3% of total)
Longest unported chain: 4/107 (96.3% progress)

port-progress bot (Jun 06 2023 at 23:14):

mathlib port progress all
Unported files: 489/3019 (83.8% of total)
Unported lines: 174077/1036526 (83.2% of total)
Longest unported chain: 16/117 (86.3% progress)

Scott Morrison (Jun 06 2023 at 23:14):

measure_theory.function.jacobian has as help-wanted

  • MeasureTheory.Decomposition.Lebesgue !4#4736

after which a linear chain of 4 files to the target!

Scott Morrison (Jun 06 2023 at 23:15):

1.3%

Amelia Livingston (Jun 06 2023 at 23:17):

Scott Morrison said:

Maybe group_cohomology can be finished today! Just three files, in a linear chain, and representation_theory.Rep is currently open for porting.

I'm going to open a PR for RepresentationTheory.Rep - it's my first port of a full file so I might slow down progress. But I have been practicing.

port-progress bot (Jun 06 2023 at 23:18):

600/3020 files completely ported (19.86%), in the sense that also all downstream dependencies are ported.

Johan Commelin (Jun 07 2023 at 00:22):

We ported another 40 files yesterday! Good numbers :smiley:

Jireh Loreaux (Jun 07 2023 at 00:37):

In the past 3 weeks we've ported 19.3% of mathlib for an average of 0.92% / day!

Scott Morrison (Jun 07 2023 at 01:14):

So we're done at , right?

Scott Morrison (Jun 07 2023 at 02:04):

I've added some extra targets for the port progress bot, which essentially get us to "the end". After all those targets are done I think there's no chain longer than 3 or 4 files.

port-progress bot (Jun 07 2023 at 02:07):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 14/677 (97.9% of total)
Unported lines: 5237/279792 (98.1% of total)
Longest unported chain: 6/84 (92.9% progress)

Scott Morrison (Jun 07 2023 at 02:11):

The top file here looks like it's ready to go, I just relaunched CI after the "disk full" fiasco. :-) After that, perhaps @Eric Wieser would like to push the Clifford algebra files along?

port-progress bot (Jun 07 2023 at 02:12):

mathlib port progress representation_theory.character
Unported files: 22/920 (97.6% of total)
Unported lines: 8286/349046 (97.6% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (Jun 07 2023 at 02:16):

mathlib port progress algebra.lie.weights
Unported files: 19/717 (97.4% of total)
Unported lines: 8588/292957 (97.1% of total)
Longest unported chain: 7/91 (92.3% progress)

Scott Morrison (Jun 07 2023 at 02:19):

Both of these last two are essentially trapped behind field_theory.adjoin, although algebra.lie.quotient is open for porting.

Scott Morrison (Jun 07 2023 at 02:20):

And for representation_theory.character we have CategoryTheory.Monoidal.Subcategory !4#4769 ready to be merged.

port-progress bot (Jun 07 2023 at 02:21):

mathlib port progress analysis.normed_space.star.continuous_functional_calculus
Unported files: 27/1182 (97.7% of total)
Unported lines: 12516/517546 (97.6% of total)
Longest unported chain: 10/111 (91.0% progress)

Scott Morrison (Jun 07 2023 at 02:23):

Ah, although I see that for finishing off Lie algebras, the portion of linear_algebra.eigenspace that we need doesn't actually rely on field_theory.is_alg_closed.spectrum (and then transitively field_theory.adjoin, so if someone wanted to refactor linear_algebra.eigenspace to split it that might be nice.

port-progress bot (Jun 07 2023 at 02:26):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 23/748 (96.9% of total)
Unported lines: 8997/297727 (97.0% of total)
Longest unported chain: 7/93 (92.5% progress)

Scott Morrison (Jun 07 2023 at 02:30):

This needs the relatively simple tactics ported. I can look at this if no one wants to jump on it!

port-progress bot (Jun 07 2023 at 02:33):

mathlib port progress number_theory.zeta_function
Unported files: 57/1240 (95.4% of total)
Unported lines: 32790/551353 (94.1% of total)
Longest unported chain: 13/116 (88.8% progress)

Scott Morrison (Jun 07 2023 at 02:37):

Lots of work still to go here!

port-progress bot (Jun 07 2023 at 02:41):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 20/933 (97.9% of total)
Unported lines: 10216/411147 (97.5% of total)
Longest unported chain: 12/112 (89.3% progress)

port-progress bot (Jun 07 2023 at 02:48):

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 15/1034 (98.5% of total)
Unported lines: 9222/448408 (97.9% of total)
Longest unported chain: 5/108 (95.4% progress)

port-progress bot (Jun 07 2023 at 02:55):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156365 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

Damiano Testa (Jun 07 2023 at 02:57):

Scott Morrison said:

This needs the relatively simple tactics ported. I can look at this if no one wants to jump on it!

Unless someone else wants to try this, I'll give RingTheory.WittVector.Basic a go for a little bit now.

port-progress bot (Jun 07 2023 at 03:00):

mathlib port progress order.category.FinBoolAlg
Unported files: 15/348 (95.7% of total)
Unported lines: 4203/129422 (96.7% of total)
Longest unported chain: 5/49 (89.8% progress)

port-progress bot (Jun 07 2023 at 03:05):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/284929 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

Scott Morrison (Jun 07 2023 at 03:07):

The graph for geometry.manifold.algebra.left_invariant_derivation is interesting. First, it's just a long chain, but secondly, it suggests a split might be possible in file#geometry/manifold/cont_mdiff_map, separating out a portion that doesn't depend on file#geometry/manifold/cont_mdiff_mfderiv. EDIT: see #19164

Scott Morrison (Jun 07 2023 at 03:08):

order.category.FinBoolAlg looks to be wide open for porting if someone doesn't feel like struggling with existing problems. :-)

port-progress bot (Jun 07 2023 at 03:10):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/804 (98.6% of total)
Unported lines: 4541/346402 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

Scott Morrison (Jun 07 2023 at 03:12):

Scott Morrison said:

Ah, although I see that for finishing off Lie algebras, the portion of linear_algebra.eigenspace that we need doesn't actually rely on field_theory.is_alg_closed.spectrum (and then transitively field_theory.adjoin, so if someone wanted to refactor linear_algebra.eigenspace to split it that might be nice.

I couldn't resist: #19163 is the splitting PR. It seems quite natural.

port-progress bot (Jun 07 2023 at 03:15):

mathlib port progress number_theory.pell
Unported files: 11/806 (98.6% of total)
Unported lines: 5452/344650 (98.4% of total)
Longest unported chain: 3/81 (96.3% progress)

port-progress bot (Jun 07 2023 at 03:19):

mathlib port progress topology.sheaves.locally_surjective
Unported files: 11/822 (98.7% of total)
Unported lines: 4091/329138 (98.8% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 07 2023 at 03:20):

606/3020 files completely ported (20.06%), in the sense that also all downstream dependencies are ported.

Kevin Buzzard (Jun 07 2023 at 06:33):

Under 500 files to go!

Jeremy Tan (Jun 07 2023 at 14:50):

umm… the bot went bonkers on https://tqft.net/mathlib4/latest/number_theory.legendre_symbol.quadratic_reciprocity.pdf

Ruben Van de Velde (Jun 07 2023 at 14:58):

Pretty

Patrick Massot (Jun 07 2023 at 17:50):

The port is really doing great! It looks like we'll be able to restore the integration chapter of MIL very soon. The remaining targets are https://leanprover-community.github.io/mathlib-port-status/file/measure_theory/function/jacobian, https://leanprover-community.github.io/mathlib-port-status/file/analysis/convolution and https://leanprover-community.github.io/mathlib-port-status/file/analysis/special_functions/integrals if I'm counting right.

port-progress bot (Jun 07 2023 at 19:04):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/279798 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 07 2023 at 19:08):

mathlib port progress representation_theory.character
Unported files: 19/920 (97.9% of total)
Unported lines: 7473/349061 (97.9% of total)
Longest unported chain: 7/91 (92.3% progress)

port-progress bot (Jun 07 2023 at 19:11):

mathlib port progress algebra.lie.weights
Unported files: 15/573 (97.4% of total)
Unported lines: 6212/234268 (97.3% of total)
Longest unported chain: 4/74 (94.6% progress)

port-progress bot (Jun 07 2023 at 19:16):

mathlib port progress analysis.normed_space.star.continuous_functional_calculus
Unported files: 26/1182 (97.8% of total)
Unported lines: 11202/517614 (97.8% of total)
Longest unported chain: 9/111 (91.9% progress)

port-progress bot (Jun 07 2023 at 19:20):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 23/748 (96.9% of total)
Unported lines: 8997/297730 (97.0% of total)
Longest unported chain: 7/93 (92.5% progress)

port-progress bot (Jun 07 2023 at 19:25):

mathlib port progress number_theory.zeta_function
Unported files: 53/1252 (95.8% of total)
Unported lines: 29183/557043 (94.8% of total)
Longest unported chain: 11/116 (90.5% progress)

port-progress bot (Jun 07 2023 at 19:29):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/922 (98.4% of total)
Unported lines: 6695/404474 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 07 2023 at 19:33):

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 14/1034 (98.6% of total)
Unported lines: 8654/448467 (98.1% of total)
Longest unported chain: 5/108 (95.4% progress)

port-progress bot (Jun 07 2023 at 19:37):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156365 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 07 2023 at 19:40):

mathlib port progress order.category.FinBoolAlg
Unported files: 15/348 (95.7% of total)
Unported lines: 4203/129422 (96.7% of total)
Longest unported chain: 5/49 (89.8% progress)

port-progress bot (Jun 07 2023 at 19:44):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/284963 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 07 2023 at 19:48):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/804 (98.6% of total)
Unported lines: 4541/346449 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 07 2023 at 19:52):

mathlib port progress number_theory.pell
Unported files: 11/806 (98.6% of total)
Unported lines: 5452/344684 (98.4% of total)
Longest unported chain: 3/81 (96.3% progress)

port-progress bot (Jun 07 2023 at 19:56):

mathlib port progress topology.sheaves.locally_surjective
Unported files: 10/822 (98.8% of total)
Unported lines: 3870/329172 (98.8% of total)
Longest unported chain: 2/80 (97.5% progress)

port-progress bot (Jun 07 2023 at 19:57):

616/3022 files completely ported (20.38%), in the sense that also all downstream dependencies are ported.

Scott Morrison (Jun 07 2023 at 20:04):

Oops, it only ran on the new targets! Follow up run starting now.

port-progress bot (Jun 07 2023 at 20:14):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 35/1052 (96.7% of total)
Unported lines: 14138/446269 (96.8% of total)
Longest unported chain: 13/97 (86.6% progress)

port-progress bot (Jun 07 2023 at 20:18):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4664/380374 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

Ruben Van de Velde (Jun 07 2023 at 20:23):

port-progress bot said:

mathlib port progress number_theory.zeta_function
Unported files: 53/1252 (95.8% of total)
Unported lines: 29183/557043 (94.8% of total)
Longest unported chain: 11/116 (90.5% progress)

Hmm, seems like number_theory.modular_forms.jacobi_theta pulls in a bunch of manifold stuff for the one lemma mdifferentiable_jacobi_theta. Not sure if that's worth changing

port-progress bot (Jun 07 2023 at 20:23):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 22/978 (97.8% of total)
Unported lines: 11326/398601 (97.2% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 07 2023 at 20:28):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 13/1112 (98.8% of total)
Unported lines: 6972/496414 (98.6% of total)
Longest unported chain: 3/105 (97.1% progress)

port-progress bot (Jun 07 2023 at 20:33):

mathlib port progress analysis.fourier.add_circle
Unported files: 12/1108 (98.9% of total)
Unported lines: 6196/495057 (98.7% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 07 2023 at 20:39):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 25/1125 (97.8% of total)
Unported lines: 13992/505795 (97.2% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 07 2023 at 20:44):

mathlib port progress measure_theory.function.jacobian
Unported files: 11/1097 (99.0% of total)
Unported lines: 6577/496091 (98.7% of total)
Longest unported chain: 2/107 (98.1% progress)

Kevin Buzzard (Jun 07 2023 at 20:46):

Subtracting the 7 manually makes it look much more exciting: all targets look like they're 10+ files away whereas some of them are just 3 or 4.

Johan Commelin (Jun 07 2023 at 20:47):

You can also look at the height of all.pdf ... that's pretty encouraging!!

Heather Macbeth (Jun 07 2023 at 20:48):

Ruben Van de Velde said:

Hmm, seems like number_theory.modular_forms.jacobi_theta pulls in a bunch of manifold stuff for the one lemma mdifferentiable_jacobi_theta. Not sure if that's worth changing

I don't think it will be possible to avoid the manifold stuff as we get deeper into complex analysis, so I don't think it's worth changing now.

port-progress bot (Jun 07 2023 at 20:49):

mathlib port progress all
Unported files: 456/3023 (84.9% of total)
Unported lines: 161478/1037467 (84.4% of total)
Longest unported chain: 16/117 (86.3% progress)

port-progress bot (Jun 07 2023 at 20:49):

616/3024 files completely ported (20.37%), in the sense that also all downstream dependencies are ported.

Kevin Buzzard (Jun 07 2023 at 20:59):

Presumably the height is highly correlated with the length of the longest unported chain.

Patrick Stevens (Jun 07 2023 at 21:04):

I'd be mildly interested to know from the peanut gallery why it seems to be going so fast at the moment - is it more people, improvements to the porting process, better parallelism, more enthusiasm, more dedicated time people are setting aside for it, something else?

Jireh Loreaux (Jun 07 2023 at 21:05):

1.2%

Scott Morrison (Jun 07 2023 at 21:06):

  • We got past the etaExperiment bottleneck ~3 weeks ago
  • A lot of people active in porting were at Banff 2 weeks ago, and had a lot of time to allocate to it
  • We're getting near the end and people are excited
  • We've dealt with a lot of problems and many files are now porting very smoothly

Allocate percentages as you see fit. :-)

Matthew Ballard (Jun 07 2023 at 21:07):

  • Lessened teaching demands in the summer

Kevin Buzzard (Jun 07 2023 at 21:09):

More people learning the skill.

Yury G. Kudryashov (Jun 07 2023 at 21:28):

@Jireh Loreaux 's #18854 semi-broke #port-status: now we have a new file with 500+ reverse dependencies. It can't be ported before it goes through mathport and files that depend on it are not in the green area.

Yury G. Kudryashov (Jun 07 2023 at 21:28):

Also, e.g., https://leanprover-community.github.io/mathlib-port-status/file/measure_theory/integral/divergence_theorem has no dependency graph.

Yury G. Kudryashov (Jun 07 2023 at 21:29):

BTW, how often is #port-status updated?

Jireh Loreaux (Jun 07 2023 at 21:29):

@Yury G. Kudryashov If you want, I could manually forward port it now. It shouldn't be that bad (at least, the parts that will make everything work again).

Yury G. Kudryashov (Jun 07 2023 at 21:31):

I think that we should wait for mathport.

Yury G. Kudryashov (Jun 07 2023 at 21:32):

We have enough in-progress files to fill the gap.

Jireh Loreaux (Jun 07 2023 at 21:34):

Alright, I'll forward port as soon as the next mathport comes through. When is the next mathlib3 run scheduled? (EDIT: in about 6 hours it should be ready)

Eric Wieser (Jun 07 2023 at 22:02):

Yury G. Kudryashov said:

BTW, how often is #port-status updated?

Every half hour, but there's another 20 minutes or so of latency as it uses the output from another script that is run every 10 minutes

Eric Wieser (Jun 07 2023 at 22:03):

Yury G. Kudryashov said:

Also, e.g., https://leanprover-community.github.io/mathlib-port-status/file/measure_theory/integral/divergence_theorem has no dependency graph.

This means you can port it after all!

Eric Wieser (Jun 07 2023 at 22:05):

Yury G. Kudryashov said:

Jireh Loreaux 's #18854 semi-broke #port-status: now we have a new file with 500+ reverse dependencies.

This is just a bug in #port-dashboard; it counts unported dependences rather than pruning ported dependencies recursively and _then_ counting unported dependencies

Yury G. Kudryashov (Jun 07 2023 at 22:34):

Eric Wieser said:

Yury G. Kudryashov said:

Also, e.g., https://leanprover-community.github.io/mathlib-port-status/file/measure_theory/integral/divergence_theorem has no dependency graph.

Already done: !4#4814.
This means you can port it after all!

Yury G. Kudryashov (Jun 07 2023 at 22:35):

Eric Wieser said:

Yury G. Kudryashov said:

BTW, how often is #port-status updated?

Every half hour, but there's another 20 minutes or so of latency as it uses the output from another script that is run every 10 minutes

!4#4773 was merged ~4h ago but is still on the list of "in-progress" files.

Eric Wieser (Jun 07 2023 at 22:38):

#port-wiki hasn't been updated for 7 hours

Eric Wieser (Jun 07 2023 at 22:39):

And the dashboard just consumes that to know what's ported

Yury G. Kudryashov (Jun 07 2023 at 22:45):

So, we should ping @Johan Commelin to run his script?

Eric Wieser (Jun 07 2023 at 22:55):

I suspect the script crashed, but only Johan can see its traceback

Pol'tta / Miyahara Kō (Jun 08 2023 at 03:04):

MeasureTheory.Function.Jacobian is ready to review except a dependent file.

Johan Commelin (Jun 08 2023 at 03:45):

somehow my server ended up in a borked state after testing the tweaks to the script yesterday. It should be running again

Johan Commelin (Jun 08 2023 at 04:01):

script seems to have completed succesfully

Johan Commelin (Jun 08 2023 at 04:26):

and we have a fresh #port-status

Yury G. Kudryashov (Jun 08 2023 at 05:24):

Is it intentional that #port-status leads to the /old URL?

Jireh Loreaux (Jun 08 2023 at 05:30):

!4#4840 is the forward port of #18854, as promised.

Johan Commelin (Jun 08 2023 at 05:34):

#port-dashboard should give the new one

David Loeffler (Jun 08 2023 at 05:53):

Ruben Van de Velde said:

Hmm, seems like number_theory.modular_forms.jacobi_theta pulls in a bunch of manifold stuff for the one lemma mdifferentiable_jacobi_theta. Not sure if that's worth changing

This is kind of irrelevant for the applications of jacobi_theta to zeta values; it's there in order to link up with the general modular forms code. So I wouldn't lose any sleep if it were removed. But the manifold stuff has to get ported sooner or later anyway so it's debatable whether removing it is a real gain.

Yury G. Kudryashov (Jun 08 2023 at 13:06):

You can also move this lemma to a new file.

port-progress bot (Jun 08 2023 at 19:04):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 32/1052 (97.0% of total)
Unported lines: 12241/446344 (97.3% of total)
Longest unported chain: 12/97 (87.6% progress)

port-progress bot (Jun 08 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4664/380449 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 08 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 22/978 (97.8% of total)
Unported lines: 11326/398670 (97.2% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 08 2023 at 19:17):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 9/1112 (99.2% of total)
Unported lines: 4618/496486 (99.1% of total)
Longest unported chain: 1/105 (99.0% progress)

port-progress bot (Jun 08 2023 at 19:22):

mathlib port progress analysis.fourier.add_circle
Unported files: 10/1108 (99.1% of total)
Unported lines: 4528/495138 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 08 2023 at 19:27):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 24/1125 (97.9% of total)
Unported lines: 13813/505870 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 08 2023 at 19:30):

mathlib port progress measure_theory.function.jacobian
Unported files: 7/1097 (99.4% of total)
Unported lines: 3409/496166 (99.3% of total)
Longest unported chain: 1/107 (99.1% progress)

port-progress bot (Jun 08 2023 at 19:34):

mathlib port progress all
Unported files: 417/3023 (86.2% of total)
Unported lines: 146645/1037654 (85.9% of total)
Longest unported chain: 15/117 (87.2% progress)

Johan Commelin (Jun 08 2023 at 19:35):

1.5%

port-progress bot (Jun 08 2023 at 19:35):

638/3024 files completely ported (21.09%), in the sense that also all downstream dependencies are ported.

Johan Commelin (Jun 08 2023 at 19:36):

39 files ported today

port-progress bot (Jun 08 2023 at 23:09):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/279803 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 08 2023 at 23:13):

mathlib port progress representation_theory.character
Unported files: 17/920 (98.2% of total)
Unported lines: 6019/349072 (98.3% of total)
Longest unported chain: 6/91 (93.4% progress)

port-progress bot (Jun 08 2023 at 23:18):

mathlib port progress algebra.lie.weights
Unported files: 11/573 (98.1% of total)
Unported lines: 5024/234270 (97.9% of total)
Longest unported chain: 2/74 (97.3% progress)

port-progress bot (Jun 09 2023 at 00:49):

mathlib port progress analysis.normed_space.star.continuous_functional_calculus
Unported files: 19/1183 (98.4% of total)
Unported lines: 7258/517801 (98.6% of total)
Longest unported chain: 7/111 (93.7% progress)

port-progress bot (Jun 09 2023 at 00:53):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 19/748 (97.5% of total)
Unported lines: 6908/297732 (97.7% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 09 2023 at 00:59):

mathlib port progress number_theory.zeta_function
Unported files: 44/1253 (96.5% of total)
Unported lines: 23035/557254 (95.9% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 09 2023 at 01:03):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6695/404657 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 09 2023 at 01:27):

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 14/1035 (98.6% of total)
Unported lines: 8654/448654 (98.1% of total)
Longest unported chain: 5/108 (95.4% progress)

port-progress bot (Jun 09 2023 at 01:31):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156365 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 09 2023 at 01:35):

mathlib port progress order.category.FinBoolAlg
Unported files: 15/348 (95.7% of total)
Unported lines: 4203/129422 (96.7% of total)
Longest unported chain: 5/49 (89.8% progress)

port-progress bot (Jun 09 2023 at 01:59):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/284960 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 09 2023 at 02:03):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346633 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 09 2023 at 02:06):

mathlib port progress number_theory.pell
Unported files: 11/807 (98.6% of total)
Unported lines: 5452/344867 (98.4% of total)
Longest unported chain: 3/81 (96.3% progress)

port-progress bot (Jun 09 2023 at 02:10):

mathlib port progress topology.sheaves.locally_surjective
Unported files: 10/822 (98.8% of total)
Unported lines: 3870/329177 (98.8% of total)
Longest unported chain: 2/80 (97.5% progress)

port-progress bot (Jun 09 2023 at 02:11):

639/3024 files completely ported (21.13%), in the sense that also all downstream dependencies are ported.

Kevin Buzzard (Jun 09 2023 at 06:46):

Where is "all"? I was going to post something of the form "three days ago there were under 500 files to go, now there are under 400" (assuming there are under 400 to go...)

Johan Commelin (Jun 09 2023 at 06:47):

There are now two different runs. all is posted about 15 posts up.

Johan Commelin (Jun 09 2023 at 06:48):

You'll have to wait one day with posting your intended message

Kevin Buzzard (Jun 09 2023 at 06:48):

Ok I'll wait!

Scott Morrison (Jun 09 2023 at 06:52):

(There are not really meant to be two runs, that's just me being silly. Going forward there should be one run each day, ending with all.)

port-progress bot (Jun 09 2023 at 19:07):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 30/1052 (97.1% of total)
Unported lines: 11447/446360 (97.4% of total)
Longest unported chain: 11/97 (88.7% progress)

port-progress bot (Jun 09 2023 at 19:12):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4664/380456 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 09 2023 at 19:18):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 22/978 (97.8% of total)
Unported lines: 11326/398677 (97.2% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 09 2023 at 19:22):

mathlib port progress analysis.complex.cauchy_integral
Unported files: 7/1112 (99.4% of total)
Unported lines: 3409/496505 (99.3% of total)
Longest unported chain: 1/105 (99.0% progress)

port-progress bot (Jun 09 2023 at 19:28):

mathlib port progress analysis.fourier.add_circle
Unported files: 10/1108 (99.1% of total)
Unported lines: 4528/495151 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 09 2023 at 19:34):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 24/1125 (97.9% of total)
Unported lines: 13813/505880 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 09 2023 at 19:39):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/279810 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 09 2023 at 19:44):

mathlib port progress representation_theory.character
Unported files: 16/920 (98.3% of total)
Unported lines: 5562/349085 (98.4% of total)
Longest unported chain: 5/91 (94.5% progress)

port-progress bot (Jun 09 2023 at 19:49):

mathlib port progress algebra.lie.weights
Unported files: 11/573 (98.1% of total)
Unported lines: 5024/234289 (97.9% of total)
Longest unported chain: 2/74 (97.3% progress)

port-progress bot (Jun 09 2023 at 19:55):

mathlib port progress analysis.normed_space.star.continuous_functional_calculus
Unported files: 15/1183 (98.7% of total)
Unported lines: 5467/517832 (98.9% of total)
Longest unported chain: 5/111 (95.5% progress)

port-progress bot (Jun 09 2023 at 20:01):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 18/748 (97.6% of total)
Unported lines: 6451/297751 (97.8% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 09 2023 at 20:07):

mathlib port progress number_theory.zeta_function
Unported files: 37/1253 (97.0% of total)
Unported lines: 20078/557291 (96.4% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 09 2023 at 20:12):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6695/404667 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 09 2023 at 20:18):

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 14/1035 (98.6% of total)
Unported lines: 8654/448664 (98.1% of total)
Longest unported chain: 5/108 (95.4% progress)

port-progress bot (Jun 09 2023 at 20:23):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156365 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 09 2023 at 20:28):

mathlib port progress order.category.FinBoolAlg
Unported files: 15/348 (95.7% of total)
Unported lines: 4203/129422 (96.7% of total)
Longest unported chain: 5/49 (89.8% progress)

port-progress bot (Jun 09 2023 at 20:33):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/284967 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 09 2023 at 20:39):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346643 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 09 2023 at 20:44):

mathlib port progress number_theory.pell
Unported files: 11/807 (98.6% of total)
Unported lines: 5452/344877 (98.4% of total)
Longest unported chain: 3/81 (96.3% progress)

port-progress bot (Jun 09 2023 at 20:49):

mathlib port progress topology.sheaves.locally_surjective
Unported files: 10/822 (98.8% of total)
Unported lines: 3870/329184 (98.8% of total)
Longest unported chain: 2/80 (97.5% progress)

port-progress bot (Jun 09 2023 at 20:55):

mathlib port progress probability.borel_cantelli
Unported files: 23/1062 (97.8% of total)
Unported lines: 11502/479860 (97.6% of total)
Longest unported chain: 10/113 (91.2% progress)

port-progress bot (Jun 09 2023 at 21:01):

mathlib port progress probability.kernel.condexp
Unported files: 16/1044 (98.5% of total)
Unported lines: 9270/473298 (98.0% of total)
Longest unported chain: 5/108 (95.4% progress)

port-progress bot (Jun 09 2023 at 21:07):

mathlib port progress all
Unported files: 385/3024 (87.3% of total)
Unported lines: 137343/1038375 (86.8% of total)
Longest unported chain: 14/117 (88.0% progress)

port-progress bot (Jun 09 2023 at 21:08):

656/3025 files completely ported (21.68%), in the sense that also all downstream dependencies are ported.

Johan Commelin (Jun 09 2023 at 21:09):

0.9%

Johan Commelin (Jun 09 2023 at 21:10):

32 files ported today

Ruben Van de Velde (Jun 09 2023 at 21:11):

We're slacking off!

Ruben Van de Velde (Jun 09 2023 at 23:36):

389(*) unported, 65 in progress

(*) including archive and some data structure files that don't need porting

Yury G. Kudryashov (Jun 09 2023 at 23:37):

Am I right that archive counts towards "unported" but we can't port it yet?

Ruben Van de Velde (Jun 09 2023 at 23:42):

I thought we could? But I haven't tried any yet

James Gallicchio (Jun 10 2023 at 00:04):

https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/mk_all.2Esh

James Gallicchio (Jun 10 2023 at 00:04):

i'm assuming this means the archive is portable now? :joy: maybe i'll try to port one of the short freek theorems tonight

Yury G. Kudryashov (Jun 10 2023 at 00:36):

start_port.sh still doesn't support paths outside of Mathlib.

Eric Wieser (Jun 10 2023 at 00:59):

!4#4811 adds support for that

Eric Wieser (Jun 10 2023 at 00:59):

But we shouldn't merge it until we teach mathlib4 CI to actually build things in the archive directory

Eric Wieser (Jun 10 2023 at 01:00):

Otherwise we're just going to end up having people port code that doesn't work

Scott Morrison (Jun 10 2023 at 01:34):

It seems like there's a chicken and egg problem here. No one is going to update the CI until there is a file to test / we know where it lives, etc.

Scott Morrison (Jun 10 2023 at 01:35):

I propose that someone makes the first PR of an Archive file, and we'll just make sure not to actually merge it until it has proper CI.

Scott Morrison (Jun 10 2023 at 01:35):

i.e. so we should merge !4#4811 now.

Eric Wieser (Jun 10 2023 at 01:41):

I already made a first PR of an archive file, !4#4812

Eric Wieser (Jun 10 2023 at 01:43):

The sequence should be:

  • Push some lakefile config to !4#4812 and convince ourselves that it's really being built in CI
  • Merge !4#4812, the porting PR
  • Merge !4#4811, the script PR

Eric Wieser (Jun 10 2023 at 01:43):

Merging the script PR first isn't going to do us any favors, especially if it turns out we need to modify the script to make CI work

Eric Wieser (Jun 10 2023 at 01:46):

It seems like there's a chicken and egg problem here

The chicken doesn't have to be on the master branch to produce an egg :)

Yury G. Kudryashov (Jun 10 2023 at 03:00):

!4#4812 should not depend on !4#4811, if we're going to merge it first.

Johan Commelin (Jun 10 2023 at 05:48):

https://tqft.net/mathlib4/2023-06-10/all shows that number_theory/wilson is now at the end of the longest chain... :rofl:
It also suggests that this can easily be solved by some refactor.

Ruben Van de Velde (Jun 10 2023 at 08:33):

Johan Commelin said:

https://tqft.net/mathlib4/2023-06-10/all shows that number_theory/wilson is now at the end of the longest chain... :rofl:
It also suggests that this can easily be solved by some refactor.

A refactor that was hinted at in a todo in the source, even: https://github.com/leanprover-community/mathlib/pull/19172

Scott Morrison (Jun 10 2023 at 08:34):

#19173

Scott Morrison (Jun 10 2023 at 08:34):

:racecar:

Ruben Van de Velde (Jun 10 2023 at 08:47):

:racecar: :race:

port-progress bot (Jun 10 2023 at 19:05):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 29/1052 (97.2% of total)
Unported lines: 10919/446384 (97.6% of total)
Longest unported chain: 11/97 (88.7% progress)

port-progress bot (Jun 10 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4664/380456 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 10 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 22/978 (97.8% of total)
Unported lines: 11326/398692 (97.2% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 10 2023 at 19:18):

mathlib port progress analysis.fourier.add_circle
Unported files: 9/1108 (99.2% of total)
Unported lines: 4331/495169 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 10 2023 at 19:22):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1125 (98.0% of total)
Unported lines: 13616/505898 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 10 2023 at 19:26):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/279825 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 10 2023 at 19:30):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4639/349106 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 10 2023 at 19:34):

mathlib port progress algebra.lie.weights
Unported files: 9/573 (98.4% of total)
Unported lines: 4191/234295 (98.2% of total)
Longest unported chain: 1/74 (98.6% progress)

port-progress bot (Jun 10 2023 at 19:39):

mathlib port progress analysis.normed_space.star.continuous_functional_calculus
Unported files: 12/1183 (99.0% of total)
Unported lines: 4738/517862 (99.1% of total)
Longest unported chain: 3/111 (97.3% progress)

port-progress bot (Jun 10 2023 at 19:43):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5923/297772 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 10 2023 at 19:48):

mathlib port progress number_theory.zeta_function
Unported files: 33/1253 (97.4% of total)
Unported lines: 19252/557339 (96.5% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 10 2023 at 19:52):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6695/404682 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 10 2023 at 19:56):

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 14/1035 (98.6% of total)
Unported lines: 8654/448679 (98.1% of total)
Longest unported chain: 5/108 (95.4% progress)

port-progress bot (Jun 10 2023 at 20:00):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156365 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 10 2023 at 20:03):

mathlib port progress order.category.FinBoolAlg
Unported files: 15/348 (95.7% of total)
Unported lines: 4203/129422 (96.7% of total)
Longest unported chain: 5/49 (89.8% progress)

port-progress bot (Jun 10 2023 at 20:07):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/284967 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 10 2023 at 20:11):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346643 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 10 2023 at 20:15):

mathlib port progress number_theory.pell
Unported files: 11/807 (98.6% of total)
Unported lines: 5452/344892 (98.4% of total)
Longest unported chain: 3/81 (96.3% progress)

port-progress bot (Jun 10 2023 at 20:19):

mathlib port progress topology.sheaves.locally_surjective
Unported files: 9/822 (98.9% of total)
Unported lines: 3714/329199 (98.9% of total)
Longest unported chain: 1/80 (98.8% progress)

port-progress bot (Jun 10 2023 at 20:24):

mathlib port progress probability.borel_cantelli
Unported files: 23/1062 (97.8% of total)
Unported lines: 11502/479875 (97.6% of total)
Longest unported chain: 10/113 (91.2% progress)

port-progress bot (Jun 10 2023 at 20:28):

mathlib port progress probability.kernel.condexp
Unported files: 16/1044 (98.5% of total)
Unported lines: 9270/473316 (98.0% of total)
Longest unported chain: 5/108 (95.4% progress)

port-progress bot (Jun 10 2023 at 20:33):

mathlib port progress all
Unported files: 366/3025 (87.9% of total)
Unported lines: 132899/1038756 (87.2% of total)
Longest unported chain: 14/117 (88.0% progress)

port-progress bot (Jun 10 2023 at 20:34):

676/3026 files completely ported (22.33%), in the sense that also all downstream dependencies are ported.

Chris Hughes (Jun 10 2023 at 21:44):

0.4%

port-progress bot (Jun 11 2023 at 19:05):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 29/1052 (97.2% of total)
Unported lines: 10919/446393 (97.6% of total)
Longest unported chain: 11/97 (88.7% progress)

port-progress bot (Jun 11 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4664/380465 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 11 2023 at 19:14):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 22/978 (97.8% of total)
Unported lines: 11326/398692 (97.2% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 11 2023 at 19:19):

mathlib port progress analysis.fourier.add_circle
Unported files: 9/1108 (99.2% of total)
Unported lines: 4331/495178 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 11 2023 at 19:24):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1125 (98.0% of total)
Unported lines: 13616/505907 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 11 2023 at 19:28):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/279825 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 11 2023 at 19:32):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4639/349112 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 11 2023 at 19:37):

mathlib port progress algebra.lie.weights
Unported files: 9/573 (98.4% of total)
Unported lines: 4191/234295 (98.2% of total)
Longest unported chain: 1/74 (98.6% progress)

port-progress bot (Jun 11 2023 at 19:42):

mathlib port progress analysis.normed_space.star.continuous_functional_calculus
Unported files: 9/1183 (99.2% of total)
Unported lines: 3911/517877 (99.2% of total)
Longest unported chain: 1/111 (99.1% progress)

port-progress bot (Jun 11 2023 at 19:46):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5923/297772 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 11 2023 at 19:52):

mathlib port progress number_theory.zeta_function
Unported files: 33/1253 (97.4% of total)
Unported lines: 19252/557551 (96.5% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 11 2023 at 19:56):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6695/404691 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 11 2023 at 20:01):

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 14/1035 (98.6% of total)
Unported lines: 8654/448688 (98.1% of total)
Longest unported chain: 5/108 (95.4% progress)

port-progress bot (Jun 11 2023 at 20:05):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156365 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 11 2023 at 20:09):

mathlib port progress order.category.FinBoolAlg
Unported files: 15/348 (95.7% of total)
Unported lines: 4203/129422 (96.7% of total)
Longest unported chain: 5/49 (89.8% progress)

port-progress bot (Jun 11 2023 at 20:14):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/284976 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 11 2023 at 20:18):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346652 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 11 2023 at 20:23):

mathlib port progress number_theory.pell
Unported files: 11/807 (98.6% of total)
Unported lines: 5452/344901 (98.4% of total)
Longest unported chain: 3/81 (96.3% progress)

port-progress bot (Jun 11 2023 at 20:27):

mathlib port progress topology.sheaves.locally_surjective
Unported files: 8/822 (99.0% of total)
Unported lines: 3533/329202 (98.9% of total)
Longest unported chain: 1/80 (98.8% progress)

port-progress bot (Jun 11 2023 at 20:32):

mathlib port progress probability.borel_cantelli
Unported files: 23/1062 (97.8% of total)
Unported lines: 11502/479884 (97.6% of total)
Longest unported chain: 10/113 (91.2% progress)

port-progress bot (Jun 11 2023 at 20:37):

mathlib port progress probability.kernel.condexp
Unported files: 16/1044 (98.5% of total)
Unported lines: 9270/473325 (98.0% of total)
Longest unported chain: 5/108 (95.4% progress)

port-progress bot (Jun 11 2023 at 20:43):

mathlib port progress all
Unported files: 356/3026 (88.2% of total)
Unported lines: 128936/1039084 (87.6% of total)
Longest unported chain: 14/117 (88.0% progress)

port-progress bot (Jun 11 2023 at 20:44):

684/3027 files completely ported (22.59%), in the sense that also all downstream dependencies are ported.

Scott Morrison (Jun 11 2023 at 22:47):

0.4%

Yury G. Kudryashov (Jun 12 2023 at 01:34):

@Eric Wieser I started !4#4978 and I'm experimenting with the build system there. For some reason, lake exe cache get failed to fetch a single file, so it's rebuilding everything.

Scott Morrison (Jun 12 2023 at 02:08):

Modifying the lakefile.lean invalidates the entire olean cache.

Yury G. Kudryashov (Jun 12 2023 at 03:13):

So, should we host examples in the main repo?

Yury G. Kudryashov (Jun 12 2023 at 03:14):

Or create new repos for IMO (or, more generally, math contest problems), 100-theorems, and misc?

Yury G. Kudryashov (Jun 12 2023 at 03:28):

If we host them with mathlib, will it make them available to any package that adds mathlib as a dependency?

Scott Morrison (Jun 12 2023 at 03:52):

Aren't we just keeping the structure from mathlib3? I'd prefer not to change anything that doesn't immediately need changing.

Yury G. Kudryashov (Jun 12 2023 at 04:12):

If hosting archive/... with mathlib4 has more implications than in lean3 case, then we can reconsider.

Yury G. Kudryashov (Jun 12 2023 at 04:12):

Instead, we can move the current archive etc to new repo(s) and consider it one of the "projects".

Yury G. Kudryashov (Jun 12 2023 at 04:19):

I mean, in Lean 3 it was possible to host some files in the same repo and build them in CI without making them a part of the official package.

Eric Wieser (Jun 12 2023 at 07:48):

In mathlib 3 they're packaged as an "official package" too

Yury G. Kudryashov (Jun 12 2023 at 14:21):

I opened a tmp file in sphere-eversion. import archive.arithcc fails, import algebra.algebra.basic works.

Yury G. Kudryashov (Jun 12 2023 at 14:25):

In a a fresh lake init tmp math project,

import Mathlib.Algebra.Algebra.Basic
import MathlibExtras.Rewrites

both work.

Yury G. Kudryashov (Jun 12 2023 at 14:26):

So, if we have Archive/, Counterexamples/ etc, then we make them available for import in projects that depend on mathlib.

port-progress bot (Jun 12 2023 at 19:04):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 29/1052 (97.2% of total)
Unported lines: 10919/446401 (97.6% of total)
Longest unported chain: 11/97 (88.7% progress)

port-progress bot (Jun 12 2023 at 19:08):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4664/380473 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 12 2023 at 19:12):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 22/978 (97.8% of total)
Unported lines: 11326/398700 (97.2% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 12 2023 at 19:17):

mathlib port progress analysis.fourier.add_circle
Unported files: 9/1108 (99.2% of total)
Unported lines: 4331/495186 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 12 2023 at 19:21):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1125 (98.0% of total)
Unported lines: 13616/505915 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 12 2023 at 19:25):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/279833 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 12 2023 at 19:29):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4639/349120 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 12 2023 at 19:33):

mathlib port progress algebra.lie.weights
Unported files: 8/573 (98.6% of total)
Unported lines: 3906/234303 (98.3% of total)
Longest unported chain: 1/74 (98.6% progress)

port-progress bot (Jun 12 2023 at 19:36):

mathlib port progress analysis.normed_space.star.continuous_functional_calculus
Unported files: 7/1183 (99.4% of total)
Unported lines: 3409/517897 (99.3% of total)
Longest unported chain: 1/111 (99.1% progress)

port-progress bot (Jun 12 2023 at 19:40):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5923/297780 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 12 2023 at 19:45):

mathlib port progress number_theory.zeta_function
Unported files: 33/1253 (97.4% of total)
Unported lines: 19252/557559 (96.5% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 12 2023 at 19:49):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6695/404699 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 12 2023 at 19:54):

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 14/1035 (98.6% of total)
Unported lines: 8654/448696 (98.1% of total)
Longest unported chain: 5/108 (95.4% progress)

port-progress bot (Jun 12 2023 at 19:58):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156373 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 12 2023 at 20:01):

mathlib port progress order.category.FinBoolAlg
Unported files: 15/348 (95.7% of total)
Unported lines: 4203/129422 (96.7% of total)
Longest unported chain: 5/49 (89.8% progress)

port-progress bot (Jun 12 2023 at 20:06):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/284984 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 12 2023 at 20:11):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346660 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 12 2023 at 20:15):

mathlib port progress number_theory.pell
Unported files: 11/807 (98.6% of total)
Unported lines: 5452/344909 (98.4% of total)
Longest unported chain: 3/81 (96.3% progress)

port-progress bot (Jun 12 2023 at 20:20):

mathlib port progress topology.sheaves.locally_surjective
Unported files: 8/822 (99.0% of total)
Unported lines: 3533/329213 (98.9% of total)
Longest unported chain: 1/80 (98.8% progress)

port-progress bot (Jun 12 2023 at 20:25):

mathlib port progress probability.borel_cantelli
Unported files: 27/1066 (97.5% of total)
Unported lines: 11657/480047 (97.6% of total)
Longest unported chain: 14/116 (87.9% progress)

port-progress bot (Jun 12 2023 at 20:30):

mathlib port progress probability.kernel.condexp
Unported files: 20/1048 (98.1% of total)
Unported lines: 9425/473488 (98.0% of total)
Longest unported chain: 7/109 (93.6% progress)

port-progress bot (Jun 12 2023 at 20:35):

mathlib port progress all
Unported files: 350/3030 (88.4% of total)
Unported lines: 126323/1039250 (87.8% of total)
Longest unported chain: 15/117 (87.2% progress)

port-progress bot (Jun 12 2023 at 20:35):

0/3031 files completely ported (0%), in the sense that also all downstream dependencies are ported.

Scott Morrison (Jun 12 2023 at 20:45):

0.2%

Yury G. Kudryashov (Jun 12 2023 at 20:53):

We're too slow. Why 0 files are completely ported?

Jireh Loreaux (Jun 12 2023 at 21:51):

FYI: analysis.normed_space.star.continuous_functional_calculus is done (which I think you saw, but just emphasizing it can be removed from the bot @Scott Morrison). I guess this is sort of a big milestone since it was at one point the end of the longest chain!

Scott Morrison (Jun 12 2023 at 22:21):

Yury G. Kudryashov said:

We're too slow. Why 0 files are completely ported?

Sorry, the bot that does this computation is unreliable for a reason I haven't understood yet.

port-progress bot (Jun 13 2023 at 19:04):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 29/1052 (97.2% of total)
Unported lines: 10915/446420 (97.6% of total)
Longest unported chain: 11/97 (88.7% progress)

port-progress bot (Jun 13 2023 at 19:08):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4636/380445 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 13 2023 at 19:12):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 22/978 (97.8% of total)
Unported lines: 11326/398722 (97.2% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 13 2023 at 19:17):

mathlib port progress analysis.fourier.add_circle
Unported files: 9/1108 (99.2% of total)
Unported lines: 4331/495208 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 13 2023 at 19:21):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1125 (98.0% of total)
Unported lines: 13616/505937 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 13 2023 at 19:25):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/279855 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 13 2023 at 19:29):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4611/349115 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 13 2023 at 19:33):

mathlib port progress algebra.lie.weights
Unported files: 8/573 (98.6% of total)
Unported lines: 3906/234306 (98.3% of total)
Longest unported chain: 1/74 (98.6% progress)

port-progress bot (Jun 13 2023 at 19:37):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5923/297803 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 13 2023 at 19:42):

mathlib port progress number_theory.zeta_function
Unported files: 33/1253 (97.4% of total)
Unported lines: 19252/557581 (96.5% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 13 2023 at 19:46):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6695/404721 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 13 2023 at 19:50):

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 12/1035 (98.8% of total)
Unported lines: 6972/448718 (98.4% of total)
Longest unported chain: 3/108 (97.2% progress)

port-progress bot (Jun 13 2023 at 19:54):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156373 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 13 2023 at 19:58):

mathlib port progress order.category.FinBoolAlg
Unported files: 13/348 (96.3% of total)
Unported lines: 3972/129422 (96.9% of total)
Longest unported chain: 4/49 (91.8% progress)

port-progress bot (Jun 13 2023 at 20:01):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/284984 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 13 2023 at 20:05):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346660 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 13 2023 at 20:09):

mathlib port progress number_theory.pell
Unported files: 11/807 (98.6% of total)
Unported lines: 5452/344931 (98.4% of total)
Longest unported chain: 3/81 (96.3% progress)

port-progress bot (Jun 13 2023 at 20:13):

mathlib port progress topology.sheaves.locally_surjective
Unported files: 8/822 (99.0% of total)
Unported lines: 3533/329235 (98.9% of total)
Longest unported chain: 1/80 (98.8% progress)

port-progress bot (Jun 13 2023 at 20:18):

mathlib port progress probability.borel_cantelli
Unported files: 26/1066 (97.6% of total)
Unported lines: 10959/480069 (97.7% of total)
Longest unported chain: 13/116 (88.8% progress)

port-progress bot (Jun 13 2023 at 20:22):

mathlib port progress probability.kernel.condexp
Unported files: 19/1048 (98.2% of total)
Unported lines: 8727/473510 (98.2% of total)
Longest unported chain: 6/109 (94.5% progress)

port-progress bot (Jun 13 2023 at 20:27):

mathlib port progress all
Unported files: 336/3030 (88.9% of total)
Unported lines: 122396/1039547 (88.2% of total)
Longest unported chain: 14/117 (88.0% progress)

port-progress bot (Jun 13 2023 at 20:28):

721/3031 files completely ported (23.78%), in the sense that also all downstream dependencies are ported.

Scott Morrison (Jun 13 2023 at 22:07):

0.4%

port-progress bot (Jun 14 2023 at 19:04):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 29/1052 (97.2% of total)
Unported lines: 10915/446423 (97.6% of total)
Longest unported chain: 11/97 (88.7% progress)

port-progress bot (Jun 14 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4636/380448 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 14 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 19/978 (98.1% of total)
Unported lines: 10244/398725 (97.4% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 14 2023 at 19:18):

mathlib port progress analysis.fourier.add_circle
Unported files: 9/1117 (99.2% of total)
Unported lines: 4331/499308 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 14 2023 at 19:22):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1125 (98.0% of total)
Unported lines: 13688/506015 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 14 2023 at 19:27):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/279858 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 14 2023 at 19:31):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4611/349118 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 14 2023 at 19:34):

mathlib port progress algebra.lie.weights
Unported files: 7/573 (98.8% of total)
Unported lines: 3409/234306 (98.5% of total)
Longest unported chain: 1/74 (98.6% progress)

port-progress bot (Jun 14 2023 at 19:38):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5923/297806 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 14 2023 at 19:43):

mathlib port progress number_theory.zeta_function
Unported files: 28/1253 (97.8% of total)
Unported lines: 16708/557745 (97.0% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 14 2023 at 19:47):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6761/404790 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 14 2023 at 19:51):

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 8/1035 (99.2% of total)
Unported lines: 3837/448727 (99.1% of total)
Longest unported chain: 1/108 (99.1% progress)

port-progress bot (Jun 14 2023 at 19:55):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156373 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 14 2023 at 19:59):

mathlib port progress order.category.FinBoolAlg
Unported files: 12/348 (96.6% of total)
Unported lines: 3808/129428 (97.1% of total)
Longest unported chain: 3/49 (93.9% progress)

port-progress bot (Jun 14 2023 at 20:03):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/284984 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 14 2023 at 20:08):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346660 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 14 2023 at 20:12):

mathlib port progress number_theory.pell
Unported files: 11/807 (98.6% of total)
Unported lines: 5452/344934 (98.4% of total)
Longest unported chain: 3/81 (96.3% progress)

Ruben Van de Velde (Jun 14 2023 at 20:12):

port-progress bot said:

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346660 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

This one's stuck on an extension to positivity in !4#4409, in case anyone wants to look at it. (@Damiano Testa as my usual suspect? :innocent: )

port-progress bot (Jun 14 2023 at 20:16):

mathlib port progress topology.sheaves.locally_surjective
Unported files: 8/822 (99.0% of total)
Unported lines: 3533/329238 (98.9% of total)
Longest unported chain: 1/80 (98.8% progress)

port-progress bot (Jun 14 2023 at 20:20):

mathlib port progress probability.borel_cantelli
Unported files: 25/1066 (97.7% of total)
Unported lines: 10746/480227 (97.8% of total)
Longest unported chain: 12/116 (89.7% progress)

port-progress bot (Jun 14 2023 at 20:25):

mathlib port progress probability.kernel.condexp
Unported files: 17/1048 (98.4% of total)
Unported lines: 8197/473668 (98.3% of total)
Longest unported chain: 5/109 (95.4% progress)

port-progress bot (Jun 14 2023 at 20:30):

mathlib port progress all
Unported files: 312/3031 (89.7% of total)
Unported lines: 112836/1040034 (89.2% of total)
Longest unported chain: 14/117 (88.0% progress)

port-progress bot (Jun 14 2023 at 20:31):

742/3032 files completely ported (24.47%), in the sense that also all downstream dependencies are ported.

Ruben Van de Velde (Jun 14 2023 at 20:35):

port-progress bot said:

mathlib port progress all
Unported files: 312/3031 (89.7% of total)
Unported lines: 112836/1040034 (89.2% of total)
Longest unported chain: 14/117 (88.0% progress)

Let's get to 90!

Ruben Van de Velde (Jun 14 2023 at 20:43):

port-progress bot said:

mathlib port progress topology.sheaves.locally_surjective
Unported files: 8/822 (99.0% of total)
Unported lines: 3533/329238 (98.9% of total)
Longest unported chain: 1/80 (98.8% progress)

!4#4980 up for review

Ruben Van de Velde (Jun 14 2023 at 20:44):

port-progress bot said:

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 8/1035 (99.2% of total)
Unported lines: 3837/448727 (99.1% of total)
Longest unported chain: 1/108 (99.1% progress)

!4#5054 up for review

Jireh Loreaux (Jun 14 2023 at 20:44):

1.0%

Damiano Testa (Jun 14 2023 at 21:19):

Ruben Van de Velde said:

This one's stuck on an extension to positivity in !4#4409, in case anyone wants to look at it. (Damiano Testa as my usual suspect? :innocent: )

I'd be happy to take it on, but I am still struggling with finding the time to properly port the ghost tactics of Witt. In case no one else does it before, I will look at this once ghost is ported. If you think that this is a priority over ghost, then I can switch the processing order, though!

Yaël Dillies (Jun 14 2023 at 21:22):

I have one or two PRs to this file, so I'd say no rush!

Damiano Testa (Jun 14 2023 at 21:24):

Anyway, my scheduling is just chronological order in which I said I would do it, but I am happy to change, also at a later time. I do try to process these things sequentially though, rather than in parallel.

Ruben Van de Velde (Jun 14 2023 at 21:28):

I have no priorities here (except splitting fields, but those are up for review :tada: )

Patrick Massot (Jun 14 2023 at 21:38):

@Yury G. Kudryashov do you need help with convolution? I guess @Floris van Doorn would be happy to help.

Yury G. Kudryashov (Jun 14 2023 at 22:11):

Yes. I'm sorry for not marking it as help-wanted. I'll do it now.

Mauricio Collares (Jun 15 2023 at 08:14):

Currently there are 316 unported files on the dashboard, but only 248 of them are portable at the moment. The other 68 (21.5% of remaining files) are in archive/counterexamples.

Eric Wieser (Jun 15 2023 at 08:19):

Those are blocked by configuring the lakefile correctly

Eric Wieser (Jun 15 2023 at 08:20):

!4#4978 is where this needs to be solved

Eric Wieser (Jun 15 2023 at 08:22):

In particular, there's the question of whether we need a Counterexamples.lean, or if lake can just be told to build everything in the directory.

Scott Morrison (Jun 15 2023 at 08:42):

Let's just have a Counterexamples.lean. Why not?

Eric Wieser (Jun 15 2023 at 08:42):

Because we're already complaining elsewhere that (conflicts in) the Mathlib.lean is annoying, and it's going to be worse if we have have 15 simultaneous counterexample PRs appear on the same day

Scott Morrison (Jun 15 2023 at 08:50):

Okay, solve that when we get there. That's certainly not a blocker.

Scott Morrison (Jun 15 2023 at 08:50):

I've just pushed changes to !4#4978 that will hopefully make it work. awaiting-CI.

Eric Wieser (Jun 15 2023 at 08:55):

Should we put in the Archive config at the same time?

Scott Morrison (Jun 15 2023 at 11:08):

Done!

Scott Morrison (Jun 15 2023 at 11:09):

It looks like CI is doing its thing on !4#4978, there are errors in the ported file.

Eric Wieser (Jun 15 2023 at 11:50):

Should I split the CI to its own PR so that that doesn't block anything?

Eric Wieser (Jun 15 2023 at 11:55):

!4#5078

Eric Wieser (Jun 15 2023 at 12:00):

I've merged that into both !4#4978 and !4#4812 to check it works in both Archive and Counterexamples

Ruben Van de Velde (Jun 15 2023 at 12:05):

Ruben Van de Velde said:

port-progress bot said:

mathlib port progress topology.sheaves.locally_surjective
Unported files: 8/822 (99.0% of total)
Unported lines: 3533/329238 (98.9% of total)
Longest unported chain: 1/80 (98.8% progress)

!4#4980 up for review

Merged @Scott Morrison

Jeremy Tan (Jun 15 2023 at 14:07):

port-progress bot said:

mathlib port progress all
Unported files: 312/3031 (89.7% of total)
Unported lines: 112836/1040034 (89.2% of total)
Longest unported chain: 14/117 (88.0% progress)

Wait a minute. The longest unported chain output over here shows a long list of hyphens at the beginning

Riccardo Brasca (Jun 15 2023 at 14:11):

Those files are surely needed.

Yury G. Kudryashov (Jun 15 2023 at 14:27):

I fixed some IMO files in a local repo. Once they become portable, I'm going to make PRs for these files.

Eric Wieser (Jun 15 2023 at 14:53):

Eric Wieser said:

!4#5078

This should be ready to go, which will unblock Yury

Johan Commelin (Jun 15 2023 at 15:19):

Kicked it on the queue

port-progress bot (Jun 15 2023 at 19:04):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 28/1052 (97.3% of total)
Unported lines: 10430/446322 (97.7% of total)
Longest unported chain: 10/97 (89.7% progress)

Yury G. Kudryashov (Jun 15 2023 at 19:07):

https://leanprover-community.github.io/mathlib-port-status/file/category_theory/limits/constructions/over/default is the only default file we may want to port because it contains some code other than imports.

port-progress bot (Jun 15 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4636/380448 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 15 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 19/978 (98.1% of total)
Unported lines: 10244/398746 (97.4% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 15 2023 at 19:17):

mathlib port progress analysis.fourier.add_circle
Unported files: 9/1117 (99.2% of total)
Unported lines: 4331/499316 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 15 2023 at 19:22):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1125 (98.0% of total)
Unported lines: 13688/506023 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 15 2023 at 19:26):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/279866 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 15 2023 at 19:30):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4611/349126 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 15 2023 at 19:35):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5923/297814 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 15 2023 at 19:39):

mathlib port progress number_theory.zeta_function
Unported files: 28/1253 (97.8% of total)
Unported lines: 16708/557765 (97.0% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 15 2023 at 19:44):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6761/404798 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 15 2023 at 19:47):

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 7/1035 (99.3% of total)
Unported lines: 3409/448747 (99.2% of total)
Longest unported chain: 1/108 (99.1% progress)

Ruben Van de Velde (Jun 15 2023 at 19:50):

port-progress bot said:

mathlib port progress geometry.euclidean.angle.sphere
Unported files: 7/1035 (99.3% of total)
Unported lines: 3409/448747 (99.2% of total)
Longest unported chain: 1/108 (99.1% progress)

Done

port-progress bot (Jun 15 2023 at 19:51):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156373 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 15 2023 at 19:55):

mathlib port progress order.category.FinBoolAlg
Unported files: 8/348 (97.7% of total)
Unported lines: 3511/129437 (97.3% of total)
Longest unported chain: 1/49 (98.0% progress)

port-progress bot (Jun 15 2023 at 19:59):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/284984 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 15 2023 at 20:03):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346663 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 15 2023 at 20:08):

mathlib port progress number_theory.pell
Unported files: 11/807 (98.6% of total)
Unported lines: 5452/344942 (98.4% of total)
Longest unported chain: 3/81 (96.3% progress)

Jon Eugster (Jun 15 2023 at 20:09):

port-progress bot said:

mathlib port progress order.category.FinBoolAlg
Unported files: 8/348 (97.7% of total)
Unported lines: 3511/129437 (97.3% of total)
Longest unported chain: 1/49 (98.0% progress)

there's one single error left in this one if anybody wants to have a look. !4#5052

Jireh Loreaux (Jun 15 2023 at 20:10):

I just had a look, but didn't see the solution. The FunLike instance seemed suspicious to me though.

port-progress bot (Jun 15 2023 at 20:11):

mathlib port progress topology.sheaves.locally_surjective
Unported files: 7/822 (99.1% of total)
Unported lines: 3409/329246 (99.0% of total)
Longest unported chain: 1/80 (98.8% progress)

port-progress bot (Jun 15 2023 at 20:15):

mathlib port progress probability.borel_cantelli
Unported files: 25/1066 (97.7% of total)
Unported lines: 10746/480238 (97.8% of total)
Longest unported chain: 12/116 (89.7% progress)

port-progress bot (Jun 15 2023 at 20:20):

mathlib port progress probability.kernel.condexp
Unported files: 17/1048 (98.4% of total)
Unported lines: 8197/473682 (98.3% of total)
Longest unported chain: 5/109 (95.4% progress)

port-progress bot (Jun 15 2023 at 20:24):

mathlib port progress all
Unported files: 296/3031 (90.2% of total)
Unported lines: 109440/1040021 (89.5% of total)
Longest unported chain: 13/117 (88.9% progress)

Ruben Van de Velde (Jun 15 2023 at 20:25):

port-progress bot said:

mathlib port progress all
Unported files: 296/3031 (90.2% of total)
Unported lines: 109440/1040021 (89.5% of total)
Longest unported chain: 13/117 (88.9% progress)

First 90% achieved

port-progress bot (Jun 15 2023 at 20:25):

764/3032 files completely ported (25.19%), in the sense that also all downstream dependencies are ported.

Jireh Loreaux (Jun 15 2023 at 20:29):

0.3%

Kevin Buzzard (Jun 15 2023 at 21:03):

Under 300 files to go!

Eric Wieser (Jun 15 2023 at 22:08):

Yury G. Kudryashov said:

I fixed some IMO files in a local repo. Once they become portable, I'm going to make PRs for these files.

#port-wiki doesn't seem to be counting these just yet, but I've made !4#5108 to hopefully fix that

port-progress bot (Jun 16 2023 at 19:07):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 22/1054 (97.9% of total)
Unported lines: 8322/446646 (98.1% of total)
Longest unported chain: 9/97 (90.7% progress)

port-progress bot (Jun 16 2023 at 19:11):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4636/380704 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 16 2023 at 19:15):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 19/978 (98.1% of total)
Unported lines: 10244/399002 (97.4% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 16 2023 at 19:20):

mathlib port progress analysis.fourier.add_circle
Unported files: 9/1117 (99.2% of total)
Unported lines: 4331/499572 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 16 2023 at 23:42):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/280122 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 16 2023 at 23:47):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4611/349382 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 16 2023 at 23:52):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5923/298070 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 16 2023 at 23:57):

mathlib port progress number_theory.zeta_function
Unported files: 28/1253 (97.8% of total)
Unported lines: 16708/558021 (97.0% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 17 2023 at 00:02):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6761/405054 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 17 2023 at 00:07):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156490 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 17 2023 at 00:11):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285240 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 17 2023 at 00:16):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346919 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 17 2023 at 00:19):

mathlib port progress number_theory.pell
Unported files: 7/807 (99.1% of total)
Unported lines: 3409/345201 (99.0% of total)
Longest unported chain: 1/81 (98.8% progress)

port-progress bot (Jun 17 2023 at 00:25):

mathlib port progress probability.borel_cantelli
Unported files: 25/1066 (97.7% of total)
Unported lines: 10746/480494 (97.8% of total)
Longest unported chain: 12/116 (89.7% progress)

port-progress bot (Jun 17 2023 at 00:30):

mathlib port progress probability.kernel.condexp
Unported files: 15/1048 (98.6% of total)
Unported lines: 6320/473938 (98.7% of total)
Longest unported chain: 5/109 (95.4% progress)

port-progress bot (Jun 17 2023 at 00:35):

mathlib port progress all
Unported files: 274/3034 (91.0% of total)
Unported lines: 101732/1040487 (90.2% of total)
Longest unported chain: 13/117 (88.9% progress)

port-progress bot (Jun 17 2023 at 00:37):

796/3035 files completely ported (26.22%), in the sense that also all downstream dependencies are ported.

Scott Morrison (Jun 17 2023 at 00:59):

0.7%, and we're 90% done!

David Michael Roberts (Jun 17 2023 at 01:17):

port-progress bot said:

mathlib port progress number_theory.pell
Unported files: 7/807 (99.1% of total)
Unported lines: 3409/345201 (99.0% of total)
Longest unported chain: 1/81 (98.8% progress)

Is this done, now?

Eric Wieser (Jun 17 2023 at 16:35):

port-progress bot said:

mathlib port progress all
Unported files: 274/3034 (91.0% of total)
Unported lines: 101732/1040487 (90.2% of total)
Longest unported chain: 13/117 (88.9% progress)

#port-dashboard says there are 3109 total files, not 3034; so I assume this is not counting the archive/counterexamples?

Eric Wieser (Jun 17 2023 at 16:36):

(either way the 90% figure is still true!)

Ruben Van de Velde (Jun 17 2023 at 16:36):

Either that or the lean core files

Ryan McCorvie (Jun 17 2023 at 17:03):

What happens when the port gets to 100%? Are there more steps involved in porting other than getting all the files ported? Also, is there a party planned?

Eric Wieser (Jun 17 2023 at 17:09):

My suggestion would be something along the lines of

  • Freeze mathlib3 for feature PRs
  • Finish up any backport PRs in mathlib3 (these will help downstream projects upgrade)
  • Freeze mathlib3 completely
  • Empty #outofsync
  • Make some kind of release tag
  • Open mathlib4 up to refactors

port-progress bot (Jun 17 2023 at 19:05):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 21/1054 (98.0% of total)
Unported lines: 8001/446670 (98.2% of total)
Longest unported chain: 9/97 (90.7% progress)

port-progress bot (Jun 17 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4636/380704 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 17 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 19/978 (98.1% of total)
Unported lines: 10244/399002 (97.4% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 17 2023 at 19:18):

mathlib port progress analysis.fourier.add_circle
Unported files: 9/1117 (99.2% of total)
Unported lines: 4331/499572 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 17 2023 at 19:23):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1125 (98.0% of total)
Unported lines: 13688/506279 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

Joseph Myers (Jun 17 2023 at 19:26):

There's also the suggestion of putting both histories in the same repository with merge commits.

port-progress bot (Jun 17 2023 at 19:27):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/280122 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 17 2023 at 19:31):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4611/349382 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 17 2023 at 19:36):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5923/298070 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 17 2023 at 19:41):

mathlib port progress number_theory.zeta_function
Unported files: 28/1253 (97.8% of total)
Unported lines: 16708/558021 (97.0% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 17 2023 at 19:45):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6761/405054 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 17 2023 at 19:49):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156490 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 17 2023 at 19:53):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285240 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 17 2023 at 19:57):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346919 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 17 2023 at 20:02):

mathlib port progress probability.borel_cantelli
Unported files: 18/1066 (98.3% of total)
Unported lines: 8486/480494 (98.2% of total)
Longest unported chain: 7/116 (94.0% progress)

port-progress bot (Jun 17 2023 at 20:06):

mathlib port progress probability.kernel.condexp
Unported files: 11/1048 (99.0% of total)
Unported lines: 4737/473944 (99.0% of total)
Longest unported chain: 3/109 (97.2% progress)

Eric Wieser (Jun 17 2023 at 20:08):

Joseph Myers said:

There's also the suggestion of putting both histories in the same repository with merge commits.

I don't think the timing on this is essential, we can always merge into the "released" version of mathlib 4, then merge _that_ merge back into master at whatever point it's at by the time the history is unified

port-progress bot (Jun 17 2023 at 20:11):

mathlib port progress all
Unported files: 261/3034 (91.4% of total)
Unported lines: 97637/1040559 (90.6% of total)
Longest unported chain: 12/117 (89.7% progress)

port-progress bot (Jun 17 2023 at 20:12):

816/3035 files completely ported (26.88%), in the sense that also all downstream dependencies are ported.

Jireh Loreaux (Jun 18 2023 at 00:30):

0.4%

port-progress bot (Jun 18 2023 at 19:05):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 20/1054 (98.1% of total)
Unported lines: 7703/446670 (98.3% of total)
Longest unported chain: 9/97 (90.7% progress)

port-progress bot (Jun 18 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4636/380704 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 18 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 19/978 (98.1% of total)
Unported lines: 10244/399002 (97.4% of total)
Longest unported chain: 7/90 (92.2% progress)

port-progress bot (Jun 18 2023 at 19:18):

mathlib port progress analysis.fourier.add_circle
Unported files: 9/1117 (99.2% of total)
Unported lines: 4331/499572 (99.1% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 18 2023 at 19:23):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1125 (98.0% of total)
Unported lines: 13688/506279 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 18 2023 at 19:27):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/280122 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 18 2023 at 19:31):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4611/349382 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 18 2023 at 19:36):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5923/298070 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 18 2023 at 19:41):

mathlib port progress number_theory.zeta_function
Unported files: 28/1253 (97.8% of total)
Unported lines: 16708/558021 (97.0% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 18 2023 at 19:45):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6761/405054 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 18 2023 at 19:49):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156490 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 18 2023 at 19:53):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285240 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 18 2023 at 19:57):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346919 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 18 2023 at 20:02):

mathlib port progress probability.borel_cantelli
Unported files: 15/1066 (98.6% of total)
Unported lines: 6640/480494 (98.6% of total)
Longest unported chain: 4/116 (96.6% progress)

port-progress bot (Jun 18 2023 at 20:06):

mathlib port progress probability.kernel.condexp
Unported files: 11/1048 (99.0% of total)
Unported lines: 4737/473944 (99.0% of total)
Longest unported chain: 3/109 (97.2% progress)

port-progress bot (Jun 18 2023 at 20:10):

mathlib port progress all
Unported files: 257/3034 (91.5% of total)
Unported lines: 95625/1040559 (90.8% of total)
Longest unported chain: 12/117 (89.7% progress)

port-progress bot (Jun 18 2023 at 20:11):

816/3035 files completely ported (26.88%), in the sense that also all downstream dependencies are ported.

Scott Morrison (Jun 18 2023 at 22:08):

0.2%

port-progress bot (Jun 19 2023 at 19:05):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 19/1054 (98.2% of total)
Unported lines: 7435/446676 (98.3% of total)
Longest unported chain: 8/97 (91.8% progress)

port-progress bot (Jun 19 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4636/380704 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 19 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 18/978 (98.2% of total)
Unported lines: 9163/399002 (97.7% of total)
Longest unported chain: 6/90 (93.3% progress)

port-progress bot (Jun 19 2023 at 19:18):

mathlib port progress analysis.fourier.add_circle
Unported files: 8/1117 (99.3% of total)
Unported lines: 3950/499572 (99.2% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 19 2023 at 19:23):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1125 (98.0% of total)
Unported lines: 13688/506279 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

Ruben Van de Velde (Jun 19 2023 at 19:23):

port-progress bot said:

mathlib port progress analysis.fourier.add_circle
Unported files: 8/1117 (99.3% of total)
Unported lines: 3950/499572 (99.2% of total)
Longest unported chain: 1/104 (99.0% progress)

Who wants to start this port?

port-progress bot (Jun 19 2023 at 19:27):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/280122 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 19 2023 at 19:31):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4611/349382 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 19 2023 at 19:36):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5923/298070 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 19 2023 at 19:41):

mathlib port progress number_theory.zeta_function
Unported files: 26/1253 (97.9% of total)
Unported lines: 15415/558021 (97.2% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 19 2023 at 19:45):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6761/405054 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 19 2023 at 19:49):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156490 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 19 2023 at 19:53):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285240 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 19 2023 at 19:58):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346919 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 19 2023 at 20:03):

mathlib port progress probability.borel_cantelli
Unported files: 12/1066 (98.9% of total)
Unported lines: 5533/480524 (98.8% of total)
Longest unported chain: 3/116 (97.4% progress)

port-progress bot (Jun 19 2023 at 20:08):

mathlib port progress probability.kernel.condexp
Unported files: 10/1048 (99.0% of total)
Unported lines: 4457/473956 (99.1% of total)
Longest unported chain: 2/109 (98.2% progress)

port-progress bot (Jun 19 2023 at 20:14):

mathlib port progress all
Unported files: 242/3034 (92.0% of total)
Unported lines: 89650/1040607 (91.4% of total)
Longest unported chain: 11/117 (90.6% progress)

Kevin Buzzard (Jun 19 2023 at 20:15):

Under 250 files to go!

port-progress bot (Jun 19 2023 at 20:15):

828/3035 files completely ported (27.28%), in the sense that also all downstream dependencies are ported.

Eric Wieser (Jun 19 2023 at 20:16):

Kevin Buzzard said:

Under 250 files to go!

#port-dashboard says we have over 250, I think the above doesn't count the archive

Scott Morrison (Jun 19 2023 at 21:08):

0.6%

Scott Morrison (Jun 19 2023 at 21:11):

(That's 3.2% over the last week, so linearly extrapolating we are now done at . :-)

Matthew Ballard (Jun 19 2023 at 21:12):

Is there data to make a plot of the progress?

Scott Morrison (Jun 19 2023 at 21:13):

I think you'd have to scrape this topic, unfortunately.

Oliver Nash (Jun 19 2023 at 21:20):

Jireh Loreaux said:

0.5%. That makes 6.5% in the past two weeks. On track for mid-July at that pace.

This is beginning to look quite prescient.

Jeremy Tan (Jun 20 2023 at 03:16):

port-progress bot said:

mathlib port progress analysis.fourier.add_circle
Unported files: 8/1117 (99.3% of total)
Unported lines: 3950/499572 (99.2% of total)
Longest unported chain: 1/104 (99.0% progress)

!4#5273 is ready for review; I've taken over it. Can I add the awaiting-review label @David Loeffler?

David Loeffler (Jun 20 2023 at 06:52):

!4#5273 is ready for review; I've taken over it. Can I add the awaiting-review label @David Loeffler?

@Parcly-Taxel: You seem to have force-pushed a new branch on top of the PR I'd already made. I tagged the PR with "help wanted" because I was hoping for some suggestions and input that I could have used to learn to solve the problems in that file for myself – not to have the whole PR casually overwritten with no comment or explanation.

Johan Commelin (Jun 20 2023 at 06:57):

Maybe help-wanted is too ambiguous. For a sizable chunk of the community, over time, it seems to have acquired the meaning of

I'm stuck. If anyone sees a way to make progress, please push fixes.

Johan Commelin (Jun 20 2023 at 06:58):

Especially on porting PRs, we have mostly been hyper-collaborative on the varying PRs...

Eric Wieser (Jun 20 2023 at 07:00):

Force pushing with new mathport output is probably not the worst thing in the world for PRs that have been stale for some time

Eric Wieser (Jun 20 2023 at 07:00):

Though I guess this one was only 9 hours old...

David Loeffler (Jun 20 2023 at 07:00):

"Stale for some time"? I made the PR fresh at 23.30 last night and I got up this morning to find it had been overwritten!

Eric Wieser (Jun 20 2023 at 07:01):

Yeah, I misread the timestamp

Eric Wieser (Jun 20 2023 at 07:02):

I agree force pushing was a little strange here, though I don't think it matters too much. I'd be interested to hear why @Jeremy Tan did it though.

David Loeffler (Jun 20 2023 at 07:24):

Especially on porting PRs, we have mostly been hyper-collaborative on the varying PRs...

In my mind "collaboration" involves learning from other people, and sharing your knowledge and experience with others so they can learn too. Overwriting somebody else's work seems to me the opposite of "collaboration".

Mario Carneiro (Jun 20 2023 at 07:26):

Without making any claims about the benefits you mention, I don't think that's what "collaboration" literally means. A collaboration is a jointly produced work, it does not usually come with teaching connotations

Mario Carneiro (Jun 20 2023 at 07:33):

and I think the "hyper-" in hyper-collaborative in this case is that there are more people involved than communication one would expect of that many people, meaning that there will be some repeated and/or clobbered work

Jeremy Tan (Jun 20 2023 at 08:03):

port-progress bot said:

mathlib port progress probability.borel_cantelli
Unported files: 12/1066 (98.9% of total)
Unported lines: 5533/480524 (98.8% of total)
Longest unported chain: 3/116 (97.4% progress)

!4#5286 is ready for review

Chris Hughes (Jun 20 2023 at 10:10):

Matthew Ballard said:

Is there data to make a plot of the progress?

@Sebastian Ullrich showed me a graph of the progress yesterday

Sebastian Ullrich (Jun 20 2023 at 14:27):

I only have ported lines, it doesn't estimate where we will end up at 100%: http://speedcenter.informatik.kit.edu/mathlib4/repo-detail/e7b27246-a3e6-496a-b552-ff4b45c7236e?zoomXStart=1667257200000&dimensions=size%3A.lean&dayEquidistant=true

Sebastian Ullrich (Jun 20 2023 at 14:27):

Also the benchmarking machine seems to have died a few days ago

Johan Commelin (Jun 20 2023 at 14:37):

Not Found

The requested URL was not found on this server.

Johan Commelin (Jun 20 2023 at 14:37):

@Sebastian Ullrich link is broken for me

Floris van Doorn (Jun 20 2023 at 14:38):

I can view it:
image.png

Johan Commelin (Jun 20 2023 at 14:38):

Very weird...

Riccardo Brasca (Jun 20 2023 at 14:40):

Johan Commelin said:

Not Found

The requested URL was not found on this server.

Same for me

Sebastian Ullrich (Jun 20 2023 at 14:42):

I didn't think the infrastructure would crumble that fast after I leave the group

Jeremy Tan (Jun 20 2023 at 15:39):

"Last Skyfall" has happened – the last file with 10 or more immediate dependencies, RingTheory.Norm, has been ported

Floris van Doorn (Jun 20 2023 at 15:41):

and it's the last file with >= 30 total dependencies :tada:

Jeremy Tan (Jun 20 2023 at 16:38):

port-progress bot said:

mathlib port progress probability.kernel.condexp
Unported files: 10/1048 (99.0% of total)
Unported lines: 4457/473956 (99.1% of total)
Longest unported chain: 2/109 (98.2% progress)

I have an open PR for the sole dependent of this file, !4#5293

port-progress bot (Jun 20 2023 at 19:05):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 17/1054 (98.4% of total)
Unported lines: 6486/446690 (98.5% of total)
Longest unported chain: 7/97 (92.8% progress)

port-progress bot (Jun 20 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 10/968 (99.0% of total)
Unported lines: 4636/380704 (98.8% of total)
Longest unported chain: 2/79 (97.5% progress)

port-progress bot (Jun 20 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 17/978 (98.3% of total)
Unported lines: 8860/399005 (97.8% of total)
Longest unported chain: 5/90 (94.4% progress)

port-progress bot (Jun 20 2023 at 19:17):

mathlib port progress analysis.fourier.add_circle
Unported files: 7/1117 (99.4% of total)
Unported lines: 3409/499575 (99.3% of total)
Longest unported chain: 1/104 (99.0% progress)

port-progress bot (Jun 20 2023 at 19:22):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1125 (98.0% of total)
Unported lines: 13688/506279 (97.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 20 2023 at 19:26):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 13/677 (98.1% of total)
Unported lines: 4958/280122 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 20 2023 at 19:30):

mathlib port progress representation_theory.character
Unported files: 13/920 (98.6% of total)
Unported lines: 4611/349382 (98.7% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 20 2023 at 19:35):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5924/298077 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 20 2023 at 19:40):

mathlib port progress number_theory.zeta_function
Unported files: 25/1253 (98.0% of total)
Unported lines: 14874/558027 (97.3% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 20 2023 at 19:44):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/923 (98.4% of total)
Unported lines: 6761/405054 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 20 2023 at 19:48):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156490 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 20 2023 at 19:52):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285240 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 20 2023 at 19:56):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/346919 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 20 2023 at 20:01):

mathlib port progress probability.kernel.condexp
Unported files: 9/1048 (99.1% of total)
Unported lines: 3899/473959 (99.2% of total)
Longest unported chain: 1/109 (99.1% progress)

port-progress bot (Jun 20 2023 at 20:05):

mathlib port progress all
Unported files: 230/3034 (92.4% of total)
Unported lines: 84067/1040667 (91.9% of total)
Longest unported chain: 10/117 (91.5% progress)

port-progress bot (Jun 20 2023 at 20:06):

844/3035 files completely ported (27.80%), in the sense that also all downstream dependencies are ported.

Jireh Loreaux (Jun 20 2023 at 21:42):

0.5%

Jeremy Tan (Jun 21 2023 at 04:18):

port-progress bot said:

mathlib port progress probability.kernel.condexp
Unported files: 10/1048 (99.0% of total)
Unported lines: 4457/473956 (99.1% of total)
Longest unported chain: 2/109 (98.2% progress)

!4#5324 is ready and will close this target

Jeremy Tan (Jun 21 2023 at 11:38):

Probability is free! All files under the Probability folder have been ported to mathlib4

Jeremy Tan (Jun 21 2023 at 11:38):

And now I can take an indefinite but well-deserved break

Scott Morrison (Jun 21 2023 at 11:44):

Quick, somebody move all the remaining files to be ported into the Probability/ folder. :-)

Johan Commelin (Jun 21 2023 at 12:34):

@Jeremy Tan Thanks a lot for your contributions to the porting effort!

port-progress bot (Jun 21 2023 at 19:08):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 14/1055 (98.7% of total)
Unported lines: 5820/446862 (98.7% of total)
Longest unported chain: 5/97 (94.8% progress)

port-progress bot (Jun 21 2023 at 19:12):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 9/968 (99.1% of total)
Unported lines: 4150/380766 (98.9% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jun 21 2023 at 19:17):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 17/978 (98.3% of total)
Unported lines: 8860/399088 (97.8% of total)
Longest unported chain: 5/90 (94.4% progress)

port-progress bot (Jun 21 2023 at 19:22):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 23/1126 (98.0% of total)
Unported lines: 12161/506550 (97.6% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 21 2023 at 19:26):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 14/678 (97.9% of total)
Unported lines: 5049/280238 (98.2% of total)
Longest unported chain: 5/84 (94.0% progress)

port-progress bot (Jun 21 2023 at 19:31):

mathlib port progress representation_theory.character
Unported files: 12/920 (98.7% of total)
Unported lines: 4125/349431 (98.8% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 21 2023 at 19:36):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5924/298126 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 21 2023 at 19:41):

mathlib port progress number_theory.zeta_function
Unported files: 23/1254 (98.2% of total)
Unported lines: 12716/558613 (97.7% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 21 2023 at 19:46):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 16/924 (98.3% of total)
Unported lines: 6934/405333 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 21 2023 at 19:50):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156539 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 21 2023 at 19:54):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285302 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 21 2023 at 19:59):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/347015 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 21 2023 at 20:03):

mathlib port progress all
Unported files: 206/3036 (93.2% of total)
Unported lines: 74601/1041443 (92.8% of total)
Longest unported chain: 9/117 (92.3% progress)

port-progress bot (Jun 21 2023 at 20:05):

892/3037 files completely ported (29.37%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jun 21 2023 at 20:05):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jun 21 2023 at 20:15):

0.9%

Kevin Buzzard (Jun 21 2023 at 21:43):

Can we start counting down instead of up? 6.8% to go!

Ruben Van de Velde (Jun 21 2023 at 21:46):

We can unless we look at the unported file with the largest number of dependents; up to 366 from 20-something

Eric Wieser (Jun 22 2023 at 00:47):

I can resolve that tomorrow once mathport has run

Scott Morrison (Jun 22 2023 at 04:12):

geometry.manifold.cont_mdiff has retaken the lead!

Yury G. Kudryashov (Jun 22 2023 at 04:20):

I will rebase it on top of the current mathport output tomorrow.

Yury G. Kudryashov (Jun 22 2023 at 04:20):

Then we can try to fix it.

port-progress bot (Jun 22 2023 at 19:05):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 11/1055 (99.0% of total)
Unported lines: 4482/447041 (99.0% of total)
Longest unported chain: 3/97 (96.9% progress)

port-progress bot (Jun 22 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 9/968 (99.1% of total)
Unported lines: 4150/380895 (98.9% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jun 22 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 15/978 (98.5% of total)
Unported lines: 7426/399176 (98.1% of total)
Longest unported chain: 5/90 (94.4% progress)

port-progress bot (Jun 22 2023 at 19:18):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 22/1126 (98.0% of total)
Unported lines: 12070/506723 (97.6% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 22 2023 at 19:23):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 12/678 (98.2% of total)
Unported lines: 4602/280333 (98.4% of total)
Longest unported chain: 4/84 (95.2% progress)

port-progress bot (Jun 22 2023 at 19:27):

mathlib port progress representation_theory.character
Unported files: 12/920 (98.7% of total)
Unported lines: 4125/349529 (98.8% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 22 2023 at 19:32):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5924/298221 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 22 2023 at 19:37):

mathlib port progress number_theory.zeta_function
Unported files: 22/1254 (98.2% of total)
Unported lines: 12625/558789 (97.7% of total)
Longest unported chain: 8/116 (93.1% progress)

port-progress bot (Jun 22 2023 at 19:42):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/924 (98.4% of total)
Unported lines: 6843/405503 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 22 2023 at 19:46):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156566 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 22 2023 at 19:50):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285379 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 22 2023 at 19:55):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/347151 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 22 2023 at 19:59):

mathlib port progress all
Unported files: 188/3036 (93.8% of total)
Unported lines: 68267/1041691 (93.4% of total)
Longest unported chain: 9/117 (92.3% progress)

port-progress bot (Jun 22 2023 at 20:00):

917/3037 files completely ported (30.19%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jun 22 2023 at 20:00):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Jireh Loreaux (Jun 22 2023 at 20:38):

0.6%

Kevin Buzzard (Jun 22 2023 at 21:32):

Under 200 files to go!

port-progress bot (Jun 23 2023 at 19:05):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 10/1055 (99.1% of total)
Unported lines: 4064/447050 (99.1% of total)
Longest unported chain: 2/97 (97.9% progress)

port-progress bot (Jun 23 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 9/968 (99.1% of total)
Unported lines: 4150/380895 (98.9% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jun 23 2023 at 19:14):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 14/978 (98.6% of total)
Unported lines: 6807/399182 (98.3% of total)
Longest unported chain: 4/90 (95.6% progress)

port-progress bot (Jun 23 2023 at 19:18):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 21/1126 (98.1% of total)
Unported lines: 11520/506726 (97.7% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 23 2023 at 19:23):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 10/678 (98.5% of total)
Unported lines: 4106/280339 (98.5% of total)
Longest unported chain: 2/84 (97.6% progress)

port-progress bot (Jun 23 2023 at 19:27):

mathlib port progress representation_theory.character
Unported files: 12/920 (98.7% of total)
Unported lines: 4125/349529 (98.8% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 23 2023 at 19:31):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5924/298221 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 23 2023 at 19:36):

mathlib port progress number_theory.zeta_function
Unported files: 15/1238 (98.8% of total)
Unported lines: 6624/546577 (98.8% of total)
Longest unported chain: 3/116 (97.4% progress)

port-progress bot (Jun 23 2023 at 19:41):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 15/924 (98.4% of total)
Unported lines: 6843/405506 (98.3% of total)
Longest unported chain: 7/107 (93.5% progress)

port-progress bot (Jun 23 2023 at 19:45):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156566 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 23 2023 at 19:49):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285379 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 23 2023 at 19:53):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/347151 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 23 2023 at 19:57):

mathlib port progress all
Unported files: 175/3038 (94.2% of total)
Unported lines: 63989/1041785 (93.9% of total)
Longest unported chain: 8/117 (93.2% progress)

port-progress bot (Jun 23 2023 at 19:59):

923/3039 files completely ported (30.37%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jun 23 2023 at 19:59):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Scott Morrison (Jun 23 2023 at 23:32):

0.5%

Johan Commelin (Jun 24 2023 at 05:42):

all.pdf is starting to look very encouraging!

port-progress bot (Jun 24 2023 at 19:04):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 10/1055 (99.1% of total)
Unported lines: 4064/447053 (99.1% of total)
Longest unported chain: 2/97 (97.9% progress)

port-progress bot (Jun 24 2023 at 19:09):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 9/968 (99.1% of total)
Unported lines: 4150/380895 (98.9% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jun 24 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 14/978 (98.6% of total)
Unported lines: 6807/399185 (98.3% of total)
Longest unported chain: 4/90 (95.6% progress)

port-progress bot (Jun 24 2023 at 19:18):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 15/1126 (98.7% of total)
Unported lines: 7972/506729 (98.4% of total)
Longest unported chain: 4/107 (96.3% progress)

port-progress bot (Jun 24 2023 at 19:22):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 9/678 (98.7% of total)
Unported lines: 3897/280345 (98.6% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jun 24 2023 at 19:27):

mathlib port progress representation_theory.character
Unported files: 12/920 (98.7% of total)
Unported lines: 4125/349529 (98.8% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 24 2023 at 19:31):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5924/298221 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 24 2023 at 19:36):

mathlib port progress number_theory.zeta_function
Unported files: 15/1238 (98.8% of total)
Unported lines: 6624/546577 (98.8% of total)
Longest unported chain: 3/116 (97.4% progress)

port-progress bot (Jun 24 2023 at 19:41):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 12/924 (98.7% of total)
Unported lines: 4362/405506 (98.9% of total)
Longest unported chain: 4/107 (96.3% progress)

port-progress bot (Jun 24 2023 at 19:45):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156566 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 24 2023 at 19:49):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285379 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 24 2023 at 19:53):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/347151 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 24 2023 at 19:57):

mathlib port progress all
Unported files: 160/3039 (94.7% of total)
Unported lines: 58440/1042212 (94.4% of total)
Longest unported chain: 6/117 (94.9% progress)

port-progress bot (Jun 24 2023 at 19:58):

947/3040 files completely ported (31.15%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jun 24 2023 at 19:58):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jun 24 2023 at 20:03):

0.5%

Johan Commelin (Jun 24 2023 at 20:04):

The game theorists now have the longest chain!

Scott Morrison (Jun 25 2023 at 05:41):

Wow! We are really getting to the end...

Scott Morrison (Jun 25 2023 at 05:50):

From memory the combinatorial game theory files are mostly broken because of termination_by clauses that need writing.

Scott Morrison (Jun 25 2023 at 07:17):

I did some work on #4311, our current longest chain about combinatorial games. Some problems were easily fixable, but I've run into two problems:

  • an error I simply don't understand yet, at negMulRelabelling
  • in quot_left_distrib and quot_mul_assoc, the goals that appear in decreasing_by don't seem to accurately reflect the actual recursive calls made in the body (which, perhaps unusually, were via simp).

Scott Morrison (Jun 25 2023 at 07:44):

I suspect this second point may be a bug in the way the goals for decreasing_by are being collected, so if someone else could take a look at this one that would be much appreciated. We'd need to find a minimisation.

Scott Morrison (Jun 25 2023 at 08:04):

My evidence that there is a bug in the way that goals are collected is that if you fill in the arguments in simp [quot_left_distrib], then the decreasing_by goals change (to become the correct ones). I'm dubious, however, as I don't understand how that could be happening!

Mario Carneiro (Jun 25 2023 at 08:09):

that sounds expected

Mario Carneiro (Jun 25 2023 at 08:10):

I think simp is creating an unapplied reference to quot_left_distrib, lambda abstracting and then applying it again

Mario Carneiro (Jun 25 2023 at 08:11):

does quot_left_distrib .. work?

Scott Morrison (Jun 25 2023 at 08:18):

That changes the names of the fake hypotheses that end up in the decreasing_by goal, but doesn't make them be what they should be.

Mario Carneiro (Jun 25 2023 at 08:18):

quot_left_distrib _ ..?

Scott Morrison (Jun 25 2023 at 08:19):

I guess I can fill in all the arguments by hand. It's a little tedious here, as there are 24 different applications of this simp lemma, all of which need different explicit arguments.

Scott Morrison (Jun 25 2023 at 08:20):

_ .. has the same effect as ... (Similarly _ _ _ and _ _ _ ...)

Mario Carneiro (Jun 25 2023 at 08:21):

Why does #4311 change 1520 files?

Mario Carneiro (Jun 25 2023 at 08:22):

could you rebase it / clean up the history?

Scott Morrison (Jun 25 2023 at 08:23):

Ugh... I don't think I did anything scarier than merging master, but I will rebase.

Mario Carneiro (Jun 25 2023 at 08:23):

you could also just cherry pick the commits that are actually part of the PR

Scott Morrison (Jun 25 2023 at 08:25):

Rebasing wanted to tell me about lots of conflicts. Simply merging master again seems to have fixed the diff.

Mario Carneiro (Jun 25 2023 at 08:26):

although I'm not sure it won't look like a 100 person coauthored PR when it lands

Scott Morrison (Jun 25 2023 at 08:27):

This is a very old PR. I'm worried it dates back to that time we had to rewrite history.

Mario Carneiro (Jun 25 2023 at 08:28):

in that case you should definitely rebase

Scott Morrison (Jun 25 2023 at 08:28):

How? It's going to make me walk through hundreds of diffs, no?

Mario Carneiro (Jun 25 2023 at 08:29):

create a new branch, cherry pick all the commits that look like they are actually supposed to be in the PR in order, and then change the old branch to point to the new one and force push

Mario Carneiro (Jun 25 2023 at 08:30):

I can try doing this if you like

Scott Morrison (Jun 25 2023 at 08:30):

I'm worried it has 100s of commits since diverging from master, and I'd never work out which to cherry pick. Particularly since the early work on this PR was done by someone else.

Scott Morrison (Jun 25 2023 at 08:31):

If you could that would be great. I'm happy to try to learn how to do this, but I just don't know at the moment.

Scott Morrison (Jun 25 2023 at 08:31):

I mean, I can just discard history...

Scott Morrison (Jun 25 2023 at 08:32):

run start_port again, and then merge --squash the current messy branch onto that?

Patrick Massot (Jun 25 2023 at 08:32):

Shouldn't we wait until everything else is ported before porting game theory?

Scott Morrison (Jun 25 2023 at 08:32):

Patrick, why?

Scott Morrison (Jun 25 2023 at 08:33):

Just that you don't like game theory? :-) I was looking at it because it is now the longest unported chain of imports...

Patrick Massot (Jun 25 2023 at 08:33):

This isn't for anything else, isn't used by any external project and wasn't very active.

Scott Morrison (Jun 25 2023 at 08:35):

I think we have reached, or are very very close to, the point of just cleaning up the stray junk. (Like these files.)

Scott Morrison (Jun 25 2023 at 08:35):

And there is a lean3 vs lean4 regression here, so better to look at it sooner rather than later.

Patrick Massot (Jun 25 2023 at 08:35):

What about working on differential geometry or analytic number theory?

Scott Morrison (Jun 25 2023 at 08:36):

@Mario Carneiro, have you already started on the history? If not I will do the merge --squash approach.

Mario Carneiro (Jun 25 2023 at 08:37):

I'd rather do the rebase

Patrick Massot (Jun 25 2023 at 08:37):

About regressions, as far as I understand, there is still a lot more important work to do on understanding issues with simp.

Scott Morrison (Jun 25 2023 at 08:39):

I agree -- I've been working on that too, but it's Sunday evening and I felt like doing some game theory. :woman_shrugging:

Ruben Van de Velde (Jun 25 2023 at 08:43):

That makes sense to me, Sunday night is game night

Scott Morrison (Jun 25 2023 at 08:44):

Here's what's left of differential geometry:
Screen-Shot-2023-06-25-at-6.37.17-pm.png

Scott Morrison (Jun 25 2023 at 08:44):

and analytic number theory:
Screen-Shot-2023-06-25-at-6.43.58-pm.png

Mario Carneiro (Jun 25 2023 at 08:45):

history fixed

David Renshaw (Jun 25 2023 at 14:31):

Scott Morrison said:

I guess I can fill in all the arguments by hand. It's a little tedious here, as there are 24 different applications of this simp lemma, all of which need different explicit arguments.

I went ahead and filled in all the arguments: https://github.com/leanprover-community/mathlib4/pull/4311/commits/c008589ce87a01496e3db16d9ea78f4b86ee7bf9

David Renshaw (Jun 25 2023 at 14:34):

Looks like all that's left to do on this PR is fix some simpNF linter issues.

port-progress bot (Jun 25 2023 at 19:06):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 10/1055 (99.1% of total)
Unported lines: 4064/447053 (99.1% of total)
Longest unported chain: 2/97 (97.9% progress)

port-progress bot (Jun 25 2023 at 19:11):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 8/968 (99.2% of total)
Unported lines: 3593/380895 (99.1% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jun 25 2023 at 19:15):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 14/978 (98.6% of total)
Unported lines: 6807/399185 (98.3% of total)
Longest unported chain: 4/90 (95.6% progress)

port-progress bot (Jun 25 2023 at 19:20):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 12/1126 (98.9% of total)
Unported lines: 7293/506729 (98.6% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jun 25 2023 at 19:25):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 9/678 (98.7% of total)
Unported lines: 3897/280345 (98.6% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jun 25 2023 at 19:29):

mathlib port progress representation_theory.character
Unported files: 12/920 (98.7% of total)
Unported lines: 4125/349529 (98.8% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 25 2023 at 19:34):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5924/298221 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 25 2023 at 19:39):

mathlib port progress number_theory.zeta_function
Unported files: 15/1238 (98.8% of total)
Unported lines: 6624/546577 (98.8% of total)
Longest unported chain: 3/116 (97.4% progress)

port-progress bot (Jun 25 2023 at 19:43):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 10/924 (98.9% of total)
Unported lines: 4087/405506 (99.0% of total)
Longest unported chain: 2/107 (98.1% progress)

port-progress bot (Jun 25 2023 at 19:47):

mathlib port progress set_theory.game.domineering
Unported files: 13/387 (96.6% of total)
Unported lines: 5020/156566 (96.8% of total)
Longest unported chain: 5/63 (92.1% progress)

port-progress bot (Jun 25 2023 at 19:51):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285379 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 25 2023 at 19:55):

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/347151 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

port-progress bot (Jun 25 2023 at 19:59):

mathlib port progress all
Unported files: 156/3039 (94.9% of total)
Unported lines: 57238/1042212 (94.5% of total)
Longest unported chain: 6/117 (94.9% progress)

port-progress bot (Jun 25 2023 at 20:00):

951/3040 files completely ported (31.28%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jun 25 2023 at 20:00):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Scott Morrison (Jun 25 2023 at 23:46):

0.1%

Jeremy Tan (Jun 26 2023 at 10:01):

port-progress bot said:

mathlib port progress combinatorics.simple_graph.regularity.lemma
Unported files: 11/805 (98.6% of total)
Unported lines: 4541/347151 (98.7% of total)
Longest unported chain: 3/93 (96.8% progress)

!4#5477 will finish this (and free combinatorics)

Jeremy Tan (Jun 26 2023 at 10:20):

And now combinatorics is free

Yaël Dillies (Jun 26 2023 at 11:23):

...so long, we have a few open PRs on the mathlib side

Jeremy Tan (Jun 26 2023 at 13:21):

port-progress bot said:

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 10/1055 (99.1% of total)
Unported lines: 4064/447053 (99.1% of total)
Longest unported chain: 2/97 (97.9% progress)

And this is done too

port-progress bot (Jun 26 2023 at 19:04):

mathlib port progress number_theory.legendre_symbol.quadratic_reciprocity
Unported files: 7/1055 (99.3% of total)
Unported lines: 3409/447240 (99.2% of total)
Longest unported chain: 1/97 (99.0% progress)

port-progress bot (Jun 26 2023 at 19:08):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 8/968 (99.2% of total)
Unported lines: 3593/381085 (99.1% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jun 26 2023 at 19:13):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 14/978 (98.6% of total)
Unported lines: 6807/399372 (98.3% of total)
Longest unported chain: 4/90 (95.6% progress)

port-progress bot (Jun 26 2023 at 19:18):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 12/1126 (98.9% of total)
Unported lines: 7293/506943 (98.6% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jun 26 2023 at 19:22):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 9/678 (98.7% of total)
Unported lines: 3897/280535 (98.6% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jun 26 2023 at 19:27):

mathlib port progress representation_theory.character
Unported files: 11/920 (98.8% of total)
Unported lines: 3934/349716 (98.9% of total)
Longest unported chain: 3/91 (96.7% progress)

port-progress bot (Jun 26 2023 at 19:31):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 17/748 (97.7% of total)
Unported lines: 5924/298408 (98.0% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 26 2023 at 19:37):

mathlib port progress number_theory.zeta_function
Unported files: 13/1238 (98.9% of total)
Unported lines: 5505/546764 (99.0% of total)
Longest unported chain: 3/116 (97.4% progress)

port-progress bot (Jun 26 2023 at 19:42):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 10/924 (98.9% of total)
Unported lines: 4087/405708 (99.0% of total)
Longest unported chain: 2/107 (98.1% progress)

port-progress bot (Jun 26 2023 at 19:46):

mathlib port progress set_theory.game.domineering
Unported files: 11/387 (97.2% of total)
Unported lines: 4245/156651 (97.3% of total)
Longest unported chain: 3/63 (95.2% progress)

port-progress bot (Jun 26 2023 at 19:50):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 11/701 (98.4% of total)
Unported lines: 4159/285464 (98.5% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jun 26 2023 at 19:54):

mathlib port progress all
Unported files: 137/3040 (95.5% of total)
Unported lines: 51089/1042672 (95.1% of total)
Longest unported chain: 6/117 (94.9% progress)

Johan Commelin (Jun 26 2023 at 19:55):

0.6%

port-progress bot (Jun 26 2023 at 19:55):

994/3041 files completely ported (32.68%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jun 26 2023 at 19:55):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Ruben Van de Velde (Jun 27 2023 at 08:16):

Dashboard claims we're down to 89 unported files :exploding_head:

Scott Morrison (Jun 27 2023 at 08:18):

It's probably finally time for me to diagnose that N+7 thing.

Johan Commelin (Jun 27 2023 at 08:19):

@Ruben Van de Velde during the porting meeting yesterday we identified a whole bunch of low-level files that either could be ported with a few #align statements, or shouldn't be ported at all, or were already ported but were missing a porting header, etc...

port-progress bot (Jun 27 2023 at 08:28):

1000/3041 files completely ported (32.88%), in the sense that also all downstream dependencies are ported.

Scott Morrison (Jun 27 2023 at 08:29):

(Sorry, expect some bot noise on this channel, debugging.)

port-progress bot (Jun 27 2023 at 08:42):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 4/1126 (99.6% of total)
Unported lines: 1805/506943 (99.6% of total)
Longest unported chain: 2/107 (98.1% progress)

Scott Morrison (Jun 27 2023 at 08:42):

Hurrah! Without any hacky -7s, the number of unported files seems to match the graph.

Scott Morrison (Jun 27 2023 at 08:43):

I think I will add 1 to the "longest unported chain" number, so it matches the number of vertices, not the number of edges.

Johan Commelin (Jun 27 2023 at 09:20):

Great! Where did the 7 come from?

Scott Morrison (Jun 27 2023 at 09:25):

Disconnected components "above" stuff that had already been ported. We were already removing these to display the graph and compute the longest path, I just had to remove the line that killed these components to before the code that counted files and lines.

David Michael Roberts (Jun 27 2023 at 10:22):

Scott Morrison said:

Hurrah! Without any hacky -7s, the number of unported files seems to match the graph.

What's the correct number for all, currently?

port-progress bot (Jun 27 2023 at 10:36):

mathlib port progress all
Unported files: 115/3040 (96.2% of total)
Unported lines: 40183/1042672 (96.1% of total)
Longest unported chain: 7/117 (94.0% progress)

Scott Morrison (Jun 27 2023 at 11:47):

(Let's remember not to include this one in the daily progress count: it's just an answer to @David Michael Roberts.)

Johan Commelin (Jun 27 2023 at 11:49):

It would be quite sad to leave it out, indeed!

port-progress bot (Jun 27 2023 at 19:04):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 1/968 (99.9% of total)
Unported lines: 184/381085 (100.0% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jun 27 2023 at 19:08):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 7/978 (99.3% of total)
Unported lines: 3398/399372 (99.1% of total)
Longest unported chain: 5/90 (94.4% progress)

port-progress bot (Jun 27 2023 at 19:13):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 4/1126 (99.6% of total)
Unported lines: 1805/506943 (99.6% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jun 27 2023 at 19:17):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 2/678 (99.7% of total)
Unported lines: 488/280535 (99.8% of total)
Longest unported chain: 2/84 (97.6% progress)

port-progress bot (Jun 27 2023 at 19:22):

mathlib port progress representation_theory.character
Unported files: 4/920 (99.6% of total)
Unported lines: 525/349716 (99.8% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 27 2023 at 19:26):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 7/748 (99.1% of total)
Unported lines: 1796/298408 (99.4% of total)
Longest unported chain: 5/93 (94.6% progress)

port-progress bot (Jun 27 2023 at 19:31):

mathlib port progress number_theory.zeta_function
Unported files: 5/1238 (99.6% of total)
Unported lines: 1470/546764 (99.7% of total)
Longest unported chain: 4/116 (96.6% progress)

port-progress bot (Jun 27 2023 at 19:36):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 3/924 (99.7% of total)
Unported lines: 678/405708 (99.8% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jun 27 2023 at 19:40):

mathlib port progress set_theory.game.domineering
Unported files: 4/387 (99.0% of total)
Unported lines: 836/156651 (99.5% of total)
Longest unported chain: 4/63 (93.7% progress)

port-progress bot (Jun 27 2023 at 19:44):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 4/701 (99.4% of total)
Unported lines: 750/285464 (99.7% of total)
Longest unported chain: 4/80 (95.0% progress)

port-progress bot (Jun 27 2023 at 19:48):

mathlib port progress all
Unported files: 107/3040 (96.5% of total)
Unported lines: 38448/1042672 (96.3% of total)
Longest unported chain: 6/117 (94.9% progress)

port-progress bot (Jun 27 2023 at 19:49):

1011/3041 files completely ported (33.24%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jun 27 2023 at 19:49):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jun 27 2023 at 19:49):

1.2%

Johan Commelin (Jun 27 2023 at 19:50):

longest chain is still witt vectors! I guess we had a backlog...

Mario Carneiro (Jun 27 2023 at 19:57):

Wow, if we keep that rate we'll be done by friday

Kevin Buzzard (Jun 27 2023 at 21:05):

there might be some boss levels at the end

Jeremy Tan (Jun 28 2023 at 04:10):

Johan Commelin said:

longest chain is still witt vectors! I guess we had a backlog...

This should change with !4#5538

Jeremy Tan (Jun 28 2023 at 04:13):

I wouldn't be surprised if we're still not done by , though I consider that time likely

Scott Morrison (Jun 28 2023 at 06:56):

There's a list of boss levels, already ordered by an estimate of how tough they are (=how long the author has been ignoring it and hoping it goes away), at #help-wanted!

Antoine Chambert-Loir (Jun 28 2023 at 07:24):

I have tried to work on RingTheory.Jacobson, but I don't understand what happens, and I would have proved the result in a different way. For example, the missing result has to reprove basically that if an algebra is generated by elements, then it is integral iff these elements are integral.

Scott Morrison (Jun 28 2023 at 08:17):

We could ping the original author @Devon Tuma and see if they'd like to help? :-)

Devon Tuma (Jun 28 2023 at 09:53):

I could definitely take a look, but I've only gone through the basics of Lean 4, so I'll have some up-time on that first (and probably on relearning some commutative algebra after being in computer science for grad school)

Scott Morrison (Jun 28 2023 at 11:33):

Sorry everyone, we've had to move up the schedule, and are now planning to be done at . (Linearly interpolating the last 14 days progress.)

Johan Commelin (Jun 28 2023 at 11:49):

Your previous guess was Jul 8, I think.

Antoine Chambert-Loir (Jun 28 2023 at 13:41):

Devon Tuma said:

I could definitely take a look, but I've only gone through the basics of Lean 4, so I'll have some up-time on that first (and probably on relearning some commutative algebra after being in computer science for grad school)

I'll try to do something in the forthcoming days. If you happen to make modifications meanwhile, please tell me so!

Johan Commelin (Jun 28 2023 at 14:41):

My working day is over, but I just want to point out that number_theory.zeta_function is now portable!

Scott Morrison (Jun 28 2023 at 20:55):

Apologies for the delay with the bot today. zulip-send was hard-coded to use an ancient version of python that I had deleted yesterday.

port-progress bot (Jun 28 2023 at 20:59):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 1/968 (99.9% of total)
Unported lines: 184/381085 (100.0% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jun 28 2023 at 21:03):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 7/978 (99.3% of total)
Unported lines: 3398/399372 (99.1% of total)
Longest unported chain: 5/90 (94.4% progress)

port-progress bot (Jun 28 2023 at 21:08):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 3/1126 (99.7% of total)
Unported lines: 1271/506946 (99.7% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jun 28 2023 at 21:12):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 2/678 (99.7% of total)
Unported lines: 488/280535 (99.8% of total)
Longest unported chain: 2/84 (97.6% progress)

port-progress bot (Jun 28 2023 at 21:16):

mathlib port progress representation_theory.character
Unported files: 4/920 (99.6% of total)
Unported lines: 525/349719 (99.8% of total)
Longest unported chain: 4/91 (95.6% progress)

port-progress bot (Jun 28 2023 at 21:21):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 2/748 (99.7% of total)
Unported lines: 480/298408 (99.8% of total)
Longest unported chain: 2/93 (97.8% progress)

port-progress bot (Jun 28 2023 at 21:26):

mathlib port progress number_theory.zeta_function
Unported files: 1/1238 (99.9% of total)
Unported lines: 767/546770 (99.9% of total)
Longest unported chain: 1/116 (99.1% progress)

port-progress bot (Jun 28 2023 at 21:30):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 3/924 (99.7% of total)
Unported lines: 678/405708 (99.8% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jun 28 2023 at 21:35):

mathlib port progress set_theory.game.domineering
Unported files: 3/387 (99.2% of total)
Unported lines: 678/156657 (99.6% of total)
Longest unported chain: 3/63 (95.2% progress)

port-progress bot (Jun 28 2023 at 21:39):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 4/701 (99.4% of total)
Unported lines: 750/285464 (99.7% of total)
Longest unported chain: 4/80 (95.0% progress)

port-progress bot (Jun 28 2023 at 21:44):

mathlib port progress all
Unported files: 88/3040 (97.1% of total)
Unported lines: 32464/1042735 (96.9% of total)
Longest unported chain: 6/117 (94.9% progress)

port-progress bot (Jun 28 2023 at 21:45):

1029/3041 files completely ported (33.83%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jun 28 2023 at 21:45):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Jireh Loreaux (Jun 28 2023 at 21:46):

0.6%

Kevin Buzzard (Jun 28 2023 at 22:41):

Under 100 to go!

Jeremy Tan (Jun 29 2023 at 03:17):

Both remaining files at level 5, in algebraic geometry, are passing CI and ready for review: !4#5394 and !4#5446

Jeremy Tan (Jun 29 2023 at 03:24):

Scott Morrison said:

Sorry everyone, we've had to move up the schedule, and are now planning to be done at . (Linearly interpolating the last 14 days progress.)

If you're trying to merge new features into mathlib4 that are unrelated to the port, how can you possibly meet that deadline?

As Tedros said: port, port, port

Jeremy Tan (Jun 29 2023 at 03:27):

Jeremy Tan said:

I wouldn't be surprised if we're still not done by , though I consider that time likely

If you don't go full focus on the port, my prediction here is going to be more accurate

Johan Commelin (Jun 29 2023 at 03:52):

@Jeremy Tan I think that almost all Scott's new features are there to debug issues that are coming up during the port, like debugging why simp is sometimes less powerful.

port-progress bot (Jun 29 2023 at 19:04):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 1/968 (99.9% of total)
Unported lines: 184/381085 (100.0% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jun 29 2023 at 19:08):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 4/978 (99.6% of total)
Unported lines: 1551/399372 (99.6% of total)
Longest unported chain: 3/90 (96.7% progress)

port-progress bot (Jun 29 2023 at 19:13):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 3/1126 (99.7% of total)
Unported lines: 1271/506949 (99.7% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jun 29 2023 at 19:17):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 1/678 (99.9% of total)
Unported lines: 247/280535 (99.9% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jun 29 2023 at 19:21):

mathlib port progress representation_theory.character
Unported files: 3/920 (99.7% of total)
Unported lines: 448/349719 (99.9% of total)
Longest unported chain: 3/91 (96.7% progress)

port-progress bot (Jun 29 2023 at 19:26):

mathlib port progress ring_theory.witt_vector.isocrystal
Unported files: 1/748 (99.9% of total)
Unported lines: 204/298432 (99.9% of total)
Longest unported chain: 1/93 (98.9% progress)

port-progress bot (Jun 29 2023 at 19:34):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 3/924 (99.7% of total)
Unported lines: 678/405708 (99.8% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jun 29 2023 at 19:38):

mathlib port progress set_theory.game.domineering
Unported files: 3/387 (99.2% of total)
Unported lines: 678/156660 (99.6% of total)
Longest unported chain: 3/63 (95.2% progress)

port-progress bot (Jun 29 2023 at 19:42):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 4/701 (99.4% of total)
Unported lines: 750/285464 (99.7% of total)
Longest unported chain: 4/80 (95.0% progress)

port-progress bot (Jun 29 2023 at 19:46):

mathlib port progress all
Unported files: 75/3040 (97.5% of total)
Unported lines: 27664/1042914 (97.3% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jun 29 2023 at 19:47):

1099/3041 files completely ported (36.13%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jun 29 2023 at 19:47):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jun 29 2023 at 19:49):

0.4%

Ruben Van de Velde (Jun 30 2023 at 07:36):

https://leanprover-community.github.io/mathlib-port-status says under 50 unported and under 50 in progress :tada:

port-progress bot (Jun 30 2023 at 19:04):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 1/968 (99.9% of total)
Unported lines: 184/381052 (100.0% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jun 30 2023 at 19:08):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 2/978 (99.8% of total)
Unported lines: 819/399328 (99.8% of total)
Longest unported chain: 2/90 (97.8% progress)

port-progress bot (Jun 30 2023 at 19:13):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 3/1126 (99.7% of total)
Unported lines: 1271/506888 (99.7% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jun 30 2023 at 19:18):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 1/678 (99.9% of total)
Unported lines: 247/280501 (99.9% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jun 30 2023 at 19:22):

mathlib port progress representation_theory.character
Unported files: 3/920 (99.7% of total)
Unported lines: 448/349689 (99.9% of total)
Longest unported chain: 3/91 (96.7% progress)

port-progress bot (Jun 30 2023 at 19:34):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 3/924 (99.7% of total)
Unported lines: 678/405646 (99.8% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jun 30 2023 at 19:38):

mathlib port progress set_theory.game.domineering
Unported files: 3/387 (99.2% of total)
Unported lines: 678/156629 (99.6% of total)
Longest unported chain: 3/63 (95.2% progress)

port-progress bot (Jun 30 2023 at 19:41):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 4/701 (99.4% of total)
Unported lines: 750/285431 (99.7% of total)
Longest unported chain: 4/80 (95.0% progress)

port-progress bot (Jun 30 2023 at 19:46):

mathlib port progress all
Unported files: 69/3040 (97.7% of total)
Unported lines: 26087/1042895 (97.5% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jun 30 2023 at 19:47):

1136/3041 files completely ported (37.35%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jun 30 2023 at 19:47):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Scott Morrison (Jul 01 2023 at 02:32):

0.2%

Jeremy Tan (Jul 01 2023 at 03:51):

Ruben Van de Velde said:

https://leanprover-community.github.io/mathlib-port-status says under 50 unported and under 50 in progress :tada:

There are now more in progress files than unported files on the dashboard (42 vs 41)

Jeremy Tan (Jul 01 2023 at 04:02):

Also !4#3961 is ready for review

Jeremy Tan (Jul 01 2023 at 04:56):

And now, I think, I'm really going to take the break I promised when I declared that probability is free. There just aren't that many files left to port, I'm feeling a bit of burnout and there are other things in life for me to do

Johan Commelin (Jul 01 2023 at 05:02):

Take care! Enjoy your break. And once again: thanks for all your help

Timo Carlin-Burns (Jul 01 2023 at 09:01):

My first file! #5551 will be ready for initial review once I get push permissions (or someone cherrypicks the commits from my fork). It compiles, but I left a few porting notes where I'm guessing I'm doing something wrong

Johan Commelin (Jul 01 2023 at 14:01):

Both lists are below 40 now!

port-progress bot (Jul 01 2023 at 19:04):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 1/968 (99.9% of total)
Unported lines: 184/381052 (100.0% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jul 01 2023 at 19:09):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 2/978 (99.8% of total)
Unported lines: 819/399328 (99.8% of total)
Longest unported chain: 2/90 (97.8% progress)

port-progress bot (Jul 01 2023 at 19:14):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 3/1126 (99.7% of total)
Unported lines: 1271/506888 (99.7% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jul 01 2023 at 19:18):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 1/678 (99.9% of total)
Unported lines: 247/280501 (99.9% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jul 01 2023 at 19:23):

mathlib port progress representation_theory.character
Unported files: 3/920 (99.7% of total)
Unported lines: 448/349689 (99.9% of total)
Longest unported chain: 3/91 (96.7% progress)

port-progress bot (Jul 01 2023 at 19:34):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 1/924 (99.9% of total)
Unported lines: 200/405646 (100.0% of total)
Longest unported chain: 1/107 (99.1% progress)

port-progress bot (Jul 01 2023 at 19:39):

mathlib port progress set_theory.game.domineering
Unported files: 3/387 (99.2% of total)
Unported lines: 678/156629 (99.6% of total)
Longest unported chain: 3/63 (95.2% progress)

port-progress bot (Jul 01 2023 at 19:43):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 3/701 (99.6% of total)
Unported lines: 497/285431 (99.8% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jul 01 2023 at 19:48):

mathlib port progress all
Unported files: 61/3040 (98.0% of total)
Unported lines: 24622/1042895 (97.6% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jul 01 2023 at 19:49):

1145/3041 files completely ported (37.65%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 01 2023 at 19:49):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jul 01 2023 at 19:54):

0.1%

Johan Commelin (Jul 01 2023 at 20:07):

I've been going through the list of PRs that are help-wanted. Some files are now compiling. Let's see what CI says.

Johan Commelin (Jul 01 2023 at 20:07):

ModelTheory.DirectLimit #4391

This one is help-wanted, but the file builds. It's just that some new names are suboptimal.

Johan Commelin (Jul 01 2023 at 20:08):

Algebra.Category.Algebra.Basic #4504

File now builds, but there are 3 linter failures.

Johan Commelin (Jul 01 2023 at 20:11):

AlgebraicGeometry.ProjectiveSpectrum.StructureSheaf #5224

This one compiles, but needs some help from someone who knows how to set up Lean 4 notation.

Johan Commelin (Jul 01 2023 at 20:13):

basic big operator plugin for norm_num #4350

compiles, and is awaiting-review from a metaxpert.

Antoine Chambert-Loir (Jul 02 2023 at 09:15):

Antoine Chambert-Loir said:

I have tried to work on RingTheory.Jacobson, but I don't understand what happens, and I would have proved the result in a different way. For example, the missing result has to reprove basically that if an algebra is generated by elements, then it is integral iff these elements are integral.

Some progress on that file, I managed to make a proof that was broken, but it requires 300000 heartbeats.
(I could try to split it into two shorter ones…)
Many complicated terms are repeated, and I wonder whether introducing intermediate definitions (let mystuff := <complicated term>) within the proof would help.
That's isIntegral_isLocalization_polynomial_quotient in branch#port/RingTheory.Jacobson

Antoine Chambert-Loir (Jul 02 2023 at 11:51):

Johan Commelin said:

Algebra.Category.Algebra.Basic #4504

File now builds, but there are 3 linter failures.

This is [simps] creating nonoptimal lemmas (“Left-hand side simplifies from…”).
I rewrote the two theorems that made the linter complain. Let's see whether that suffices.

Antoine Chambert-Loir (Jul 02 2023 at 14:27):

That doesn't work, @Johan Commelin , because the lemma I created duplicates the one that is automatically created.

Antoine Chambert-Loir (Jul 02 2023 at 14:37):

Meanwhile, I found about initialize_simps_projection.

port-progress bot (Jul 02 2023 at 19:04):

mathlib port progress representation_theory.group_cohomology.basic
Unported files: 1/968 (99.9% of total)
Unported lines: 184/381059 (100.0% of total)
Longest unported chain: 1/79 (98.7% progress)

port-progress bot (Jul 02 2023 at 19:09):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 2/978 (99.8% of total)
Unported lines: 819/399328 (99.8% of total)
Longest unported chain: 2/90 (97.8% progress)

port-progress bot (Jul 02 2023 at 19:14):

mathlib port progress geometry.manifold.whitney_embedding
Unported files: 3/1126 (99.7% of total)
Unported lines: 1272/506867 (99.7% of total)
Longest unported chain: 3/107 (97.2% progress)

port-progress bot (Jul 02 2023 at 19:18):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 1/678 (99.9% of total)
Unported lines: 247/280501 (99.9% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jul 02 2023 at 19:22):

mathlib port progress representation_theory.character
Unported files: 1/920 (99.9% of total)
Unported lines: 115/349696 (100.0% of total)
Longest unported chain: 1/91 (98.9% progress)

port-progress bot (Jul 02 2023 at 19:34):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 1/924 (99.9% of total)
Unported lines: 200/405646 (100.0% of total)
Longest unported chain: 1/107 (99.1% progress)

port-progress bot (Jul 02 2023 at 19:41):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 3/701 (99.6% of total)
Unported lines: 497/285431 (99.8% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jul 02 2023 at 19:46):

mathlib port progress all
Unported files: 54/3040 (98.2% of total)
Unported lines: 23684/1043008 (97.7% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jul 02 2023 at 19:47):

1257/3041 files completely ported (41.33%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 02 2023 at 19:47):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Scott Morrison (Jul 02 2023 at 23:14):

0.1%

Johan Commelin (Jul 03 2023 at 15:19):

Progress is slowing down, but we are getting closer to the above targets

  • rt.gc.b is done
  • ag.m.qs is one file closer to being done
  • g.m.we is done
  • la.ca.ee didn't move
  • rt.c is done
  • g.m.a.lid didn't move
  • at.fg.sc is still 3 files away from being done

Henrik Böving (Jul 03 2023 at 16:39):

Its not slowing done, you're merely making it exciting for the end!

port-progress bot (Jul 03 2023 at 19:08):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 1/978 (99.9% of total)
Unported lines: 481/399331 (99.9% of total)
Longest unported chain: 1/90 (98.9% progress)

port-progress bot (Jul 03 2023 at 19:16):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 1/678 (99.9% of total)
Unported lines: 247/280501 (99.9% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jul 03 2023 at 19:32):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 1/924 (99.9% of total)
Unported lines: 200/405652 (100.0% of total)
Longest unported chain: 1/107 (99.1% progress)

port-progress bot (Jul 03 2023 at 19:39):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 3/701 (99.6% of total)
Unported lines: 497/285434 (99.8% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jul 03 2023 at 19:44):

mathlib port progress all
Unported files: 46/3040 (98.5% of total)
Unported lines: 20800/1043065 (98.0% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jul 03 2023 at 19:45):

1486/3041 files completely ported (48.86%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 03 2023 at 19:45):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jul 03 2023 at 19:57):

0.3%

port-progress bot (Jul 04 2023 at 19:04):

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 1/978 (99.9% of total)
Unported lines: 481/399303 (99.9% of total)
Longest unported chain: 1/90 (98.9% progress)

port-progress bot (Jul 04 2023 at 19:08):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 1/678 (99.9% of total)
Unported lines: 247/280501 (99.9% of total)
Longest unported chain: 1/84 (98.8% progress)

Ruben Van de Velde (Jul 04 2023 at 19:12):

port-progress bot said:

mathlib port progress algebraic_geometry.morphisms.quasi_separated
Unported files: 1/978 (99.9% of total)
Unported lines: 481/399303 (99.9% of total)
Longest unported chain: 1/90 (98.9% progress)

Speaking of... This is done

port-progress bot (Jul 04 2023 at 19:20):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 1/924 (99.9% of total)
Unported lines: 200/405652 (100.0% of total)
Longest unported chain: 1/107 (99.1% progress)

port-progress bot (Jul 04 2023 at 19:28):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 3/701 (99.6% of total)
Unported lines: 497/285434 (99.8% of total)
Longest unported chain: 3/80 (96.2% progress)

Johan Commelin (Jul 04 2023 at 19:30):

Do we need new targets?

Mario Carneiro (Jul 04 2023 at 19:31):

LTE?

Johan Commelin (Jul 04 2023 at 19:32):

No, I meant mathlib targets

Mario Carneiro (Jul 04 2023 at 19:32):

BTW the completely ported number is really starting to pick up now, it jumped by 7% yesterday

port-progress bot (Jul 04 2023 at 19:32):

mathlib port progress all
Unported files: 42/3040 (98.6% of total)
Unported lines: 19126/1043037 (98.2% of total)
Longest unported chain: 5/117 (95.7% progress)

Ruben Van de Velde (Jul 04 2023 at 19:33):

Next target is all :)

port-progress bot (Jul 04 2023 at 19:33):

1510/3041 files completely ported (49.65%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 04 2023 at 19:33):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jul 04 2023 at 19:34):

Mario Carneiro said:

BTW the completely ported number is really starting to pick up now, it jumped by 7% yesterday

This time it jumped up a bit less: 0.8% or so

Johan Commelin (Jul 04 2023 at 19:34):

0.2%

Johan Commelin (Jul 04 2023 at 19:38):

4 files were ported today.

Scott Morrison (Jul 04 2023 at 23:00):

Interesting there are some additional targets in my scripts, but the bot is not running on them.

Scott Morrison (Jul 04 2023 at 23:01):

In any case, they have already been ported!

Johan Commelin (Jul 05 2023 at 04:59):

yeah, I noticed that your bot stopped posting about stuff that was ported. I thought you added that as a feature :rofl:

port-progress bot (Jul 05 2023 at 19:04):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 1/678 (99.9% of total)
Unported lines: 247/280501 (99.9% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jul 05 2023 at 19:08):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 1/924 (99.9% of total)
Unported lines: 200/405652 (100.0% of total)
Longest unported chain: 1/107 (99.1% progress)

port-progress bot (Jul 05 2023 at 19:12):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 3/701 (99.6% of total)
Unported lines: 497/285434 (99.8% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jul 05 2023 at 19:17):

mathlib port progress all
Unported files: 38/3040 (98.8% of total)
Unported lines: 18528/1043037 (98.2% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jul 05 2023 at 19:18):

1558/3041 files completely ported (51.23%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 05 2023 at 19:18):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Ruben Van de Velde (Jul 05 2023 at 19:22):

port-progress bot said:

1558/3041 files completely ported (51.23%), in the sense that also all downstream dependencies are ported.

+1.58%

Johan Commelin (Jul 05 2023 at 19:24):

0.0%

Johan Commelin (Jul 05 2023 at 19:24):

4 files were ported

Mario Carneiro (Jul 06 2023 at 02:15):

4 files with 0 lines in them?

Scott Morrison (Jul 06 2023 at 02:31):

Apparently 598 lines, but you need ~1000 to get a 0.1% achievement.

Johan Commelin (Jul 06 2023 at 04:21):

I expect that today we'll have more than 0.0%.

Johan Commelin (Jul 06 2023 at 13:44):

I'm hoping that we'll have 6 ported files today.

Johan Commelin (Jul 06 2023 at 13:51):

Jeremy Tan said:

I wouldn't be surprised if we're still not done by , though I consider that time likely

I'm starting to believe this estimate. Looking at the remaining list of PRs, I think we should expect to finish at most 1 PR per day, on average.

port-progress bot (Jul 06 2023 at 19:04):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 1/678 (99.9% of total)
Unported lines: 247/280501 (99.9% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jul 06 2023 at 19:08):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 1/924 (99.9% of total)
Unported lines: 200/405678 (100.0% of total)
Longest unported chain: 1/107 (99.1% progress)

port-progress bot (Jul 06 2023 at 19:12):

mathlib port progress algebraic_topology.fundamental_groupoid.simply_connected
Unported files: 3/701 (99.6% of total)
Unported lines: 497/285434 (99.8% of total)
Longest unported chain: 3/80 (96.2% progress)

port-progress bot (Jul 06 2023 at 19:16):

mathlib port progress all
Unported files: 30/3040 (99.0% of total)
Unported lines: 15390/1043059 (98.5% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jul 06 2023 at 19:18):

1625/3041 files completely ported (53.43%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 06 2023 at 19:18):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Jireh Loreaux (Jul 06 2023 at 19:24):

0.3%, 8 files ported

David Michael Roberts (Jul 07 2023 at 00:11):

Heh, https://leanprover-community.github.io/mathlib-port-status/ tells me :37: files to go. But perhaps 7 of those are not "real" outstanding files?

Johan Commelin (Jul 07 2023 at 05:25):

There are various "zombies" on the dashboard. For technical reasons the dashboard doesnt realise they are already ported.

Johan Commelin (Jul 07 2023 at 05:25):

30 is certainly a more realistic nr

Pol'tta / Miyahara Kō (Jul 07 2023 at 06:06):

The dashboard doesn't recognize !4#5751.

Johan Commelin (Jul 07 2023 at 06:19):

Let's "solve" that problem by getting the PR merged :grinning:

port-progress bot (Jul 07 2023 at 19:04):

mathlib port progress linear_algebra.clifford_algebra.even_equiv
Unported files: 1/678 (99.9% of total)
Unported lines: 247/280501 (99.9% of total)
Longest unported chain: 1/84 (98.8% progress)

port-progress bot (Jul 07 2023 at 19:08):

mathlib port progress geometry.manifold.algebra.left_invariant_derivation
Unported files: 1/924 (99.9% of total)
Unported lines: 200/405678 (100.0% of total)
Longest unported chain: 1/107 (99.1% progress)

port-progress bot (Jul 07 2023 at 19:15):

mathlib port progress all
Unported files: 22/3040 (99.3% of total)
Unported lines: 13272/1043059 (98.7% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jul 07 2023 at 19:16):

1671/3041 files completely ported (54.94%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 07 2023 at 19:16):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jul 07 2023 at 19:41):

0.2%

Johan Commelin (Jul 07 2023 at 19:41):

8 files ported

Matthew Ballard (Jul 07 2023 at 21:14):

Finish Him!!

Jeremy Tan (Jul 07 2023 at 21:40):

To further hasten the end of the port I suggest that non-porting mathlib4 PRs be slapped with after-port (i.e. don't even start reviewing them for merge) unless they are meant to ease porting problems (in which case the PR(s) it is intended to help should be explicitly stated in the description)

Jeremy Tan (Jul 07 2023 at 21:41):

This is to reduce the effect of the many new feature distractions that have recently arrived

Jeremy Tan (Jul 07 2023 at 23:50):

Johan Commelin said:

I'm starting to believe this estimate.

Frankly I chose that time simply because it's my country's National Day

Jireh Loreaux (Jul 08 2023 at 00:15):

I disagree. I've looked at several of the files left, and haven't been able to make progress really. That shouldn't prevent me from working on new feature PRs or reviewing those of others. I won't stop contributing to the port entirely, but I've reduced my effort a bit.

Scott Morrison (Jul 08 2023 at 01:27):

I think the after-port label is working perfectly: you can filter it out (and indeed I recently changed the #help-wanted linkifier to do so) if you want to concentrate on finishing the port, but people are free to get started on those PRs too.

The end of the port is still going to take some work, but we're getting there. The critical thing is not hitting 100% asap, but instead to enable everyone to get on with the real work --- formalizing new maths and writing new automation! We don't want to lose people's enthusiasm for contributing because there's nothing to do but difficult porting. .

Johan Commelin (Jul 08 2023 at 03:59):

There is some value in getting to 100% sooner. Once we have 100% of mathlib compiling in Lean 4, people can start refactors and be certain that they don't suddenly put the port in limbo because of it.

Yury G. Kudryashov (Jul 08 2023 at 05:05):

IMHO, after-port is for refactors that are not allowed before we reach 100%.

Yury G. Kudryashov (Jul 08 2023 at 05:05):

And possibly cleanup #queue3 and #outofsync

Yury G. Kudryashov (Jul 08 2023 at 05:08):

But not everyone's goal is to have 100% of files ported ASAP. Some people are not interested in porting other people's work and some people (like me) want to alternate between writing new code and porting the remaining files.

Yury G. Kudryashov (Jul 08 2023 at 05:11):

And since people volunteer their time, we can't force each other to do what we want to have done (e.g., I would vote for a quick expansion of Geometry.Manifold and Dynamics but I know that other people have their own agenda).

Yaël Dillies (Jul 08 2023 at 07:16):

Johan Commelin said:

There is some value in getting to 100% sooner. Once we have 100% of mathlib compiling in Lean 4, people can start refactors and be certain that they don't suddenly put the port in limbo because of it.

Hmm, I hope that's not how it's going to work because that means all non-mathlib projects can't be accurately mathported anymore.

Yaël Dillies (Jul 08 2023 at 07:17):

Again, hitting 100% of the port on mathlib does not equate with finishing the port.

Ruben Van de Velde (Jul 08 2023 at 07:24):

Depends on what you mean by "the port", of course

Eric Wieser (Jul 08 2023 at 07:48):

@Yaël Dillies, I don't understand your point; once mathlib4 hits 100% ported (which should include #outofsync), then we tag the commit and tell downstream projects to run mathport against that commit first.

Eric Wieser (Jul 08 2023 at 07:49):

Mathport isn't going to be able to translate old mathlib3 to new mathlib4; the only place where we can hope for reliable success is for mathport to help make the jump from final mathlib3 to "100% ported" mathlib4; then we're back in the normal "bump mathlib(4)" territory that is already part of maintaining Lean 3 projects

Scott Morrison (Jul 08 2023 at 09:42):

Hmm... it occurs to me that Eric's suggestion that the 100% tag "should include #outofsync" may be problematic. We have approximately 60 PRs at the moment to mathlib3, which will not be marked as too-late next week. I don't think it is reasonable to wait to start work on refactoring for all of those. Yet for those PRs, while hopefully some we can just translate directly to mathlib4 PRs, for at least some it may make more sense to merge them to mathlib3 and then use #outofsync to manage bringing them to mathlib4.

Eric Wieser (Jul 08 2023 at 09:47):

I think it should include everything that is out of sync at the point that we hit 100%, but not necessarily anything after that

Eric Wieser (Jul 08 2023 at 09:48):

What matters is that the mathlib3 "final" tag is in sync with the mathlib4 "100% complete" tag

Eric Wieser (Jul 08 2023 at 09:48):

If mathlib3 picks up a few extra commits after the final tag, because that makes it easier to forward-port them, I think that's ok

Eric Wieser (Jul 08 2023 at 09:49):

I think it would make sense to start ramping down the allowed size of #outofsync

Yaël Dillies (Jul 08 2023 at 10:44):

Nobody is reviewing mathlib PRs anyway, so I'm not sure this is gonna change much.

Scott Morrison (Jul 08 2023 at 11:46):

Once the port is done (and I'm finished vacation :-) I'm keen to work on #outofsync and the not too-late PRs to mathlib3. They've just been lower priority for a while, in part because working on them induces more working being done in Lean 3. :-) Once June 14 and the too-late label arrives, the incentives change!

Johan Commelin (Jul 08 2023 at 11:47):

s/June/July/

Mauricio Collares (Jul 08 2023 at 12:00):

Exactly a week to go!

Kevin Buzzard (Jul 08 2023 at 14:32):

port-progress bot said:

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Why did the linkifier for #help-wanted not work? Edit: it didn't work in the post I'm quoting, but works when I quote it :-) Maybe someone was fiddling with the linkifiers the moment the post was made?

Kevin Buzzard (Jul 08 2023 at 14:34):

o_O only 7 PRs on the list!

Patrick Massot (Jul 08 2023 at 14:40):

If you need help to choose one, I suggest #5496

Yury G. Kudryashov (Jul 08 2023 at 14:48):

Please let me try the "no simp on extChartAt" first.

Kevin Buzzard (Jul 08 2023 at 14:54):

I was just trying that one. The first error is with a ⁻¹' and it can be fixed by changing π (TangentSpace I) to (fun x ↦ π (TangentSpace I) x) (and also once in the proof) but then I get

argument
  TangentSpace I
has type
  ?m.67664  Type ?u.64688 : Type (max ?u.67646 (?u.64688 + 1))
but is expected to have type
  Type ?u.67643 : Type (?u.67643 + 1)

and by this point the fact that I don't understand how tangent spaces are set up means I don't really know how to go further. I assume I've made a wrong turn.

Kevin Buzzard (Jul 08 2023 at 14:55):

What surprises me is that there's already a porting note in the proof, meaning that at some point it was compiling?

Yury G. Kudryashov (Jul 08 2023 at 15:01):

I'll come home in a few hours, then force-push a rebase of this branch on top of a new mathport output.

port-progress bot (Jul 08 2023 at 19:13):

mathlib port progress all
Unported files: 18/3040 (99.4% of total)
Unported lines: 11704/1043155 (98.9% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jul 08 2023 at 19:14):

1709/3041 files completely ported (56.19%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 08 2023 at 19:14):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jul 08 2023 at 19:32):

0.2%

port-progress bot (Jul 09 2023 at 19:13):

mathlib port progress all
Unported files: 18/3040 (99.4% of total)
Unported lines: 11704/1043155 (98.9% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jul 09 2023 at 19:14):

1709/3041 files completely ported (56.19%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 09 2023 at 19:14):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jul 10 2023 at 06:35):

0.0%

Kevin Buzzard (Jul 10 2023 at 09:41):

yeah but: 18 to go!

port-progress bot (Jul 10 2023 at 19:13):

mathlib port progress all
Unported files: 15/3040 (99.5% of total)
Unported lines: 11008/1043155 (98.9% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jul 10 2023 at 19:14):

1735/3041 files completely ported (57.05%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 10 2023 at 19:14):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jul 10 2023 at 19:17):

0.0%

Patrick Stevens (Jul 10 2023 at 19:46):

The real progress was the friends we made along the way

Kevin Buzzard (Jul 10 2023 at 21:31):

This 0.0% is misleading. 3/18 remaining files were merged

Ruben Van de Velde (Jul 10 2023 at 21:39):

Lies, damn lies and statistics?

Yury G. Kudryashov (Jul 11 2023 at 00:42):

#5727 compiles

Pol'tta / Miyahara Kō (Jul 11 2023 at 02:05):

The Traversable deriving handler is awaiting review from @Kyle Miller which is requested from @Scott Morrison. Any news?

David Michael Roberts (Jul 11 2023 at 02:12):

Out of curiosity, which files are https://leanprover-community.github.io/mathlib-port-status/ are zombies?

Eric Wieser (Jul 11 2023 at 05:07):

#5768 (slim_check stuff) almost compiles too, but has grown a dependency that needs review

Johan Commelin (Jul 11 2023 at 06:23):

@David Michael Roberts The zombies have mostly been removed yesterday.

Johan Commelin (Jul 11 2023 at 06:23):

There were entries called .decision_nec etc, but they are gone now.

Johan Commelin (Jul 11 2023 at 06:24):

I think that all the remaining entries are non-zombie

Johan Commelin (Jul 11 2023 at 06:24):

But there's still a debate about how/when/if certain entries should be ported.

David Michael Roberts (Jul 11 2023 at 06:35):

True. Especially the ones that are more "meta". Thanks!

David Michael Roberts (Jul 11 2023 at 06:40):

Though there are 18 files at the port-status page, but 15 reported for 'all' by the bot. I guess things like system.io are not being ported? And data.buffer.basic, marked "not needed"? Perhaps I shouldn't have said zombies, but something else...

David Michael Roberts (Jul 11 2023 at 06:41):

And technically, one of those 15 files is all.

Kyle Miller (Jul 11 2023 at 07:05):

@Pol'tta / Miyahara Kō I'll take a look today

port-progress bot (Jul 11 2023 at 19:13):

mathlib port progress all
Unported files: 13/3040 (99.6% of total)
Unported lines: 10486/1043260 (99.0% of total)
Longest unported chain: 5/117 (95.7% progress)

port-progress bot (Jul 11 2023 at 19:14):

1738/3041 files completely ported (57.15%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 11 2023 at 19:14):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Floris van Doorn (Jul 11 2023 at 19:16):

2 more ported files. 6 files remaining (assuming that the remaining files in data/testing are not counted)

Johan Commelin (Jul 11 2023 at 19:23):

0.1%

Tobias Grosser (Jul 11 2023 at 19:26):

99%!

Matthew Ballard (Jul 11 2023 at 19:26):

I've been banging my head against #5663 but not much productive has happened since yesterday. Please feel encouraged to take a look.

Jeremy Tan (Jul 12 2023 at 00:40):

Apparently #5088 passes CI now

Scott Morrison (Jul 12 2023 at 00:57):

@Matthew Ballard, nice work on #5088. I've left a few comments.

Matthew Ballard (Jul 12 2023 at 01:23):

:ping_pong: Two oddities:

  • the instance synthesis failure config for apply doesn't seem to always work (but perhaps I did something wrong)
  • local notation "F" := left_adjoint G in ml3 allowed for F.obj F.map... to parse. Here notation and notation3 don't (again perhaps it's me)

Scott Morrison (Jul 12 2023 at 01:55):

@Kyle Miller, any chance you could look at the notation issues in #5088? It's not a blocker, so low priority.

Matthew Ballard (Jul 12 2023 at 02:21):

I restored the notation (using notation3). It was a hygiene issue

Matthew Ballard (Jul 12 2023 at 02:29):

Off to sleep. Hopefully I will wake up to #5663 :check: :wink: :prayer_beads:

Scott Morrison (Jul 12 2023 at 03:39):

I pushed a few clean-ups to #5088, and then hit :merge:.

Kyle Miller (Jul 12 2023 at 06:55):

Matthew Ballard said:

local notation "F" := left_adjoint G in ml3 allowed for F.obj F.map... to parse. Here notation and notation3 don't

In mathlib3, neither of these parsed; you had to write F .obj and F .map.

For notation3, the trick to using it is to write notation3 and not notation :wink: (notation3 allows you to refer to local variables if you write local notation3. Though it gives sort of obscure errors about not being able to generate delaborators if you forget local or get the names of variables wrong...)

port-progress bot (Jul 12 2023 at 19:53):

mathlib port progress all
Unported files: 10/3040 (99.7% of total)
Unported lines: 9336/1043379 (99.1% of total)
Longest unported chain: 4/117 (96.6% progress)

port-progress bot (Jul 12 2023 at 19:55):

1761/3041 files completely ported (57.90%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 12 2023 at 19:55):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Jeremy Tan (Jul 13 2023 at 03:53):

Analysis.Analytic.Inverse #5032 is ready for review

Scott Morrison (Jul 13 2023 at 04:58):

Just four real files to go!

Johan Commelin (Jul 13 2023 at 05:29):

0.1%

Scott Morrison (Jul 13 2023 at 06:36):

#5846 adds a porting header to Data.HashMap, along with a comment saying that everything has been reimplemented in Std.

Scott Morrison (Jul 13 2023 at 06:49):

and #5848 proposes empty ports of the Data/Buffer/Parser files, on the basis that these should be ported as needed in the manner of tactics, rather than as part of the main port.

Johan Commelin (Jul 13 2023 at 09:31):

#port-dashboard now says 99.8%. Thanks @Scott Morrison :octopus:

Eric Wieser (Jul 13 2023 at 09:46):

If that's dangerously high we could merge mathlib-port-status#21 to bring it back down to a more manageable 96%! :upside_down:

Eric Wieser (Jul 13 2023 at 10:29):

The above might be worth doing briefly, as a lot of those files _are_ ported but missing porting headers

Johan Commelin (Jul 13 2023 at 10:30):

Can you autogenerate a patch that adds the headers? Or is that complicated for some reason?

Eric Wieser (Jul 13 2023 at 10:30):

Well a lot of the files are ad-hoc

Eric Wieser (Jul 13 2023 at 10:31):

So the header would be a lie anyway

Eric Wieser (Jul 13 2023 at 10:33):

I just re-ported two of them in #5857 and #5859

port-progress bot (Jul 13 2023 at 19:14):

mathlib port progress all
Unported files: 5/3041 (99.8% of total)
Unported lines: 4811/1043953 (99.5% of total)
Longest unported chain: 3/117 (97.4% progress)

Johan Commelin (Jul 13 2023 at 19:14):

0.4%

port-progress bot (Jul 13 2023 at 19:15):

1775/3042 files completely ported (58.34%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 13 2023 at 19:15):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Kevin Buzzard (Jul 13 2023 at 21:37):

So five non-All files between them import over 40% of mathlib?

David Michael Roberts (Jul 13 2023 at 22:26):

@Kevin Buzzard https://leanprover-community.github.io/mathlib-port-status/file/algebraic_geometry/morphisms/finite_type alone depends on 946 other files!

Eric Wieser (Jul 13 2023 at 22:30):

Eric Wieser said:

I just re-ported two of them in #5857 and #5859

These are now both green, but they're not visible on the dashboard

port-progress bot (Jul 14 2023 at 19:14):

mathlib port progress all
Unported files: 4/3041 (99.9% of total)
Unported lines: 4432/1043953 (99.6% of total)
Longest unported chain: 3/117 (97.4% progress)

port-progress bot (Jul 14 2023 at 19:15):

1776/3042 files completely ported (58.38%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 14 2023 at 19:15):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Johan Commelin (Jul 14 2023 at 19:55):

0.1%

Matthew Ballard (Jul 14 2023 at 20:37):

Of the count above only #5571 remains (count is one less due to all)

Yury G. Kudryashov (Jul 14 2023 at 21:43):

I'm sorry for a delay with #5571. If someone wants to port is as is, you may take over that file. I don't want to port it today and rewrite it tomorrow.

Eric Wieser (Jul 15 2023 at 07:58):

Note that there are two new files on the dashboard; algebra.expr and data.matrix.auto. Both are meta files, so can be ported as just a SHA header (or ignored) Edit: I've made porting PRs

port-progress bot (Jul 15 2023 at 19:14):

mathlib port progress all
Unported files: 2/3043 (99.9% of total)
Unported lines: 3780/1044558 (99.6% of total)
Longest unported chain: 2/117 (98.3% progress)

port-progress bot (Jul 15 2023 at 19:15):

2028/3044 files completely ported (66.62%), in the sense that also all downstream dependencies are ported.

port-progress bot (Jul 15 2023 at 19:15):

Please remember that the PRs on #help-wanted are high priority as we approach completion. Please also check #stalled occasionally to see if you have anything there, or know how to help.

Heather Macbeth (Jul 15 2023 at 20:54):

#5571 passes CI.

Kevin Buzzard (Jul 15 2023 at 20:55):

ooh so it does :-)

Matthew Ballard (Jul 15 2023 at 20:55):

But it is not 3870 lines...

Heather Macbeth (Jul 15 2023 at 20:57):

Are the remaining lines the list of all files in all?

Matthew Ballard (Jul 15 2023 at 21:01):

Looks right

Kevin Buzzard (Jul 15 2023 at 21:02):

Yeah all is 3209 lines on this recent mathlib and the circle file is 660, it doesn't quite add up but fingers crossed...

Yury G. Kudryashov (Jul 15 2023 at 21:02):

One of my recently merged PRs can make linter fail in #5571

Yury G. Kudryashov (Jul 15 2023 at 21:02):

Merging master.

Patrick Massot (Jul 15 2023 at 23:23):

The port is officially done since two minutes ago!

Patrick Massot (Jul 15 2023 at 23:23):

Every file from mathlib has been ported to Lean 4!

Patrick Massot (Jul 15 2023 at 23:24):

Of course there is still a lot of work to do to polish Mathlib 4, but today is the day of Mathlib 4!

Patrick Massot (Jul 15 2023 at 23:25):

Huge congratulations to everyone who has been involved in the port!

Patrick Massot (Jul 15 2023 at 23:27):

The full list of people who directly contributed to the port is at https://github.com/leanprover-community/mathlib4/graphs/contributors. But don't forget the crucial mathport infrastructure at https://github.com/leanprover-community/mathport/graphs/contributors, and of course the amazing work of @Leonardo de Moura, @Sebastian Ullrich and @Gabriel Ebner on Lean 4 itself!

Patrick Massot (Jul 15 2023 at 23:29):

As a first celebration item, I recorded a video showing some stuff I like about Lean 4 for formalized mathematics. We will probably move it to the Lean community Youtube channel soon, but right now you can watch it at http://pat.perso.ens-lyon.org/lean4_overview_for_mathlib_users.m4v

Jeremy Tan (Jul 15 2023 at 23:30):

:congratulations:

Scott Morrison (Jul 16 2023 at 05:02):

@Patrick Massot's new video will be on the Youtube channel shortly at https://youtu.be/8MFGhOWeCNE.

Johan Commelin (Jul 16 2023 at 05:27):

@Patrick Massot you mention Leo's talk at ICERM last year. Did you notice that is was also on exactly July 15?

Yury G. Kudryashov (Jul 16 2023 at 05:33):

It looks like Lean community has a long tradition of celebrating my wife's birthday without knowing about it.

Arthur Paulino (Jul 16 2023 at 05:59):

This is epic. What a nicely coordinated effort. Congrats everyone!

Johan Commelin (Jul 16 2023 at 06:53):

@Patrick Massot Thank you so much for making this video. A very nice idea, and a great showcase!

Patrick Massot (Jul 16 2023 at 08:52):

I just realized that I intended to mention goal diffs in my video but I missed the moment I wanted to discuss it. Depending on your color theme, this really nice and useful feature can be easy to miss. It changes the background color of the part of the goal that is about to change or has just changed.

Eric Wieser (Jul 16 2023 at 09:11):

Fix it in post!

Johan Commelin (Jul 17 2023 at 07:53):

I really want those calc and conv widgets! They look awesome

Patrick Massot (Jul 17 2023 at 08:38):

People who want those widgets can start with upvoting https://github.com/EdAyers/ProofWidgets4/pull/16 I guess.

Johan Commelin (Jul 18 2023 at 11:46):

#outofsync is empty!

Richard L Ford (Jul 21 2023 at 17:32):

At mathlib-port-status, there had been only one remaining file, and essentially at 100%, but then a bunch of core.* files were added. Nothing seems to have changed for the last few days. What is happening?

Johan Commelin (Jul 21 2023 at 17:36):

Many of these core files are effectively ported, but in a more ad-hoc manner than mathlib. So there is the remaining task of adding #align statements that document which lean 4 declarations correspond to which lean 3 declarations. I think that is most of what needs to be done.

What is happening?

Currently, it is of higher priority to finalize the porting path from ml3 to ml4 for projects that depend on mathlib. And in the past week there has also been a higher activity to work through the queue of PRs to mathlib3 that made the freezing deadline.

Eric Wieser (Jul 21 2023 at 17:53):

I don't think aligning those core files is very urgent; I put them on the dashboard because we tracked down a few that were missing

Eric Wieser (Jul 21 2023 at 17:53):

But I think it's still basically accurate to claim "mathlib is 100% ported", as strictly speaking those files are not mathlib at all!

Scott Morrison (Jul 22 2023 at 07:29):

Moreover some of those files are very old, are intended to support language features that have been completely replaced, or otherwise probably wouldn't be included in Mathlib today. So porting them just because they are there is pretty low priority, especially given the prima facie evidence that they are useless (i.e. not needed to port Mathlib).

Patrick Massot (Jul 22 2023 at 08:21):

Why don't we simply remove them from the dashboard? They are only confusing.

Eric Wieser (Jul 22 2023 at 08:54):

They're useful for if someone finds a file that we forgot that actually is useful

Eric Wieser (Jul 22 2023 at 08:55):

Also, if we removed them the page would just be empty which doesn't really achieve anything

Eric Wieser (Jul 22 2023 at 08:56):

Perhaps a banner at the top explaining the situation is a good compromise? Maybe we need a blog post to link to :)

Patrick Massot (Jul 22 2023 at 09:16):

Eric Wieser said:

Also, if we removed them the page would just be empty which doesn't really achieve anything

It achieves telling people there are no more files to port.

Yaël Dillies (Jul 23 2023 at 08:19):

Eric Wieser said:

They're useful for if someone finds a file that we forgot that actually is useful

This happened just five days ago FYI

Eric Wieser (Jul 23 2023 at 08:51):

Eric Wieser said:

Perhaps a banner at the top explaining the situation is a good compromise? Maybe we need a blog post to link to :)

I added such a banner

Richard L Ford (Jul 26 2023 at 18:09):

Patrick Massot said:

The port is officially done since two minutes ago!

Perhaps since the port of mathlib4 is considered complete, the GitHub README should be changed to no longer say that it is a port in progress.

Patrick Massot (Jul 26 2023 at 18:10):

That's a good point!


Last updated: Dec 20 2023 at 11:08 UTC