src/Pure/Syntax/syn_trans.ML
changeset 15421 fcf747c0b6b8
parent 14981 e73f8140af78
child 15531 08c8dad8e399
--- a/src/Pure/Syntax/syn_trans.ML	Fri Dec 17 12:43:12 2004 +0100
+++ b/src/Pure/Syntax/syn_trans.ML	Sat Dec 18 17:10:49 2004 +0100
@@ -132,9 +132,14 @@
 (* meta implication *)
 
 fun bigimpl_ast_tr (*"_bigimpl"*) [asms, concl] =
+      Ast.fold_ast_p "==>" (Ast.unfold_ast2 "_asms" "_asm" asms, concl)
+  | bigimpl_ast_tr (*"_bigimpl"*) asts = raise Ast.AST ("bigimpl_ast_tr", asts);
+
+(*
+fun bigimpl_ast_tr (*"_bigimpl"*) [asms, concl] =
       Ast.fold_ast_p "==>" (Ast.unfold_ast "_asms" asms, concl)
   | bigimpl_ast_tr (*"_bigimpl"*) asts = raise Ast.AST ("bigimpl_ast_tr", asts);
-
+*)
 
 (* type reflection *)
 
@@ -348,9 +353,18 @@
   else
     (case Ast.unfold_ast_p "==>" (Ast.Appl (Ast.Constant "==>" :: asts)) of
       (asms as _ :: _ :: _, concl)
+        => Ast.Appl [Ast.Constant "_bigimpl", Ast.fold_ast2 "_asms" "_asm" asms, concl]
+    | _ => raise Match);
+
+(*
+fun impl_ast_tr' (*"==>"*) asts =
+  if TypeExt.no_brackets () then raise Match
+  else
+    (case Ast.unfold_ast_p "==>" (Ast.Appl (Ast.Constant "==>" :: asts)) of
+      (asms as _ :: _ :: _, concl)
         => Ast.Appl [Ast.Constant "_bigimpl", Ast.fold_ast "_asms" asms, concl]
     | _ => raise Match);
-
+*)
 
 (* meta conjunction *)