src/Sequents/S43.thy
changeset 52143 36ffe23b25f8
parent 51309 473303ef6e34
child 54742 7a86358a3c0b
--- a/src/Sequents/S43.thy	Sat May 25 15:00:53 2013 +0200
+++ b/src/Sequents/S43.thy	Sat May 25 15:37:53 2013 +0200
@@ -21,7 +21,7 @@
     val tr  = seq_tr;
     fun s43pi_tr [s1, s2, s3, s4, s5, s6] =
       Const (@{const_syntax S43pi}, dummyT) $ tr s1 $ tr s2 $ tr s3 $ tr s4 $ tr s5 $ tr s6;
-  in [(@{syntax_const "_S43pi"}, s43pi_tr)] end
+  in [(@{syntax_const "_S43pi"}, K s43pi_tr)] end
 *}
 
 print_translation {*
@@ -29,7 +29,7 @@
   val tr' = seq_tr';
   fun s43pi_tr' [s1, s2, s3, s4, s5, s6] =
     Const(@{syntax_const "_S43pi"}, dummyT) $ tr' s1 $ tr' s2 $ tr' s3 $ tr' s4 $ tr' s5 $ tr' s6;
-in [(@{const_syntax S43pi}, s43pi_tr')] end
+in [(@{const_syntax S43pi}, K s43pi_tr')] end
 *}
 
 axiomatization where