Skip to content

Commit

Permalink
Bump mathlib
Browse files Browse the repository at this point in the history
Signed-off-by: zeramorphic <[email protected]>
  • Loading branch information
zeramorphic committed Mar 25, 2024
1 parent a10b390 commit 10b1ae2
Show file tree
Hide file tree
Showing 3 changed files with 6 additions and 6 deletions.
4 changes: 2 additions & 2 deletions ConNF/Mathlib/Logic/Equiv/PartialPerm.lean
Original file line number Diff line number Diff line change
Expand Up @@ -150,10 +150,10 @@ theorem image_domain : π '' π.domain = π.domain :=
π.bijOn.image_eq

theorem forall_mem_domain {p : α → Prop} : (∀ y ∈ π.domain, p y) ↔ ∀ x ∈ π.domain, p (π x) := by
conv_lhs => rw [← image_domain, ball_image_iff]
conv_lhs => rw [← image_domain, forall_mem_image]

theorem exists_mem_domain {p : α → Prop} : (∃ y ∈ π.domain, p y) ↔ ∃ x ∈ π.domain, p (π x) := by
conv_lhs => rw [← image_domain, bex_image_iff]
conv_lhs => rw [← image_domain, exists_mem_image]

/-- A set `s` is *stable* under a partial equivalence `π` if it preserved by it. -/
def IsStable (s : Set α) : Prop :=
Expand Down
2 changes: 1 addition & 1 deletion ConNF/NewTangle/NewAllowable.lean
Original file line number Diff line number Diff line change
Expand Up @@ -267,7 +267,7 @@ theorem isAllowable_pow (h : ρ.IsAllowable) (n : ℕ) : (ρ ^ n).IsAllowable :=
theorem isAllowable_zpow (h : ρ.IsAllowable) (n : ℤ) : (ρ ^ n).IsAllowable := by
cases n with
| ofNat n =>
rw [Int.ofNat_eq_coe, zpow_coe_nat]
rw [Int.ofNat_eq_coe, zpow_natCast]
exact isAllowable_pow h n
| negSucc n =>
rw [zpow_negSucc]
Expand Down
6 changes: 3 additions & 3 deletions lake-manifest.json
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@
[{"url": "https://github.com/leanprover/std4",
"type": "git",
"subDir": null,
"rev": "f3447c3732c9d6e8df3bdad78e5ecf7e8b353bbc",
"rev": "e5306c3b0edefe722370b7387ee9bcd4631d6c17",
"name": "std",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand Down Expand Up @@ -49,7 +49,7 @@
{"url": "https://github.com/leanprover-community/import-graph.git",
"type": "git",
"subDir": null,
"rev": "bbcffbcc19d69e13d5eea716283c76169db524ba",
"rev": "61a79185b6582573d23bf7e17f2137cd49e7e662",
"name": "importGraph",
"manifestFile": "lake-manifest.json",
"inputRev": "main",
Expand All @@ -58,7 +58,7 @@
{"url": "https://github.com/leanprover-community/mathlib4.git",
"type": "git",
"subDir": null,
"rev": "0c4d96e6b94d1d61c45658d569d6e4a56fa68535",
"rev": "103d868920c23be42cde493246a7da660149bd8b",
"name": "mathlib",
"manifestFile": "lake-manifest.json",
"inputRev": null,
Expand Down

0 comments on commit 10b1ae2

Please sign in to comment.