src/HOL/HOL.thy
changeset 19607 07eeb832f28d
parent 19598 d68dd20af31f
child 19656 09be06943252
equal deleted inserted replaced
19606:01e23aa70d3a 19607:07eeb832f28d
  1408 
  1408 
  1409 code_syntax_const
  1409 code_syntax_const
  1410   "op =" (* an intermediate solution for polymorphic equality *)
  1410   "op =" (* an intermediate solution for polymorphic equality *)
  1411     ml (infixl 6 "=")
  1411     ml (infixl 6 "=")
  1412     haskell (infixl 4 "==")
  1412     haskell (infixl 4 "==")
  1413   arbitrary
       
  1414     ml ("raise/ (Fail/ \"non-defined-result\")")
       
  1415     haskell ("error/ \"non-defined result\"")
       
  1416 
  1413 
  1417 end
  1414 end