--- a/src/HOL/MicroJava/Comp/TranslCompTp.thy Sat Oct 17 01:05:59 2009 +0200
+++ b/src/HOL/MicroJava/Comp/TranslCompTp.thy Sat Oct 17 14:43:18 2009 +0200
@@ -1,5 +1,4 @@
(* Title: HOL/MicroJava/Comp/TranslCompTp.thy
- ID: $Id$
Author: Martin Strecker
*)
@@ -43,8 +42,8 @@
(**********************************************************************)
syntax
- mt_of :: "method_type \<times> state_type \<Rightarrow> method_type"
- sttp_of :: "method_type \<times> state_type \<Rightarrow> state_type"
+ mt_of :: "method_type \<times> state_type \<Rightarrow> method_type"
+ sttp_of :: "method_type \<times> state_type \<Rightarrow> state_type"
translations
"mt_of" => "fst"