--- a/src/HOL/Bali/Basis.thy Wed Apr 11 08:28:13 2007 +0200
+++ b/src/HOL/Bali/Basis.thy Wed Apr 11 08:28:14 2007 +0200
@@ -246,7 +246,7 @@
"the_In1r" == "the_Inr \<circ> the_In1"
ML {*
-fun sum3_instantiate thm = map (fn s => simplify(simpset()delsimps[not_None_eq])
+fun sum3_instantiate thm = map (fn s => simplify(simpset()delsimps[@{thm not_None_eq}])
(read_instantiate [("t","In"^s^" ?x")] thm)) ["1l","2","3","1r"]
*}
(* e.g. lemmas is_stmt_rews = is_stmt_def [of "In1l x", simplified] *)
--- a/src/HOL/List.thy Wed Apr 11 08:28:13 2007 +0200
+++ b/src/HOL/List.thy Wed Apr 11 08:28:14 2007 +0200
@@ -299,8 +299,6 @@
ML_setup {*
local
-val neq_if_length_neq = thm "neq_if_length_neq";
-
fun len (Const("List.list.Nil",_)) acc = acc
| len (Const("List.list.Cons",_) $ _ $ xs) (ts,n) = len xs (ts,n+1)
| len (Const("List.op @",_) $ xs $ ys) acc = len xs (len ys acc)
@@ -308,8 +306,6 @@
| len (Const("List.map",_) $ _ $ xs) acc = len xs acc
| len t (ts,n) = (t::ts,n);
-val list_ss = simpset_of(the_context());
-
fun list_eq ss (Const(_,eqT) $ lhs $ rhs) =
let
val (ls,m) = len lhs ([],0) and (rs,n) = len rhs ([],0);
@@ -320,8 +316,8 @@
val eq_len = HOLogic.mk_eq (size $ lhs, size $ rhs);
val neq_len = HOLogic.mk_Trueprop (HOLogic.Not $ eq_len);
val thm = Goal.prove (Simplifier.the_context ss) [] [] neq_len
- (K (simp_tac (Simplifier.inherit_context ss list_ss) 1));
- in SOME (thm RS neq_if_length_neq) end
+ (K (simp_tac (Simplifier.inherit_context ss @{simpset}) 1));
+ in SOME (thm RS @{thm neq_if_length_neq}) end
in
if m < n andalso gen_submultiset (op aconv) (ls,rs) orelse
n < m andalso gen_submultiset (op aconv) (rs,ls)
@@ -331,7 +327,7 @@
in
val list_neq_simproc =
- Simplifier.simproc (the_context ()) "list_neq" ["(xs::'a list) = ys"] (K list_eq);
+ Simplifier.simproc @{theory} "list_neq" ["(xs::'a list) = ys"] (K list_eq);
end;
@@ -441,12 +437,6 @@
ML_setup {*
local
-val append_assoc = thm "append_assoc";
-val append_Nil = thm "append_Nil";
-val append_Cons = thm "append_Cons";
-val append1_eq_conv = thm "append1_eq_conv";
-val append_same_eq = thm "append_same_eq";
-
fun last (cons as Const("List.list.Cons",_) $ _ $ xs) =
(case xs of Const("List.list.Nil",_) => cons | _ => last xs)
| last (Const("List.op @",_) $ _ $ ys) = last ys
@@ -460,7 +450,8 @@
| butlast ((app as Const("List.op @",_) $ xs) $ ys) = app $ butlast ys
| butlast xs = Const("List.list.Nil",fastype_of xs);
-val rearr_ss = HOL_basic_ss addsimps [append_assoc, append_Nil, append_Cons];
+val rearr_ss = HOL_basic_ss addsimps [@{thm append_assoc},
+ @{thm append_Nil}, @{thm append_Cons}];
fun list_eq ss (F as (eq as Const(_,eqT)) $ lhs $ rhs) =
let
@@ -478,15 +469,15 @@
in SOME ((conv RS (thm RS trans)) RS eq_reflection) end;
in
- if list1 lastl andalso list1 lastr then rearr append1_eq_conv
- else if lastl aconv lastr then rearr append_same_eq
+ if list1 lastl andalso list1 lastr then rearr @{thm append1_eq_conv}
+ else if lastl aconv lastr then rearr @{thm append_same_eq}
else NONE
end;
in
val list_eq_simproc =
- Simplifier.simproc (the_context ()) "list_eq" ["(xs::'a list) = ys"] (K list_eq);
+ Simplifier.simproc @{theory} "list_eq" ["(xs::'a list) = ys"] (K list_eq);
end;
--- a/src/HOL/MicroJava/J/WellForm.thy Wed Apr 11 08:28:13 2007 +0200
+++ b/src/HOL/MicroJava/J/WellForm.thy Wed Apr 11 08:28:14 2007 +0200
@@ -505,7 +505,7 @@
apply( rotate_tac -1, frule ssubst, erule_tac [2] asm_rl)
prefer 2
apply( rotate_tac -1, frule ssubst, erule_tac [2] asm_rl)
-apply( tactic "asm_full_simp_tac (HOL_ss addsimps [not_None_eq RS sym]) 1")
+apply( tactic "asm_full_simp_tac (HOL_ss addsimps [@{thm not_None_eq} RS sym]) 1")
apply( simp_all (no_asm_simp) del: split_paired_Ex)
apply( frule (1) class_wf)
apply( simp (no_asm_simp) only: split_tupled_all)