print_translation: does not handle _idtdummy;
authorwenzelm
Fri, 07 Oct 2005 22:59:18 +0200
changeset 17781 32bb237158a5
parent 17780 274eaa114c6d
child 17782 b3846df9d643
print_translation: does not handle _idtdummy;
src/CCL/Term.thy
src/HOL/Hoare/Hoare.thy
src/HOL/Hoare/HoareAbort.thy
src/HOL/Hoare/Separation.thy
src/HOL/Library/FuncSet.thy
--- a/src/CCL/Term.thy	Fri Oct 07 22:59:17 2005 +0200
+++ b/src/CCL/Term.thy	Fri Oct 07 22:59:18 2005 +0200
@@ -56,6 +56,7 @@
 ML {*
 (** Quantifier translations: variable binding **)
 
+(* FIXME does not handle "_idtdummy" *)
 (* FIXME should use Syntax.mark_bound(T), Syntax.variant_abs' *)
 
 fun let_tr [Free(id,T),a,b] = Const("let",dummyT) $ a $ absfree(id,T,b);
--- a/src/HOL/Hoare/Hoare.thy	Fri Oct 07 22:59:17 2005 +0200
+++ b/src/HOL/Hoare/Hoare.thy	Fri Oct 07 22:59:18 2005 +0200
@@ -101,7 +101,7 @@
   | com_tr t _ = t (* if t is just a Free/Var *)
 *}
 
-(* triple_tr *)
+(* triple_tr *)    (* FIXME does not handle "_idtdummy" *)
 ML{*
 local
 
--- a/src/HOL/Hoare/HoareAbort.thy	Fri Oct 07 22:59:17 2005 +0200
+++ b/src/HOL/Hoare/HoareAbort.thy	Fri Oct 07 22:59:18 2005 +0200
@@ -103,7 +103,7 @@
   | com_tr t _ = t (* if t is just a Free/Var *)
 *}
 
-(* triple_tr *)
+(* triple_tr *)  (* FIXME does not handle "_idtdummy" *)
 ML{*
 local
 
--- a/src/HOL/Hoare/Separation.thy	Fri Oct 07 22:59:17 2005 +0200
+++ b/src/HOL/Hoare/Separation.thy	Fri Oct 07 22:59:18 2005 +0200
@@ -55,6 +55,7 @@
  "@star" :: "bool \<Rightarrow> bool \<Rightarrow> bool" (infixl "**" 60)
  "@wand" :: "bool \<Rightarrow> bool \<Rightarrow> bool" (infixl "-*" 60)
 
+(* FIXME does not handle "_idtdummy" *)
 ML{*
 (* free_tr takes care of free vars in the scope of sep. logic connectives:
    they are implicitly applied to the heap *)
--- a/src/HOL/Library/FuncSet.thy	Fri Oct 07 22:59:17 2005 +0200
+++ b/src/HOL/Library/FuncSet.thy	Fri Oct 07 22:59:18 2005 +0200
@@ -35,7 +35,7 @@
 
 translations
   "PI x:A. B" => "Pi A (%x. B)"
-  "A -> B" => "Pi A (_K B)"
+  "A -> B" => "Pi A (%_. B)"
   "%x:A. f" == "restrict (%x. f) A"
 
 constdefs