equal
deleted
inserted
replaced
1405 "op *" "HOL.op_times" |
1405 "op *" "HOL.op_times" |
1406 Not "HOL.not" |
1406 Not "HOL.not" |
1407 uminus "HOL.uminus" |
1407 uminus "HOL.uminus" |
1408 arbitrary "HOL.arbitrary" |
1408 arbitrary "HOL.arbitrary" |
1409 |
1409 |
1410 code_syntax_tyco bool |
|
1411 ml (target_atom "bool") |
|
1412 haskell (target_atom "Bool") |
|
1413 |
|
1414 code_syntax_const |
1410 code_syntax_const |
1415 Not |
|
1416 ml (target_atom "not") |
|
1417 haskell (target_atom "not") |
|
1418 "op &" |
|
1419 ml (infixl 1 "andalso") |
|
1420 haskell (infixl 3 "&&") |
|
1421 "op |" |
|
1422 ml (infixl 0 "orelse") |
|
1423 haskell (infixl 2 "||") |
|
1424 If |
|
1425 ml (target_atom "(if __/ then __/ else __)") |
|
1426 haskell (target_atom "(if __/ then __/ else __)") |
|
1427 "op =" (* an intermediate solution for polymorphic equality *) |
1411 "op =" (* an intermediate solution for polymorphic equality *) |
1428 ml (infixl 6 "=") |
1412 ml (infixl 6 "=") |
1429 haskell (infixl 4 "==") |
1413 haskell (infixl 4 "==") |
1430 arbitrary |
1414 arbitrary |
1431 ml ("raise/ (Fail/ \"non-defined-result\")") |
1415 ml ("raise/ (Fail/ \"non-defined-result\")") |