Skip to content

Commit 1d6ac29

Browse files
committed
Do not register pre-datatype MRBNFs
ISSUES FIXED: #121
1 parent 3f17a44 commit 1d6ac29

File tree

4 files changed

+7
-3
lines changed

4 files changed

+7
-3
lines changed

Tools/mrbnf_comp.ML

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1431,7 +1431,6 @@ fun seal_mrbnf qualify (unfold_set : unfold_set) b force_out_of_line Ds all_Ds m
14311431
|> map (fn (b, def) => ((b, []), [([def], [])]))
14321432
val (noted, lthy'') = lthy'
14331433
|> Local_Theory.notes notes
1434-
||> (if repTA = TA then I else register_mrbnf_raw (fst (dest_Type TA)) mrbnf'')
14351434
in
14361435
((morph_mrbnf (substitute_noted_thm noted) mrbnf'', the info_opt, (all_Ds, absT_info)), lthy'')
14371436
end;

case_studies/Pi_Calculus/Commitment.thy

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -84,7 +84,7 @@ abbreviation "bvars \<equiv> bns"
8484
abbreviation "fvars \<equiv> fns"
8585

8686
lemma bns_bound: "|bns \<alpha>| <o |UNIV::'a::var set|"
87-
by (cases \<alpha>) (auto simp: emp_bound infinite_UNIV)
87+
by (cases \<alpha>) auto
8888

8989
local_setup \<open>Binder_Sugar.register_binder_sugar "Commitment.commit" {
9090
ctors = [
@@ -111,7 +111,7 @@ local_setup \<open>Binder_Sugar.register_binder_sugar "Commitment.commit" {
111111
pset_ctors = [],
112112
strong_induct = NONE,
113113
inject = @{thms commit.inject},
114-
mrbnf = the (MRBNF_Def.mrbnf_of @{context} "Commitment.commit_pre"),
114+
mrbnf = #mrbnf (the (Binder_Sugar.binder_sugar_of @{context} @{type_name commit})),
115115
set_simpss = [],
116116
subst_simps = NONE,
117117
IImsupp_Diffs = NONE,

operations/Composition.thy

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -75,6 +75,9 @@ let
7575
val ((mrbnf2, _, (Ds, info)), lthy) = MRBNF_Comp.seal_mrbnf I (snd accum) (Binding.name (name2 ^ "_pre")) true (fst tys2) [] mrbnf2 NONE lthy
7676
val _ = @{print} "seal2"
7777
78+
val lthy = MRBNF_Def.register_mrbnf_raw "Composition.T1_pre" mrbnf1 lthy
79+
val lthy = MRBNF_Def.register_mrbnf_raw "Composition.T2_pre" mrbnf2 lthy
80+
7881
(* Step 3: Register the pre-MRBNF as a BNF in its live variables *)
7982
val (bnf1, lthy) = MRBNF_Def.register_mrbnf_as_bnf mrbnf1 lthy
8083
val (bnf2, lthy) = MRBNF_Def.register_mrbnf_as_bnf mrbnf2 lthy

operations/Greatest_Fixpoint.thy

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -46,6 +46,8 @@ local_setup \<open>fn lthy =>
4646
val ((mrbnf1, _, (Ds, info)), lthy) = MRBNF_Comp.seal_mrbnf I (snd accum) (Binding.name (name1 ^ "_pre")) true (fst tys1) [] mrbnf1 NONE lthy
4747
val _ = @{print} "seal"
4848
49+
val lthy = MRBNF_Def.register_mrbnf_raw "Greatest_Fixpoint.term_pre" mrbnf1 lthy;
50+
4951
(* Step 3: Register the pre-MRBNF as a BNF in its live variables *)
5052
val (bnf1, lthy) = MRBNF_Def.register_mrbnf_as_bnf mrbnf1 lthy
5153
val _ = @{print} "register"

0 commit comments

Comments
 (0)