Skip to content

Commit

Permalink
Use Sort* and Type* slightly more.
Browse files Browse the repository at this point in the history
  • Loading branch information
grunweg committed Jul 8, 2024
1 parent 406babb commit 9c93648
Show file tree
Hide file tree
Showing 3 changed files with 5 additions and 3 deletions.
2 changes: 1 addition & 1 deletion SphereEversion/ToMathlib/Data/Set/Lattice.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,7 @@ theorem const_prod_iUnion {s : ι → Set α} {t : Set β} : (t ×ˢ ⋃ i, s i)
ext; simp

-- Put next to Union₂_prod_const...
theorem const_prod_iUnion₂ {κ : ι → Sort _} {s : ∀ i, κ i → Set α} {t : Set β} :
theorem const_prod_iUnion₂ {κ : ι → Sort*} {s : ∀ i, κ i → Set α} {t : Set β} :
(t ×ˢ ⋃ (i) (j), s i j) = ⋃ (i) (j), t ×ˢ s i j := by simp_rw [const_prod_iUnion]

-- the next 2 lemmas should be generalized from `Set α` to a `CompleteLattice`
Expand Down
4 changes: 3 additions & 1 deletion SphereEversion/ToMathlib/Logic/Basic.lean
Original file line number Diff line number Diff line change
@@ -1,4 +1,6 @@
import Mathlib.Tactic.TypeStar

-- `by simp [forall_and]` works in Lean 4
theorem forall₂_and_distrib {α β : Sort _} {p q : α → β → Prop} :
theorem forall₂_and_distrib {α β : Sort*} {p q : α → β → Prop} :
(∀ x y, p x y ∧ q x y) ↔ (∀ x y, p x y) ∧ ∀ x y, q x y :=
(forall_congr' fun x : α ↦ @forall_and _ (p x) (q x)).trans forall_and
Original file line number Diff line number Diff line change
Expand Up @@ -7,7 +7,7 @@ We no longer intend to use this file in the sphere eversion project.
-/
namespace Function

variable {ι : Sort _} [DecidableEq ι] {α β : ι → Type*}
variable {ι : Sort*} [DecidableEq ι] {α β : ι → Type*}

/-- Special case of `function.apply_update`. Useful for `rw`/`simp`. -/
theorem update_fst (g : ∀ i, α i × β i) (i : ι) (v : α i × β i) (j : ι) :
Expand Down

0 comments on commit 9c93648

Please sign in to comment.