diff -r be8c0e039a5e -r bc936d3d8b45 src/Cube/Cube.thy --- a/src/Cube/Cube.thy Sun Aug 25 15:02:19 2024 +0200 +++ b/src/Cube/Cube.thy Sun Aug 25 15:07:22 2024 +0200 @@ -39,6 +39,13 @@ "_Lam" :: "[idt, term, term] \ term" ("(3\<^bold>\_:_./ _)" [0, 0, 0] 10) "_Pi" :: "[idt, term, term] \ term" ("(3\_:_./ _)" [0, 0] 10) "_arrow" :: "[term, term] \ term" (infixr "\" 10) +syntax_consts + "_Trueprop" \ Trueprop and + "_MT_context" \ MT_context and + "_Context" \ Context and + "_Has_type" \ Has_type and + "_Lam" \ Abs and + "_Pi" "_arrow" \ Prod translations "_Trueprop(G, t)" \ "CONST Trueprop(G, t)" ("prop") "x:X" \ ("prop") "\ x:X" @@ -52,13 +59,6 @@ [(\<^const_syntax>\Prod\, fn _ => Syntax_Trans.dependent_tr' (\<^syntax_const>\_Pi\, \<^syntax_const>\_arrow\))] \ -syntax_consts - "_Trueprop" \ Trueprop and - "_MT_context" \ MT_context and - "_Context" \ Context and - "_Has_type" \ Has_type and - "_Lam" \ Abs and - "_Pi" "_arrow" \ Prod axiomatization where s_b: "*: \" and