Translation of Nondeterministic Automata for finite strings into Deterministic Automata #
This file implements the standard subset construction.
def
Cslib.Automata.NA.FinAcc.toDAFinAcc
{State : Type u_1}
{Symbol : Type u_2}
(a : FinAcc State Symbol)
:
Converts an NA.FinAcc into a DA.FinAcc using the subset construction.
Instances For
theorem
Cslib.Automata.NA.FinAcc.toDAFinAcc_language_eq
{State : Type u_1}
{Symbol : Type u_2}
{na : FinAcc State Symbol}
:
The DA constructed from an NA has the same language.