removed split_all_tac from claset() globally within IOA
authoroheimb
Tue, 21 Apr 1998 17:21:42 +0200
changeset 4815 b8a32ef742d9
parent 4814 0277a026f99d
child 4816 64f075872f69
removed split_all_tac from claset() globally within IOA
src/HOLCF/IOA/NTP/Correctness.ML
src/HOLCF/IOA/meta_theory/TLS.ML
src/HOLCF/IOA/meta_theory/Traces.ML
--- a/src/HOLCF/IOA/NTP/Correctness.ML	Tue Apr 21 17:20:54 1998 +0200
+++ b/src/HOLCF/IOA/NTP/Correctness.ML	Tue Apr 21 17:21:42 1998 +0200
@@ -6,6 +6,8 @@
 The main correctness proof: Impl implements Spec
 *)
 
+(* repeated from Traces.ML *)
+claset_ref() := claset() delSWrapper "split_all_tac";
 
 
 val hom_ioas = [Spec.ioa_def, Spec.trans_def,
--- a/src/HOLCF/IOA/meta_theory/TLS.ML	Tue Apr 21 17:20:54 1998 +0200
+++ b/src/HOLCF/IOA/meta_theory/TLS.ML	Tue Apr 21 17:21:42 1998 +0200
@@ -6,6 +6,12 @@
 Temporal Logic of Steps -- tailored for I/O automata
 *)   
 
+(* global changes to simpset() and claset(), repeated from Traces.ML *)
+Delsimps (ex_simps @ all_simps);
+Delsimps [split_paired_Ex];
+Addsimps [Let_def];
+claset_ref() := claset() delSWrapper "split_all_tac";
+
 
 (* ---------------------------------------------------------------- *)
 (*                                 ex2seqC                          *)
--- a/src/HOLCF/IOA/meta_theory/Traces.ML	Tue Apr 21 17:20:54 1998 +0200
+++ b/src/HOLCF/IOA/meta_theory/Traces.ML	Tue Apr 21 17:21:42 1998 +0200
@@ -6,8 +6,11 @@
 Theorems about Executions and Traces of I/O automata in HOLCF.
 *)   
 
+(* global changes to simpset() and claset(), see also TLS.ML *)
 Delsimps (ex_simps @ all_simps);
 Delsimps [split_paired_Ex];
+Addsimps [Let_def];
+claset_ref() := claset() delSWrapper "split_all_tac";
 
 val exec_rws = [executions_def,is_exec_frag_def];