Skip to content

Commit

Permalink
re-fix
Browse files Browse the repository at this point in the history
  • Loading branch information
vihdzp committed Jan 15, 2025
1 parent 64d6dc3 commit a7597d1
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/Init/Core.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1908,11 +1908,11 @@ instance Pi.instSubsingleton {α : Sort u} {β : α → Sort v} [∀ a, Subsingl

/-! # Squash -/

theorem true_equivalence : @Equivalence α fun _ _ ↦ True :=
theorem true_equivalence (α : Sort u) : Equivalence fun _ _ : α ↦ True :=
fun _ ↦ trivial, fun _ ↦ trivial, fun _ _ ↦ trivial⟩

/-- Always-true relation as a `Setoid`. -/
def trueSetoid : Setoid α :=
def trueSetoid (α : Sort u) : Setoid α :=
⟨_, true_equivalence⟩

/--
Expand All @@ -1929,7 +1929,7 @@ represents an element of `Squash α` the same as `α` itself
`Squash.lift` will extract a value in any subsingleton `β` from a function on `α`,
while `Nonempty.rec` can only do the same when `β` is a proposition.
-/
def Squash (α : Sort u) := @Quotient α trueSetoid
def Squash (α : Sort u) := Quotient (trueSetoid α)

/-- The canonical quotient map into `Squash α`. -/
def Squash.mk {α : Sort u} (x : α) : Squash α := Quot.mk _ x
Expand Down

0 comments on commit a7597d1

Please sign in to comment.