src/Doc/Codegen/Evaluation.thy
changeset 63175 d191892b1c23
parent 63161 2660ba498798
child 63670 8e0148e1f5f4
--- a/src/Doc/Codegen/Evaluation.thy	Sun May 29 14:43:17 2016 +0200
+++ b/src/Doc/Codegen/Evaluation.thy	Sun May 29 14:43:18 2016 +0200
@@ -344,7 +344,7 @@
 \<close>
 
 code_reflect %quote Rat
-  datatypes rat = Frct
+  datatypes rat
   functions Fract
     "(plus :: rat \<Rightarrow> rat \<Rightarrow> rat)" "(minus :: rat \<Rightarrow> rat \<Rightarrow> rat)"
     "(times :: rat \<Rightarrow> rat \<Rightarrow> rat)" "(divide :: rat \<Rightarrow> rat \<Rightarrow> rat)"