src/HOL/HOL.thy
changeset 18867 f8e4322c9567
parent 18832 6ab4de872a70
child 18887 6ad81e3fa478
equal deleted inserted replaced
18866:378c0cb028a8 18867:f8e4322c9567
  1374   "op +" "IntDef.op_add"
  1374   "op +" "IntDef.op_add"
  1375   "op -" "IntDef.op_minus"
  1375   "op -" "IntDef.op_minus"
  1376   "op *" "IntDef.op_times"
  1376   "op *" "IntDef.op_times"
  1377   Not "HOL.not"
  1377   Not "HOL.not"
  1378   uminus "HOL.uminus"
  1378   uminus "HOL.uminus"
       
  1379   arbitrary "HOL.arbitrary"
  1379 
  1380 
  1380 code_syntax_tyco bool
  1381 code_syntax_tyco bool
  1381   ml (target_atom "bool")
  1382   ml (target_atom "bool")
  1382   haskell (target_atom "Bool")
  1383   haskell (target_atom "Bool")
  1383 
  1384 
  1395     ml ("if __/ then __/ else __")
  1396     ml ("if __/ then __/ else __")
  1396     haskell ("if __/ then __/ else __")
  1397     haskell ("if __/ then __/ else __")
  1397   "op =" (* an intermediate solution *)
  1398   "op =" (* an intermediate solution *)
  1398     ml (infixl 6 "=")
  1399     ml (infixl 6 "=")
  1399     haskell (infixl 4 "==")
  1400     haskell (infixl 4 "==")
       
  1401   arbitrary
       
  1402     ml ("raise/ (Fail/ \"non-defined-result\")")
       
  1403     haskell ("error/ \"non-defined result\"")
  1400 
  1404 
  1401 end
  1405 end