src/HOL/Bali/AxSem.thy
changeset 61424 c3658c18b7bc
parent 60754 02924903a6fd
child 61989 ba8c284d4725
--- a/src/HOL/Bali/AxSem.thy	Tue Oct 13 09:21:14 2015 +0200
+++ b/src/HOL/Bali/AxSem.thy	Tue Oct 13 09:21:15 2015 +0200
@@ -969,7 +969,7 @@
 done
 
 lemma ax_methods_spec: 
-"\<lbrakk>G,(A::'a triple set)|\<turnstile>split f ` ms; (C,sig) \<in> ms\<rbrakk>\<Longrightarrow> G,A\<turnstile>((f C sig)::'a triple)"
+"\<lbrakk>G,(A::'a triple set)|\<turnstile>case_prod f ` ms; (C,sig) \<in> ms\<rbrakk>\<Longrightarrow> G,A\<turnstile>((f C sig)::'a triple)"
 apply (erule ax_derivs.weaken)
 apply (force del: image_eqI intro: rev_image_eqI)
 done
@@ -977,7 +977,7 @@
 (* this version is used to avoid using the cut rule *)
 lemma ax_finite_pointwise_lemma [rule_format]: "\<lbrakk>F \<subseteq> ms; finite ms\<rbrakk> \<Longrightarrow>  
   ((\<forall>(C,sig)\<in>F. G,(A::'a triple set)\<turnstile>(f C sig::'a triple)) \<longrightarrow> (\<forall>(C,sig)\<in>ms. G,A\<turnstile>(g C sig::'a triple))) \<longrightarrow>  
-      G,A|\<turnstile>split f ` F \<longrightarrow> G,A|\<turnstile>split g ` F"
+      G,A|\<turnstile>case_prod f ` F \<longrightarrow> G,A|\<turnstile>case_prod g ` F"
 apply (frule (1) finite_subset)
 apply (erule rev_mp)
 apply (erule thin_rl)