| author | huffman | 
| Sun, 17 Sep 2006 16:44:05 +0200 | |
| changeset 20561 | 6a6d8004322f | 
| parent 19048 | 2b875dd5eb4c | 
| child 26435 | bdce320cd426 | 
| permissions | -rw-r--r-- | 
| 15804 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 1 | (* Title: Pure/CPure.thy | 
| 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 2 | ID: $Id$ | 
| 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 3 | |
| 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 4 | The CPure theory -- Pure with alternative application syntax. | 
| 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 5 | *) | 
| 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 6 | |
| 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 7 | theory CPure | 
| 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 8 | imports Pure | 
| 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 9 | begin | 
| 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 10 | |
| 19048 | 11 | setup  -- {* Some syntax modifications, see ROOT.ML *}
 | 
| 15804 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 12 | |
| 
3a55e6e26c8a
The CPure theory -- Pure with alternative application syntax.
 wenzelm parents: diff
changeset | 13 | end |