doc-src/IsarAdvanced/Codegen/Thy/Adaption.thy
changeset 28714 1992553cccfe
parent 28679 d7384e8e99b3
equal deleted inserted replaced
28713:135317cd34d6 28714:1992553cccfe
   299   for the class @{class eq} (by command @{command code_class}) and its operation
   299   for the class @{class eq} (by command @{command code_class}) and its operation
   300   @{const HOL.eq}
   300   @{const HOL.eq}
   301 *}
   301 *}
   302 
   302 
   303 code_class %quotett eq
   303 code_class %quotett eq
   304   (Haskell "Eq" where "HOL.eq" \<equiv> "(==)")
   304   (Haskell "Eq")
   305 
   305 
   306 code_const %quotett "op ="
   306 code_const %quotett "op ="
   307   (Haskell infixl 4 "==")
   307   (Haskell infixl 4 "==")
   308 
   308 
   309 text {*
   309 text {*