Skip to content

Upgrade Lean and mathlib #148

Upgrade Lean and mathlib

Upgrade Lean and mathlib #148

Triggered via pull request October 23, 2023 21:53
Status Success
Total duration 12m 21s
Artifacts

ci.yml

on: pull_request
Fit to window
Zoom out
Zoom in

Annotations

11 warnings and 10 notices
Build project
The following actions uses node12 which is deprecated and will be forced to run on node16: actions/checkout@v2, actions/setup-python@v1. For more info: https://github.blog/changelog/2023-06-13-github-actions-all-actions-will-run-on-node16-instead-of-node12-by-default/
Build project: src/hints/category_theory/exercise1/hint1.lean#L9
/home/runner/work/lftcm2020/lftcm2020/src/hints/category_theory/exercise1/hint1.lean:9:0: declaration 'iso_of_hom_iso_attempt_1' uses sorry
Build project: src/hints/category_theory/exercise2/hint1.lean#L13
/home/runner/work/lftcm2020/lftcm2020/src/hints/category_theory/exercise2/hint1.lean:13:0: declaration 'CommRing.polynomial' uses sorry
Build project: src/hints/category_theory/exercise2/hint3.lean#L35
/home/runner/work/lftcm2020/lftcm2020/src/hints/category_theory/exercise2/hint3.lean:35:0: declaration 'CommRing.polynomial' uses sorry
Build project: src/hints/category_theory/exercise2/hint2.lean#L21
/home/runner/work/lftcm2020/lftcm2020/src/hints/category_theory/exercise2/hint2.lean:21:0: declaration 'CommRing.polynomial' uses sorry
Build project: src/exercises_sources/thursday/category_theory/exercise2.lean#L15
/home/runner/work/lftcm2020/lftcm2020/src/exercises_sources/thursday/category_theory/exercise2.lean:15:0: declaration 'Ring.polynomial' uses sorry
Build project: src/hints/category_theory/exercise2/hint5.lean#L12
/home/runner/work/lftcm2020/lftcm2020/src/hints/category_theory/exercise2/hint5.lean:12:0: declaration 'CommRing.polynomial' uses sorry
Build project: src/exercises_sources/thursday/category_theory/exercise2.lean#L18
/home/runner/work/lftcm2020/lftcm2020/src/exercises_sources/thursday/category_theory/exercise2.lean:18:0: declaration 'CommRing.polynomial' uses sorry
Build project: src/exercises_sources/monday/metaprogramming.lean#L41
/home/runner/work/lftcm2020/lftcm2020/src/exercises_sources/monday/metaprogramming.lean:41:0: declaration '[anonymous]' uses sorry
Build project: src/exercises_sources/tuesday/numbers.lean#L23
/home/runner/work/lftcm2020/lftcm2020/src/exercises_sources/tuesday/numbers.lean:23:0: declaration '[anonymous]' uses sorry
Build project: src/hints/category_theory/exercise2/hint1.lean#L18
/home/runner/work/lftcm2020/lftcm2020/src/hints/category_theory/exercise2/hint1.lean:18:0: declaration 'commutes' uses sorry
Build project: src/demos/linalg.lean#L23
/home/runner/work/lftcm2020/lftcm2020/src/demos/linalg.lean:23:0: @[_ext_core id.{1} name module.ext, class, ext option.none.{0} name, protect_proj list.nil.{0} name] structure module : Π (R : Type u) (M : Type v) [_inst_1 : semiring R] [_inst_2 : add_comm_monoid M], Type (max u v) fields: module.to_distrib_mul_action : Π {R : Type u} {M : Type v} [_inst_1 : semiring R] [_inst_2 : add_comm_monoid M] [self : module R M], distrib_mul_action R M module.add_smul : ∀ {R : Type u} {M : Type v} [_inst_1 : semiring R] [_inst_2 : add_comm_monoid M] [self : module R M] (r s : R) (x : M), (r + s) • x = r • x + s • x module.zero_smul : ∀ {R : Type u} {M : Type v} [_inst_1 : semiring R] [_inst_2 : add_comm_monoid M] [self : module R M] (x : M), 0 • x = 0
Build project: src/demos/linalg.lean#L32
/home/runner/work/lftcm2020/lftcm2020/src/demos/linalg.lean:32:0: add_smul : ∀ (r s : ?M_1) (x : ?M_2), (r + s) • x = r • x + s • x
Build project: src/demos/linalg.lean#L33
/home/runner/work/lftcm2020/lftcm2020/src/demos/linalg.lean:33:0: smul_add : ∀ (a : ?M_1) (b₁ b₂ : ?M_2), a • (b₁ + b₂) = a • b₁ + a • b₂
Build project: src/demos/linalg.lean#L34
/home/runner/work/lftcm2020/lftcm2020/src/demos/linalg.lean:34:0: mul_smul : ∀ (x y : ?M_1) (b : ?M_2), (x * y) • b = x • y • b
Build project: src/demos/linalg.lean#L35
/home/runner/work/lftcm2020/lftcm2020/src/demos/linalg.lean:35:0: one_smul : ∀ (M : Type u_1) {α : Type u_2} [_inst_1 : monoid M] [_inst_2 : mul_action M α] (b : α), 1 • b = b
Build project: src/demos/linalg.lean#L36
/home/runner/work/lftcm2020/lftcm2020/src/demos/linalg.lean:36:0: zero_smul : ∀ (R : Type u_1) {M : Type u_2} [_inst_1 : has_zero R] [_inst_2 : has_zero M] [_inst_3 : smul_with_zero R M] (m : M), 0 • m = 0
Build project: src/solutions/friday/topology.lean#L97
/home/runner/work/lftcm2020/lftcm2020/src/solutions/friday/topology.lean:97:0: sets_of_superset : ∀ {α : Type u_1} (self : filter α) {x y : set α}, x ∈ self.sets → x ⊆ y → y ∈ self.sets
Build project: src/demos/linalg.lean#L37
/home/runner/work/lftcm2020/lftcm2020/src/demos/linalg.lean:37:0: smul_zero : ∀ (a : ?M_1), a • 0 = 0
Build project: src/exercises_sources/friday/topology.lean#L56
/home/runner/work/lftcm2020/lftcm2020/src/exercises_sources/friday/topology.lean:56:0: sets_of_superset : ∀ {α : Type u_1} (self : filter α) {x y : set α}, x ∈ self.sets → x ⊆ y → y ∈ self.sets
Build project: src/solutions/friday/topology.lean#L98
/home/runner/work/lftcm2020/lftcm2020/src/solutions/friday/topology.lean:98:0: mem_of_superset : ∀ {α : Type u_1} {f : filter α} {x y : set α}, x ∈ f → x ⊆ y → y ∈ f