Strings #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Supplementary theorems about the string
type.
<
on string iterators. This coincides with <
on strings as lists.
@[protected, instance]
Equations
- string.has_lt' = {lt := λ (s₁ s₂ : string), ↥(string.ltb s₁.mk_iterator s₂.mk_iterator)}
@[protected, instance]
Equations
- string.decidable_lt = λ (a b : string), bool.decidable_eq (string.ltb a.mk_iterator b.mk_iterator) bool.tt
@[protected, instance]
Equations
- string.decidable_le = λ (a b : string), ne.decidable (string.ltb b.mk_iterator a.mk_iterator) bool.tt
@[protected, instance]
Equations
- string.linear_order = {le := has_le.le string.has_le, lt := has_lt.lt string.has_lt', le_refl := string.linear_order._proof_1, le_trans := string.linear_order._proof_2, lt_iff_le_not_le := string.linear_order._proof_3, le_antisymm := string.linear_order._proof_4, le_total := string.linear_order._proof_5, decidable_le := string.decidable_le, decidable_eq := λ (a b : string), string.has_decidable_eq a b, decidable_lt := λ (a b : string), string.decidable_lt a b, max := max_default (λ (a b : string), string.decidable_le a b), max_def := string.linear_order._proof_10, min := min_default (λ (a b : string), string.decidable_le a b), min_def := string.linear_order._proof_11}