1 (**************************************************************************)
4 (* ||A|| A project by Andrea Asperti *)
6 (* ||I|| Developers: *)
7 (* ||T|| The HELM team. *)
8 (* ||A|| http://helm.cs.unibo.it *)
10 (* \ / This file is distributed under the terms of the *)
11 (* v GNU General Public License Version 2 *)
13 (**************************************************************************)
28 notation "#" with precedence 90 for @{ 'foo }.
29 interpretation "a" 'foo = a.
30 interpretation "b" 'foo = b.
31 interpretation "c" 'foo = c.
32 interpretation "d" 'foo = d.
34 alias symbol "foo" = "c".
35 alias symbol "foo" = "b".
36 alias symbol "foo" = "d".
37 alias symbol "foo" = "b".
39 lemma xx : ∀P: A → B → Prop. P # #. (* NON STAMPA GLI ALIAS *)