src/HOL/HOL.thy
changeset 20380 14f9f2a1caa6
parent 20223 89d2758ecddf
child 20453 855f07fabd76
equal deleted inserted replaced
20379:154d8c155a65 20380:14f9f2a1caa6
  1418 
  1418 
  1419 setup {*
  1419 setup {*
  1420   CodegenTheorems.init_obj ((TrueI, FalseE), (conjI, thm "HOL.atomize_eq" |> Thm.symmetric))
  1420   CodegenTheorems.init_obj ((TrueI, FalseE), (conjI, thm "HOL.atomize_eq" |> Thm.symmetric))
  1421 *}
  1421 *}
  1422 
  1422 
  1423 code_alias
       
  1424   bool "HOL.bool"
       
  1425   True "HOL.True"
       
  1426   False "HOL.False"
       
  1427   "op =" "HOL.op_eq"
       
  1428   "op -->" "HOL.op_implies"
       
  1429   "op &" "HOL.op_and"
       
  1430   "op |" "HOL.op_or"
       
  1431   Not "HOL.not"
       
  1432   arbitrary "HOL.arbitrary"
       
  1433 
       
  1434 code_constapp
  1423 code_constapp
  1435   "op =" (* an intermediate solution for polymorphic equality *)
  1424   "op =" (* an intermediate solution for polymorphic equality *)
  1436     ml (infixl 6 "=")
  1425     ml (infixl 6 "=")
  1437     haskell (infixl 4 "==")
  1426     haskell (infixl 4 "==")
  1438 
  1427