From 5655750e12d3459c1237588f8dec3fc883a966b7 Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Mon, 28 Jun 2021 16:06:19 +0100 Subject: 1. Thm/def statement display. 2. Syntax + computation proof. --- mltt/core/MLTT.thy | 12 ++++++------ 1 file changed, 6 insertions(+), 6 deletions(-) (limited to 'mltt/core/MLTT.thy') diff --git a/mltt/core/MLTT.thy b/mltt/core/MLTT.thy index 29c7248..96cbe96 100644 --- a/mltt/core/MLTT.thy +++ b/mltt/core/MLTT.thy @@ -63,15 +63,15 @@ typedecl lvl axiomatization O :: \lvl\ and S :: \lvl \ lvl\ and - lt :: \lvl \ lvl \ prop\ (infix "<" 900) + lt :: \lvl \ lvl \ prop\ (infix "<\<^sub>U" 900) where - O_min: "O < S i" and - lt_S: "i < S i" and - lt_trans: "i < j \ j < k \ i < k" + O_min: "O <\<^sub>U S i" and + lt_S: "i <\<^sub>U S i" and + lt_trans: "i <\<^sub>U j \ j <\<^sub>U k \ i <\<^sub>U k" axiomatization U :: \lvl \ o\ where - Ui_in_Uj: "i < j \ U i: U j" and - U_cumul: "A: U i \ i < j \ A: U j" + Ui_in_Uj: "i <\<^sub>U j \ U i: U j" and + U_cumul: "A: U i \ i <\<^sub>U j \ A: U j" lemma Ui_in_USi: "U i: U (S i)" -- cgit v1.2.3