src/Pure/CPure.thy
changeset 15804 3a55e6e26c8a
child 18019 d1ff9ebb8bcb
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/Pure/CPure.thy	Thu Apr 21 22:06:18 2005 +0200
@@ -0,0 +1,16 @@
+(*  Title:      Pure/CPure.thy
+    ID:         $Id$
+    Author:     Makarius
+
+The CPure theory -- Pure with alternative application syntax.
+*)
+
+theory CPure
+imports Pure
+begin
+
+setup
+"[Theory.del_modesyntax Syntax.default_mode Syntax.pure_appl_syntax,
+  Theory.add_syntax Syntax.pure_applC_syntax]"
+
+end