src/HOL/IOA/meta_theory/Asig.ML
changeset 3077 750b766645b8
parent 3076 3e8d80cdd3e7
child 3078 984866a8f905
--- a/src/HOL/IOA/meta_theory/Asig.ML	Wed Apr 30 11:53:30 1997 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,19 +0,0 @@
-(*  Title:      HOL/IOA/meta_theory/Asig.ML
-    ID:         $Id$
-    Author:     Tobias Nipkow & Konrad Slind
-    Copyright   1994  TU Muenchen
-
-Action signatures
-*)
-
-open Asig;
-
-val asig_projections = [asig_inputs_def, asig_outputs_def, asig_internals_def];
-
-goal Asig.thy "!!a.[| a~:internals(S) ;a~:externals(S)|] ==> a~:actions(S)";
-by (asm_full_simp_tac (!simpset addsimps [externals_def,actions_def]) 1);
-qed"int_and_ext_is_act";
-
-goal Asig.thy "!!a.[|a:externals(S)|] ==> a:actions(S)";
-by (asm_full_simp_tac (!simpset addsimps [externals_def,actions_def]) 1);
-qed"ext_is_act";