From e513fc2958133e3a00c06ebcd1214741843acf08 Mon Sep 17 00:00:00 2001 From: Josh Chen Date: Wed, 3 Jun 2020 13:09:30 +0200 Subject: 1. Type information context data 2. Small reformulations of rules 3. Bool --- spartan/core/Spartan.thy | 5 +++-- 1 file changed, 3 insertions(+), 2 deletions(-) (limited to 'spartan/core/Spartan.thy') 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 \ A: U (S i)" by (erule U_cumulative, rule lt_S) @@ -154,6 +154,7 @@ named_theorems typechk ML_file \lib/lib.ML\ ML_file \lib/goals.ML\ ML_file \lib/focus.ML\ +ML_file \lib/types.ML\ section \Congruence automation\ @@ -322,7 +323,7 @@ lemma lift_universe_codomain: shows "f: A \ 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 \Function composition\ -- cgit v1.2.3