theorem
func_subsingleton_iff_to_empty
{α : Type u}
{β : Type v}
(h : α → Empty)
:
Subsingleton (α → β)
Equations
- PUnit.unique = { default := PUnit.unit, uniq := PUnit.unique.proof_1 }
Every provable proposition is unique, as all proofs are equal.
Equations
- uniqueProp h = { default := h, uniq := ⋯ }
Instances For
True
has a unique term.
Equations
@[instance 100]
Equations
- ⋯ = ⋯
Equations
- Unique.ExistsUnique p = ∃ (x : α), p x ∧ ∀ (y : α), p y → y = x
Instances For
Checks to see that xs
has only one binder.
Equations
- One or more equations did not get rendered due to their size.
Instances For
∃! x : α, p x
means that there exists a unique x
in α
such that p x
.
This is notation for ExistsUnique (fun (x : α) ↦ p x)
.
This notation does not allow multiple binders like ∃! (x : α) (y : β), p x y
as a shorthand for ∃! (x : α), ∃! (y : β), p x y
since it is liable to be misunderstood.
Often, the intended meaning is instead ∃! q : α × β, p q.1 q.2
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
∃! x ∈ s, p x
means ∃! x, x ∈ s ∧ p x
, which is to say that there exists a unique x ∈ s
such that p x
.
Similarly, notations such as ∃! x ≤ n, p n
are supported,
using any relation defined using the binder_predicate
command.
Equations
- One or more equations did not get rendered due to their size.