Type Definition validus::vstr::vstr

source ·
pub type vstr<Rule> = VStr<Rule>;
Expand description

Create a validated string slice.

See VStr for more information.

Trait Implementations§

source§

impl<R: ValidateString> ToOwned for vstr<R>

§

type Owned = Box<VStr<R>, Global>

The resulting type after obtaining ownership.
source§

fn to_owned(&self) -> Self::Owned

Creates owned data from borrowed data, usually by cloning. Read more
1.63.0 · source§

fn clone_into(&self, target: &mut Self::Owned)

Uses borrowed data to replace owned data, usually by cloning. Read more
source§

impl<'a: 'b, 'b, R: ValidateString> TryFrom<&'a VCow<'b, R>> for &'b vstr<R>

§

type Error = <R as ValidateString>::Error

The type returned in the event of a conversion error.
source§

fn try_from(cow: &'a VCow<'b, R>) -> Result<Self, Self::Error>

Performs the conversion.