author | Christian Urban <urbanc@in.tum.de> |
Sun, 29 Aug 2010 12:14:40 +0800 | |
changeset 2452 | 39f8d405d7a2 |
parent 2436 | 3885dc2669f9 |
permissions | -rw-r--r-- |
theory Term8 imports "../NewParser" begin (* example 8 *) atom_decl name nominal_datatype foo = Foo0 "name" | Foo1 b::"bar" f::"foo" bind (set) "bv b" in f and bar = Bar0 "name" | Bar1 "name" s::"name" b::"bar" bind (set) s in b binder bv where "bv (Bar0 x) = {}" | "bv (Bar1 v x b) = {atom v}" (* thm foo_bar.supp *) end