Semiquotients #
A data type for semiquotients, which are classically equivalent to
nonempty sets, but are useful for programming; the idea is that
a semiquotient set S
represents some (particular but unknown)
element of S
. This can be used to model nondeterministic functions,
which return something in a range of values (represented by the
predicate S
) but are not completely determined.
A member of Semiquot α
is classically a nonempty Set α
,
and in the VM is represented by an element of α
; the relation
between these is that the VM element is required to be a member
of the set s
. The specific element of s
that the VM computes
is hidden by a quotient construction, allowing for the representation
of nondeterministic functions.
Instances For
Equations
- Semiquot.instMembership = { mem := fun (q : Semiquot α) (a : α) => a ∈ q.s }
Equations
- One or more equations did not get rendered due to their size.
Equations
- Semiquot.partialOrder = { le := fun (s t : Semiquot α) => ∀ ⦃x : α⦄, x ∈ s → x ∈ t, le_refl := ⋯, le_trans := ⋯, lt_iff_le_not_le := ⋯, le_antisymm := ⋯ }
Equations
- Semiquot.instSemilatticeSup = { toPartialOrder := Semiquot.partialOrder, sup := fun (s : Semiquot α) => Semiquot.blur s.s, le_sup_left := ⋯, le_sup_right := ⋯, sup_le := ⋯ }
Equations
- Semiquot.instInhabited = { default := Semiquot.univ }
@[simp]
Equations
- Semiquot.instOrderTopOfInhabited = { top := Semiquot.univ, le_top := ⋯ }