summaryrefslogtreecommitdiff
path: root/Everything.agda
diff options
context:
space:
mode:
Diffstat (limited to 'Everything.agda')
-rw-r--r--Everything.agda20
1 files changed, 20 insertions, 0 deletions
diff --git a/Everything.agda b/Everything.agda
new file mode 100644
index 0000000..5f0a173
--- /dev/null
+++ b/Everything.agda
@@ -0,0 +1,20 @@
+------------------------------------------------------------------------
+-- Agda Helium
+--
+-- All library modules, along with short descriptions.
+------------------------------------------------------------------------
+
+{-# OPTIONS --safe --without-K #-}
+
+module Everything where
+
+-- Definition of types and operations used by the Armv8-M pseudocode.
+import Helium.Data.Pseudocode
+
+-- Definitions of a subset of Armv8-M instructions.
+import Helium.Instructions
+
+import Helium.Semantics.Denotational
+
+-- Base definitions for the denotational semantics.
+import Helium.Semantics.Denotational.Core