Theory Simple_Network_Language_Export_Code
section ‹Assembling the Model Checker and Generating Code›
text ‹
We assemble the model checker:
▪ A parser is added to parse JSON files
▪ The resulting JSON data is validated and converted to the simple networks language
▪ The verified model checker is run on this input, and the output is printed
▪ The verified part includes a ``renaming'' step to normalize identifiers in the input
Then the code is exported:
▪ We add some logging utilities (via code printings)
▪ Code generation is setup
▪ We export this to SML via reflection
▪ And test it on a few small examples
›
theory Simple_Network_Language_Export_Code
imports
Munta_Model_Checker.JSON_Parsing
Munta_Model_Checker.Simple_Network_Language_Renaming
Munta_Model_Checker.Simple_Network_Language_Deadlock_Checking
Shortest_SCC_Paths
Munta_Base.Error_List_Monad
begin