diff -r 33f81e980c93 -r 7c8d1c7c876d src/HOL/ex/Antiquote.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/ex/Antiquote.thy Mon Aug 24 18:17:25 1998 +0200 @@ -0,0 +1,27 @@ +(* Title: HOL/ex/Antiquote.thy + ID: $Id$ + Author: Markus Wenzel, TU Muenchen + +Simple quote / antiquote example. +*) + +Antiquote = Arith + + +syntax + "_Expr" :: "'a => 'a" ("EXPR _" [1000] 999) + +constdefs + var :: "'a => ('a => nat) => nat" ("VAR _" [1000] 999) + "var x env == env x" + + Expr :: "'a => 'a" + (*"(('a => nat) => nat) => (('a => nat) => nat)"*) + "Expr == (%x. x)" + +end + + +ML + +val parse_translation = [Syntax.quote_antiquote_tr "_Expr" "var" "Expr"]; +val print_translation = [Syntax.quote_antiquote_tr' "_Expr" "var" "Expr"];