src/HOL/Bali/State.thy
changeset 80768 c7723cc15de8
parent 77645 7edbb16bc60f
child 80914 d97fdabd9e2b
--- a/src/HOL/Bali/State.thy	Sun Aug 25 20:54:20 2024 +0200
+++ b/src/HOL/Bali/State.thy	Sun Aug 25 21:10:01 2024 +0200
@@ -135,6 +135,10 @@
   Heap  :: "loc   \<Rightarrow> oref"
   Stat  :: "qtname \<Rightarrow> oref"
 
+syntax_consts
+  Heap == Inl and
+  Stat == Inr
+
 translations
   "Heap" => "CONST Inl"
   "Stat" => "CONST Inr"