changeset 17782 | b3846df9d643 |
parent 17260 | df7c3b1f390a |
child 22809 | 3cf5df73d50a |
--- a/src/Cube/Cube.thy Fri Oct 07 22:59:18 2005 +0200 +++ b/src/Cube/Cube.thy Fri Oct 07 22:59:19 2005 +0200 @@ -39,7 +39,7 @@ ("prop") "x:X" == ("prop") "|- x:X" "Lam x:A. B" == "Abs(A, %x. B)" "Pi x:A. B" => "Prod(A, %x. B)" - "A -> B" => "Prod(A, _K(B))" + "A -> B" => "Prod(A, %_. B)" syntax (xsymbols) Trueprop :: "[context_, typing_] => prop" ("(_/ \<turnstile> _)")