src/Cube/Cube.thy
changeset 80754 701912f5645a
parent 69593 3dda49e08b9d
child 80761 bc936d3d8b45
--- a/src/Cube/Cube.thy	Fri Aug 23 22:47:51 2024 +0200
+++ b/src/Cube/Cube.thy	Fri Aug 23 23:14:39 2024 +0200
@@ -52,6 +52,13 @@
   [(\<^const_syntax>\<open>Prod\<close>,
     fn _ => Syntax_Trans.dependent_tr' (\<^syntax_const>\<open>_Pi\<close>, \<^syntax_const>\<open>_arrow\<close>))]
 \<close>
+syntax_consts
+  "_Trueprop" \<rightleftharpoons> Trueprop and
+  "_MT_context" \<rightleftharpoons> MT_context and
+  "_Context" \<rightleftharpoons> Context and
+  "_Has_type" \<rightleftharpoons> Has_type and
+  "_Lam" \<rightleftharpoons> Abs and
+  "_Pi" "_arrow" \<rightleftharpoons> Prod
 
 axiomatization where
   s_b: "*: \<box>"  and