Theory Interpreter
text‹
Interpreter.thy defines a simple programming language over interval-valued variables and executable
semantics (interpreter) for that language. We then prove that the interpretation of interval terms
is a sound over-approximation of a real-valued semantics of the same language.
Our language is a version of first order dynamic logic-style regular programs.
We use a finite identifier space for compatibility with Differential-Dynamic-Logic, where identifier
finiteness is required to treat program states as Banach spaces to enable differentiation.
›
theory Interpreter
imports
Complex_Main
Finite_String
Interval_Word32
begin
section‹Syntax›
text‹Our term language supports variables, polynomial arithmetic, and extrema. This choice was made
based on the needs of the original paper and could be extended if necessary.›