src/ZF/Coind/Static.thy
changeset 12610 8b9845807f77
parent 12595 0480d02221b8
child 16417 9bc16273c2d4
--- a/src/ZF/Coind/Static.thy	Sat Dec 29 18:35:27 2001 +0100
+++ b/src/ZF/Coind/Static.thy	Sat Dec 29 18:36:12 2001 +0100
@@ -54,11 +54,12 @@
   type_intros te_appI Exp.intros Ty.intros
 
 
-inductive_cases elab_constE [elim!]: "<te,e_const(c),t> \<in> ElabRel"
-inductive_cases elab_varE   [elim!]: "<te,e_var(x),t> \<in> ElabRel"
-inductive_cases elab_fnE    [elim]:  "<te,e_fn(x,e),t> \<in> ElabRel"
-inductive_cases elab_fixE   [elim!]: "<te,e_fix(f,x,e),t> \<in> ElabRel"
-inductive_cases elab_appE   [elim]:  "<te,e_app(e1,e2),t> \<in> ElabRel"
+inductive_cases
+    elab_constE [elim!]: "<te,e_const(c),t> \<in> ElabRel"
+  and elab_varE [elim!]: "<te,e_var(x),t> \<in> ElabRel"
+  and elab_fnE [elim]:   "<te,e_fn(x,e),t> \<in> ElabRel"
+  and elab_fixE [elim!]: "<te,e_fix(f,x,e),t> \<in> ElabRel"
+  and elab_appE [elim]:  "<te,e_app(e1,e2),t> \<in> ElabRel"
 
 declare ElabRel.dom_subset [THEN subsetD, dest]