aboutsummaryrefslogtreecommitdiff
path: root/spartan/core/Spartan.thy
diff options
context:
space:
mode:
authorJosh Chen2020-06-03 13:10:35 +0200
committerJosh Chen2020-06-03 13:10:35 +0200
commit9050b7414021db31b23a034567ebc6da3f6c5f67 (patch)
tree2f5928e275c3e8ae7d99fef65e7fddf31f11d2f6 /spartan/core/Spartan.thy
parentccc26cf8073071698f333107fd7443a6af7fb3de (diff)
parent515c142828e66dcb1c273e53816ef8b6e1bb3f01 (diff)
Merge branch 'dev'
Diffstat (limited to 'spartan/core/Spartan.thy')
-rw-r--r--spartan/core/Spartan.thy5
1 files changed, 3 insertions, 2 deletions
diff --git a/spartan/core/Spartan.thy b/spartan/core/Spartan.thy
index 9a6d884..55eb657 100644
--- a/spartan/core/Spartan.thy
+++ b/spartan/core/Spartan.thy
@@ -56,7 +56,7 @@ lemma U_in_U:
"U i: U (S i)"
by (rule U_hierarchy, rule lt_S)
-lemma lift_universe:
+lemma lift_U:
"A: U i \<Longrightarrow> A: U (S i)"
by (erule U_cumulative, rule lt_S)
@@ -154,6 +154,7 @@ named_theorems typechk
ML_file \<open>lib/lib.ML\<close>
ML_file \<open>lib/goals.ML\<close>
ML_file \<open>lib/focus.ML\<close>
+ML_file \<open>lib/types.ML\<close>
section \<open>Congruence automation\<close>
@@ -322,7 +323,7 @@ lemma lift_universe_codomain:
shows "f: A \<rightarrow> U (S j)"
apply (sub eta_exp)
apply known
- apply (Pure.rule intros; rule lift_universe)
+ apply (Pure.rule intros; rule lift_U)
done
subsection \<open>Function composition\<close>