Regular languages #
theorem
Language.IsRegular.iff_cslib_dfa
{Symbol : Type u_1}
{l : Language Symbol}
:
l.IsRegular ↔ ∃ (State : Type) (_ : Finite State) (dfa : Cslib.Automata.DA.FinAcc State Symbol),
Cslib.Automata.Acceptor.language dfa = l
A characterization of Language.IsRegular using Cslib.DA
theorem
Language.IsRegular.iff_cslib_nfa
{Symbol : Type u_1}
{l : Language Symbol}
:
l.IsRegular ↔ ∃ (State : Type) (_ : Finite State) (nfa : Cslib.Automata.NA.FinAcc State Symbol),
Cslib.Automata.Acceptor.language nfa = l
A characterization of Language.IsRegular using Cslib.NA