Skip to content

Commit ca41e2e

Browse files
committed
Adapt operations theory
1 parent 34e2740 commit ca41e2e

File tree

2 files changed

+1
-8
lines changed

2 files changed

+1
-8
lines changed

operations/BMV_Fixpoint.thy

Lines changed: 1 addition & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -10,8 +10,6 @@ type_synonym ('tv, 'v, 'btv, 'bv, 'c, 'd) FTerm_pre' =
1010
+ 'bv * 'tv FType * 'c \<comment>\<open>Lam x::'v \<open>'tv FType\<close> t::\<open>('tv, 'v) FTerm\<close> binds x in t\<close>
1111
+ 'btv * 'c \<comment>\<open>TyLam a::'tv t::\<open>('tv, 'v) FTerm\<close> binds a in t\<close>"
1212

13-
ML_file \<open>../Tools/mrsbnf_comp.ML\<close>
14-
1513
local_setup \<open>fn lthy =>
1614
let
1715
val T = @{typ "('tv, 'v, 'btv, 'bv, 'c, 'd) FTerm_pre'"};
@@ -1531,8 +1529,6 @@ lemma FTerm_subst:
15311529
apply (rule refl)
15321530
done
15331531

1534-
ML_file \<open>../Tools/tvsubst.ML\<close>
1535-
15361532
local_setup \<open>fn lthy =>
15371533
let
15381534
@@ -1551,7 +1547,7 @@ val x = TVSubst.create_tvsubst_of_mrsbnf
15511547
eta_compl_free = fn ctxt => etac ctxt @{thm eta_compl_free} 1,
15521548
eta_inj = fn ctxt => etac ctxt @{thm eta_inj} 1,
15531549
eta_natural = fn ctxt => HEADGOAL (rtac ctxt @{thm eta_natural} THEN_ALL_NEW assume_tac ctxt),
1554-
eta_Sb = fn ctxt => HEADGOAL (etac ctxt @{thm eta_Sb[rotated -1]} THEN_ALL_NEW assume_tac ctxt)
1550+
eta_Sb = fn ctxt => HEADGOAL (etac ctxt @{thm eta_Sb[unfolded FTerm_pre.Map_map, rotated -1]} THEN_ALL_NEW assume_tac ctxt)
15551551
}
15561552
}] "BMV_Fixpoint.QREC_fixed_FTerm" lthy
15571553

operations/BMV_Monad.thy

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1,8 +1,5 @@
11
theory BMV_Monad
22
imports "Binders.MRBNF_Recursor"
3-
keywords "print_pbmv_monads" :: diag and
4-
"pbmv_monad" :: thy_goal and
5-
"mrsbnf" :: thy_goal
63
begin
74

85
declare [[mrbnf_internals]]

0 commit comments

Comments
 (0)