equal
deleted
inserted
replaced
36 "{l<..u} == {l<..} Int {..u}" |
36 "{l<..u} == {l<..} Int {..u}" |
37 |
37 |
38 atLeastAtMost :: "['a::ord, 'a] => 'a set" ("(1{_.._})") |
38 atLeastAtMost :: "['a::ord, 'a] => 'a set" ("(1{_.._})") |
39 "{l..u} == {l..} Int {..u}" |
39 "{l..u} == {l..} Int {..u}" |
40 |
40 |
41 (* Old syntax, will disappear! *) |
41 (* Old syntax, no longer supported: |
42 syntax |
42 syntax |
43 "_lessThan" :: "('a::ord) => 'a set" ("(1{.._'(})") |
43 "_lessThan" :: "('a::ord) => 'a set" ("(1{.._'(})") |
44 "_greaterThan" :: "('a::ord) => 'a set" ("(1{')_..})") |
44 "_greaterThan" :: "('a::ord) => 'a set" ("(1{')_..})") |
45 "_greaterThanLessThan" :: "['a::ord, 'a] => 'a set" ("(1{')_.._'(})") |
45 "_greaterThanLessThan" :: "['a::ord, 'a] => 'a set" ("(1{')_.._'(})") |
46 "_atLeastLessThan" :: "['a::ord, 'a] => 'a set" ("(1{_.._'(})") |
46 "_atLeastLessThan" :: "['a::ord, 'a] => 'a set" ("(1{_.._'(})") |
49 "{..m(}" => "{..<m}" |
49 "{..m(}" => "{..<m}" |
50 "{)m..}" => "{m<..}" |
50 "{)m..}" => "{m<..}" |
51 "{)m..n(}" => "{m<..<n}" |
51 "{)m..n(}" => "{m<..<n}" |
52 "{m..n(}" => "{m..<n}" |
52 "{m..n(}" => "{m..<n}" |
53 "{)m..n}" => "{m<..n}" |
53 "{)m..n}" => "{m<..n}" |
54 |
54 *) |
55 |
55 |
56 text{* A note of warning when using @{term"{..<n}"} on type @{typ |
56 text{* A note of warning when using @{term"{..<n}"} on type @{typ |
57 nat}: it is equivalent to @{term"{0::nat..<n}"} but some lemmas involving |
57 nat}: it is equivalent to @{term"{0::nat..<n}"} but some lemmas involving |
58 @{term"{m..<n}"} may not exist in @{term"{..<n}"}-form as well. *} |
58 @{term"{m..<n}"} may not exist in @{term"{..<n}"}-form as well. *} |
59 |
59 |